Skip to content

Commit

Permalink
feat(order/conditionally_complete_lattice): cInf_le variant without…
Browse files Browse the repository at this point in the history
… redundant assumption (#11863)

We prove `cInf_le'` on a `conditionally_complete_linear_order_bot`. We no longer need the boundedness assumption.
  • Loading branch information
vihdzp committed Feb 10, 2022
1 parent 66d9cc1 commit efa3157
Showing 1 changed file with 7 additions and 0 deletions.
7 changes: 7 additions & 0 deletions src/order/conditionally_complete_lattice.lean
Expand Up @@ -687,6 +687,13 @@ is_lub_le_iff (is_lub_cSup' hs)
lemma cSup_le' {s : set α} {a : α} (h : a ∈ upper_bounds s) : Sup s ≤ a :=
(cSup_le_iff' ⟨a, h⟩).2 h

theorem le_cInf_iff'' {s : set α} {a : α} (ne : s.nonempty) :
a ≤ Inf s ↔ ∀ (b : α), b ∈ s → a ≤ b :=
le_cInf_iff ⟨⊥, λ a _, bot_le⟩ ne

theorem cInf_le' {s : set α} {a : α} (h : a ∈ s) : Inf s ≤ a :=
cInf_le ⟨⊥, λ a _, bot_le⟩ h

lemma exists_lt_of_lt_cSup' {s : set α} {a : α} (h : a < Sup s) : ∃ b ∈ s, a < b :=
by { contrapose! h, exact cSup_le' h }

Expand Down

0 comments on commit efa3157

Please sign in to comment.