Documentation

Mathlib.CategoryTheory.Bicategory.Adjunction

Adjunctions in bicategories #

For 1-morphisms f : a ⟶ b and g : b ⟶ a in a bicategory, an adjunction between f and g consists of a pair of 2-morphism η : 𝟙 a ⟶ f ≫ g and ε : g ≫ f ⟶ 𝟙 b satisfying the triangle identities. The 2-morphism η is called the unit and ε is called the counit.

Main definitions #

TODO #

structure CategoryTheory.Bicategory.Adjunction {B : Type u} [CategoryTheory.Bicategory B] {a b : B} (f : a b) (g : b a) :

Adjunction between two 1-morphisms.

Instances For

    Adjunction between two 1-morphisms.

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

      Adjunction between identities.

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

        Auxiliary definition for adjunction.comp.

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

          Auxiliary definition for adjunction.comp.

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

            Composition of adjunctions.

            Equations
            • adj₁.comp adj₂ = { unit := adj₁.compUnit adj₂, counit := adj₁.compCounit adj₂, left_triangle := , right_triangle := }
            Instances For
              @[simp]
              theorem CategoryTheory.Bicategory.Adjunction.comp_unit {B : Type u} [CategoryTheory.Bicategory B] {a b c : B} {f₁ : a b} {g₁ : b a} {f₂ : b c} {g₂ : c b} (adj₁ : CategoryTheory.Bicategory.Adjunction f₁ g₁) (adj₂ : CategoryTheory.Bicategory.Adjunction f₂ g₂) :
              (adj₁.comp adj₂).unit = adj₁.compUnit adj₂
              @[simp]
              theorem CategoryTheory.Bicategory.Adjunction.comp_counit {B : Type u} [CategoryTheory.Bicategory B] {a b c : B} {f₁ : a b} {g₁ : b a} {f₂ : b c} {g₂ : c b} (adj₁ : CategoryTheory.Bicategory.Adjunction f₁ g₁) (adj₂ : CategoryTheory.Bicategory.Adjunction f₂ g₂) :
              (adj₁.comp adj₂).counit = adj₁.compCounit adj₂

              Adjoint equivalences between two objects.

              Instances For

                Adjoint equivalences between two objects.

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

                  The identity 1-morphism is an equivalence.

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

                    Construct an adjoint equivalence from 2-isomorphisms by upgrading ε to a counit.

                    Equations
                    Instances For
                      structure CategoryTheory.Bicategory.RightAdjoint {B : Type u} [CategoryTheory.Bicategory B] {a b : B} (left : a b) :
                      Type (max v w)

                      A structure giving a chosen right adjoint of a 1-morphism left.

                      Instances For

                        The existence of a right adjoint of f.

                        Instances
                          structure CategoryTheory.Bicategory.LeftAdjoint {B : Type u} [CategoryTheory.Bicategory B] {a b : B} (right : b a) :
                          Type (max v w)

                          A structure giving a chosen left adjoint of a 1-morphism right.

                          Instances For

                            The existence of a left adjoint of f.

                            Instances