Checking the sheaf condition on the underlying presheaf of types. #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
If G : C ⥤ D
is a functor which reflects isomorphisms and preserves limits
(we assume all limits exist in both C
and D
),
then checking the sheaf condition for a presheaf F : presheaf C X
is equivalent to checking the sheaf condition for F ⋙ G
.
The important special case is when
C
is a concrete category with a forgetful functor
that preserves limits and reflects isomorphisms.
Then to check the sheaf condition it suffices
to check it on the underlying sheaf of types.
References #
When G
preserves limits, the sheaf condition diagram for F
composed with G
is
naturally isomorphic to the sheaf condition diagram for F ⋙ G
.
Equations
- Top.presheaf.sheaf_condition.diagram_comp_preserves_limits G F U = category_theory.nat_iso.of_components (λ (X_1 : category_theory.limits.walking_parallel_pair), X_1.cases_on (category_theory.limits.preserves_product.iso G (λ (i : ι), F.obj (opposite.op (U i)))) (category_theory.limits.preserves_product.iso G (λ (p : ι × ι), F.obj (opposite.op (U p.fst ⊓ U p.snd))))) _
When G
preserves limits, the image under G
of the sheaf condition fork for F
is the sheaf condition fork for F ⋙ G
,
postcomposed with the inverse of the natural isomorphism diagram_comp_preserves_limits
.
If G : C ⥤ D
is a functor which reflects isomorphisms and preserves limits
(we assume all limits exist in both C
and D
),
then checking the sheaf condition for a presheaf F : presheaf C X
is equivalent to checking the sheaf condition for F ⋙ G
.
The important special case is when
C
is a concrete category with a forgetful functor
that preserves limits and reflects isomorphisms.
Then to check the sheaf condition it suffices to check it on the underlying sheaf of types.
Another useful example is the forgetful functor TopCommRing ⥤ Top
.
See https://stacks.math.columbia.edu/tag/0073. In fact we prove a stronger version with arbitrary complete target category.
As an example, we now have everything we need to check the sheaf condition for a presheaf of commutative rings, merely by checking the sheaf condition for the underlying sheaf of types.