Skip to content

Commit

Permalink
feat(Order/ConditionallyCompleteLattice/Basic): not_mem_of_lt_csInf' (
Browse files Browse the repository at this point in the history
  • Loading branch information
vihdzp committed Sep 21, 2024
1 parent 94533cc commit ddb07e5
Showing 1 changed file with 3 additions and 0 deletions.
3 changes: 3 additions & 0 deletions Mathlib/Order/ConditionallyCompleteLattice/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1212,6 +1212,9 @@ theorem exists_lt_of_lt_ciSup' {f : ι → α} {a : α} (h : a < ⨆ i, f i) :
contrapose! h
exact ciSup_le' h

theorem not_mem_of_lt_csInf' {x : α} {s : Set α} (h : x < sInf s) : x ∉ s :=
not_mem_of_lt_csInf h (OrderBot.bddBelow s)

theorem ciSup_mono' {ι'} {f : ι → α} {g : ι' → α} (hg : BddAbove (range g))
(h : ∀ i, ∃ i', f i ≤ g i') : iSup f ≤ iSup g :=
ciSup_le' fun i => Exists.elim (h i) (le_ciSup_of_le hg)
Expand Down

0 comments on commit ddb07e5

Please sign in to comment.