Documentation

Mathlib.Algebra.Module.PID

Structure of finitely generated modules over a PID #

Main statements #

Notation #

Implementation details #

We first prove (Submodule.isInternal_prime_power_torsion_of_pid) that a finitely generated torsion module is the internal direct sum of its p i ^ e i-torsion submodules for some (finitely many) prime powers p i ^ e i. This is proved in more generality for a Dedekind domain at Submodule.isInternal_prime_power_torsion.

Then we treat the case of a p ^ ∞-torsion module (that is, a module where all elements are cancelled by scalar multiplication by some power of p) and apply it to the p i ^ e i-torsion submodules (that are p i ^ ∞-torsion) to get the result for torsion modules.

Then we get the general result using that a torsion free module is free (which has been proved at Module.free_of_finite_type_torsion_free' at LinearAlgebra.FreeModule.PID.)

Tags #

Finitely generated module, principal ideal domain, classification, structure theorem

A finitely generated torsion module over a PID is an internal direct sum of its p i ^ e i-torsion submodules for some primes p i and numbers e i.

theorem Submodule.exists_isInternal_prime_power_torsion_of_pid {R : Type u} [CommRing R] [IsDomain R] [IsPrincipalIdealRing R] {M : Type v} [AddCommGroup M] [Module R M] [Module.Finite R M] (hM : Module.IsTorsion R M) :
∃ (ι : Type u) (x : Fintype ι) (x : DecidableEq ι) (p : ιR) (_ : ∀ (i : ι), Irreducible (p i)) (e : ι), DirectSum.IsInternal fun (i : ι) => Submodule.torsionBy R M (p i ^ e i)

A finitely generated torsion module over a PID is an internal direct sum of its p i ^ e i-torsion submodules for some primes p i and numbers e i.

theorem Ideal.torsionOf_eq_span_pow_pOrder {R : Type u} [CommRing R] [IsDomain R] [IsPrincipalIdealRing R] {M : Type v} [AddCommGroup M] [Module R M] {p : R} (hp : Irreducible p) (hM : Module.IsTorsion' M (Submonoid.powers p)) [dec : (x : M) → Decidable (x = 0)] (x : M) :
theorem Module.p_pow_smul_lift {R : Type u} [CommRing R] [IsDomain R] [IsPrincipalIdealRing R] {M : Type v} [AddCommGroup M] [Module R M] {p : R} (hp : Irreducible p) (hM : Module.IsTorsion' M (Submonoid.powers p)) [dec : (x : M) → Decidable (x = 0)] {x : M} {y : M} {k : } (hM' : Module.IsTorsionBy R M (p ^ Submodule.pOrder hM y)) (h : p ^ k x Submodule.span R {y}) :
∃ (a : R), p ^ k x = p ^ k a y
theorem Module.exists_smul_eq_zero_and_mk_eq {R : Type u} [CommRing R] [IsDomain R] [IsPrincipalIdealRing R] {M : Type v} [AddCommGroup M] [Module R M] {p : R} (hp : Irreducible p) (hM : Module.IsTorsion' M (Submonoid.powers p)) [dec : (x : M) → Decidable (x = 0)] {z : M} (hz : Module.IsTorsionBy R M (p ^ Submodule.pOrder hM z)) {k : } (f : R Submodule.span R {p ^ k} →ₗ[R] M Submodule.span R {z}) :
∃ (x : M), p ^ k x = 0 Submodule.Quotient.mk x = f 1
theorem Module.torsion_by_prime_power_decomposition {R : Type u} [CommRing R] [IsDomain R] [IsPrincipalIdealRing R] {N : Type (max u v)} [AddCommGroup N] [Module R N] {p : R} (hp : Irreducible p) (hN : Module.IsTorsion' N (Submonoid.powers p)) [h' : Module.Finite R N] :
∃ (d : ) (k : Fin d), Nonempty (N ≃ₗ[R] DirectSum (Fin d) fun (i : Fin d) => R Submodule.span R {p ^ k i})

A finitely generated p ^ ∞-torsion module over a PID is isomorphic to a direct sum of some R ⧸ R ∙ (p ^ e i) for some e i.

theorem Module.equiv_directSum_of_isTorsion {R : Type u} [CommRing R] [IsDomain R] [IsPrincipalIdealRing R] {N : Type (max u v)} [AddCommGroup N] [Module R N] [h' : Module.Finite R N] (hN : Module.IsTorsion R N) :
∃ (ι : Type u) (x : Fintype ι) (p : ιR) (_ : ∀ (i : ι), Irreducible (p i)) (e : ι), Nonempty (N ≃ₗ[R] DirectSum ι fun (i : ι) => R Submodule.span R {p i ^ e i})

A finitely generated torsion module over a PID is isomorphic to a direct sum of some R ⧸ R ∙ (p i ^ e i) where the p i ^ e i are prime powers.

theorem Module.equiv_free_prod_directSum {R : Type u} [CommRing R] [IsDomain R] [IsPrincipalIdealRing R] {N : Type (max u v)} [AddCommGroup N] [Module R N] [h' : Module.Finite R N] :
∃ (n : ) (ι : Type u) (x : Fintype ι) (p : ιR) (_ : ∀ (i : ι), Irreducible (p i)) (e : ι), Nonempty (N ≃ₗ[R] (Fin n →₀ R) × DirectSum ι fun (i : ι) => R Submodule.span R {p i ^ e i})

Structure theorem of finitely generated modules over a PID : A finitely generated module over a PID is isomorphic to the product of a free module and a direct sum of some R ⧸ R ∙ (p i ^ e i) where the p i ^ e i are prime powers.