Documentation

Mathlib.AlgebraicGeometry.SpreadingOut

Spreading out morphisms #

Under certain conditions, a morphism on stalks Spec 𝒪_{X, x} ⟶ Spec 𝒪_{Y, y} can be spread out into a neighborhood of x.

Main result #

Given S-schemes X Y and points x : X y : Y over s : S. Suppose we have the following diagram of S-schemes

Spec 𝒪_{X, x} ⟶ X
    |
  Spec(φ)
    ↓
Spec 𝒪_{Y, y} ⟶ Y

We would like to spread Spec(φ) out to an S-morphism on an open subscheme U ⊆ X

Spec 𝒪_{X, x} ⟶ U ⊆ X
    |             |
  Spec(φ)         |
    ↓             ↓
Spec 𝒪_{Y, y} ⟶ Y

TODO #

Show that certain morphism properties can also be spread out.

The germ map at x is injective if there exists some affine U ∋ x such that the map Γ(X, U) ⟶ X_x is injective

Instances
    @[reducible, inline]

    The class of schemes such that for each x : X, Γ(X, U) ⟶ X_x is injective for some affine U containing x.

    This is typically satisfied when X is integral or locally noetherian.

    Equations
    Instances For
      theorem AlgebraicGeometry.Scheme.IsGermInjective.Spec {R : CommRingCat} (H : ∀ (I : Ideal R), I.IsPrimefI, ∀ (x y : R), y * x = 0yI∃ (n : ), f ^ n * x = 0) :

      Let x : X and f g : X ⟶ Y be two morphisms such that f x = g x. If f and g agree on the stalk of x, then they agree on an open neighborhood of x, provided X is "germ-injective" at x (e.g. when it's integral or locally noetherian).

      TODO: The condition on X is unnecessary when Y is locally of finite type.

      Stacks Tag 0BX6

      A variant of spread_out_unique_of_isGermInjective whose condition is an equality of scheme morphisms instead of ring homomorphisms.

      theorem AlgebraicGeometry.exists_lift_of_germInjective_aux {X : Scheme} {R A : CommRingCat} {U : X.Opens} {x : X} (hxU : x U) (φ : A X.presheaf.stalk x) (φRA : R A) (φRX : R X.presheaf.obj (Opposite.op U)) (hφRA : (CommRingCat.Hom.hom φRA).FiniteType) (e : CategoryTheory.CategoryStruct.comp φRA φ = CategoryTheory.CategoryStruct.comp φRX (X.presheaf.germ U x hxU)) :
      ∃ (V : X.Opens) (hxV : x V), V U (CommRingCat.Hom.hom φ).range (CommRingCat.Hom.hom (X.presheaf.germ V x hxV)).range

      Suppose X is a scheme, x : X such that the germ map at x is (locally) injective, and U is a neighborhood of x. Given a commutative diagram of CommRingCat

      R ⟶ Γ(X, U)
      ↓    ↓
      A ⟶ 𝒪_{X, x}
      

      such that R is of finite type over A, we may lift A ⟶ 𝒪_{X, x} to some A ⟶ Γ(X, V).

      Given S-schemes X Y and points x : X y : Y over s : S. Suppose we have the following diagram of S-schemes

      Spec 𝒪_{X, x} ⟶ X
          |
        Spec(φ)
          ↓
      Spec 𝒪_{Y, y} ⟶ Y
      

      Then the map Spec(φ) spreads out to an S-morphism on an open subscheme U ⊆ X,

      Spec 𝒪_{X, x} ⟶ U ⊆ X
          |             |
        Spec(φ)         |
          ↓             ↓
      Spec 𝒪_{Y, y} ⟶ Y
      

      provided that Y is locally of finite type over S and X is "germ-injective" at x (e.g. when it's integral or locally noetherian).

      TODO: The condition on X is unnecessary when Y is locally of finite presentation.

      Stacks Tag 0BX6

      Given S-schemes X Y, a point x : X, and a S-morphism φ : Spec 𝒪_{X, x} ⟶ Y, we may spread it out to an S-morphism f : U ⟶ Y provided that Y is locally of finite type over S and X is "germ-injective" at x (e.g. when it's integral or locally noetherian).

      TODO: The condition on X is unnecessary when Y is locally of finite presentation.