Yoneda embedding of Mon C
#
We show that monoid objects in Cartesian monoidal categories 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.
Equations
- One or more equations did not get rendered due to their size.
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 MonObj.ofRepresentableBy
.
If X
represents a presheaf of monoids, then X
is a monoid object.
Equations
Instances For
Alias of MonObj.ofRepresentableBy
.
If X
represents a presheaf of monoids, then X
is a monoid object.
Equations
Instances For
Alias of MonObj.ofRepresentableBy
.
Alias of MonObj.ofRepresentableBy
.
If X
represents a presheaf of monoids, then X
is a monoid object.
Equations
Instances For
If M
is a monoid object, then Hom(X, M)
has a monoid structure.
Equations
- One or more equations did not get rendered due to their size.
Instances For
If M
is a commutative monoid object, then Hom(X, M)
has a commutative monoid structure.
Equations
- Hom.commMonoid = { toMonoid := Hom.monoid, mul_comm := ⋯ }
Instances For
If M
is a monoid object, then Hom(-, M)
is a presheaf of monoids.
Equations
- One or more equations did not get rendered due to their size.
Instances For
If X
represents a presheaf of monoids F
, then Hom(-, X)
is isomorphic to F
as
a presheaf of monoids.
Equations
- yonedaMonObjIsoOfRepresentableBy X F α = CategoryTheory.NatIso.ofComponents (fun (Y : Cᵒᵖ) => (let __Equiv := α.homEquiv; { toEquiv := __Equiv, 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
If M
is a monoid object, then Hom(-, M)
as a presheaf of monoids is represented by M
.
Equations
Instances For
Alias of MonObj.ofRepresentableBy_yonedaMonObjRepresentableBy
.
Alias of MonObj.ofRepresentableBy_yonedaMonObjRepresentableBy
.
Alias of MonObj.ofRepresentableBy_yonedaMonObjRepresentableBy
.
Alias of MonObj.ofRepresentableBy_yonedaMonObjRepresentableBy
.
The yoneda embedding for Mon_C
is fully faithful.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Alias of MonObj.one_comp
.
Alias of MonObj.mul_comp
.
Alias of MonObj.pow_comp
.
Alias of MonObj.comp_one
.
Alias of MonObj.comp_mul
.
Alias of MonObj.comp_pow
.
Alias of MonObj.one_eq_one
.
Alias of MonObj.mul_eq_mul
.