Basic properties of the scheme Proj A #
The scheme Proj 𝒜 for a graded algebra 𝒜 is constructed in
AlgebraicGeometry/ProjectiveSpectrum/Scheme.lean.
In this file we provide basic properties of the scheme.
Main results #
AlgebraicGeometry.Proj.toSpecZero: The structure mapProj A ⟶ Spec (A 0).AlgebraicGeometry.Proj.basicOpenIsoSpec: The canonical isomorphismProj A |_ D₊(f) ≅ Spec (A_f)₀whenfis homogeneous of positive degree.AlgebraicGeometry.Proj.awayι: The open immersionSpec (A_f)₀ ⟶ Proj A.AlgebraicGeometry.Proj.affineOpenCover: The open cover ofProj AbySpec (A_f)₀for all homogeneousfof positive degree.AlgebraicGeometry.Proj.stalkIso: The stalk ofProj Aatxis the degree0part of the localization ofAatx.AlgebraicGeometry.Proj.fromOfGlobalSections: Given a mapf : A →+* Γ(X, ⊤)such that the image of the irrelevant ideal underfgenerates the whole ring, we can construct a mapX ⟶ Proj 𝒜.
The basic open set D₊(f) associated to f : A.
Equations
Instances For
If { xᵢ } spans the irrelevant ideal of A, then D₊(xᵢ) covers Proj A.
If { xᵢ } are homogeneous and span A as an A₀ algebra, then D₊(xᵢ) covers Proj A.
The canonical map (A_f)₀ ⟶ Γ(Proj A, D₊(f)).
This is an isomorphism when f is homogeneous of positive degree. See basicOpenIsoAway below.
Equations
Instances For
The canonical map Proj A |_ D₊(f) ⟶ Spec (A_f)₀.
This is an isomorphism when f is homogeneous of positive degree. See basicOpenIsoSpec below.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The structure map Proj A ⟶ Spec A₀.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The canonical isomorphism Proj A |_ D₊(f) ≅ Spec (A_f)₀
when f is homogeneous of positive degree.
Equations
Instances For
The canonical isomorphism (A_f)₀ ≅ Γ(Proj A, D₊(f))
when f is homogeneous of positive degree.
Equations
Instances For
The open immersion Spec (A_f)₀ ⟶ Proj A.
Equations
- AlgebraicGeometry.Proj.awayι 𝒜 f f_deg hm = CategoryTheory.CategoryStruct.comp (AlgebraicGeometry.Proj.basicOpenIsoSpec 𝒜 f f_deg hm).inv (AlgebraicGeometry.Proj.basicOpen 𝒜 f).ι
Instances For
The isomorphism D₊(f) ×[Proj 𝒜] D₊(g) ≅ D₊(fg).
Equations
- One or more equations did not get rendered due to their size.
Instances For
Given a family of homogeneous elements f of positive degree that spans the irrelevant ideal,
Spec (A_f)₀ ⟶ Proj A forms an affine open cover of Proj A.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Alias of AlgebraicGeometry.Proj.affineOpenCoverOfIrrelevantLESpan.
Given a family of homogeneous elements f of positive degree that spans the irrelevant ideal,
Spec (A_f)₀ ⟶ Proj A forms an affine open cover of Proj A.
Equations
Instances For
Proj A is covered by Spec (A_f)₀ for all homogeneous elements of positive degree.
Equations
- AlgebraicGeometry.Proj.affineOpenCover 𝒜 = AlgebraicGeometry.Proj.affineOpenCoverOfIrrelevantLESpan 𝒜 (fun (i : (i : ℕ+) × ↥(𝒜 ↑i)) => ↑i.snd) ⋯ ⋯ ⋯
Instances For
The stalk of Proj A at x is the degree 0 part of the localization of A at x.
Equations
Instances For
Given a graded ring A and a map f : A →+* Γ(X, ⊤),
for each homogeneous t of positive degree, it induces a map from D(f(t)) ⟶ D₊(t).
Equations
- One or more equations did not get rendered due to their size.
Instances For
Given a graded ring A and a map f : A →+* Γ(X, ⊤) such that the image of the
irrelevant ideal under f generates the whole ring, the set of D(f(r)) for homogeneous r
of positive degree forms an open cover on X.
Equations
- AlgebraicGeometry.Proj.openCoverOfMapIrrelevantEqTop 𝒜 f hf = X.openCoverOfIsOpenCover (fun (ir : (i : ℕ) ×' (r : A) ×' 0 < i ∧ r ∈ 𝒜 i) => X.basicOpen (f ir.snd.fst)) ⋯
Instances For
Alias of AlgebraicGeometry.Proj.openCoverOfMapIrrelevantEqTop.
Given a graded ring A and a map f : A →+* Γ(X, ⊤) such that the image of the
irrelevant ideal under f generates the whole ring, the set of D(f(r)) for homogeneous r
of positive degree forms an open cover on X.
Equations
Instances For
Given a graded ring A and a map f : A →+* Γ(X, ⊤) such that the image of the
irrelevant ideal under f generates the whole ring, we can construct a map X ⟶ Proj 𝒜.
Equations
- One or more equations did not get rendered due to their size.