Documentation

Mathlib.CategoryTheory.Monad.Equalizer

Special equalizers associated to a comonad #

Associated to a comonad T : C ⥤ C we have important equalizer constructions: Any coalgebra is an equalizer (in the category of coalgebras) of cofree coalgebras. Furthermore, this equalizer is coreflexive. In C, this fork diagram is a split equalizer (in particular, it is still an equalizer). This split equalizer is known as the Beck equalizer (as it features heavily in Beck's comonadicity theorem).

This file is adapted from Mathlib.CategoryTheory.Monad.Coequalizer. Please try to keep them in sync.

Show that any coalgebra is an equalizer of cofree coalgebras.

def CategoryTheory.Comonad.CofreeEqualizer.topMap {C : Type u₁} [CategoryTheory.Category.{v₁, u₁} C] {T : CategoryTheory.Comonad C} (X : T.Coalgebra) :
T.cofree.obj X.A T.cofree.obj (T.obj X.A)

The top map in the equalizer diagram we will construct.

Equations
Instances For
    def CategoryTheory.Comonad.CofreeEqualizer.bottomMap {C : Type u₁} [CategoryTheory.Category.{v₁, u₁} C] {T : CategoryTheory.Comonad C} (X : T.Coalgebra) :
    T.cofree.obj X.A T.cofree.obj (T.obj X.A)

    The bottom map in the equalizer diagram we will construct.

    Equations
    Instances For

      The fork map in the equalizer diagram we will construct.

      Equations
      Instances For

        The fork constructed is a limit. This shows that any coalgebra is a (coreflexive) equalizer of cofree coalgebras.

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

          The Beck fork is a split equalizer.

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

            This is the Beck fork. It is a split equalizer, in particular a equalizer.

            Equations
            Instances For