Mates in bicategories #
This file establishes the bijection between the 2-cells
l₁ r₁
c --→ d c ←-- d
g ↓ ↗ ↓ h g ↓ ↘ ↓ h
e --→ f e ←-- f
l₂ r₂
where l₁ ⊣ r₁
and l₂ ⊣ r₂
. The corresponding natural transformations are called mates.
For the bicategory Cat
, the definitions in this file are provided in
Mathlib/CategoryTheory/Adjunction/Mates.lean
, where you can find more detailed documentation
about mates.
Remarks #
To be precise, the definitions in Mathlib/CategoryTheory/Adjunction/Mates.lean
are universe
polymorphic, so they are not simple specializations of the definitions in this file.
Suppose we have a square of 1-morphisms (where the top and bottom are adjunctions l₁ ⊣ r₁
and l₂ ⊣ r₂
respectively).
c ↔ d
g ↓ ↓ h
e ↔ f
Then we have a bijection between natural transformations g ≫ l₂ ⟶ l₁ ≫ h
and
r₁ ≫ g ⟶ h ≫ r₂
. This can be seen as a bijection of the 2-cells:
l₁ r₁
c --→ d c ←-- d
g ↓ ↗ ↓ h g ↓ ↘ ↓ h
e --→ f e ←-- f
L₂ R₂
Note that if one of the transformations is an iso, it does not imply the other is an iso.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Squares between left adjoints can be composed "vertically" by pasting.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Squares between right adjoints can be composed "vertically" by pasting.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The mates equivalence commutes with vertical composition.
Squares between left adjoints can be composed "horizontally" by pasting.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Squares between right adjoints can be composed "horizontally" by pasting.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The mates equivalence commutes with horizontal composition of squares.
Squares of squares between left adjoints can be composed by iterating vertical and horizontal composition.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Horizontal and vertical composition of squares commutes.
Squares of squares between right adjoints can be composed by iterating vertical and horizontal composition.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Horizontal and vertical composition of squares commutes.
The mates equivalence commutes with composition of squares of squares. These results form the basis for an isomorphism of double categories to be proven later.
Given two adjunctions l₁ ⊣ r₁
and l₂ ⊣ r₂
both between objects c
, d
, there is a
bijection between 2-morphisms l₂ ⟶ l₁
and 2-morphisms r₁ ⟶ r₂
. This is
defined as a special case of mateEquiv
, where the two "vertical" 1-morphisms are identities.
Corresponding 2-morphisms are called conjugateEquiv
.
Furthermore, this bijection preserves (and reflects) isomorphisms, i.e. a 2-morphism is an iso iff its image under the bijection is an iso.
Equations
- One or more equations did not get rendered due to their size.
Instances For
If α
is an isomorphism between left adjoints, then its conjugate transformation is an
isomorphism. The converse is given in conjugateEquiv_of_iso
.
If α
is an isomorphism between right adjoints, then its conjugate transformation is an
isomorphism. The converse is given in conjugateEquiv_symm_of_iso
.
If α
is a natural transformation between left adjoints whose conjugate natural transformation
is an isomorphism, then α
is an isomorphism. The converse is given in Conjugate_iso
.
If α
is a natural transformation between right adjoints whose conjugate natural transformation is
an isomorphism, then α
is an isomorphism. The converse is given in conjugateEquiv_symm_iso
.
Thus conjugation defines an equivalence between natural isomorphisms.
Equations
- One or more equations did not get rendered due to their size.
Instances For
When all four morphisms in a square are left adjoints, the mates operation can be iterated: l₁ r₁ r₁ c --→ d c ←-- d c ←-- d f₁ ↓ ↗ ↓ f₂ f₁ ↓ ↘ ↓ f₂ u₁ ↑ ↙ ↑ u₂ a --→ b a ←-- b a ←-- b l₂ r₂ r₂ In this case the iterated mate equals the conjugate of the original 2-morphism and is thus an isomorphism if and only if the original 2-morphism is. This explains why some Beck-Chevalley 2-morphisms are isomorphisms.
Composition of a squares between left adjoints with a conjugate square.
Equations
Instances For
Composition of a squares between right adjoints with a conjugate square.
Equations
Instances For
The mates equivalence commutes with this composition, essentially by mateEquiv_vcomp
.
Composition of a conjugate square with a squares between left adjoints.
Equations
Instances For
Composition of a conjugate square with a squares between right adjoints.
Equations
Instances For
The mates equivalence commutes with this composition, essentially by mateEquiv_vcomp
.