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.
Equations
- CategoryTheory.Grp.homMk f = { hom := f, isMonHom_hom := inst✝ }
Instances For
Alias of CategoryTheory.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 CategoryTheory.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 CategoryTheory.GrpObj.ofRepresentableBy.
If X represents a presheaf of monoids, then X is a monoid object.
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 CategoryTheory.GrpObj.ofRepresentableBy_yonedaGrpObjRepresentableBy.
If X represents a presheaf of groups F, then Hom(-, X) is isomorphic to F as
a presheaf of groups.
Equations
- One or more equations did not get rendered due to their size.
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 CategoryTheory.GrpObj.inv_comp.
Alias of CategoryTheory.GrpObj.div_comp.
Alias of CategoryTheory.GrpObj.zpow_comp.
Alias of CategoryTheory.GrpObj.comp_inv.
Alias of CategoryTheory.GrpObj.comp_div.
Alias of CategoryTheory.GrpObj.comp_zpow.
Alias of CategoryTheory.GrpObj.inv_eq_inv.
Equations
- CategoryTheory.Grp.instMonObj = { one := CategoryTheory.MonObj.one, mul := CategoryTheory.MonObj.mul, one_mul := ⋯, mul_one := ⋯, mul_assoc := ⋯ }
A commutative group object is a group object in the category of group objects.
Equations
- CategoryTheory.Grp.instGrpObj = { toMonObj := CategoryTheory.Grp.instMonObj, inv := { hom := CategoryTheory.GrpObj.inv, isMonHom_hom := ⋯ }, left_inv := ⋯, right_inv := ⋯ }
A commutative group object is a commutative group object in the category of group objects.
If G is a commutative group object, then Hom(X, G) has a commutative group structure.
Equations
- CategoryTheory.Hom.commGroup = { toGroup := CategoryTheory.Hom.group, mul_comm := ⋯ }