Subscheme associated to an ideal sheaf #
We construct the subscheme associated to an ideal sheaf.
Main definition #
AlgebraicGeometry.Scheme.IdealSheafData.subscheme
: The subscheme associated to an ideal sheaf.AlgebraicGeometry.Scheme.IdealSheafData.subschemeι
: The inclusion from the subscheme.AlgebraicGeometry.Scheme.Hom.image
: The scheme theoretical image of a morphism.AlgebraicGeometry.Scheme.kerAdjunction
: The adjunction between taking kernels and taking the associated subscheme.
Note #
Some instances are in Mathlib/AlgebraicGeometry/Morphisms/ClosedImmersion
and
Mathlib/AlgebraicGeometry/Morphisms/Separated
because they need more API to prove.
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 underlying space of Spec (𝒪ₓ(U)/I(U))
is homeomorphic to its image in X
.
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 subscheme associated to an ideal sheaf.
Equations
Instances For
The inclusion from the subscheme associated to an ideal sheaf.
Equations
- One or more equations did not get rendered due to their size.
Instances For
See AlgebraicGeometry.Morphisms.ClosedImmersion
for the closed immersion version.
The subscheme associated to an ideal sheaf I
is covered by Spec(Γ(X, U)/I(U))
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Γ(𝒪ₓ/I, U) ≅ 𝒪ₓ(U)/I(U)
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Given I ≤ J
, this is the map Spec(Γ(X, U)/J(U)) ⟶ Spec(Γ(X, U)/I(U))
.
Equations
Instances For
The inclusion of ideal sheaf induces an inclusion of subschemes
Equations
- One or more equations did not get rendered due to their size.
Instances For
The functor taking an ideal sheaf to its associated subscheme.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The embedding from the scheme theoretic image to the codomain.
Equations
- f.imageι = f.ker.subschemeι
Instances For
The morphism from the domain to the scheme theoretic image.
Equations
- f.toImage = AlgebraicGeometry.Scheme.Hom.copyBase (AlgebraicGeometry.Scheme.Hom.toImageAux✝ f) (fun (x : ↑↑X.toPresheafedSpace) => ⟨(CategoryTheory.ConcreteCategory.hom f.base) x, ⋯⟩) ⋯
Instances For
The adjunction between Y.IdealSheafData
and (Over Y)ᵒᵖ
given by taking kernels.
Equations
- One or more equations did not get rendered due to their size.