Documentation

Mathlib.AlgebraicGeometry.GammaSpecAdjunction

Adjunction between Γ and Spec #

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 #

The canonical map from the underlying set to the prime spectrum of Γ(X).

Equations
Instances For

    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).

    The canonical (bundled) continuous map from the underlying topological space of X to the prime spectrum of its global sections.

    Equations
    Instances For
      @[reducible, inline]

      The preimage in X of a basic open in Spec Γ(X) (as an open set).

      Equations
      Instances For

        The preimage is the basic open in X defined by the same element r.

        @[reducible, inline]

        The map from the global sections Γ(X) to the sections on the (preimage of) a basic open.

        Equations
        Instances For

          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
          • One or more equations did not get rendered due to their size.
          Instances For

            The canonical morphism of sheafed spaces from X to the spectrum of its global sections.

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For

              The canonical morphism from X to the spectrum of its global sections.

              Equations
              Instances For

                On a locally ringed space X, the preimage of the zero locus of the prime spectrum of Γ(X, ⊤) under toΓSpec agrees with the associated zero locus on X.

                The adjunction Γ ⊣ Spec from CommRingᵒᵖ to LocallyRingedSpace.

                Equations
                • One or more equations did not get rendered due to their size.
                Instances For

                  The adjunction Γ ⊣ Spec from CommRingᵒᵖ to Scheme.

                  Equations
                  • One or more equations did not get rendered due to their size.
                  Instances For

                    The canonical map X ⟶ Spec Γ(X, ⊤). This is the unit of the Γ-Spec adjunction.

                    Equations
                    Instances For
                      @[deprecated AlgebraicGeometry.Scheme.toSpecΓ_appTop (since := "2024-11-23")]

                      Alias of AlgebraicGeometry.Scheme.toSpecΓ_appTop.

                      Immediate consequences of the adjunction.

                      Spec is a full functor.

                      Spec is a faithful functor.

                      theorem AlgebraicGeometry.Spec.map_inj {R S : CommRingCat} {φ ψ : R S} :
                      map φ = map ψ φ = ψ
                      @[simp]
                      theorem AlgebraicGeometry.Spec.preimage_map {R S : CommRingCat} (φ : R S) :
                      preimage (map φ) = φ

                      Useful for replacing f by Spec.map φ everywhere in proofs.

                      Spec is fully faithful

                      Equations
                      Instances For