Prime ideals #
Main definitions #
Throughout this file, P
is at least a preorder, but some sections require more
structure, such as a bottom element, a top element, or a join-semilattice structure.
Order.Ideal.PrimePair
: A pair of anOrder.Ideal
and anOrder.PFilter
which form a partition ofP
. This is useful as giving the data of a prime ideal is the same as giving the data of a prime filter.Order.Ideal.IsPrime
: a predicate for prime ideals. Dual to the notion of a prime filter.Order.PFilter.IsPrime
: a predicate for prime filters. Dual to the notion of a prime ideal.
References #
Tags #
ideal, prime
A pair of an Order.Ideal
and an Order.PFilter
which form a partition of P
.
Instances For
theorem
Order.Ideal.PrimePair.I_isProper
{P : Type u_1}
[Preorder P]
(IF : PrimePair P)
:
IF.I.IsProper
Create an element of type Order.Ideal.PrimePair
from an ideal satisfying the predicate
Order.Ideal.IsPrime
.
Equations
- h.toPrimePair = { I := I, F := ⋯.toPFilter, isCompl_I_F := ⋯ }
Instances For
theorem
Order.Ideal.PrimePair.I_isPrime
{P : Type u_1}
[Preorder P]
(IF : PrimePair P)
:
IF.I.IsPrime
theorem
Order.Ideal.IsPrime.mem_or_mem
{P : Type u_1}
[SemilatticeInf P]
{I : Ideal P}
(hI : I.IsPrime)
{x y : P}
:
theorem
Order.Ideal.IsPrime.of_mem_or_mem
{P : Type u_1}
[SemilatticeInf P]
{I : Ideal P}
[I.IsProper]
(hI : ∀ {x y : P}, x ⊓ y ∈ I → x ∈ I ∨ y ∈ I)
:
I.IsPrime
@[instance 100]
instance
Order.Ideal.IsMaximal.isPrime
{P : Type u_1}
[DistribLattice P]
{I : Ideal P}
[I.IsMaximal]
:
I.IsPrime
theorem
Order.Ideal.IsPrime.mem_or_compl_mem
{P : Type u_1}
[BooleanAlgebra P]
{x : P}
{I : Ideal P}
(hI : I.IsPrime)
:
theorem
Order.Ideal.IsPrime.mem_compl_of_not_mem
{P : Type u_1}
[BooleanAlgebra P]
{x : P}
{I : Ideal P}
(hI : I.IsPrime)
(hxnI : x ∉ I)
:
theorem
Order.Ideal.isPrime_of_mem_or_compl_mem
{P : Type u_1}
[BooleanAlgebra P]
{I : Ideal P}
[I.IsProper]
(h : ∀ {x : P}, x ∈ I ∨ xᶜ ∈ I)
:
I.IsPrime
theorem
Order.Ideal.isPrime_iff_mem_or_compl_mem
{P : Type u_1}
[BooleanAlgebra P]
{I : Ideal P}
[I.IsProper]
:
@[instance 100]
instance
Order.Ideal.IsPrime.isMaximal
{P : Type u_1}
[BooleanAlgebra P]
{I : Ideal P}
[I.IsPrime]
:
I.IsMaximal
Create an element of type Order.Ideal.PrimePair
from a filter satisfying the predicate
Order.PFilter.IsPrime
.
Equations
- h.toPrimePair = { I := ⋯.toIdeal, F := F, isCompl_I_F := ⋯ }
Instances For
theorem
Order.Ideal.PrimePair.F_isPrime
{P : Type u_1}
[Preorder P]
(IF : PrimePair P)
:
IF.F.IsPrime