Documentation

Mathlib.CategoryTheory.Monoidal.CommMon_

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

A commutative monoid object internal to a monoidal category.

  • X : C

    The underlying object in the ambient monoidal category

  • mon : Mon_Class self.X
  • comm : IsCommMon self.X
Instances For

    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
        @[deprecated CommMon_.forget₂Mon_map_hom (since := "2025-02-07")]

        Alias of CommMon_.forget₂Mon_map_hom.

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

        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
              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

                    Natural isomorphisms between functors lift to monoid objects.

                    Equations
                    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

                          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