Smooth morphisms #
An R-algebra A is formally smooth if Ω[A⁄R] is A-projective and H¹(L_{A/R}) = 0.
This is equivalent to the standard definition that "for every R-algebra B,
every square-zero ideal I : Ideal B and f : A →ₐ[R] B ⧸ I, there exists
at least one lift A →ₐ[R] B".
An R-algebra A is smooth if it is formally smooth and of finite presentation.
We show that the property of being formally smooth extends onto nilpotent ideals,
and that it is stable under R-algebra homomorphisms and compositions.
We show that smooth is stable under algebra isomorphisms, composition and localization at an element.
Main results #
Algebra.FormallySmooth: The class of formally smooth algebras.Algebra.formallySmooth_iff: Formally smooth iffΩ[A⁄R]isA-projective andH¹(L_{A/R}) = 0.Algebra.FormallySmooth.lift: IfAis formally smooth andIis nilpotent, any mapA →ₐ[R] B ⧸ Ilifts toA →ₐ[R] B.Algebra.FormallySmooth.iff_comp_surjective:Ais formally smooth iff any mapA →ₐ[R] B ⧸ Ilifts toA →ₐ[R] Bfor any square zeroI.
Suppose P is a formally smooth R algebra that surjects onto A with kernel I, then
Algebra.FormallySmooth.iff_split_surjection:Ais formally smooth iff the algebra mapP ⧸ I² →ₐ[R] Ahas anR-algebra section.Algebra.Extension.equivH1CotangentOfFormallySmooth:H¹(L_{A/R})is isomorphic toker(I/I² → A ⊗[P] Ω[P⁄R]).Algebra.FormallySmooth.iff_split_injection:Ais formally smooth iff theP-linear mapI/I² → A ⊗[P] Ω[P⁄R]is split injective.
An R-algebra A is formally smooth if Ω[A⁄R] is A-projective and H¹(L_{A/R}) = 0.
For the infinitesimal lifting definition,
see FormallySmooth.lift and FormallySmooth.iff_comp_surjective.
- projective_kaehlerDifferential : Module.Projective A Ω[A⁄R]
- subsingleton_h1Cotangent : Subsingleton (H1Cotangent R A)
Instances
Alias of Algebra.formallySmooth_iff.
For a formally smooth R-algebra A and a map f : A →ₐ[R] B ⧸ I with I square-zero,
this is an arbitrary lift A →ₐ[R] B.
Equations
- Algebra.FormallySmooth.lift I hI g = ⋯.choose
Instances For
For a formally smooth R-algebra A and a map f : A →ₐ[R] B ⧸ I with I nilpotent,
this is an arbitrary lift A →ₐ[R] B.
Equations
- Algebra.FormallySmooth.liftOfSurjective f g hg hg' = Algebra.FormallySmooth.lift (RingHom.ker ↑g) hg' ((↑(Ideal.quotientKerAlgEquivOfSurjective hg).symm).comp f)
Instances For
Given extensions 0 → I₁ → P₁ → A → 0 and 0 → I₂ → P₂ → A → 0 with P₁ formally smooth,
this is an arbitrarily chosen map P₁/I₁² → P₂/I₂² of extensions.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Formally smooth extensions have isomorphic H¹(L_P).
Equations
- One or more equations did not get rendered due to their size.
Instances For
Any formally smooth extension can be used to calculate H¹(L_{A/R}).
Equations
Instances For
Given a formally smooth R-algebra P and a surjective algebra homomorphism f : P →ₐ[R] A
with kernel I (typically a presentation R[X] → A),
A is formally smooth iff the P-linear map I/I² → A ⊗[P] Ω[P⁄R] is split injective.
Also see Algebra.Extension.formallySmooth_iff_split_injection
for the version in terms of Extension.
Given a formally smooth R-algebra P and a surjective algebra homomorphism f : P →ₐ[R] S
with kernel I (typically a presentation R[X] → S),
S is formally smooth iff the P-linear map I/I² → S ⊗[P] Ω[P⁄R] is split injective.
Let P →ₐ[R] A be a surjection with kernel J, and P a formally smooth R-algebra,
then A is formally smooth over R iff the surjection P ⧸ J ^ 2 →ₐ[R] A has a section.
Geometric intuition: we require that a first-order thickening of Spec A inside Spec P admits
a retraction.
An R-algebra A is formally smooth iff "for every R-algebra B,
every square-zero ideal I : Ideal B and f : A →ₐ[R] B ⧸ I, there exists
at least one lift A →ₐ[R] B".
An R algebra A is smooth if it is formally smooth and of finite presentation.
- formallySmooth : FormallySmooth R A
- finitePresentation : FinitePresentation R A
Instances
Localization at an element is smooth.