Documentation

Mathlib.RingTheory.Flat.Localization

Flatness and localization #

In this file we show that localizations are flat, and flatness is a local property (TODO).

Main result #

theorem IsLocalization.flat {R : Type u_1} (S : Type u_2) [CommRing R] [CommRing S] [Algebra R S] (p : Submonoid R) [IsLocalization p S] :
instance Localization.flat {R : Type u_1} [CommRing R] (p : Submonoid R) :
Equations
  • =