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 refactored 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)
- a subset of
X
equal to the support.
Also see Scheme.IdealSheafData.mkOfMemSupportIff
for a constructor with the condition on the
support being (usually) easier to prove.
- 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)
- supportSet : Set โโX.toPresheafedSpace
The support of an ideal sheaf. Use
IdealSheafData.support
instead for most occasions. - supportSet_eq_iInter_zeroLocus : self.supportSet = โ (U : โX.affineOpens), X.zeroLocus โ(self.ideal U)
Instances For
Equations
- One or more equations did not get rendered due to their size.
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
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
A form of map_ideal
that is easier to rewrite with.
The support of an ideal sheaf. Also see IdealSheafData.mem_support_iff_of_mem
.
Equations
- I.support = { carrier := I.supportSet, isClosed' := โฏ }
Instances For
Custom simps projection for IdealSheafData
.
Equations
Instances For
A useful constructor of IdealSheafData
with the condition on supportSet
being easier to check.
Equations
- One or more equations did not get rendered due to their size.
Instances For
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 radical of a ideal sheaf.
Equations
- I.radical = AlgebraicGeometry.Scheme.IdealSheafData.mkOfMemSupportIff (fun (U : โX.affineOpens) => (I.ideal U).radical) โฏ I.supportSet โฏ
Instances For
The nilradical of a scheme.
Equations
Instances For
The vanishing ideal sheaf of a closed set, which is the largest ideal sheaf whose support is equal to it. The reduced induced scheme structure on the closed set 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
The functor taking a morphism into Y
to its kernel as an ideal sheaf on Y
.
Equations
- One or more equations did not get rendered due to their size.