The category of commutative squares #
In this file, we define a bundled version of CommSq
which allows to consider commutative squares as
objects in a category Square C.
The four objects in a commutative square are numbered as follows:
X₁ --> X₂
|      |
v      v
X₃ --> X₄
We define the flip functor, and two equivalences with
the category Arrow (Arrow C), depending on whether
we consider a commutative square as a horizontal
morphism between two vertical maps (arrowArrowEquivalence)
or a vertical morphism between two horizontal
maps (arrowArrowEquivalence').
The category of commutative squares in a category.
- X₁ : Cthe top-left object 
- X₂ : Cthe top-right object 
- X₃ : Cthe bottom-left object 
- X₄ : Cthe bottom-right object 
- the top morphism 
- the left morphism 
- the right morphism 
- the bottom morphism 
Instances For
A morphism between two commutative squares consists of 4 morphisms which extend these two squares into a commuting cube.
- the top-left morphism 
- the top-right morphism 
- the bottom-left morphism 
- the bottom-right morphism 
Instances For
The identity of a commutative square.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The composition of morphisms of squares.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Constructor for isomorphisms in Square c
Equations
- One or more equations did not get rendered due to their size.
Instances For
Flipping a square by switching the top-right and the bottom-left objects.
Equations
Instances For
The functor which flips commutative squares.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Flipping commutative squares is an auto-equivalence.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The functor Square C ⥤ Arrow (Arrow C) which sends a
commutative square sq to the obvious arrow from the left morphism of sq
to the right morphism of sq.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The functor Arrow (Arrow C) ⥤ Square C which sends
a morphism Arrow.mk f ⟶ Arrow.mk g to the commutative square
with f on the left side and g on the right side.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The equivalence Square C ≌ Arrow (Arrow C) which sends a
commutative square sq to the obvious arrow from the left morphism of sq
to the right morphism of sq.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The functor Square C ⥤ Arrow (Arrow C) which sends a
commutative square sq to the obvious arrow from the top morphism of sq
to the bottom morphism of sq.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The functor Arrow (Arrow C) ⥤ Square C which sends
a morphism Arrow.mk f ⟶ Arrow.mk g to the commutative square
with f on the top side and g on the bottom side.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The equivalence Square C ≌ Arrow (Arrow C) which sends a
commutative square sq to the obvious arrow from the top morphism of sq
to the bottom morphism of sq.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The top-left evaluation Square C ⥤ C.
Equations
- CategoryTheory.Square.evaluation₁ = { obj := fun (sq : CategoryTheory.Square C) => sq.X₁, map := fun {X Y : CategoryTheory.Square C} (φ : X ⟶ Y) => φ.τ₁, map_id := ⋯, map_comp := ⋯ }
Instances For
The top-right evaluation Square C ⥤ C.
Equations
- CategoryTheory.Square.evaluation₂ = { obj := fun (sq : CategoryTheory.Square C) => sq.X₂, map := fun {X Y : CategoryTheory.Square C} (φ : X ⟶ Y) => φ.τ₂, map_id := ⋯, map_comp := ⋯ }
Instances For
The bottom-left evaluation Square C ⥤ C.
Equations
- CategoryTheory.Square.evaluation₃ = { obj := fun (sq : CategoryTheory.Square C) => sq.X₃, map := fun {X Y : CategoryTheory.Square C} (φ : X ⟶ Y) => φ.τ₃, map_id := ⋯, map_comp := ⋯ }
Instances For
The bottom-right evaluation Square C ⥤ C.
Equations
- CategoryTheory.Square.evaluation₄ = { obj := fun (sq : CategoryTheory.Square C) => sq.X₄, map := fun {X Y : CategoryTheory.Square C} (φ : X ⟶ Y) => φ.τ₄, map_id := ⋯, map_comp := ⋯ }
Instances For
The functor (Square C)ᵒᵖ ⥤ Square Cᵒᵖ.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The functor (Square Cᵒᵖ)ᵒᵖ ⥤ Square Cᵒᵖ.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The equivalence (Square C)ᵒᵖ ≌ Square Cᵒᵖ.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The image of a commutative square by a functor.
Equations
Instances For
The functor Square C ⥤ Square D induced by a functor C ⥤ D.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The natural transformation F.mapSquare ⟶ G.mapSquare induces
by a natural transformation F ⟶ G.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The functor (C ⥤ D) ⥤ Square C ⥤ Square D.
Equations
- One or more equations did not get rendered due to their size.