Documentation

Mathlib.CategoryTheory.Monoidal.Discrete

Monoids as discrete monoidal categories #

The discrete category on a monoid is a monoidal category. Multiplicative morphisms induced monoidal functors.

@[simp]
@[simp]
theorem CategoryTheory.Discrete.monoidal_associator (M : Type u) [Monoid M] (x✝ x✝¹ x✝² : Discrete M) :
@[simp]

A multiplicative morphism between monoids gives a monoidal functor between the corresponding discrete monoidal categories.

Equations
Instances For

    An additive morphism between add_monoids gives a monoidal functor between the corresponding discrete monoidal categories.

    Equations
    Instances For
      @[simp]
      theorem CategoryTheory.Discrete.monoidalFunctor_obj {M : Type u} [Monoid M] {N : Type u'} [Monoid N] (F : M →* N) (m : M) :
      (monoidalFunctor F).obj { as := m } = { as := F m }
      @[simp]
      theorem CategoryTheory.Discrete.addMonoidalFunctor_obj {M : Type u} [AddMonoid M] {N : Type u'} [AddMonoid N] (F : M →+ N) (m : M) :
      (addMonoidalFunctor F).obj { as := m } = { as := F m }
      instance CategoryTheory.Discrete.monoidalFunctorMonoidal {M : Type u} [Monoid M] {N : Type u'} [Monoid N] (F : M →* N) :
      (monoidalFunctor F).Monoidal
      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.
      def CategoryTheory.Discrete.monoidalFunctorComp {M : Type u} [Monoid M] {N : Type u'} [Monoid N] {K : Type u} [Monoid K] (F : M →* N) (G : N →* K) :

      The monoidal natural isomorphism corresponding to composing two multiplicative morphisms.

      Equations
      Instances For

        The monoidal natural isomorphism corresponding to composing two additive morphisms.

        Equations
        Instances For