Order ideals, cofinal sets, and the Rasiowa–Sikorski lemma
Main definitions
We work with a preorder P
throughout.
ideal P
: the type of upward directed, downward closed subsets ofP
. Dual to the notion of a filter on a preorder.cofinal P
: the type of subsets ofP
containing arbitrarily large elements. Dual to the notion of 'dense set' used in forcing.ideal_of_cofinals p 𝒟
, wherep : P
, and𝒟
is a countable family of cofinal subsets of P: an ideal inP
which containsp
and intersects every set in𝒟
.
References
- https://en.wikipedia.org/wiki/Ideal_(order_theory)
- https://en.wikipedia.org/wiki/Cofinal_(mathematics)
- https://en.wikipedia.org/wiki/Rasiowa–Sikorski_lemma
Note that for the Rasiowa–Sikorski lemma, Wikipedia uses the opposite ordering on P
,
in line with most presentations of forcing.
Tags
ideal, cofinal, dense, countable, generic
The smallest ideal containing a given element.
Equations
Equations
- order.ideal.has_mem = {mem := λ (x : P) (I : order.ideal P), x ∈ I.carrier}
For a preorder P
, cofinal P
is the type of subsets of P
containing arbitrarily large elements. They are the dense sets in
the topology whose open sets are terminal segments.
Equations
- order.has_mem = {mem := λ (x : P) (D : order.cofinal P), x ∈ D.carrier}
A (noncomputable) element of a cofinal set lying above a given element.
Equations
- D.above x = classical.some _
Given a starting point, and a countable family of cofinal sets, this is an increasing sequence that intersects each cofinal set.
Equations
- order.sequence_of_cofinals p 𝒟 (n + 1) = order.sequence_of_cofinals._match_1 𝒟 (order.sequence_of_cofinals p 𝒟 n) (order.sequence_of_cofinals p 𝒟 n) (encodable.decode ι n)
- order.sequence_of_cofinals p 𝒟 0 = p
- order.sequence_of_cofinals._match_1 𝒟 _f_1 _f_2 (some i) = (𝒟 i).above _f_2
- order.sequence_of_cofinals._match_1 𝒟 _f_1 _f_2 none = _f_1
Given an element p : P
and a family 𝒟
of cofinal subsets of a preorder P
,
indexed by a countable type, ideal_of_cofinals p 𝒟
is an ideal in P
which
- contains
p
, according tomem_ideal_of_cofinals p 𝒟
, and - intersects every set in
𝒟
, according tocofinal_meets_ideal_of_cofinals p 𝒟
.
This proves the Rasiowa–Sikorski lemma.
Equations
- order.ideal_of_cofinals p 𝒟 = {carrier := {x : P | ∃ (n : ℕ), x ≤ order.sequence_of_cofinals p 𝒟 n}, nonempty := _, directed := _, mem_of_le := _}
ideal_of_cofinals p 𝒟
is 𝒟
-generic.