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.

structure Grp_ (C : Type u₁) [CategoryTheory.Category.{v₁, u₁} C] [CategoryTheory.ChosenFiniteProducts C] extends Mon_ C :
Type (max u₁ v₁)

A group object in a cartesian monoidal category.

Instances For

    The trivial group object.

    Equations
    Instances For
      theorem Grp_.hom_ext {C : Type u₁} [CategoryTheory.Category.{v₁, u₁} C] [CategoryTheory.ChosenFiniteProducts C] {A B : Grp_ C} (f g : A B) (h : f.hom = g.hom) :
      f = g

      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.

      The forgetful functor from group objects to the ambient category.

      Equations
      Instances For
        @[simp]
        theorem Grp_.forget_map (C : Type u₁) [CategoryTheory.Category.{v₁, u₁} C] [CategoryTheory.ChosenFiniteProducts C] {X✝ Y✝ : Grp_ C} (f : X✝ Y✝) :
        (forget C).map f = f.hom

        Constructor for isomorphisms in the category Grp_ C.

        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

            mapGrp is functorial in the left-exact functor.

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