Documentation

Mathlib.CategoryTheory.Monoidal.CommMon_

The category of commutative monoids in a braided monoidal category. #

structure CategoryTheory.CommMon (C : Type u₁) [Category.{v₁, u₁} C] [MonoidalCategory C] [BraidedCategory C] :
Type (max u₁ v₁)

A commutative monoid object internal to a monoidal category.

  • X : C

    The underlying object in the ambient monoidal category

  • mon : MonObj self.X
  • comm : IsCommMonObj self.X
Instances For
    @[deprecated CategoryTheory.CommMon (since := "2025-09-15")]

    Alias of CategoryTheory.CommMon.


    A commutative monoid object internal to a monoidal category.

    Equations
    Instances For

      A commutative monoid object is a monoid object.

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

        Alias of CategoryTheory.CommMon.toMon.


        A commutative monoid object is a monoid object.

        Equations
        Instances For

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

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

            The forgetful functor from commutative monoid objects to monoid objects.

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

              Alias of CategoryTheory.CommMon.forget₂Mon.


              The forgetful functor from commutative monoid objects to monoid objects.

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

                Alias of CategoryTheory.CommMon.fullyFaithfulForget₂Mon.


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

                Equations
                Instances For

                  The forgetful functor from commutative monoid objects to the ambient category.

                  Equations
                  Instances For
                    @[simp]
                    theorem CategoryTheory.CommMon.forget_map (C : Type u₁) [Category.{v₁, u₁} C] [MonoidalCategory C] [BraidedCategory C] {X✝ Y✝ : CommMon C} (f : X✝ Y✝) :
                    (forget C).map f = f.hom
                    def CategoryTheory.CommMon.mkIso' {C : Type u₁} [Category.{v₁, u₁} C] [MonoidalCategory C] [BraidedCategory C] {M N : C} (e : M N) [MonObj M] [IsCommMonObj M] [MonObj N] [IsCommMonObj N] [IsMonHom e.hom] :
                    { X := M, mon := inst✝, comm := inst✝¹ } { X := N, mon := inst✝², comm := inst✝³ }

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

                    Equations
                    Instances For
                      @[reducible, inline]

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

                      Equations
                      Instances For

                        A lax braided functor takes commutative monoid objects to commutative monoid objects.

                        That is, a lax braided functor F : C ⥤ D induces a functor CommMon C ⥤ CommMon D.

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

                          The identity functor is also the identity on commutative monoid objects.

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

                            The composition functor is also the composition on commutative monoid objects.

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

                              mapCommMon is functorial in the lax braided functor.

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

                                Natural transformations between functors lift to monoid objects.

                                Equations
                                Instances For

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

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

                                    An adjunction of braided functors lifts to an adjunction of their lifts to commutative monoid 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 commutative monoid objects.

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

                                        Implementation of CommMon.equivLaxBraidedFunctorPUnit.

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

                                          Implementation of CommMon.equivLaxBraidedFunctorPUnit.

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

                                            Implementation of CommMon.equivLaxBraidedFunctorPUnit.

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

                                              Commutative monoid objects in C are "just" braided lax monoidal functors from the trivial braided monoidal category to C.

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