Documentation

Mathlib.RingTheory.Ideal.KrullsHeightTheorem

Krull's Height Theorem #

In this file, we prove Krull's principal ideal theorem (also known as Krullscher Hauptidealsatz), and Krull's height theorem (also known as Krullscher Höhensatz).

Main Results #

Krull's principal ideal theorem (also known as Krullscher Hauptidealsatz) : In a commutative Noetherian ring R, any prime ideal that is minimal over a principal ideal has height at most 1.

theorem Ideal.mem_minimalPrimes_span_of_mem_minimalPrimes_span_insert {R : Type u_1} [CommRing R] [IsNoetherianRing R] {q p : Ideal R} [q.IsPrime] (hqp : q < p) (x : R) (s : Set R) (hp : p (span (insert x s)).minimalPrimes) (t : Set R) (htq : t q) (hsp : s (span (insert x t)).radical) :

If q < p are prime ideals such that p is minimal over span (s ∪ {x}) and t is a set contained in q such that s ⊆ √span (t ∪ {x}), then q is minimal over span t. This is used in the induction step for the proof of Krull's height theorem.

Krull's height theorem (also known as Krullscher Höhensatz) : In a commutative Noetherian ring R, any prime ideal that is minimal over an ideal generated by n elements has height at most n.

In a commutative Noetherian ring R, the height of a (finitely-generated) ideal is smaller than or equal to the minimum number of generators for this ideal.

In a commutative Noetherian ring R, a prime ideal p has height no greater than n if and only if it is a minimal ideal over some ideal generated by no more than n elements.

If p is a prime in a Noetherian ring R, there exists a p-primary ideal I spanned by p.height elements.