Finitely generated module over noetherian ring have finitely many associated primes. #
In this file we proved that any finitely generated module over a noetherian ring have finitely many associated primes.
Main results #
IsNoetherianRing.exists_relSeries_isQuotientEquivQuotientPrime
: IfA
is a Noetherian ring andM
is a finitely generatedA
-module, then there exists a chain of submodules0 = M₀ ≤ M₁ ≤ M₂ ≤ ... ≤ Mₙ = M
ofM
, such that for each0 ≤ i < n
,Mᵢ₊₁ / Mᵢ
is isomorphic toA / pᵢ
for some prime idealpᵢ
ofA
.IsNoetherianRing.induction_on_isQuotientEquivQuotientPrime
: If a property on finitely generated modules over a Noetherian ring satisfies that:- it holds for zero module,
- it holds for any module isomorphic to some
A ⧸ p
wherep
is a prime ideal ofA
, - it is stable by short exact sequences,
then the property holds for every finitely generated modules.
associatedPrimes.finite
: There are only finitely many associated primes of a finitely generated module over a Noetherian ring.
A Prop
asserting that two submodules N₁, N₂
satisfy N₁ ≤ N₂
and
N₂ / N₁
is isomorphic to A / p
for some prime ideal p
of A
.
Equations
- N₁.IsQuotientEquivQuotientPrime N₂ = (N₁ ≤ N₂ ∧ ∃ (p : PrimeSpectrum A), Nonempty ((↥N₂ ⧸ N₁.submoduleOf N₂) ≃ₗ[A] A ⧸ p.asIdeal))
Instances For
If A
is a Noetherian ring and M
is a finitely generated A
-module, then there exists
a chain of submodules 0 = M₀ ≤ M₁ ≤ M₂ ≤ ... ≤ Mₙ = M
of M
, such that for each 0 ≤ i < n
,
Mᵢ₊₁ / Mᵢ
is isomorphic to A / pᵢ
for some prime ideal pᵢ
of A
.
If a property on finitely generated modules over a Noetherian ring satisfies that:
- it holds for zero module (it's formalized as it holds for any module which is subsingleton),
- it holds for
A ⧸ p
for every prime idealp
ofA
(to avoid universe problem, it's formalized as it holds for any module isomorphic toA ⧸ p
), - it is stable by short exact sequences,
then the property holds for every finitely generated modules.
NOTE: This should be the induction principle for M
, but due to the bug
https://github.com/leanprover/lean4/issues/4246
currently it is induction for Module.Finite A M
.
There are only finitely many associated primes of a finitely generated module over a Noetherian ring.