Documentation

Mathlib.RingTheory.RingHom.Flat

Flat ring homomorphisms #

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

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

A ring homomorphism f : R →+* S is flat if S is flat as an R module.

Equations
Instances For
    theorem RingHom.Flat.id (R : Type u_1) [CommRing R] :
    (RingHom.id R).Flat

    The identity of a ring is flat.

    theorem RingHom.Flat.comp {R : Type u_1} {S : Type u_2} {T : Type u_3} [CommRing R] [CommRing S] [CommRing T] {f : R →+* S} {g : S →+* T} (hf : f.Flat) (hg : g.Flat) :
    (g.comp f).Flat

    Composition of flat ring homomorphisms is flat.

    theorem RingHom.Flat.of_bijective {R : Type u_1} {S : Type u_2} [CommRing R] [CommRing S] {f : R →+* S} (hf : Function.Bijective f) :
    f.Flat

    Bijective ring maps are flat.

    theorem RingHom.Flat.respectsIso :
    RingHom.RespectsIso fun {R S : Type u_4} [CommRing R] [CommRing S] => RingHom.Flat