Documentation

Mathlib.CategoryTheory.Bicategory.Kan.Adjunction

Adjunctions as Kan extensions #

We show that adjunctions are realized as Kan extensions or Kan lifts. We also show that a left adjoint commutes with a left Kan extension.

References #

TODO #

At the moment, the results are stated for left Kan extensions and left Kan lifts. We can prove the similar results for right Kan extensions and right Kan lifts.

For an adjuntion f ⊣ u, u is an absolute left Kan extension of the identity along f. The unit of this Kan extension is given by the unit of the adjunction.

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

    A left Kan extension of the identity along f such that f commutes with is a right adjoint to f. The unit of this adjoint is given by the unit of the Kan extension.

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

      For an adjuntion f ⊣ u, u is a left Kan extension of the identity along f. The unit of this Kan extension is given by the unit of the adjunction.

      Equations
      Instances For

        For an adjuntion f ⊣ u, f is an absolute left Kan lift of the identity along u. The unit of this Kan lift is given by the unit of the adjunction.

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

          A left Kan lift of the identity along u such that u commutes with is a left adjoint to u. The unit of this adjoint is given by the unit of the Kan lift.

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

            For an adjuntion f ⊣ u, f is a left Kan lift of the identity along u. The unit of this Kan lift is given by the unit of the adjunction.

            Equations
            Instances For
              def CategoryTheory.Bicategory.LeftExtension.isKanOfWhiskerLeftAdjoint {B : Type u} [CategoryTheory.Bicategory B] {a : B} {b : B} {c : B} {f : a b} {g : a c} {t : CategoryTheory.Bicategory.LeftExtension f g} (H : t.IsKan) {x : B} {h : c x} {u : x c} (adj : CategoryTheory.Bicategory.Adjunction h u) :
              (t.whisker h).IsKan

              A left adjoint commutes with a left Kan extension.

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