Categorical pullbacks #
This file defines the basic properties of categorical pullbacks.
Given a pair of functors (F : A ⥤ B, G : C ⥤ B)
, we define the category
CategoricalPullback F G
as the category of triples
(a : A, c : C, e : F.obj a ≅ G.obj b)
.
The category CategoricalPullback F G
sits in a canonical CatCommSq
, and we formalize that
this square is a "limit" in the following sense: functors X ⥤ CategoricalPullback F G
are
equivalent to pairs of functors (L : X ⥤ A, R : X ⥤ C)
equipped with a natural isomorphism
L ⋙ F ≅ R ⋙ G
.
We formalize this by introducing a category CatCommSqOver F G X
that encodes
exactly this data, and we prove that the category of functors X ⥤ CategoricalPullback F G
is
equivalent to CatCommSqOver F G X
.
Main declarations #
CategoricalPullback F G
: the type of the categorical pullback.π₁ F G : CategoricalPullback F G
andπ₂ F G : CategoricalPullback F G
: the canonical projections.CategoricalPullback.catCommSq
: the canonicalCatCommSq (π₁ F G) (π₂ F G) F G
which exhibitsCategoricalPullback F G
as the pullback (in the (2,1)-categorical sense) of the cospan ofF
andG
.CategoricalPullback.functorEquiv F G X
: the equivalence of categories between functorsX ⥤ CategoricalPullback F G
andCatCommSqOver F G X
, where the latter is an abbrev forCategoricalPullback (whiskeringRight X A B|>.obj F) (whiskeringRight X C B|>.obj G)
.
References #
- Kerodon: section 1.4.5.2
- Niles Johnson, Donald Yau, 2-Dimensional Categories, example 5.3.9, although we take a slightly different (equivalent) model of the object.
TODOs: #
- 2-functoriality of the construction with respect to "transformation of categorical cospans".
- Full equivalence-invariance of the notion (follows from suitable 2-functoriality).
- Define a
CatPullbackSquare
typeclass extendingCatCommSq
that encodes the fact that a givenCatCommSq
defines an equivalence between the top left corner and the categorical pullback of its legs. - Define a
IsCatPullbackSquare
propclass. - Define the "categorical fiber" of a functor at an object of the target category.
- Pasting calculus for categorical pullback squares.
- Categorical pullback squares attached to Grothendieck constructions of pseudofunctors.
- Stability of (co)fibered categories under categorical pullbacks.
The CategoricalPullback F G
is the category of triples
(a : A, c : C, F a ≅ G c)
.
Morphisms (a, c, e) ⟶ (a', c', e')
are pairs of morphisms
(f₁ : a ⟶ a', f₂ : c ⟶ c')
compatible with the specified
isomorphisms.
- fst : A
the first component element
- snd : C
the second component element
Instances For
A notation for the categorical pullback.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The Hom types for the categorical pullback are given by pairs of maps compatible with the structural isomorphisms.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Naturality square for morphisms in the inverse direction.
Extensionnality principle for morphisms in CategoricalPullback F G
.
CategoricalPullback.π₁ F G
is the first projection CategoricalPullback F G ⥤ A
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
CategoricalPullback.π₂ F G
is the second projection CategoricalPullback F G ⥤ C
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The canonical categorical commutative square in which CategoricalPullback F G
sits.
Equations
- CategoryTheory.Limits.CategoricalPullback.catCommSq F G = { iso := CategoryTheory.NatIso.ofComponents (fun (x : CategoryTheory.Limits.CategoricalPullback F G) => x.iso) ⋯ }
Constructor for isomorphisms in CategoricalPullback F G
.
Equations
Instances For
The data of a categorical commutative square over a cospan F, G
with cone point X
is
that of a functor T : X ⥤ A
, a functor L : X ⥤ C
, and a CatCommSqOver T L F G
.
Note that this is exactly what an object of
((whiskeringRight X A B).obj F) ⊡ ((whiskeringRight X C B).obj G)
is,
so CatCommSqOver F G X
is in fact an abbreviation for
((whiskeringRight X A B).obj F) ⊡ ((whiskeringRight X C B).obj G)
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Interpret a CatCommSqOver F G X X
as a CatCommSq
.
Equations
The "first projection" of a CatCommSqOver as a functor.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The "second projection" of a CatCommSqOver as a functor.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The structure isompophism of a CatCommSqOver
as a natural transformation.
Equations
Instances For
Interpret a functor to the categorical pullback as a CatCommSqOver
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Interpret a CatCommSqOver
as a functor to the categorical pullback.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The universal property of categorical pullbacks, stated as an equivalence
of categories between functors X ⥤ (F ⊡ G)
and categorical commutative squares
over X.
Equations
- One or more equations did not get rendered due to their size.
Instances For
A constructor for natural isomorphisms of functors X ⥤ CategoricalPullback
: to
construct such an isomorphism, it suffices to produce isomorphisms after whiskering with
the projections, and compatible with the canonical 2-commutative square .
Equations
- CategoryTheory.Limits.CategoricalPullback.mkNatIso e₁ e₂ coh = CategoryTheory.NatIso.ofComponents (fun (x : X) => CategoryTheory.Limits.CategoricalPullback.mkIso (e₁.app x) (e₂.app x) ⋯) ⋯
Instances For
To check equality of two natural transformations of functors to a CategoricalPullback
, it
suffices to do so after whiskering with the projections.
Comparing mkNatIso with the corresponding construction one can deduce from
functorEquiv
.