The Grothendieck construction #
Given a functor F : C ⥤ Cat
, the objects of Grothendieck F
consist of dependent pairs (b, f)
, where b : C
and f : F.obj c
,
and a morphism (b, f) ⟶ (b', f')
is a pair β : b ⟶ b'
in C
, and
φ : (F.map β).obj f ⟶ f'
Grothendieck.functor
makes the Grothendieck construction into a functor from the functor category
C ⥤ Cat
to the over category Over C
in the category of categories.
Categories such as PresheafedSpace
are in fact examples of this construction,
and it may be interesting to try to generalize some of the development there.
Implementation notes #
Really we should treat Cat
as a 2-category, and allow F
to be a 2-functor.
There is also a closely related construction starting with G : Cᵒᵖ ⥤ Cat
,
where morphisms consists again of β : b ⟶ b'
and φ : f ⟶ (F.map (op β)).obj f'
.
Notable constructions #
Grothendieck F
is the Grothendieck construction.- Elements of
Grothendieck F
whose base isc : C
can be transported alongf : c ⟶ d
usingtransport
. - A natural transformation
α : F ⟶ G
inducesmap α : Grothendieck F ⥤ Grothendieck G
. - The Grothendieck construction and
map
together form a functor (functor
) from the functor categoryE ⥤ Cat
to the over categoryOver E
. - A functor
G : D ⥤ C
inducespre F G : Grothendieck (G ⋙ F) ⥤ Grothendieck F
.
References #
See also CategoryTheory.Functor.Elements
for the category of elements of functor F : C ⥤ Type
.
- https://stacks.math.columbia.edu/tag/02XV
- https://ncatlab.org/nlab/show/Grothendieck+construction
The Grothendieck construction (often written as ∫ F
in mathematics) for a functor F : C ⥤ Cat
gives a category whose
- objects
X
consist ofX.base : C
andX.fiber : F.obj base
- morphisms
f : X ⟶ Y
consist ofbase : X.base ⟶ Y.base
andf.fiber : (F.map base).obj X.fiber ⟶ Y.fiber
- base : C
The underlying object in
C
The object in the fiber of the base object.
Instances For
A morphism in the Grothendieck category F : C ⥤ Cat
consists of
base : X.base ⟶ Y.base
and f.fiber : (F.map base).obj X.fiber ⟶ Y.fiber
.
The morphism between base objects.
The morphism from the pushforward to the source fiber object to the target fiber object.
Instances For
The identity morphism in the Grothendieck category.
Equations
- X.id = { base := CategoryTheory.CategoryStruct.id X.base, fiber := CategoryTheory.eqToHom ⋯ }
Instances For
Equations
- X.instInhabitedHom = { default := X.id }
Composition of morphisms in the Grothendieck category.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
If F : C ⥤ Cat
is a functor and t : c ⟶ d
is a morphism in C
, then transport
maps each
c
-based element of Grothendieck F
to a d
-based element.
Instances For
If F : C ⥤ Cat
is a functor and t : c ⟶ d
is a morphism in C
, then transport
maps each
c
-based element x
of Grothendieck F
to a d
-based element x.transport t
.
toTransport
is the morphism x ⟶ x.transport t
induced by t
and the identity on fibers.
Equations
- x.toTransport t = { base := t, fiber := CategoryTheory.CategoryStruct.id ((F.map t).obj x.fiber) }
Instances For
Construct an isomorphism in a Grothendieck construction from isomorphisms in its base and fiber.
Equations
- One or more equations did not get rendered due to their size.
Instances For
If F : C ⥤ Cat
and x : Grothendieck F
, then every C
-isomorphism α : x.base ≅ c
induces
an isomorphism between x
and its transport along α
Equations
- x.transportIso α = (CategoryTheory.Grothendieck.isoMk α (CategoryTheory.Iso.refl ((F.map α.hom).obj x.fiber))).symm
Instances For
The forgetful functor from Grothendieck F
to the source category.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The Grothendieck construction is functorial: a natural transformation α : F ⟶ G
induces
a functor Grothendieck.map : Grothendieck F ⥤ Grothendieck G
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The functor Grothendieck.map α : Grothendieck F ⥤ Grothendieck G
lies over C
.
Making the equality of functors into an isomorphism. Note: we should avoid equality of functors
if possible, and we should prefer mapIdIso
to map_id_eq
whenever we can.
Instances For
Making the equality of functors into an isomorphism. Note: we should avoid equality of functors
if possible, and we should prefer map_comp_iso
to map_comp_eq
whenever we can.
Equations
Instances For
The inverse functor to build the equivalence compAsSmallFunctorEquivalence
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The functor to build the equivalence compAsSmallFunctorEquivalence
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Taking the Grothendieck construction on F ⋙ asSmallFunctor
, where
asSmallFunctor : Cat ⥤ Cat
is the functor which turns each category into a small category of a
(potentiall) larger universe, is equivalent to the Grothendieck construction on F
itself.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Mapping a Grothendieck construction along the whiskering of any natural transformation
α : F ⟶ G
with the functor asSmallFunctor : Cat ⥤ Cat
is naturally isomorphic to conjugating
map α
with the equivalence between Grothendieck (F ⋙ asSmallFunctor)
and Grothendieck F
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Auxiliary definition for grothendieckTypeToCat
, to speed up elaboration.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Auxiliary definition for grothendieckTypeToCat
, to speed up elaboration.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The Grothendieck construction applied to a functor to Type
(thought of as a functor to Cat
by realising a type as a discrete category)
is the same as the 'category of elements' construction.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Applying a functor G : D ⥤ C
to the base of the Grothendieck construction induces a functor
Grothendieck (G ⋙ F) ⥤ Grothendieck F
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
An natural isomorphism between functors G ≅ H
induces a natural isomorphism between the canonical
morphism pre F G
and pre F H
, up to composition with
Grothendieck (G ⋙ F) ⥤ Grothendieck (H ⋙ F)
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Given an equivalence of categories G
, preInv _ G
is the (weak) inverse of the pre _ G.functor
.
Equations
Instances For
Let G
be an equivalence of categories. The functor induced via pre
by G.functor ⋙ G.inverse
is naturally isomorphic to the functor induced via map
by a whiskered version of G
's inverse
unit.
Equations
Instances For
Given a functor F : C ⥤ Cat
and an equivalence of categories G : D ≌ C
, the functor
pre F G.functor
is an equivalence between Grothendieck (G.functor ⋙ F)
and Grothendieck F
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Let F, F' : C ⥤ Cat
be functor, G : D ≌ C
an equivalence and α : F ⟶ F'
a natural
transformation.
Left-whiskering α
by G
and then taking the Grothendieck construction is, up to isomorphism,
the same as taking the Grothendieck construction of α
and using the equivalences pre F G
and pre F' G
to match the expected type:
Grothendieck (G.functor ⋙ F) ≌ Grothendieck F ⥤ Grothendieck F' ≌ Grothendieck (G.functor ⋙ F')
Equations
- One or more equations did not get rendered due to their size.
Instances For
The inclusion of a fiber F.obj c
of a functor F : C ⥤ Cat
into its Grothendieck
construction.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Every morphism f : X ⟶ Y
in the base category induces a natural transformation from the fiber
inclusion ι F X
to the composition F.map f ⋙ ι F Y
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Construct a functor from Grothendieck F
to another category E
by providing a family of
functors on the fibers of Grothendieck F
, a family of natural transformations on morphisms in the
base of Grothendieck F
and coherence data for this family of natural transformations.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Grothendieck.ι F c
composed with Grothendieck.functorFrom
is isomorphic a functor on a fiber
on F
supplied as the first argument to Grothendieck.functorFrom
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The fiber inclusion ι F c
composed with map α
is isomorphic to α.app c ⋙ ι F' c
.
Equations
- One or more equations did not get rendered due to their size.