Adjunction between Γ
and Spec
#
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
We define the adjunction Γ_Spec.adjunction : Γ ⊣ Spec
by defining the unit (to_Γ_Spec
,
in multiple steps in this file) and counit (done in Spec.lean) and checking that they satisfy
the left and right triangle identities. The constructions and proofs make use of
maps and lemmas defined and proved in structure_sheaf.lean extensively.
Notice that since the adjunction is between contravariant functors, you get to choose
one of the two categories to have arrows reversed, and it is equally valid to present
the adjunction as Spec ⊣ Γ
(Spec.to_LocallyRingedSpace.right_op ⊣ Γ
), in which
case the unit and the counit would switch to each other.
Main definition #
algebraic_geometry.identity_to_Γ_Spec
: The natural transformation𝟭 _ ⟶ Γ ⋙ Spec
.algebraic_geometry.Γ_Spec.LocallyRingedSpace_adjunction
: The adjunctionΓ ⊣ Spec
fromCommRingᵒᵖ
toLocallyRingedSpace
.algebraic_geometry.Γ_Spec.adjunction
: The adjunctionΓ ⊣ Spec
fromCommRingᵒᵖ
toScheme
.
The map from the global sections to a stalk.
Equations
- X.Γ_to_stalk x = X.to_SheafedSpace.to_PresheafedSpace.presheaf.germ ⟨x, trivial⟩
The canonical map from the underlying set to the prime spectrum of Γ(X)
.
Equations
- X.to_Γ_Spec_fun = λ (x : ↥X), ⇑(prime_spectrum.comap (X.Γ_to_stalk x)) (local_ring.closed_point ↥(X.to_SheafedSpace.to_PresheafedSpace.presheaf.stalk x))
The preimage of a basic open in Spec Γ(X)
under the unit is the basic
open in X
defined by the same element (they are equal as sets).
to_Γ_Spec_fun
is continuous.
The canonical (bundled) continuous map from the underlying topological
space of X
to the prime spectrum of its global sections.
Equations
- X.to_Γ_Spec_base = {to_fun := X.to_Γ_Spec_fun, continuous_to_fun := _}
The preimage in X
of a basic open in Spec Γ(X)
(as an open set).
The preimage is the basic open in X
defined by the same element r
.
The map from the global sections Γ(X)
to the sections on the (preimage of) a basic open.
r
is a unit as a section on the basic open defined by r
.
Define the sheaf hom on individual basic opens for the unit.
Equations
Characterization of the sheaf hom on basic opens, direction ← (next lemma) is used at various places, but → is not used in this file.
The sheaf hom on all basic opens, commuting with restrictions.
Equations
The canonical morphism of sheafed spaces from X
to the spectrum of its global sections.
Equations
The map on stalks induced by the unit commutes with maps from Γ(X)
to
stalks (in Spec Γ(X)
and in X
).
The canonical morphism from X
to the spectrum of its global sections.
to_Spec_Γ _
is an isomorphism so these are mutually two-sided inverses.
The unit as a natural transformation.
Equations
- algebraic_geometry.identity_to_Γ_Spec = {app := algebraic_geometry.LocallyRingedSpace.to_Γ_Spec, naturality' := algebraic_geometry.identity_to_Γ_Spec._proof_1}
Spec_Γ_identity
is iso so these are mutually two-sided inverses.
The adjunction Γ ⊣ Spec
from CommRingᵒᵖ
to LocallyRingedSpace
.
Equations
- algebraic_geometry.Γ_Spec.LocallyRingedSpace_adjunction = category_theory.adjunction.mk_of_unit_counit {unit := algebraic_geometry.identity_to_Γ_Spec, counit := (category_theory.nat_iso.op algebraic_geometry.Spec_Γ_identity).inv, left_triangle' := algebraic_geometry.Γ_Spec.LocallyRingedSpace_adjunction._proof_1, right_triangle' := algebraic_geometry.Γ_Spec.LocallyRingedSpace_adjunction._proof_2}
The adjunction Γ ⊣ Spec
from CommRingᵒᵖ
to Scheme
.
Equations
- algebraic_geometry.Γ_Spec.adjunction = category_theory.adjunction.restrict_fully_faithful algebraic_geometry.Scheme.forget_to_LocallyRingedSpace (𝟭 CommRingᵒᵖ) algebraic_geometry.Γ_Spec.LocallyRingedSpace_adjunction (category_theory.nat_iso.of_components (λ (X : algebraic_geometry.Scheme), category_theory.iso.refl ((algebraic_geometry.Scheme.forget_to_LocallyRingedSpace ⋙ algebraic_geometry.LocallyRingedSpace.Γ.right_op).obj X)) algebraic_geometry.Γ_Spec.adjunction._proof_1) (category_theory.nat_iso.of_components (λ (X : CommRingᵒᵖ), category_theory.iso.refl ((𝟭 CommRingᵒᵖ ⋙ algebraic_geometry.Spec.to_LocallyRingedSpace).obj X)) algebraic_geometry.Γ_Spec.adjunction._proof_2)
Immediate consequences of the adjunction.
Spec preserves limits.
Spec is a full functor.
Spec is a faithful functor.