Cofinality on ordinals, regular cardinals
Cofinality of a reflexive order ≼
. This is the smallest cardinality
of a subset S : set α
such that ∀ a, ∃ b ∈ S, a ≼ b
.
Equations
- order.cof r = cardinal.min _ (λ (S : {S // ∀ (a : α), ∃ (b : α) (H : b ∈ S), r a b}), cardinal.mk ↥S)
Equations
- strict_order.cof r = order.cof (λ (x y : α), ¬r y x)
Cofinality of an ordinal. This is the smallest cardinal of a
subset S
of the ordinal which is unbounded, in the sense
∀ a, ∃ b ∈ S, ¬(b > a)
. It is defined for all ordinals, but
cof 0 = 0
and cof (succ o) = 1
, so it is only really
interesting on limit ordinals (when it is an infinite cardinal).
Equations
- o.cof = quot.lift_on o (λ (_x : Well_order), ordinal.cof._match_1 _x) ordinal.cof._proof_1
- ordinal.cof._match_1 {α := α, r := r, wo := _x} = strict_order.cof r
If the union of s is unbounded and s is smaller than the cofinality, then s has an unbounded member
If the union of s is unbounded and s is smaller than the cofinality, then s has an unbounded member
The infinite pigeonhole principle
pigeonhole principle for a cardinality below the cardinality of the domain
A cardinal is regular if it is infinite and it equals its own cofinality.
Equations
- c.is_regular = (cardinal.omega ≤ c ∧ c.ord.cof = c)
A cardinal is inaccessible if it is an uncountable regular strong limit cardinal.
Equations
- c.is_inaccessible = (cardinal.omega < c ∧ c.is_regular ∧ c.is_strong_limit)