Ideal sheaves on schemes #
We define ideal sheaves of schemes and provide various constructors for it.
Main definition #
AlgebraicGeometry.Scheme.IdealSheafData
: A structure that contains the data to uniquely define an ideal sheaf, consisting of- an ideal
I(U) ≤ Γ(X, U)
for every affine openU
- a proof that
I(D(f)) = I(U)_f
for every affine openU
and every sectionf : Γ(X, U)
.
- an ideal
AlgebraicGeometry.Scheme.IdealSheafData.ofIdeals
: The largest ideal sheaf contained in a family of ideals.AlgebraicGeometry.Scheme.IdealSheafData.equivOfIsAffine
: Over affine schemes, ideal sheaves are in bijection with ideals of the global sections.AlgebraicGeometry.Scheme.IdealSheafData.support
: The support of an ideal sheaf.AlgebraicGeometry.Scheme.IdealSheafData.vanishingIdeal
: The vanishing ideal of a set.AlgebraicGeometry.Scheme.Hom.ker
: The kernel of a morphism.
Main results #
AlgebraicGeometry.Scheme.IdealSheafData.gc
:support
andvanishingIdeal
forms a galois connection.AlgebraicGeometry.Scheme.Hom.support_ker
: The support of a kernel of a quasi-compact morphism is the closure of the range.
Implementation detail #
Ideal sheaves are not yet defined in this file as actual subsheaves of 𝒪ₓ
.
Instead, for the ease of development and application,
we define the structure IdealSheafData
containing all necessary data to uniquely define an
ideal sheaf. This should be refectored as a constructor for ideal sheaves once they are introduced
into mathlib.
A structure that contains the data to uniquely define an ideal sheaf, consisting of
- an ideal
I(U) ≤ Γ(X, U)
for every affine openU
- a proof that
I(D(f)) = I(U)_f
for every affine openU
and every sectionf : Γ(X, U)
.
- ideal (U : ↑X.affineOpens) : Ideal ↑(X.presheaf.obj (Opposite.op ↑U))
The component of an ideal sheaf at an affine open.
- map_ideal_basicOpen (U : ↑X.affineOpens) (f : ↑(X.presheaf.obj (Opposite.op ↑U))) : Ideal.map (CommRingCat.Hom.hom (X.presheaf.map (CategoryTheory.homOfLE ⋯).op)) (self.ideal U) = self.ideal (X.affineBasicOpen f)
Instances For
The largest ideal sheaf contained in a family of ideals.
Equations
Instances For
The galois coinsertion between ideal sheaves and arbitrary families of ideals.
Equations
- One or more equations did not get rendered due to their size.
Instances For
A form of map_ideal
that is easier to rewrite with.
The ideal sheaf induced by an ideal of the global sections.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Over affine schemes, ideal sheaves are in bijection with ideals of the global sections.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The support of an ideal sheaf. Also see IdealSheafData.mem_support_iff_of_mem
.
Equations
- I.support = ⋂ (U : ↑X.affineOpens), X.zeroLocus ↑(I.ideal U)
Instances For
The radical of a ideal sheaf.
Equations
- I.radical = { ideal := fun (U : ↑X.affineOpens) => (I.ideal U).radical, map_ideal_basicOpen := ⋯ }
Instances For
The vanishing ideal sheaf of a set,
which is the largest ideal sheaf whose support contains a subset.
When the set Z
is closed, the reduced induced scheme structure is the quotient of this ideal.
Equations
- One or more equations did not get rendered due to their size.
Instances For
support
and vanishingIdeal
forms a galois connection.
This is the global version of PrimeSpectrum.gc
.
The kernel of a morphism,
defined as the largest (quasi-coherent) ideal sheaf contained in the component-wise kernel.
This is usually only well-behaved when f
is quasi-compact.
Equations
- f.ker = AlgebraicGeometry.Scheme.IdealSheafData.ofIdeals fun (U : ↑Y.affineOpens) => RingHom.ker (CommRingCat.Hom.hom (f.app ↑U))
Instances For
Spec (𝒪ₓ(U)/I(U))
, the object to be glued into the closed subscheme.
Equations
- I.glueDataObj U = AlgebraicGeometry.Spec (CommRingCat.of (↑(X.presheaf.obj (Opposite.op ↑U)) ⧸ I.ideal U))
Instances For
Spec (𝒪ₓ(U)/I(U)) ⟶ Spec (𝒪ₓ(U)) = U
, the closed immersion into U
.
Equations
Instances For
The open immersion Spec Γ(𝒪ₓ/I, U) ⟶ Spec Γ(𝒪ₓ/I, V)
if U ≤ V
.
Equations
- I.glueDataObjMap h = AlgebraicGeometry.Spec.map (CommRingCat.ofHom (Ideal.quotientMap (I.ideal U) (CommRingCat.Hom.hom (X.presheaf.map (CategoryTheory.homOfLE h).op)) ⋯))
Instances For
The intersections Spec Γ(𝒪ₓ/I, U) ∩ V
useful for gluing.
Equations
- I.glueDataObjPullback U V = CategoryTheory.Limits.pullback (I.glueDataObjι U) (X.homOfLE ⋯)
Instances For
(Implementation) Transition maps in the glue data for 𝒪ₓ/I
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
(Implementation) t'
in the glue data for 𝒪ₓ/I
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
(Implementation) The glue data for 𝒪ₓ/I
.
Equations
- One or more equations did not get rendered due to their size.