Yoneda embedding of Grp C #
We show that group objects are exactly those whose yoneda presheaf is a presheaf of groups,
by constructing the yoneda embedding Grp C ⥤ Cᵒᵖ ⥤ GrpCat.{v} and
showing that it is fully faithful and its (essential) image is the representable functors.
Construct a morphism G ⟶ H of Grp C C from a map f : G ⟶ H and a IsMonHom f
instance.
Instances For
Alias of Grp.homMk.
Construct a morphism G ⟶ H of Grp C C from a map f : G ⟶ H and a IsMonHom f
instance.
Equations
Instances For
Alias of Grp.homMk_hom'.
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 GrpObj.ofRepresentableBy.
If X represents a presheaf of monoids, then X is a monoid object.
Equations
Instances For
If G is a group object, then Hom(X, G) has a group structure.
Equations
- One or more equations did not get rendered due to their size.
Instances For
If G is a group object, then Hom(-, G) is a presheaf of groups.
Equations
- One or more equations did not get rendered due to their size.
Instances For
If G is a monoid object, then Hom(-, G) as a presheaf of monoids is represented by G.
Equations
Instances For
Alias of GrpObj.ofRepresentableBy_yonedaGrpObjRepresentableBy.
If X represents a presheaf of groups F, then Hom(-, X) is isomorphic to F as
a presheaf of groups.
Equations
- yonedaGrpObjIsoOfRepresentableBy X F α = CategoryTheory.NatIso.ofComponents (fun (Y : Cᵒᵖ) => (let __Equiv := α.homEquiv; { toEquiv := __Equiv, map_mul' := ⋯ }).toGrpIso) ⋯
Instances For
The yoneda embedding of Grp_C into presheaves of groups.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The yoneda embedding for Grp_C is fully faithful.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Alias of GrpObj.inv_comp.
Alias of GrpObj.div_comp.
Alias of GrpObj.zpow_comp.
Alias of GrpObj.comp_inv.
Alias of GrpObj.comp_div.
Alias of GrpObj.comp_zpow.
Alias of GrpObj.inv_eq_inv.
If G is a commutative group object, then Hom(X, G) has a commutative group structure.
Equations
- Hom.commGroup = { toGroup := Hom.group, mul_comm := ⋯ }