Small sites #
In this file we define the small sites associated to morphism properties and give generating pretopologies.
Main definitions #
AlgebraicGeometry.Scheme.overGrothendieckTopology
: the Grothendieck topology onOver S
obtained by localizing the topology onScheme
induced byP
atS
.AlgebraicGeometry.Scheme.overPretopology
: the pretopology onOver S
defined byP
-coverings ofS
-schemes. The induced topology agrees withAlgebraicGeometry.Scheme.overGrothendieckTopology
.AlgebraicGeometry.Scheme.smallGrothendieckTopology
: the by the inclusionP.Over ⊤ S ⥤ Over S
induced topology onP.Over ⊤ S
.AlgebraicGeometry.Scheme.smallPretopology
: the pretopology onP.Over ⊤ S
defined byP
-coverings ofS
-schemes withP
. The induced topology agrees withAlgebraicGeometry.Scheme.smallGrothendieckTopology
.
The presieve defined by a P
-cover of S
-schemes.
Equations
- 𝒰.toPresieveOver = CategoryTheory.Presieve.ofArrows (fun (i : 𝒰.J) => (𝒰.obj i).asOver S) fun (i : 𝒰.J) => AlgebraicGeometry.Scheme.Hom.asOver (𝒰.map i) S
Instances For
The presieve defined by a P
-cover of S
-schemes with Q
.
Equations
- 𝒰.toPresieveOverProp h = CategoryTheory.Presieve.ofArrows (fun (i : 𝒰.J) => (𝒰.obj i).asOverProp S ⋯) fun (i : 𝒰.J) => AlgebraicGeometry.Scheme.Hom.asOverProp (𝒰.map i) S
Instances For
The pretopology on Over S
induced by P
where coverings are given by P
-covers
of S
-schemes.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The topology on Over S
induced from the topology on Scheme
defined by P
.
This agrees with the topology induced by S.overPretopology P
, see
AlgebraicGeometry.Scheme.overGrothendieckTopology_eq_toGrothendieck_overPretopology
.
Equations
Instances For
If P
and Q
are morphism properties with P ≤ Q
, this is the Grothendieck topology
induced via the forgetful functor Q.Over ⊤ S ⥤ Over S
by the topology defined by P
.
Equations
- S.smallGrothendieckTopologyOfLE hPQ = (CategoryTheory.MorphismProperty.Over.forget Q ⊤ S).inducedTopology (AlgebraicGeometry.Scheme.overGrothendieckTopology P S)
Instances For
The Grothendieck topology on the category of schemes over S
with P
induced by P
, i.e.
coverings are simply surjective families. This is the induced topology by the topology on S
defined by P
via the inclusion P.Over ⊤ S ⥤ Over S
.
This is a special case of smallGrothendieckTopologyOfLE
for the case P = Q
.
Equations
Instances For
The pretopology defind on the subcategory of S
-schemes satisfying Q
where coverings
are given by P
-coverings in S
-schemes satisfying Q
.
The most common case is P = Q
. In this case, this is simply surjective families
in S
-schemes with P
.
Equations
- One or more equations did not get rendered due to their size.