Yoneda embedding of Mon_ C
#
We show that monoid objects are exactly those whose yoneda presheaf is a presheaf of monoids,
by constructing the yoneda embedding Mon_ C ⥤ Cᵒᵖ ⥤ MonCat.{v}
and
showing that it is fully faithful and its (essential) image is the representable functors.
If X
represents a presheaf of monoids, then X
is a monoid object.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Alias of Mon_Class.ofRepresentableBy
.
If X
represents a presheaf of monoids, then X
is a monoid object.
Instances For
If X
is a monoid object, then Hom(Y, X)
has a monoid structure.
Equations
- monoidOfMon_Class X Y = Monoid.mk ⋯ ⋯ npowRecAuto ⋯ ⋯
Instances For
If X
is a monoid object, then Hom(-, X)
is a presheaf of monoids.
Equations
- One or more equations did not get rendered due to their size.
Instances For
If X
is a monoid object, then Hom(-, X)
as a presheaf of monoids is represented by X
.
Equations
Instances For
Alias of Mon_Class.ofRepresentableBy_yonedaMonObjRepresentableBy
.
If X
represents a presheaf of monoids F
, then Hom(-, X)
is isomorphic to F
as
a presheaf of monoids.
Equations
- yonedaMonObjMon_Class.ofRepresentableBy X F α = CategoryTheory.NatIso.ofComponents (fun (Y : Cᵒᵖ) => { toEquiv := α.homEquiv, map_mul' := ⋯ }.toMonCatIso) ⋯
Instances For
The yoneda embedding of Mon_C
into presheaves of monoids.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The yoneda embedding for Mon_C
is fully faithful.
Equations
- One or more equations did not get rendered due to their size.
Instances For
If X
represents a presheaf of commutative groups, then X
is a commutative group object.