Documentation

Mathlib.RingTheory.Flat.TorsionFree

Relationships between flatness and torsionfreeness. #

We show that flat implies torsion-free, and that they're the same concept for rings satisfying a certain property, including Dedekind domains and valuation rings.

Main theorems #

theorem Module.Flat.isSMulRegular_of_isRegular {R : Type u_1} {M : Type u_2} [CommSemiring R] [AddCommMonoid M] [Module R M] {r : R} (hr : IsRegular r) [Flat R M] :

Scalar multiplication m ↦ r • m by a regular r is injective on a flat module.

theorem Module.Flat.isSMulRegular_of_nonZeroDivisors {R : Type u_1} {M : Type u_2} [CommRing R] [AddCommGroup M] [Module R M] {r : R} (hr : r nonZeroDivisors R) [Flat R M] :

Scalar multiplication m ↦ r • m by a nonzerodivisor r is injective on a flat module.

theorem Module.Flat.torsion_eq_bot {R : Type u_1} {M : Type u_2} [CommRing R] [AddCommGroup M] [Module R M] [Flat R M] :

Flat modules have no torsion.

If R is Bezout then an R-module is flat iff it has no torsion.

If every localization of R at a maximal ideal is a valuation ring then an R-module is flat iff it has no torsion.

If R is a Dedekind domain then an R-module is flat iff it has no torsion.