Comma categories #
A comma category is a construction in category theory, which builds a category out of two functors
with a common codomain. Specifically, for functors L : A ⥤ T
and R : B ⥤ T
, an object in
Comma L R
is a morphism hom : L.obj left ⟶ R.obj right
for some objects left : A
and
right : B
, and a morphism in Comma L R
between hom : L.obj left ⟶ R.obj right
and
hom' : L.obj left' ⟶ R.obj right'
is a commutative square
L.obj left ⟶ L.obj left'
| |
hom | | hom'
↓ ↓
R.obj right ⟶ R.obj right',
where the top and bottom morphism come from morphisms left ⟶ left'
and right ⟶ right'
,
respectively.
Main definitions #
Comma L R
: the comma category of the functorsL
andR
.Over X
: the over category of the objectX
(developed inOver.lean
).Under X
: the under category of the objectX
(also developed inOver.lean
).Arrow T
: the arrow category of the categoryT
(developed inArrow.lean
).
References #
Tags #
comma, slice, coslice, over, under, arrow
- left : A
- right : B
- hom : L.obj s.left ⟶ R.obj s.right
The objects of the comma category are triples of an object left : A
, an object
right : B
and a morphism hom : L.obj left ⟶ R.obj right
.
Instances For
- left : X.left ⟶ Y.left
- right : X.right ⟶ Y.right
- w : CategoryTheory.CategoryStruct.comp (L.map s.left) Y.hom = CategoryTheory.CategoryStruct.comp X.hom (R.map s.right)
A morphism between two objects in the comma category is a commutative square connecting the
morphisms coming from the two objects using morphisms in the image of the functors L
and R
.
Instances For
The functor sending an object X
in the comma category to X.left
.
Instances For
The functor sending an object X
in the comma category to X.right
.
Instances For
We can interpret the commutative square constituting a morphism in the comma category as a
natural transformation between the functors fst ⋙ L
and snd ⋙ R
from the comma category
to T
, where the components are given by the morphism that constitutes an object of the comma
category.
Instances For
Construct an isomorphism in the comma category given isomorphisms of the objects whose forward directions give a commutative square.
Instances For
A natural transformation L₁ ⟶ L₂
induces a functor Comma L₂ R ⥤ Comma L₁ R
.
Instances For
The functor Comma L R ⥤ Comma L R
induced by the identity natural transformation on L
is
naturally isomorphic to the identity functor.
Instances For
The functor Comma L₁ R ⥤ Comma L₃ R
induced by the composition of two natural transformations
l : L₁ ⟶ L₂
and l' : L₂ ⟶ L₃
is naturally isomorphic to the composition of the two functors
induced by these natural transformations.
Instances For
Two equal natural transformations L₁ ⟶ L₂
yield naturally isomorphic functors
Comma L₁ R ⥤ Comma L₂ R
.
Instances For
A natural isomorphism L₁ ≅ L₂
induces an equivalence of categories
Comma L₁ R ≌ Comma L₂ R
.
Instances For
A natural transformation R₁ ⟶ R₂
induces a functor Comma L R₁ ⥤ Comma L R₂
.
Instances For
The functor Comma L R ⥤ Comma L R
induced by the identity natural transformation on R
is
naturally isomorphic to the identity functor.
Instances For
The functor Comma L R₁ ⥤ Comma L R₃
induced by the composition of the natural transformations
r : R₁ ⟶ R₂
and r' : R₂ ⟶ R₃
is naturally isomorphic to the composition of the functors
induced by these natural transformations.
Instances For
Two equal natural transformations R₁ ⟶ R₂
yield naturally isomorphic functors
Comma L R₁ ⥤ Comma L R₂
.
Instances For
A natural isomorphism R₁ ≅ R₂
induces an equivalence of categories
Comma L R₁ ≌ Comma L R₂
.
Instances For
The functor (F ⋙ L, R) ⥤ (L, R)
Instances For
If F
is an equivalence, then so is preLeft F L R
.
Instances For
The functor (F ⋙ L, R) ⥤ (L, R)
Instances For
If F
is an equivalence, then so is preRight L F R
.
Instances For
The functor (L, R) ⥤ (L ⋙ F, R ⋙ F)