Covers of schemes #
This file provides the basic API for covers of schemes. A cover of a scheme X
with respect to
a morphism property P
is a jointly surjective indexed family of scheme morphisms with
target X
all satisfying P
.
Implementation details #
The definition on the pullback of a cover along a morphism depends on results that are developed later in the import tree. Hence in this file, they have additional assumptions that will be automatically satisfied in later files. The motivation here is that we already know that these assumptions are satisfied for open immersions and hence the cover API for open immersions can be used to deduce these assumptions in the general case.
A coverage K
on Scheme
is called jointly surjective if every covering family in K
is jointly surjective.
Instances
A cover of X
in the coverage K
is a 0
-hypercover for K
.
Equations
Instances For
A choice of an index i
such that x
is in the range of 𝒰.f i
.
Instances For
Given a family of schemes with morphisms to X
satisfying P
that jointly
cover X
, Cover.mkOfCovers
is an associated P
-cover of X
.
Equations
- AlgebraicGeometry.Scheme.Cover.mkOfCovers J obj map covers map_prop = { I₀ := J, X := obj, f := map, mem₀ := ⋯ }
Instances For
An isomorphism X ⟶ Y
is a P
-cover of Y
.
Equations
- AlgebraicGeometry.Scheme.coverOfIsIso f = AlgebraicGeometry.Scheme.Cover.mkOfCovers PUnit.{?u.50 + 1} (fun (x : PUnit.{?u.50 + 1}) => X) (fun (x : PUnit.{?u.50 + 1}) => f) ⋯ ⋯
Instances For
Turn a K
-cover into a Q
-cover by showing that the components satisfy Q
.
Equations
- 𝒰.changeProp h = { toPreZeroHypercover := 𝒰.toPreZeroHypercover, mem₀ := ⋯ }
Instances For
We construct a cover from another, by providing the needed fields and showing that the provided fields are isomorphic with the original cover.
Instances For
The pushforward of a cover along an isomorphism.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Adding map satisfying P
into a cover gives another cover.
Instances For
Alias of CategoryTheory.Precoverage.ZeroHypercover.pullback₁
.
Pullback of a 0
-hypercover along a morphism. The components are pullback f (E.f i)
.
Equations
Instances For
The family of morphisms from the pullback cover to the original cover.
Equations
- 𝒰.pullbackHom f i = CategoryTheory.Limits.pullback.snd f (𝒰.f i)
Instances For
Alias of CategoryTheory.Precoverage.ZeroHypercover.pullback₂
.
Pullback of a 0
-hypercover along a morphism. The components are pullback (E.f i) f
.
Equations
Instances For
An affine cover of X
consists of a jointly surjective family of maps into X
from
spectra of rings.
Note: The map_prop
field is equipped with a default argument by infer_instance
. In general
this causes worse error messages, but in practice P
is mostly defined via class
.
- I₀ : Type v
index set of an affine cover of a scheme
S
- X (j : self.I₀) : CommRingCat
the ring associated to a component of an affine cover
the components map to
S
- idx (x : ↥S) : self.I₀
given a point of
x : S
,idx x
is the index of the component which containsx
the components cover
S
the component maps satisfy
P
Instances For
Alias of AlgebraicGeometry.Scheme.AffineCover.I₀
.
index set of an affine cover of a scheme S
Instances For
Alias of AlgebraicGeometry.Scheme.AffineCover.X
.
the ring associated to a component of an affine cover
Instances For
Alias of AlgebraicGeometry.Scheme.AffineCover.f
.
the components map to S
Instances For
The cover associated to an affine cover.
Equations
Instances For
Any v
-cover 𝒰
induces a u
-cover indexed by the points of X
.
Equations
Instances For
A morphism between covers 𝒰 ⟶ 𝒱
indicates that 𝒰
is a refinement of 𝒱
.
Since covers of schemes are indexed, the definition also involves a map on the
indexing types.
The map on indexing types associated to a morphism of covers.
The morphism between open subsets associated to a morphism of covers.
Instances For
The identity morphism in the category of covers of a scheme.
Equations
- AlgebraicGeometry.Scheme.Cover.Hom.id 𝒰 = { idx := fun (j : 𝒰.I₀) => j, app := fun (x : 𝒰.I₀) => CategoryTheory.CategoryStruct.id (𝒰.X x), app_prop := ⋯, w := ⋯ }
Instances For
The composition of two morphisms in the category of covers of a scheme.
Equations
Instances For
Equations
- One or more equations did not get rendered due to their size.