Locally directed covers #
A locally directed P-cover of a scheme X is a cover 𝒰 with an ordering
on the indices and compatible transition maps 𝒰ᵢ ⟶ 𝒰ⱼ for i ≤ j such that
every x : 𝒰ᵢ ×[X] 𝒰ⱼ comes from some 𝒰ₖ for a k ≤ i and k ≤ j.
Gluing along directed covers is easier, because the intersections 𝒰ᵢ ×[X] 𝒰ⱼ can
be covered by a subcover of 𝒰. In particular, if 𝒰 is a Zariski cover,
X naturally is the colimit of the 𝒰ᵢ.
Many natural covers are naturally directed, most importantly the cover of all affine opens of a scheme.
A directed P-cover of a scheme X is a cover 𝒰 with an ordering
on the indices and compatible transition maps 𝒰ᵢ ⟶ 𝒰ⱼ for i ≤ j such that
every x : 𝒰ᵢ ×[X] 𝒰ⱼ comes from some 𝒰ₖ for a k ≤ i and k ≤ j.
The transition map
𝒰ᵢ ⟶ 𝒰ⱼfori ≤ j.- trans_id (i : 𝒰.I₀) : trans (CategoryTheory.CategoryStruct.id i) = CategoryTheory.CategoryStruct.id (𝒰.X i)
- trans_comp {i j k : 𝒰.I₀} (hij : i ⟶ j) (hjk : j ⟶ k) : trans (CategoryTheory.CategoryStruct.comp hij hjk) = CategoryTheory.CategoryStruct.comp (trans hij) (trans hjk)
- directed {i j : 𝒰.I₀} (x : ↥(CategoryTheory.Limits.pullback (𝒰.f i) (𝒰.f j))) : ∃ (k : 𝒰.I₀) (hki : k ⟶ i) (hkj : k ⟶ j) (y : ↥(𝒰.X k)), (CategoryTheory.ConcreteCategory.hom (CategoryTheory.Limits.pullback.lift (trans hki) (trans hkj) ⋯).base) y = x
Instances
The transition maps of a directed cover.
Equations
Instances For
If 𝒰 is a directed cover of X, this is the cover of 𝒰ᵢ ×[X] 𝒰ⱼ by {𝒰ₖ} where
k ≤ i and k ≤ j.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The canonical diagram induced by a locally directed cover.
Equations
Instances For
The canonical cocone with point X on the functor induced by the locally directed cover 𝒰.
If 𝒰 is an open cover, this is colimiting (see OpenCover.isColimitCoconeOfLocallyDirected).
Instances For
Equations
Equations
- One or more equations did not get rendered due to their size.
If 𝒰 is a directed open cover of X, to glue morphisms {gᵢ : 𝒰ᵢ ⟶ Y} it suffices
to check compatibility with the transition maps.
See OpenCover.isColimitCoconeOfLocallyDirected for this result stated in the language of
colimits.
Equations
Instances For
If 𝒰 is an open cover of X that is locally directed, X is
the colimit of the components of 𝒰.
Equations
- One or more equations did not get rendered due to their size.
Instances For
If 𝒰 is a directed open cover of X, to glue morphisms {gᵢ : 𝒰ᵢ ⟶ Y} over S it suffices
to check compatibility with the transition maps.
Equations
Instances For
If 𝒰 is an open cover such that the images of the components form a basis of the topology
of X, 𝒰 is directed by the ordering of subset inclusion of the images.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The directed affine open cover of X given by all affine opens.
Equations
- X.directedAffineCover = { I₀ := ↑X.affineOpens, X := fun (U : ↑X.affineOpens) => ↑↑U, f := fun (U : ↑X.affineOpens) => (↑U).ι, mem₀ := ⋯ }