Skip to content

Commit

Permalink
cof_type_lt
Browse files Browse the repository at this point in the history
  • Loading branch information
vihdzp committed Oct 22, 2024
1 parent ec3b51e commit ea21db3
Showing 1 changed file with 7 additions and 0 deletions.
7 changes: 7 additions & 0 deletions Mathlib/SetTheory/Cardinal/Cofinality.lean
Original file line number Diff line number Diff line change
Expand Up @@ -130,6 +130,13 @@ def cof (o : Ordinal.{u}) : Cardinal.{u} := by
theorem cof_type (r : α → α → Prop) [IsWellOrder α r] : (type r).cof = Order.cof (swap rᶜ) :=
rfl

theorem cof_type_lt [LinearOrder α] [IsWellOrder α (· < ·)] :
(@type α (· < ·) _).cof = @Order.cof α (· ≤ ·) := by
rw [cof_type]
congr
ext
simp [swap]

theorem le_cof_type [IsWellOrder α r] {c} : c ≤ cof (type r) ↔ ∀ S, Unbounded r S → c ≤ #S :=
(le_csInf_iff'' (Order.cof_nonempty _)).trans
fun H S h => H _ ⟨S, h, rfl⟩, by
Expand Down

0 comments on commit ea21db3

Please sign in to comment.