Documentation

Mathlib.CategoryTheory.Monoidal.Grp_

The category of groups in a Cartesian monoidal category #

We define group objects in Cartesian monoidal categories.

We show that the associativity diagram of a group object is always Cartesian and deduce that morphisms of group objects commute with taking inverses.

We show that a finite-product-preserving functor takes group objects to group objects.

@[deprecated CategoryTheory.GrpObj (since := "2025-09-13")]

Alias of CategoryTheory.GrpObj.


A group object internal to a cartesian monoidal category. Also see the bundled Grp.

Equations
Instances For

    The inverse in a group object

    Equations
    Instances For

      The inverse in a group object

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        Equations
        • One or more equations did not get rendered due to their size.
        structure CategoryTheory.Grp (C : Type u₁) [Category.{v₁, u₁} C] [CartesianMonoidalCategory C] :
        Type (max u₁ v₁)

        A group object in a Cartesian monoidal category.

        • X : C

          The underlying object in the ambient monoidal category

        • grp : GrpObj self.X
        Instances For
          @[deprecated CategoryTheory.Grp (since := "2025-10-13")]

          Alias of CategoryTheory.Grp.


          A group object in a Cartesian monoidal category.

          Equations
          Instances For

            A group object is a monoid object.

            Equations
            Instances For
              @[deprecated CategoryTheory.Grp.toMon (since := "2025-09-15")]

              Alias of CategoryTheory.Grp.toMon.


              A group object is a monoid object.

              Equations
              Instances For
                @[deprecated CategoryTheory.Grp.mk (since := "2025-06-15")]

                Alias of CategoryTheory.Grp.mk.

                Equations
                Instances For
                  theorem CategoryTheory.Grp.hom_ext {C : Type u₁} [Category.{v₁, u₁} C] [CartesianMonoidalCategory C] {A B : Grp C} (f g : A B) (h : f.hom = g.hom) :
                  f = g
                  @[simp]
                  theorem CategoryTheory.Grp.comp' {C : Type u₁} [Category.{v₁, u₁} C] [CartesianMonoidalCategory C] {A₁ A₂ A₃ : Grp C} (f : A₁ A₂) (g : A₂ A₃) :
                  @[reducible, inline]

                  Transfer GrpObj along an isomorphism.

                  Equations
                  • One or more equations did not get rendered due to their size.
                  Instances For

                    The map (· * f).

                    Equations
                    • One or more equations did not get rendered due to their size.
                    Instances For

                      The associativity diagram of a group object is Cartesian.

                      In fact, any monoid object whose associativity diagram is Cartesian can be made into a group object (we do not prove this in this file), so we should expect that many properties of group objects follow from this result.

                      @[simp]

                      Morphisms of group objects preserve inverses.

                      @[deprecated CategoryTheory.GrpObj.toMonObj_injective (since := "2025-09-09")]

                      Alias of CategoryTheory.GrpObj.toMonObj_injective.

                      theorem CategoryTheory.GrpObj.ext {C : Type u₁} [Category.{v₁, u₁} C] [CartesianMonoidalCategory C] {X : C} (h₁ h₂ : GrpObj X) (H : h₁.toMonObj = h₂.toMonObj) :
                      h₁ = h₂
                      theorem CategoryTheory.GrpObj.ext_iff {C : Type u₁} [Category.{v₁, u₁} C] [CartesianMonoidalCategory C] {X : C} {h₁ h₂ : GrpObj X} :
                      h₁ = h₂ h₁.toMonObj = h₂.toMonObj
                      Equations
                      • One or more equations did not get rendered due to their size.

                      The forgetful functor from group objects to monoid objects.

                      Equations
                      Instances For
                        @[deprecated CategoryTheory.Grp.forget₂Mon (since := "2025-09-15")]

                        Alias of CategoryTheory.Grp.forget₂Mon.


                        The forgetful functor from group objects to monoid objects.

                        Equations
                        Instances For
                          @[deprecated CategoryTheory.Grp.fullyFaithfulForget₂Mon (since := "2025-09-15")]

                          Alias of CategoryTheory.Grp.fullyFaithfulForget₂Mon.


                          The forgetful functor from group objects to monoid objects is fully faithful.

                          Equations
                          Instances For

                            The forgetful functor from group objects to the ambient category.

                            Equations
                            Instances For
                              @[simp]
                              theorem CategoryTheory.Grp.forget_map (C : Type u₁) [Category.{v₁, u₁} C] [CartesianMonoidalCategory C] {X✝ Y✝ : Grp C} (f : X✝ Y✝) :
                              (forget C).map f = f.hom
                              def CategoryTheory.Grp.mkIso' {C : Type u₁} [Category.{v₁, u₁} C] [CartesianMonoidalCategory C] {G H : C} (e : G H) [GrpObj G] [GrpObj H] [IsMonHom e.hom] :
                              { X := G, grp := inst✝ } { X := H, grp := inst✝¹ }

                              Construct an isomorphism of group objects by giving a monoid isomorphism between the underlying objects.

                              Equations
                              Instances For
                                @[reducible, inline]

                                Construct an isomorphism of group objects by giving an isomorphism between the underlying objects and checking compatibility with unit and multiplication only in the forward direction.

                                Equations
                                Instances For

                                  Grp C is cartesian-monoidal #

                                  Equations
                                  • One or more equations did not get rendered due to their size.
                                  @[simp]
                                  theorem CategoryTheory.Grp.tensorHom_hom {C : Type u₁} [Category.{v₁, u₁} C] [CartesianMonoidalCategory C] [BraidedCategory C] {X₁✝ Y₁✝ X₂✝ Y₂✝ : Grp C} (f : X₁✝.toMon Y₁✝.toMon) (g : X₂✝.toMon Y₂✝.toMon) :
                                  Equations
                                  • One or more equations did not get rendered due to their size.
                                  Equations
                                  • One or more equations did not get rendered due to their size.
                                  Equations
                                  • One or more equations did not get rendered due to their size.
                                  Equations
                                  • One or more equations did not get rendered due to their size.
                                  @[reducible, inline]

                                  The image of a group object under a monoidal functor is a group object.

                                  Equations
                                  Instances For

                                    A finite-product-preserving functor takes group objects to group objects.

                                    Equations
                                    • One or more equations did not get rendered due to their size.
                                    Instances For
                                      @[simp]
                                      theorem CategoryTheory.Functor.mapGrp_map_hom {C : Type u₁} [Category.{v₁, u₁} C] [CartesianMonoidalCategory C] {D : Type u₂} [Category.{v₂, u₂} D] [CartesianMonoidalCategory D] (F : Functor C D) [F.Monoidal] {X✝ Y✝ : Grp C} (f : X✝ Y✝) :
                                      (F.mapGrp.map f).hom = F.map f.hom

                                      If F : C ⥤ D is a fully faithful monoidal functor, then GrpCat(F) : GrpCat C ⥤ GrpCat D is fully faithful too.

                                      Equations
                                      • One or more equations did not get rendered due to their size.
                                      Instances For

                                        The identity functor is also the identity on group objects.

                                        Equations
                                        • One or more equations did not get rendered due to their size.
                                        Instances For

                                          The composition functor is also the composition on group objects.

                                          Equations
                                          • One or more equations did not get rendered due to their size.
                                          Instances For

                                            Natural transformations between functors lift to group objects.

                                            Equations
                                            Instances For

                                              Natural isomorphisms between functors lift to group objects.

                                              Equations
                                              Instances For

                                                mapGrp is functorial in the left-exact functor.

                                                Equations
                                                • One or more equations did not get rendered due to their size.
                                                Instances For
                                                  @[reducible, inline]

                                                  Pullback a group object along a fully faithful monoidal functor.

                                                  Equations
                                                  Instances For
                                                    @[deprecated CategoryTheory.Functor.FullyFaithful.grpObj (since := "2025-09-13")]

                                                    Alias of CategoryTheory.Functor.FullyFaithful.grpObj.


                                                    Pullback a group object along a fully faithful monoidal functor.

                                                    Equations
                                                    Instances For
                                                      @[simp]

                                                      The essential image of a full and faithful functor between cartesian-monoidal categories is the same on group objects as on objects.

                                                      Equations
                                                      • One or more equations did not get rendered due to their size.

                                                      An adjunction of monoidal functors lifts to an adjunction of their lifts to group objects.

                                                      Equations
                                                      • One or more equations did not get rendered due to their size.
                                                      Instances For

                                                        An equivalence of categories lifts to an equivalence of their group objects.

                                                        Equations
                                                        • One or more equations did not get rendered due to their size.
                                                        Instances For