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 #

Implementation notes #

The computation of 2-morphisms in the proof is done using calc blocks. Typically, the LHS and the RHS in each step of calc are related by simple rewriting up to associators and unitors. So the proof for each step should be of the form rw [...]; coherence. In practice, our proofs look like rw [...]; simp [bicategoricalComp]; coherence. The simp is not strictly necessary, but it speeds up the proof and allow us to avoid increasing the maxHeartbeats. The speedup is probably due to reducing the length of the expression e.g. by absorbing identity maps or applying the pentagon relation. Such a hack may not be necessary if the coherence tactic is improved. One possible way would be to perform such a simplification in the preprocessing of the coherence tactic.

Todo #

structure CategoryTheory.Bicategory.Adjunction {B : Type u} [CategoryTheory.Bicategory B] {a : B} {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
            @[simp]
            theorem CategoryTheory.Bicategory.Adjunction.comp_unit {B : Type u} [CategoryTheory.Bicategory B] {a : B} {b : 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₂) :
            @[simp]
            theorem CategoryTheory.Bicategory.Adjunction.comp_counit {B : Type u} [CategoryTheory.Bicategory B] {a : B} {b : 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₂) :

            Composition of adjunctions.

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

              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} [CategoryTheory.Bicategory B] (a : B) (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
                      Equations

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

                      Equations
                      Instances For