Minimal primes #
We provide various results concerning the minimal primes above an ideal
Main results #
Ideal.minimalPrimes
:I.minimalPrimes
is the set of ideals that are minimal primes overI
.minimalPrimes
:minimalPrimes R
is the set of minimal primes ofR
.Ideal.exists_minimalPrimes_le
: Every prime ideal overI
contains a minimal prime overI
.Ideal.radical_minimalPrimes
: The minimal primes overI.radical
are precisely the minimal primes overI
.Ideal.sInf_minimalPrimes
: The intersection of minimal primes overI
isI.radical
.Ideal.exists_minimalPrimes_comap_eq
Ifp
is a minimal prime overf ⁻¹ I
, then it is the preimage of some minimal prime overI
.Ideal.minimalPrimes_eq_comap
: The minimal primes overI
are precisely the preimages of minimal primes ofR ⧸ I
.Localization.AtPrime.prime_unique_of_minimal
: When localizing at a minimal prime idealI
, the resulting ring only has a single prime ideal.
I.minimalPrimes
is the set of ideals that are minimal primes over I
.
Instances For
minimalPrimes R
is the set of minimal primes of R
.
This is defined as Ideal.minimalPrimes ⊥
.
Equations
- minimalPrimes R = ⊥.minimalPrimes
Instances For
theorem
minimalPrimes_eq_minimals
{R : Type u_1}
[CommSemiring R]
:
minimalPrimes R = {x : Ideal R | Minimal Ideal.IsPrime x}
theorem
Ideal.exists_minimalPrimes_le
{R : Type u_1}
[CommSemiring R]
{I : Ideal R}
{J : Ideal R}
[J.IsPrime]
(e : I ≤ J)
:
∃ p ∈ I.minimalPrimes, p ≤ J
@[simp]
theorem
Ideal.radical_minimalPrimes
{R : Type u_1}
[CommSemiring R]
{I : Ideal R}
:
I.radical.minimalPrimes = I.minimalPrimes
@[simp]
theorem
Ideal.exists_comap_eq_of_mem_minimalPrimes_of_injective
{R : Type u_1}
{S : Type u_2}
[CommSemiring R]
[CommSemiring S]
{f : R →+* S}
(hf : Function.Injective ⇑f)
(p : Ideal R)
(H : p ∈ minimalPrimes R)
:
∃ (p' : Ideal S), p'.IsPrime ∧ Ideal.comap f p' = p
theorem
Ideal.exists_minimalPrimes_comap_eq
{R : Type u_1}
{S : Type u_2}
[CommRing R]
[CommRing S]
{I : Ideal S}
(f : R →+* S)
(p : Ideal R)
(H : p ∈ (Ideal.comap f I).minimalPrimes)
:
∃ p' ∈ I.minimalPrimes, Ideal.comap f p' = p
theorem
Ideal.minimal_primes_comap_of_surjective
{R : Type u_1}
{S : Type u_2}
[CommRing R]
[CommRing S]
{f : R →+* S}
(hf : Function.Surjective ⇑f)
{I : Ideal S}
{J : Ideal S}
(h : J ∈ I.minimalPrimes)
:
Ideal.comap f J ∈ (Ideal.comap f I).minimalPrimes
theorem
Ideal.comap_minimalPrimes_eq_of_surjective
{R : Type u_1}
{S : Type u_2}
[CommRing R]
[CommRing S]
{f : R →+* S}
(hf : Function.Surjective ⇑f)
(I : Ideal S)
:
(Ideal.comap f I).minimalPrimes = Ideal.comap f '' I.minimalPrimes
theorem
Ideal.minimalPrimes_eq_comap
{R : Type u_1}
[CommRing R]
{I : Ideal R}
:
I.minimalPrimes = Ideal.comap (Ideal.Quotient.mk I) '' minimalPrimes (R ⧸ I)
theorem
IsLocalization.AtPrime.prime_unique_of_minimal
{R : Type u_1}
[CommSemiring R]
{I : Ideal R}
[hI : I.IsPrime]
(hMin : I ∈ minimalPrimes R)
{S : Type u_2}
[CommSemiring S]
[Algebra R S]
[IsLocalization.AtPrime S I]
{J : Ideal S}
{K : Ideal S}
[J.IsPrime]
[K.IsPrime]
:
J = K
theorem
Localization.AtPrime.prime_unique_of_minimal
{R : Type u_1}
[CommSemiring R]
{I : Ideal R}
[hI : I.IsPrime]
(hMin : I ∈ minimalPrimes R)
(J : Ideal (Localization I.primeCompl))
[J.IsPrime]
:
J = LocalRing.maximalIdeal (Localization I.primeCompl)
theorem
Localization.AtPrime.nilpotent_iff_mem_maximal_of_minimal
{R : Type u_1}
[CommSemiring R]
{I : Ideal R}
[hI : I.IsPrime]
(hMin : I ∈ minimalPrimes R)
{x : Localization I.primeCompl}
:
IsNilpotent x ↔ x ∈ LocalRing.maximalIdeal (Localization I.primeCompl)
theorem
Localization.AtPrime.nilpotent_iff_not_unit_of_minimal
{R : Type u_1}
[CommSemiring R]
{I : Ideal R}
[hI : I.IsPrime]
(hMin : I ∈ minimalPrimes R)
{x : Localization I.primeCompl}
:
IsNilpotent x ↔ x ∈ nonunits (Localization I.primeCompl)