Documentation

Mathlib.CategoryTheory.Monad.EquivMon

The equivalence between Monad C and Mon_ (C ⥤ C). #

A monad "is just" a monoid in the category of endofunctors.

Definitions/Theorems #

  1. toMon associates a monoid object in C ⥤ C to any monad on C.
  2. monadToMon is the functorial version of toMon.
  3. ofMon associates a monad on C to any monoid object in C ⥤ C.
  4. monadMonEquiv is the equivalence between Monad C and Mon_ (C ⥤ C).

To every Monad C we associated a monoid object in C ⥤ C.

Equations
  • M.toMon = { X := M.toFunctor, one := M.η, mul := M.μ, one_mul := , mul_one := , mul_assoc := }
Instances For
    @[simp]
    @[simp]

    Passing from Monad C to Mon_ (C ⥤ C) is functorial.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      @[simp]
      theorem CategoryTheory.Monad.monadToMon_map_hom (C : Type u) [Category.{v, u} C] {X✝ Y✝ : Monad C} (f : X✝ Y✝) :

      To every monoid object in C ⥤ C we associate a Monad C.

      Equations
      Instances For
        @[simp]
        theorem CategoryTheory.Monad.ofMon_η {C : Type u} [Category.{v, u} C] (M : Mon_ (Functor C C)) :
        (ofMon M).η = M.one
        @[simp]
        theorem CategoryTheory.Monad.ofMon_μ {C : Type u} [Category.{v, u} C] (M : Mon_ (Functor C C)) :
        (ofMon M).μ = M.mul
        @[simp]
        theorem CategoryTheory.Monad.ofMon_obj {C : Type u} [Category.{v, u} C] (M : Mon_ (Functor C C)) (X : C) :
        (ofMon M).obj X = M.X.obj X

        Passing from Mon_ (C ⥤ C) to Monad C is functorial.

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

          Oh, monads are just monoids in the category of endofunctors (equivalence of categories).

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