Documentation

Mathlib.AlgebraicGeometry.ResidueField

Residue fields of points #

Main definitions #

The following are in the AlgebraicGeometry.Scheme namespace:

def AlgebraicGeometry.Scheme.residueField (X : Scheme) (x : X.toPresheafedSpace) :

The residue field of X at a point x is the residue field of the stalk of X at x.

Equations
Instances For
    instance AlgebraicGeometry.Scheme.instFieldCarrierResidueField (X : Scheme) (x : X.toPresheafedSpace) :
    Field (X.residueField x)
    Equations
    def AlgebraicGeometry.Scheme.residue (X : Scheme) (x : X.toPresheafedSpace) :
    X.presheaf.stalk x X.residueField x

    The residue map from the stalk to the residue field.

    Equations
    Instances For
      instance AlgebraicGeometry.Scheme.instIsPreimmersionMapResidue {X : Scheme} (x : X.toPresheafedSpace) :
      IsPreimmersion (Spec.map (X.residue x))

      See AlgebraicGeometry.IsClosedImmersion.Spec_map_residue for the stronger result that Spec.map (X.residue x) is a closed immersion.

      @[simp]
      theorem AlgebraicGeometry.Scheme.Spec_map_residue_apply {X : Scheme} (x : X.toPresheafedSpace) (s : (Spec (X.residueField x)).toPresheafedSpace) :
      (Spec.map (X.residue x)).base s = IsLocalRing.closedPoint (X.presheaf.stalk x)
      theorem AlgebraicGeometry.Scheme.residue_surjective (X : Scheme) (x : X.toPresheafedSpace) :
      Function.Surjective (X.residue x).hom
      instance AlgebraicGeometry.Scheme.instEpiCommRingCatResidue (X : Scheme) (x : X.toPresheafedSpace) :
      CategoryTheory.Epi (X.residue x)
      def AlgebraicGeometry.Scheme.descResidueField {K : Type u} [Field K] {X : Scheme} {x : X.toPresheafedSpace} (f : X.presheaf.stalk x CommRingCat.of K) [IsLocalHom f.hom] :
      X.residueField x CommRingCat.of K

      If K is a field and f : 𝒪_{X, x} ⟶ K is a ring map, then this is the induced map κ(x) ⟶ K.

      Equations
      Instances For
        @[simp]
        theorem AlgebraicGeometry.Scheme.residue_descResidueField {K : Type u} [Field K] {X : Scheme} {x : X.toPresheafedSpace} (f : X.presheaf.stalk x CommRingCat.of K) [IsLocalHom f.hom] :
        def AlgebraicGeometry.Scheme.evaluation (X : Scheme) (U : X.Opens) (x : X.toPresheafedSpace) (hx : x U) :
        X.presheaf.obj (Opposite.op U) X.residueField x

        If U is an open of X containing x, we have a canonical ring map from the sections over U to the residue field of x.

        If we interpret sections over U as functions of X defined on U, then this ring map corresponds to evaluation at x.

        Equations
        Instances For
          theorem AlgebraicGeometry.Scheme.germ_residue (X : Scheme) {U : X.Opens} (x : X.toPresheafedSpace) (hx : x U) :
          CategoryTheory.CategoryStruct.comp (X.presheaf.germ U x hx) (X.residue x) = X.evaluation U x hx
          theorem AlgebraicGeometry.Scheme.germ_residue_assoc (X : Scheme) {U : X.Opens} (x : X.toPresheafedSpace) (hx : x U) {Z : CommRingCat} (h : X.residueField x Z) :
          CategoryTheory.CategoryStruct.comp (X.presheaf.germ U x hx) (CategoryTheory.CategoryStruct.comp (X.residue x) h) = CategoryTheory.CategoryStruct.comp (X.evaluation U x hx) h
          @[reducible, inline]
          abbrev AlgebraicGeometry.Scheme.Γevaluation (X : Scheme) (x : X.toPresheafedSpace) :
          X.presheaf.obj (Opposite.op ) X.residueField x

          The global evaluation map from Γ(X, ⊤) to the residue field at x.

          Equations
          Instances For
            @[simp]
            theorem AlgebraicGeometry.Scheme.evaluation_eq_zero_iff_not_mem_basicOpen (X : Scheme) {U : X.Opens} (x : X.toPresheafedSpace) (hx : x U) (f : (X.presheaf.obj (Opposite.op U))) :
            (X.evaluation U x hx).hom f = 0 xX.basicOpen f
            theorem AlgebraicGeometry.Scheme.evaluation_ne_zero_iff_mem_basicOpen (X : Scheme) {U : X.Opens} (x : X.toPresheafedSpace) (hx : x U) (f : (X.presheaf.obj (Opposite.op U))) :
            (X.evaluation U x hx).hom f 0 x X.basicOpen f
            theorem AlgebraicGeometry.Scheme.basicOpen_eq_bot_iff_forall_evaluation_eq_zero (X : Scheme) {U : X.Opens} (f : (X.presheaf.obj (Opposite.op U))) :
            X.basicOpen f = ∀ (x : U), (X.evaluation U x ).hom f = 0
            def AlgebraicGeometry.Scheme.Hom.residueFieldMap {X Y : Scheme} (f : X.Hom Y) (x : X.toPresheafedSpace) :
            Y.residueField (f.base x) X.residueField x

            If X ⟶ Y is a morphism of locally ringed spaces and x a point of X, we obtain a morphism of residue fields in the other direction.

            Equations
            Instances For
              theorem AlgebraicGeometry.Scheme.residue_residueFieldMap {X Y : Scheme} (f : X Y) (x : X.toPresheafedSpace) :
              theorem AlgebraicGeometry.Scheme.evaluation_naturality {X Y : Scheme} (f : X Y) {V : Y.Opens} (x : X.toPresheafedSpace) (hx : f.base x V) :
              CategoryTheory.CategoryStruct.comp (Y.evaluation V (f.base x) hx) (Hom.residueFieldMap f x) = CategoryTheory.CategoryStruct.comp (Hom.app f V) (X.evaluation ((TopologicalSpace.Opens.map f.base).obj V) x hx)
              theorem AlgebraicGeometry.Scheme.evaluation_naturality_assoc {X Y : Scheme} (f : X Y) {V : Y.Opens} (x : X.toPresheafedSpace) (hx : f.base x V) {Z : CommRingCat} (h : X.residueField x Z) :
              theorem AlgebraicGeometry.Scheme.evaluation_naturality_apply {X Y : Scheme} (f : X Y) {V : Y.Opens} (x : X.toPresheafedSpace) (hx : f.base x V) (s : (Y.presheaf.obj (Opposite.op V))) :
              (Hom.residueFieldMap f x).hom ((Y.evaluation V (f.base x) hx).hom s) = (X.evaluation ((TopologicalSpace.Opens.map f.base).obj V) x hx).hom ((Hom.app f V).hom s)
              theorem AlgebraicGeometry.Scheme.Γevaluation_naturality {X Y : Scheme} (f : X Y) (x : X.toPresheafedSpace) :
              CategoryTheory.CategoryStruct.comp (Y.Γevaluation (f.base x)) (Hom.residueFieldMap f x) = CategoryTheory.CategoryStruct.comp (f.c.app (Opposite.op )) (X.Γevaluation x)
              theorem AlgebraicGeometry.Scheme.Γevaluation_naturality_assoc {X Y : Scheme} (f : X Y) (x : X.toPresheafedSpace) {Z : CommRingCat} (h : X.residueField x Z) :
              theorem AlgebraicGeometry.Scheme.Γevaluation_naturality_apply {X Y : Scheme} (f : X Y) (x : X.toPresheafedSpace) (a : (Y.presheaf.obj (Opposite.op ))) :
              (Hom.residueFieldMap f x).hom ((Y.Γevaluation (f.base x)).hom a) = (X.Γevaluation x).hom ((f.c.app (Opposite.op )).hom a)
              def AlgebraicGeometry.Scheme.residueFieldCongr {X : Scheme} {x y : X.toPresheafedSpace} (h : x = y) :
              X.residueField x X.residueField y

              The isomorphism between residue fields of equal points.

              Equations
              Instances For
                @[simp]
                theorem AlgebraicGeometry.Scheme.residueFieldCongr_refl {X : Scheme} {x : X.toPresheafedSpace} :
                @[simp]
                theorem AlgebraicGeometry.Scheme.residueFieldCongr_symm {X : Scheme} {x y : X.toPresheafedSpace} (e : x = y) :
                @[simp]
                theorem AlgebraicGeometry.Scheme.residueFieldCongr_inv {X : Scheme} {x y : X.toPresheafedSpace} (e : x = y) :
                @[simp]
                theorem AlgebraicGeometry.Scheme.residueFieldCongr_trans {X : Scheme} {x y z : X.toPresheafedSpace} (e : x = y) (e' : y = z) :
                @[simp]
                theorem AlgebraicGeometry.Scheme.residueFieldCongr_trans_hom (X : Scheme) {x y z : X.toPresheafedSpace} (e : x = y) (e' : y = z) :
                theorem AlgebraicGeometry.Scheme.residue_residueFieldCongr (X : Scheme) {x y : X.toPresheafedSpace} (h : x = y) :
                CategoryTheory.CategoryStruct.comp (X.residue x) (residueFieldCongr h).hom = CategoryTheory.CategoryStruct.comp (X.presheaf.stalkCongr ).hom (X.residue y)
                theorem AlgebraicGeometry.Scheme.residue_residueFieldCongr_assoc (X : Scheme) {x y : X.toPresheafedSpace} (h : x = y) {Z : CommRingCat} (h✝ : X.residueField y Z) :
                theorem AlgebraicGeometry.Scheme.Hom.residueFieldMap_congr {X Y : Scheme} {f g : X Y} (e : f = g) (x : X.toPresheafedSpace) :
                def AlgebraicGeometry.Scheme.fromSpecResidueField (X : Scheme) (x : X.toPresheafedSpace) :
                Spec (X.residueField x) X

                The canonical map Spec κ(x) ⟶ X.

                Equations
                Instances For
                  instance AlgebraicGeometry.Scheme.instIsPreimmersionFromSpecResidueField {X : Scheme} (x : X.toPresheafedSpace) :
                  IsPreimmersion (X.fromSpecResidueField x)
                  noncomputable instance AlgebraicGeometry.Scheme.instOverSpecResidueField {X : Scheme} (x : X.toPresheafedSpace) :
                  (Spec (X.residueField x)).Over X
                  Equations
                  @[simp]
                  theorem AlgebraicGeometry.Scheme.instOverSpecResidueField_over {X : Scheme} (x : X.toPresheafedSpace) :
                  Spec (X.residueField x) X = X.fromSpecResidueField x
                  @[simp]
                  theorem AlgebraicGeometry.Scheme.instCanonicallyOver_over {X : Scheme} (x : X.toPresheafedSpace) :
                  Spec (X.residueField x) X = X.fromSpecResidueField x
                  @[simp]
                  theorem AlgebraicGeometry.Scheme.residueFieldCongr_fromSpecResidueField {X : Scheme} {x y : X.toPresheafedSpace} (h : x = y) :
                  CategoryTheory.CategoryStruct.comp (Spec.map (residueFieldCongr h).hom) (X.fromSpecResidueField x) = X.fromSpecResidueField y
                  @[simp]
                  theorem AlgebraicGeometry.Scheme.residueFieldCongr_fromSpecResidueField_assoc {X : Scheme} {x y : X.toPresheafedSpace} (h : x = y) {Z : Scheme} (h✝ : X Z) :
                  @[simp]
                  theorem AlgebraicGeometry.Scheme.Hom.Spec_map_residueFieldMap_fromSpecResidueField {X Y : Scheme} (f : X Y) (x : X.toPresheafedSpace) :
                  CategoryTheory.CategoryStruct.comp (Spec.map (residueFieldMap f x)) (Y.fromSpecResidueField (f.base x)) = CategoryTheory.CategoryStruct.comp (X.fromSpecResidueField x) f
                  @[simp]
                  theorem AlgebraicGeometry.Scheme.fromSpecResidueField_apply {X : Scheme} (x : X.toPresheafedSpace) (s : (Spec (X.residueField x)).toPresheafedSpace) :
                  (X.fromSpecResidueField x).base s = x
                  theorem AlgebraicGeometry.Scheme.range_fromSpecResidueField {X : Scheme} (x : X.toPresheafedSpace) :
                  Set.range (X.fromSpecResidueField x).base = {x}
                  theorem AlgebraicGeometry.Scheme.descResidueField_fromSpecResidueField {K : Type u_1} [Field K] (X : Scheme) {x : X.toPresheafedSpace} (f : X.presheaf.stalk x CommRingCat.of K) [IsLocalHom f.hom] :
                  theorem AlgebraicGeometry.Scheme.SpecToEquivOfField_eq_iff {K : Type u_1} [Field K] {X : Scheme} {f₁ f₂ : (x : X.toPresheafedSpace) × (X.residueField x CommRingCat.of K)} :
                  f₁ = f₂ ∃ (e : f₁.fst = f₂.fst), f₁.snd = CategoryTheory.CategoryStruct.comp (residueFieldCongr e).hom f₂.snd

                  A helper lemma to work with AlgebraicGeometry.Scheme.SpecToEquivOfField.

                  def AlgebraicGeometry.Scheme.SpecToEquivOfField (K : Type u) [Field K] (X : Scheme) :
                  (Spec (CommRingCat.of K) X) (x : X.toPresheafedSpace) × (X.residueField x CommRingCat.of K)

                  For a field K and a scheme X, the morphisms Spec K ⟶ X bijectively correspond to pairs of points x of X and embeddings κ(x) ⟶ K.

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