Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 0746194

Browse files
committed
feat(set_theory/cardinal/cofinality): limit cardinal is at least ω (#14432)
1 parent 15726ee commit 0746194

File tree

1 file changed

+8
-0
lines changed

1 file changed

+8
-0
lines changed

src/set_theory/cardinal/cofinality.lean

Lines changed: 8 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -701,6 +701,14 @@ local infixr ^ := @pow cardinal.{u} cardinal cardinal.has_pow
701701
def is_limit (c : cardinal) : Prop :=
702702
c ≠ 0 ∧ ∀ x < c, succ x < c
703703

704+
theorem is_limit.omega_le {c} (h : is_limit c) : ω ≤ c :=
705+
begin
706+
by_contra' h',
707+
rcases lt_omega.1 h' with ⟨_ | n, rfl⟩,
708+
{ exact h.1.irrefl },
709+
{ simpa using h.2 n }
710+
end
711+
704712
/-- A cardinal is a strong limit if it is not zero and it is
705713
closed under powersets. Note that `ω` is a strong limit by this definition. -/
706714
def is_strong_limit (c : cardinal) : Prop :=

0 commit comments

Comments
 (0)