Documentation

Mathlib.CategoryTheory.Monoidal.Mon_

The category of monoids in a monoidal category. #

We define monoids in a monoidal category C and show that the category of monoids is equivalent to the category of lax monoidal functors from the unit monoidal category to C. We also show that if C is braided, then the category of monoids is naturally monoidal.

A monoid object internal to a monoidal category.

When the monoidal category is preadditive, this is also sometimes called an "algebra object".

Instances For

    The trivial monoid object. We later show this is initial in Mon_ C.

    Equations
    Instances For
      theorem Mon_.Hom.ext_iff {C : Type u₁} :
      ∀ {inst : CategoryTheory.Category.{v₁, u₁} C} {inst_1 : CategoryTheory.MonoidalCategory C} {M N : Mon_ C} (x y : M.Hom N), x = y x.hom = y.hom
      theorem Mon_.Hom.ext {C : Type u₁} :
      ∀ {inst : CategoryTheory.Category.{v₁, u₁} C} {inst_1 : CategoryTheory.MonoidalCategory C} {M N : Mon_ C} (x y : M.Hom N), x.hom = y.homx = y

      A morphism of monoid objects.

      Instances For
        @[simp]
        theorem Mon_.Hom.one_hom {C : Type u₁} [CategoryTheory.Category.{v₁, u₁} C] [CategoryTheory.MonoidalCategory C] {M : Mon_ C} {N : Mon_ C} (self : M.Hom N) :

        The identity morphism on a monoid object.

        Equations
        Instances For
          Equations
          • M.homInhabited = { default := M.id }
          @[simp]
          theorem Mon_.comp_hom {C : Type u₁} [CategoryTheory.Category.{v₁, u₁} C] [CategoryTheory.MonoidalCategory C] {M : Mon_ C} {N : Mon_ C} {O : Mon_ C} (f : M.Hom N) (g : N.Hom O) :
          def Mon_.comp {C : Type u₁} [CategoryTheory.Category.{v₁, u₁} C] [CategoryTheory.MonoidalCategory C] {M : Mon_ C} {N : Mon_ C} {O : Mon_ C} (f : M.Hom N) (g : N.Hom O) :
          M.Hom O

          Composition of morphisms of monoid objects.

          Equations
          Instances For
            theorem Mon_.ext {C : Type u₁} [CategoryTheory.Category.{v₁, u₁} C] [CategoryTheory.MonoidalCategory C] {X : Mon_ C} {Y : Mon_ C} {f : X Y} {g : X Y} (w : f.hom = g.hom) :
            f = g
            @[simp]
            theorem Mon_.forget_map (C : Type u₁) [CategoryTheory.Category.{v₁, u₁} C] [CategoryTheory.MonoidalCategory C] :
            ∀ {X Y : Mon_ C} (f : X Y), (Mon_.forget C).map f = f.hom

            The forgetful functor from monoid objects to the ambient category.

            Equations
            • Mon_.forget C = { obj := fun (A : Mon_ C) => A.X, map := fun {X Y : Mon_ C} (f : X Y) => f.hom, map_id := , map_comp := }
            Instances For

              The forgetful functor from monoid objects to the ambient category reflects isomorphisms.

              Equations
              • =
              @[simp]
              @[simp]

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

              Equations
              • Mon_.isoOfIso f one_f mul_f = { hom := { hom := f.hom, one_hom := one_f, mul_hom := mul_f }, inv := { hom := f.inv, one_hom := , mul_hom := }, hom_inv_id := , inv_hom_id := }
              Instances For
                Equations
                • A.uniqueHomFromTrivial = { default := { hom := A.one, one_hom := , mul_hom := }, uniq := }

                A lax monoidal functor takes monoid objects to monoid objects.

                That is, a lax monoidal functor F : C ⥤ D induces a functor Mon_ C ⥤ Mon_ D.

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

                  mapMon is functorial in the lax monoidal functor.

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

                    Monoid objects in C are "just" lax monoidal functors from the trivial monoidal category to C.

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

                      In this section, we prove that the category of monoids in a braided monoidal category is monoidal.

                      Given two monoids M and N in a braided monoidal category C, the multiplication on the tensor product M.X ⊗ N.X is defined in the obvious way: it is the tensor product of the multiplications on M and N, except that the tensor factors in the source come in the wrong order, which we fix by pre-composing with a permutation isomorphism constructed from the braiding.

                      (There is a subtlety here: in fact there are two ways to do these, using either the positive or negative crossing.)

                      A more conceptual way of understanding this definition is the following: The braiding on C gives rise to a monoidal structure on the tensor product functor from C × C to C. A pair of monoids in C gives rise to a monoid in C × C, which the tensor product functor by being monoidal takes to a monoid in C. The permutation isomorphism appearing in the definition of the multiplication on the tensor product of two monoids is an instance of a more general family of isomorphisms which together form a strength that equips the tensor product functor with a monoidal structure, and the monoid axioms for the tensor product follow from the monoid axioms for the tensor factors plus the properties of the strength (i.e., monoidal functor axioms). The strength tensor_μ of the tensor product functor has been defined in Mathlib.CategoryTheory.Monoidal.Braided. Its properties, stated as independent lemmas in that module, are used extensively in the proofs below. Notice that we could have followed the above plan not only conceptually but also as a possible implementation and could have constructed the tensor product of monoids via mapMon, but we chose to give a more explicit definition directly in terms of tensor_μ.

                      To complete the definition of the monoidal category structure on the category of monoids, we need to provide definitions of associator and unitors. The obvious candidates are the associator and unitors from C, but we need to prove that they are monoid morphisms, i.e., compatible with unit and multiplication. These properties translate to the monoidality of the associator and unitors (with respect to the monoidal structures on the functors they relate), which have also been proved in Mathlib.CategoryTheory.Monoidal.Braided.

                      Projects: