Skip to content

Commit

Permalink
feat(order/conditionally_complete_lattice.lean): two new lemmas (#12250)
Browse files Browse the repository at this point in the history
  • Loading branch information
fpvandoorn committed Feb 24, 2022
1 parent 0840629 commit ed9f73c
Showing 1 changed file with 8 additions and 0 deletions.
8 changes: 8 additions & 0 deletions src/order/conditionally_complete_lattice.lean
Expand Up @@ -463,6 +463,10 @@ begin
{ exact csupr_le (λ x, le_csupr_of_le B x (H x)) },
end

lemma le_csupr_set {f : β → α} {s : set β}
(H : bdd_above (f '' s)) {c : β} (hc : c ∈ s) : f c ≤ ⨆ i : s, f i :=
(le_cSup H $ mem_image_of_mem f hc).trans_eq Sup_image'

/--The indexed infimum of two functions are comparable if the functions are pointwise comparable-/
lemma cinfi_le_cinfi {f g : ι → α} (B : bdd_below (range f)) (H : ∀x, f x ≤ g x) :
infi f ≤ infi g :=
Expand All @@ -479,6 +483,10 @@ lemma cinfi_le {f : ι → α} (H : bdd_below (range f)) (c : ι) : infi f ≤ f
lemma cinfi_le_of_le {f : ι → α} (H : bdd_below (range f)) (c : ι) (h : f c ≤ a) : infi f ≤ a :=
@le_csupr_of_le (order_dual α) _ _ _ _ H c h

lemma cinfi_set_le {f : β → α} {s : set β}
(H : bdd_below (f '' s)) {c : β} (hc : c ∈ s) : (⨅ i : s, f i) ≤ f c :=
@le_csupr_set (order_dual α) _ _ _ _ H _ hc

@[simp] theorem csupr_const [hι : nonempty ι] {a : α} : (⨆ b:ι, a) = a :=
by rw [supr, range_const, cSup_singleton]

Expand Down

0 comments on commit ed9f73c

Please sign in to comment.