Documentation

Mathlib.RingTheory.RingHom.Smooth

Smooth ring homomorphisms #

In this file we define smooth ring homomorphisms and show their meta properties.

def RingHom.FormallySmooth {R S : Type u} [CommRing R] [CommRing S] (f : R →+* S) :

A ring homomorphism f : R →+* S is formally smooth if S is formally smooth as an R algebra.

Equations
Instances For

    Helper lemma for the algebraize tactic

    def RingHom.Smooth {R S : Type u} [CommRing R] [CommRing S] (f : R →+* S) :

    A ring homomorphism f : R →+* S is smooth if S is smooth as an R algebra.

    Equations
    Instances For
      theorem RingHom.Smooth.toAlgebra {R S : Type u} [CommRing R] [CommRing S] {f : R →+* S} (hf : f.Smooth) :

      Helper lemma for the algebraize tactic

      The identity of a ring is smooth.

      theorem RingHom.Smooth.comp {R S T : Type u} [CommRing R] [CommRing S] [CommRing T] {f : R →+* S} {g : S →+* T} (hf : f.Smooth) (hg : g.Smooth) :
      (g.comp f).Smooth

      Composition of smooth ring homomorphisms is smooth.

      Smoothness is a local property of ring homomorphisms.