Equivalent formulations of the sheaf condition #
We give an equivalent formulation of the sheaf condition.
Given any indexed type ι
, we define overlap ι
,
a category with objects corresponding to
- individual open sets,
single i
, and - intersections of pairs of open sets,
pair i j
, with morphisms frompair i j
to bothsingle i
andsingle j
.
Any open cover U : ι → Opens X
provides a functor diagram U : overlap ι ⥤ (Opens X)ᵒᵖ
.
There is a canonical cone over this functor, cone U
, whose cone point is isup U
,
and in fact this is a limit cone.
A presheaf F : Presheaf C X
is a sheaf precisely if it preserves this limit.
We express this in two equivalent ways, as
isLimit (F.mapCone (cone U))
, orpreservesLimit (diagram U) F
We show that this sheaf condition is equivalent to the OpensLeCover
sheaf condition, and
thereby also equivalent to the default sheaf condition.
An alternative formulation of the sheaf condition
(which we prove equivalent to the usual one below as
isSheaf_iff_isSheafPairwiseIntersections
).
A presheaf is a sheaf if F
sends the cone (Pairwise.cocone U).op
to a limit cone.
(Recall Pairwise.cocone U
has cone point iSup U
, mapping down to the U i
and the U i ⊓ U j
.)
Equations
- One or more equations did not get rendered due to their size.
Instances For
An alternative formulation of the sheaf condition
(which we prove equivalent to the usual one below as
isSheaf_iff_isSheafPreservesLimitPairwiseIntersections
).
A presheaf is a sheaf if F
preserves the limit of Pairwise.diagram U
.
(Recall Pairwise.diagram U
is the diagram consisting of the pairwise intersections
U i ⊓ U j
mapping into the open sets U i
. This diagram has limit iSup U
.)
Equations
- F.IsSheafPreservesLimitPairwiseIntersections = ∀ ⦃ι : Type ?u.33⦄ (U : ι → TopologicalSpace.Opens ↑X), Nonempty (CategoryTheory.Limits.PreservesLimit (CategoryTheory.Pairwise.diagram U).op F)
Instances For
Implementation detail:
the object level of pairwiseToOpensLeCover : Pairwise ι ⥤ OpensLeCover U
Equations
- TopCat.Presheaf.SheafCondition.pairwiseToOpensLeCoverObj U (CategoryTheory.Pairwise.single i) = { obj := U i, property := ⋯ }
- TopCat.Presheaf.SheafCondition.pairwiseToOpensLeCoverObj U (CategoryTheory.Pairwise.pair i j) = { obj := U i ⊓ U j, property := ⋯ }
Instances For
Implementation detail:
the morphism level of pairwiseToOpensLeCover : Pairwise ι ⥤ OpensLeCover U
Equations
- One or more equations did not get rendered due to their size.
- TopCat.Presheaf.SheafCondition.pairwiseToOpensLeCoverMap U (CategoryTheory.Pairwise.Hom.left i j) = CategoryTheory.homOfLE ⋯
- TopCat.Presheaf.SheafCondition.pairwiseToOpensLeCoverMap U (CategoryTheory.Pairwise.Hom.right i j) = CategoryTheory.homOfLE ⋯
Instances For
The category of single and double intersections of the U i
maps into the category
of open sets below some U i
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- ⋯ = ⋯
The diagram consisting of the U i
and U i ⊓ U j
is cofinal in the diagram
of all opens contained in some U i
.
Equations
- ⋯ = ⋯
The diagram in Opens X
indexed by pairwise intersections from U
is isomorphic
(in fact, equal) to the diagram factored through OpensLeCover U
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The cocone Pairwise.cocone U
with cocone point iSup U
over Pairwise.diagram U
is isomorphic
to the cocone opensLeCoverCocone U
(with the same cocone point)
after appropriate whiskering and postcomposition.
Equations
Instances For
The sheaf condition
in terms of a limit diagram over all { V : Opens X // ∃ i, V ≤ U i }
is equivalent to the reformulation
in terms of a limit diagram over U i
and U i ⊓ U j
.
The sheaf condition in terms of an equalizer diagram is equivalent
to the reformulation in terms of a limit diagram over U i
and U i ⊓ U j
.
The sheaf condition in terms of an equalizer diagram is equivalent
to the reformulation in terms of the presheaf preserving the limit of the diagram
consisting of the U i
and U i ⊓ U j
.
For a sheaf F
, F(U ⊔ V)
is the pullback of F(U) ⟶ F(U ⊓ V)
and F(V) ⟶ F(U ⊓ V)
.
This is the pullback cone.
Equations
- F.interUnionPullbackCone U V = CategoryTheory.Limits.PullbackCone.mk (F.val.map (CategoryTheory.homOfLE ⋯).op) (F.val.map (CategoryTheory.homOfLE ⋯).op) ⋯
Instances For
(Implementation).
Every cone over F(U) ⟶ F(U ⊓ V)
and F(V) ⟶ F(U ⊓ V)
factors through F(U ⊔ V)
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
For a sheaf F
, F(U ⊔ V)
is the pullback of F(U) ⟶ F(U ⊓ V)
and F(V) ⟶ F(U ⊓ V)
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
If U, V
are disjoint, then F(U ⊔ V) = F(U) × F(V)
.
Equations
- One or more equations did not get rendered due to their size.