Documentation

Mathlib.CategoryTheory.Monad.Kleisli

Kleisli category on a (co)monad #

This file defines the Kleisli category on a monad (T, η_ T, μ_ T) as well as the co-Kleisli category on a comonad (U, ε_ U, δ_ U). It also defines the Kleisli adjunction which gives rise to the monad (T, η_ T, μ_ T) as well as the co-Kleisli adjunction which gives rise to the comonad (U, ε_ U, δ_ U).

References #

The objects for the Kleisli category of the monad T : Monad C, which are the same thing as objects of the base category C.

Equations
Instances For

    The Kleisli category on a monad T. cf Definition 5.2.9 in Riehl.

    Equations

    The left adjoint of the adjunction which induces the monad (T, η_ T, μ_ T).

    Equations
    Instances For
      @[simp]
      theorem CategoryTheory.Kleisli.Adjunction.toKleisli_obj {C : Type u} [Category.{v, u} C] (T : Monad C) (X : C) :
      (toKleisli T).obj X = X
      @[simp]
      theorem CategoryTheory.Kleisli.Adjunction.toKleisli_map {C : Type u} [Category.{v, u} C] (T : Monad C) {X Y : C} (f : X Y) :
      (toKleisli T).map f = CategoryStruct.comp f (T.app Y)

      The right adjoint of the adjunction which induces the monad (T, η_ T, μ_ T).

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        @[simp]
        @[simp]
        theorem CategoryTheory.Kleisli.Adjunction.fromKleisli_map {C : Type u} [Category.{v, u} C] (T : Monad C) {x✝ Y : Kleisli T} (f : x✝ Y) :
        (fromKleisli T).map f = CategoryStruct.comp (T.map f) (T.app Y)

        The Kleisli adjunction which gives rise to the monad (T, η_ T, μ_ T). cf Lemma 5.2.11 of Riehl.

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

          The composition of the adjunction gives the original functor.

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

            The objects for the co-Kleisli category of the comonad U : Comonad C, which are the same thing as objects of the base category C.

            Equations
            Instances For

              The co-Kleisli category on a comonad U.

              Equations

              The right adjoint of the adjunction which induces the comonad (U, ε_ U, δ_ U).

              Equations
              Instances For
                @[simp]
                theorem CategoryTheory.Cokleisli.Adjunction.toCokleisli_map {C : Type u} [Category.{v, u} C] (U : Comonad C) {X x✝ : C} (f : X x✝) :
                (toCokleisli U).map f = CategoryStruct.comp (U.app X) f

                The left adjoint of the adjunction which induces the comonad (U, ε_ U, δ_ U).

                Equations
                • One or more equations did not get rendered due to their size.
                Instances For
                  @[simp]
                  theorem CategoryTheory.Cokleisli.Adjunction.fromCokleisli_map {C : Type u} [Category.{v, u} C] (U : Comonad C) {X x✝ : Cokleisli U} (f : X x✝) :
                  (fromCokleisli U).map f = CategoryStruct.comp (U.app X) (U.map f)

                  The co-Kleisli adjunction which gives rise to the monad (U, ε_ U, δ_ U).

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

                    The composition of the adjunction gives the original functor.

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