Skip to content

Commit

Permalink
feat(set_theory/cardinal/ordinal): Beth numbers form a normal family (#…
Browse files Browse the repository at this point in the history
…16853)

Prove `is_normal (λ o, (beth o).ord)`
  • Loading branch information
YaelDillies committed Oct 8, 2022
1 parent 85453a2 commit 2a528d1
Showing 1 changed file with 6 additions and 0 deletions.
6 changes: 6 additions & 0 deletions src/set_theory/cardinal/ordinal.lean
Expand Up @@ -364,6 +364,8 @@ begin
exact le_csupr (bdd_above_of_small _) (⟨_, hb.succ_lt h⟩ : Iio b) }
end

lemma beth_mono : monotone beth := beth_strict_mono.monotone

@[simp] theorem beth_lt {o₁ o₂ : ordinal} : beth o₁ < beth o₂ ↔ o₁ < o₂ :=
beth_strict_mono.lt_iff_lt

Expand Down Expand Up @@ -391,6 +393,10 @@ aleph_0_pos.trans_le $ aleph_0_le_beth o
theorem beth_ne_zero (o : ordinal) : beth o ≠ 0 :=
(beth_pos o).ne'

lemma beth_normal : is_normal.{u} (λ o, (beth o).ord) :=
(is_normal_iff_strict_mono_limit _).2 ⟨ord_strict_mono.comp beth_strict_mono, λ o ho a ha,
by { rw [beth_limit ho, ord_le], exact csupr_le' (λ b, ord_le.1 (ha _ b.2)) }⟩

/-! ### Properties of `mul` -/

/-- If `α` is an infinite type, then `α × α` and `α` have the same cardinality. -/
Expand Down

0 comments on commit 2a528d1

Please sign in to comment.