Documentation

Mathlib.RingTheory.Flat.Stability

Flatness is stable under composition and base change #

We show that flatness is stable under composition and base change.

Main theorems #

Composition #

Let R be a ring, S a flat R-algebra and M a flat S-module. To show that M is flat as an R-module, we show that the inclusion of an R-ideal I into R tensored on the left with M is injective. For this consider the composition of natural maps

M ⊗[R] I ≃ M ⊗[S] (S ⊗[R] I) ≃ M ⊗[S] J → M ⊗[S] S ≃ M ≃ M ⊗[R] R

where J is the image of S ⊗[R] I under the (by flatness of S) injective map S ⊗[R] I → S. One checks that this composition is precisely I → R tensored on the left with M and it is injective as a composition of injective maps (note that M ⊗[S] J → M ⊗[S] S is injective because M is S-flat).

theorem Module.Flat.comp (R : Type u) (S : Type v) (M : Type w) [CommRing R] [CommRing S] [Algebra R S] [AddCommGroup M] [Module R M] [Module S M] [IsScalarTower R S M] [Module.Flat R S] [Module.Flat S M] :

If S is a flat R-algebra, then any flat S-Module is also R-flat.

Base change #

Let R be a ring, M a flat R-module and S an R-algebra. To show that S ⊗[R] M is S-flat, we consider for an ideal I in S the composition of natural maps

I ⊗[S] (S ⊗[R] M) ≃ I ⊗[R] M → S ⊗[R] M ≃ S ⊗[S] (S ⊗[R] M).

One checks that this composition is precisely the inclusion I → S tensored on the right with S ⊗[R] M and that the former is injective (note that I ⊗[R] M → S ⊗[R] M is injective, since M is R-flat).

instance Module.Flat.baseChange (R : Type u) (S : Type v) (M : Type w) [CommRing R] [CommRing S] [Algebra R S] [AddCommGroup M] [Module R M] [Module.Flat R M] :

If M is a flat R-module and S is any R-algebra, S ⊗[R] M is S-flat.

Equations
  • =
theorem Module.Flat.isBaseChange (R : Type u) (S : Type v) (M : Type w) [CommRing R] [CommRing S] [Algebra R S] [AddCommGroup M] [Module R M] [Module.Flat R M] (N : Type t) [AddCommGroup N] [Module R N] [Module S N] [IsScalarTower R S N] {f : M →ₗ[R] N} (h : IsBaseChange S f) :

A base change of a flat module is flat.