Documentation

Mathlib.AlgebraicGeometry.Morphisms.Smooth

Smooth morphisms #

A morphism of schemes f : X ⟶ Y is smooth (of relative dimension n) if for each x : X there exists an affine open neighborhood V of x and an affine open neighborhood U of f.base x with V ≤ f ⁻¹ᵁ U such that the induced map Γ(Y, U) ⟶ Γ(X, V) is standard smooth (of relative dimension n).

In other words, smooth (resp. smooth of relative dimension n) for scheme morphisms is associated to the property of ring homomorphisms Locally IsStandardSmooth (resp. Locally (IsStandardSmoothOfRelativeDimension n)).

Implementation details #

The reason why we choose the definition via IsStandardSmooth, is because verifying that Algebra.IsSmooth is local in the sense of RingHom.PropertyIsLocal is a (hard) TODO.

Notes #

This contribution was created as part of the AIM workshop "Formalizing algebraic geometry" in June 2024.

class AlgebraicGeometry.IsSmooth {X Y : Scheme} (f : X Y) :

A morphism of schemes f : X ⟶ Y is smooth if for each x : X there exists an affine open neighborhood V of x and an affine open neighborhood U of f.base x with V ≤ f ⁻¹ᵁ U such that the induced map Γ(Y, U) ⟶ Γ(X, V) is standard smooth.

  • exists_isStandardSmooth (x : X.toPresheafedSpace) : ∃ (U : Y.affineOpens) (V : X.affineOpens) (_ : x V) (e : V (TopologicalSpace.Opens.map f.base).obj U), (Scheme.Hom.appLE f (↑U) (↑V) e).hom.IsStandardSmooth
Instances
    theorem AlgebraicGeometry.isSmooth_iff {X Y : Scheme} (f : X Y) :
    IsSmooth f ∀ (x : X.toPresheafedSpace), ∃ (U : Y.affineOpens) (V : X.affineOpens) (_ : x V) (e : V (TopologicalSpace.Opens.map f.base).obj U), (Scheme.Hom.appLE f (↑U) (↑V) e).hom.IsStandardSmooth

    The property of scheme morphisms IsSmooth is associated with the ring homomorphism property Locally IsStandardSmooth.{0, 0}.

    The composition of smooth morphisms is smooth.

    A morphism of schemes f : X ⟶ Y is smooth of relative dimension n if for each x : X there exists an affine open neighborhood V of x and an affine open neighborhood U of f.base x with V ≤ f ⁻¹ᵁ U such that the induced map Γ(Y, U) ⟶ Γ(X, V) is standard smooth of relative dimension n.

    Instances
      theorem AlgebraicGeometry.isSmoothOfRelativeDimension_iff (n : ) {X Y : Scheme} (f : X Y) :
      IsSmoothOfRelativeDimension n f ∀ (x : X.toPresheafedSpace), ∃ (U : Y.affineOpens) (V : X.affineOpens) (_ : x V) (e : V (TopologicalSpace.Opens.map f.base).obj U), RingHom.IsStandardSmoothOfRelativeDimension n (Scheme.Hom.appLE f (↑U) (↑V) e).hom

      If f is smooth of any relative dimension, it is smooth.

      The property of scheme morphisms IsSmoothOfRelativeDimension n is associated with the ring homomorphism property Locally (IsStandardSmoothOfRelativeDimension.{0, 0} n).

      @[instance 900]

      Open immersions are smooth of relative dimension 0.

      @[instance 900]

      Open immersions are smooth.

      If f is smooth of relative dimension n and g is smooth of relative dimension m, then f ≫ g is smooth of relative dimension n + m.

      @[instance 100]

      Smooth morphisms are locally of finite presentation.