Noetherian rings and modules
The following are equivalent for a module M over a ring R:
- Every increasing chain of submodule M₁ ⊆ M₂ ⊆ M₃ ⊆ ⋯ eventually stabilises.
- Every submodule is finitely generated.
A module satisfying these equivalent conditions is said to be a Noetherian R-module. A ring is a Noetherian ring if it is Noetherian as a module over itself.
Main definitions
Let R
be a ring and let M
and P
be R
-modules. Let N
be an R
-submodule of M
.
fg N : Prop
is the assertion thatN
is finitely generated as anR
-module.is_noetherian R M
is the proposition thatM
is a NoetherianR
-module. It is a class, implemented as the predicate that allR
-submodules ofM
are finitely generated.
Main statements
exists_sub_one_mem_and_smul_eq_zero_of_fg_of_le_smul
is Nakayama's lemma, in the following form: if N is a finitely generated submodule of an ambient R-module M and I is an ideal of R such that N ⊆ IN, then there exists r ∈ 1 + I such that rN = 0.is_noetherian_iff_well_founded
is the theorem that an R-module M is Noetherian iff>
is well-founded onsubmodule R M
.
Note that the Hilbert basis theorem, that if a commutative ring R is Noetherian then so is R[X],
is proved in ring_theory.polynomial
.
References
- [M. F. Atiyah and I. G. Macdonald, Introduction to commutative algebra][atiyah-macdonald]
Tags
Noetherian, noetherian, Noetherian ring, Noetherian module, noetherian ring, noetherian module
A submodule of M
is finitely generated if it is the span of a finite subset of M
.
Nakayama's Lemma. Atiyah-Macdonald 2.5, Eisenbud 4.7, Matsumura 2.2, Stacks 00DV
If 0 → M' → M → M'' → 0 is exact and M' and M'' are finitely generated then so is M.
is_noetherian R M
is the proposition that M
is a Noetherian R
-module,
implemented as the predicate that all R
-submodules of M
are finitely generated.
Equations
- is_noetherian_prod = _
- _ = _
Equations
A ring is Noetherian if it is Noetherian as a module over itself, i.e. all its ideals are finitely generated.
Equations
- is_noetherian_ring R = is_noetherian R R
Equations
Equations
- _ = _
In a module over a noetherian ring, the submodule generated by finitely many vectors is noetherian.
Equations
- _ = _