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 #

@[reducible, inline]

The 2-morphism defined by the following pasting diagram:

a ------ ▸ a
  \    η      ◥   \
  f \   g  /       \ f
       ◢  /     ε      ◢
        b ------ ▸ b
Equations
Instances For
    @[reducible, inline]

    The 2-morphism defined by the following pasting diagram:

            a ------ ▸ a
           ◥  \     η      ◥
      g /      \ f     / g
      /    ε      ◢   /
    b ------ ▸ b
    
    Equations
    Instances For
      structure CategoryTheory.Bicategory.Adjunction {B : Type u} [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
            def CategoryTheory.Bicategory.Adjunction.compUnit {B : Type u} [Bicategory B] {a b c : B} {f₁ : a b} {g₁ : b a} {f₂ : b c} {g₂ : c b} (adj₁ : Adjunction f₁ g₁) (adj₂ : Adjunction f₂ g₂) :

            Auxiliary definition for adjunction.comp.

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              def CategoryTheory.Bicategory.Adjunction.compCounit {B : Type u} [Bicategory B] {a b c : B} {f₁ : a b} {g₁ : b a} {f₂ : b c} {g₂ : c b} (adj₁ : Adjunction f₁ g₁) (adj₂ : Adjunction f₂ g₂) :

              Auxiliary definition for adjunction.comp.

              Equations
              • One or more equations did not get rendered due to their size.
              Instances For
                theorem CategoryTheory.Bicategory.Adjunction.comp_left_triangle_aux {B : Type u} [Bicategory B] {a b c : B} {f₁ : a b} {g₁ : b a} {f₂ : b c} {g₂ : c b} (adj₁ : Adjunction f₁ g₁) (adj₂ : Adjunction f₂ g₂) :
                leftZigzag (adj₁.compUnit adj₂) (adj₁.compCounit adj₂) = CategoryStruct.comp (leftUnitor (CategoryStruct.comp f₁ f₂)).hom (rightUnitor (CategoryStruct.comp f₁ f₂)).inv
                theorem CategoryTheory.Bicategory.Adjunction.comp_right_triangle_aux {B : Type u} [Bicategory B] {a b c : B} {f₁ : a b} {g₁ : b a} {f₂ : b c} {g₂ : c b} (adj₁ : Adjunction f₁ g₁) (adj₂ : Adjunction f₂ g₂) :
                rightZigzag (adj₁.compUnit adj₂) (adj₁.compCounit adj₂) = CategoryStruct.comp (rightUnitor (CategoryStruct.comp g₂ g₁)).hom (leftUnitor (CategoryStruct.comp g₂ g₁)).inv
                def CategoryTheory.Bicategory.Adjunction.comp {B : Type u} [Bicategory B] {a b c : B} {f₁ : a b} {g₁ : b a} {f₂ : b c} {g₂ : c b} (adj₁ : Adjunction f₁ g₁) (adj₂ : Adjunction f₂ g₂) :

                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} [Bicategory B] {a b c : B} {f₁ : a b} {g₁ : b a} {f₂ : b c} {g₂ : c b} (adj₁ : Adjunction f₁ g₁) (adj₂ : Adjunction f₂ g₂) :
                  (adj₁.comp adj₂).unit = adj₁.compUnit adj₂
                  @[simp]
                  theorem CategoryTheory.Bicategory.Adjunction.comp_counit {B : Type u} [Bicategory B] {a b c : B} {f₁ : a b} {g₁ : b a} {f₂ : b c} {g₂ : c b} (adj₁ : Adjunction f₁ g₁) (adj₂ : Adjunction f₂ g₂) :
                  (adj₁.comp adj₂).counit = adj₁.compCounit adj₂
                  @[simp]
                  theorem CategoryTheory.Bicategory.leftZigzagIso_hom {B : Type u} [Bicategory B] {a b : B} {f : a b} {g : b a} (η : CategoryStruct.id a CategoryStruct.comp f g) (ε : CategoryStruct.comp g f CategoryStruct.id b) :
                  (leftZigzagIso η ε).hom = leftZigzag η.hom ε.hom
                  @[simp]
                  theorem CategoryTheory.Bicategory.rightZigzagIso_hom {B : Type u} [Bicategory B] {a b : B} {f : a b} {g : b a} (η : CategoryStruct.id a CategoryStruct.comp f g) (ε : CategoryStruct.comp g f CategoryStruct.id b) :
                  (rightZigzagIso η ε).hom = rightZigzag η.hom ε.hom
                  @[simp]
                  theorem CategoryTheory.Bicategory.leftZigzagIso_inv {B : Type u} [Bicategory B] {a b : B} {f : a b} {g : b a} (η : CategoryStruct.id a CategoryStruct.comp f g) (ε : CategoryStruct.comp g f CategoryStruct.id b) :
                  (leftZigzagIso η ε).inv = rightZigzag ε.inv η.inv
                  @[simp]
                  theorem CategoryTheory.Bicategory.rightZigzagIso_inv {B : Type u} [Bicategory B] {a b : B} {f : a b} {g : b a} (η : CategoryStruct.id a CategoryStruct.comp f g) (ε : CategoryStruct.comp g f CategoryStruct.id b) :
                  (rightZigzagIso η ε).inv = leftZigzag ε.inv η.inv
                  @[simp]
                  theorem CategoryTheory.Bicategory.leftZigzagIso_symm {B : Type u} [Bicategory B] {a b : B} {f : a b} {g : b a} (η : CategoryStruct.id a CategoryStruct.comp f g) (ε : CategoryStruct.comp g f CategoryStruct.id b) :
                  (leftZigzagIso η ε).symm = rightZigzagIso ε.symm η.symm
                  @[simp]
                  theorem CategoryTheory.Bicategory.rightZigzagIso_symm {B : Type u} [Bicategory B] {a b : B} {f : a b} {g : b a} (η : CategoryStruct.id a CategoryStruct.comp f g) (ε : CategoryStruct.comp g f CategoryStruct.id b) :
                  (rightZigzagIso η ε).symm = leftZigzagIso ε.symm η.symm

                  An auxiliary definition for mkOfAdjointifyCounit.

                  Equations
                  • One or more equations did not get rendered due to their size.
                  Instances For
                    structure CategoryTheory.Bicategory.Equivalence {B : Type u} [Bicategory B] (a b : B) :
                    Type (max v w)

                    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
                          theorem CategoryTheory.Bicategory.Equivalence.left_triangle_hom {B : Type u} [Bicategory B] {a b : B} (e : Equivalence a b) :
                          leftZigzag e.unit.hom e.counit.hom = CategoryStruct.comp (leftUnitor e.hom).hom (rightUnitor e.hom).inv
                          theorem CategoryTheory.Bicategory.Equivalence.right_triangle {B : Type u} [Bicategory B] {a b : B} (e : Equivalence a b) :
                          rightZigzagIso e.unit e.counit = rightUnitor e.inv ≪≫ (leftUnitor e.inv).symm
                          theorem CategoryTheory.Bicategory.Equivalence.right_triangle_hom {B : Type u} [Bicategory B] {a b : B} (e : Equivalence a b) :
                          rightZigzag e.unit.hom e.counit.hom = CategoryStruct.comp (rightUnitor e.inv).hom (leftUnitor e.inv).inv

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

                          Equations
                          Instances For
                            structure CategoryTheory.Bicategory.RightAdjoint {B : Type u} [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
                              class CategoryTheory.Bicategory.IsLeftAdjoint {B : Type u} [Bicategory B] {a b : B} (left : a b) :

                              The existence of a right adjoint of f.

                              Instances
                                theorem CategoryTheory.Bicategory.IsLeftAdjoint.mk {B : Type u} [Bicategory B] {a b : B} {f : a b} {g : b a} (adj : Adjunction f g) :

                                Use the axiom of choice to extract a right adjoint from an IsLeftAdjoint instance.

                                Equations
                                Instances For
                                  def CategoryTheory.Bicategory.rightAdjoint {B : Type u} [Bicategory B] {a b : B} (f : a b) [IsLeftAdjoint f] :
                                  b a

                                  The right adjoint of a 1-morphism.

                                  Equations
                                  Instances For
                                    structure CategoryTheory.Bicategory.LeftAdjoint {B : Type u} [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
                                      class CategoryTheory.Bicategory.IsRightAdjoint {B : Type u} [Bicategory B] {a b : B} (right : b a) :

                                      The existence of a left adjoint of f.

                                      Instances
                                        theorem CategoryTheory.Bicategory.IsRightAdjoint.mk {B : Type u} [Bicategory B] {a b : B} {f : a b} {g : b a} (adj : Adjunction f g) :

                                        Use the axiom of choice to extract a left adjoint from an IsRightAdjoint instance.

                                        Equations
                                        Instances For
                                          def CategoryTheory.Bicategory.leftAdjoint {B : Type u} [Bicategory B] {a b : B} (f : b a) [IsRightAdjoint f] :
                                          a b

                                          The left adjoint of a 1-morphism.

                                          Equations
                                          Instances For