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.

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) :
      (CategoryTheory.Discrete.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) :
      (CategoryTheory.Discrete.addMonoidalFunctor F).obj { as := m } = { as := F m }
      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.