Documentation

Mathlib.Algebra.GroupWithZero.Torsion

Torsion-free monoids with zero #

We prove that if M is an UniqueFactorizationMonoid that can be equipped with a NormalizationMonoid structure and such that is torsion-free, then M is torsion-free.

Note. You need to import this file to get that the monoid of ideals of a Dedekind domain is torsion-free.

theorem IsMulTorsionFree.mk' {M : Type u_1} [CancelCommMonoidWithZero M] (ih : ∀ (x : M), x 0∀ (y : M), y 0∀ (n : ), n 0x ^ n = y ^ nx = y) :