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)₀
whenf
is homogeneous of positive degree.AlgebraicGeometry.Proj.awayι
: The open immersionSpec (A_f)₀ ⟶ Proj A
.AlgebraicGeometry.Proj.affineOpenCover
: The open cover ofProj A
bySpec (A_f)₀
for all homogeneousf
of positive degree.AlgebraicGeometry.Proj.stalkIso
: The stalk ofProj A
atx
is the degree0
part of the localization ofA
atx
.
The basic open set D₊(f)
associated to f : A
.
Equations
Instances For
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
Equations
- ⋯ = ⋯
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 irrelavent 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
Proj A
is covered by Spec (A_f)₀
for all homogeneous elements of positive degree.
Equations
- AlgebraicGeometry.Proj.affineOpenCover 𝒜 = AlgebraicGeometry.Proj.openCoverOfISupEqTop 𝒜 (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
- AlgebraicGeometry.Proj.stalkIso 𝒜 x = (AlgebraicGeometry.Proj.stalkIso' 𝒜 x).toCommRingCatIso