Skip to content

Commit

Permalink
fixed def/lemma
Browse files Browse the repository at this point in the history
  • Loading branch information
joelriou committed Feb 13, 2025
1 parent ff381c2 commit f7edaaf
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/SetTheory/Cardinal/Cofinality.lean
Original file line number Diff line number Diff line change
Expand Up @@ -920,7 +920,7 @@ theorem isRegular_cof {o : Ordinal} (h : o.IsLimit) : IsRegular o.cof :=
⟨aleph0_le_cof.2 h, (cof_cof o).ge⟩

/-- If `c` is a regular cardinal, then `c.ord.toType` has a least element. -/
noncomputable def IsRegular.ne_zero {c : Cardinal} (H : c.IsRegular) : c ≠ 0 :=
lemma IsRegular.ne_zero {c : Cardinal} (H : c.IsRegular) : c ≠ 0 :=
H.pos.ne.symm

theorem isRegular_aleph0 : IsRegular ℵ₀ :=
Expand Down

0 comments on commit f7edaaf

Please sign in to comment.