Skip to content

Commit

Permalink
feat(order/conditionally_complete_lattice,data/real/nnreal): add 2 le…
Browse files Browse the repository at this point in the history
…mmas (#14545)

Add `cInf_univ` and `nnreal.Inf_empty`.
  • Loading branch information
urkud committed Jun 4, 2022
1 parent 72ac40e commit 85fffda
Show file tree
Hide file tree
Showing 2 changed files with 5 additions and 0 deletions.
3 changes: 3 additions & 0 deletions src/data/real/nnreal.lean
Original file line number Diff line number Diff line change
Expand Up @@ -318,6 +318,9 @@ by rw [supr, supr, coe_Sup, set.range_comp]
eq.symm $ @subset_Inf_of_within ℝ (set.Ici 0) _ ⟨(0 : ℝ≥0)⟩ s $
real.Inf_nonneg _ $ λ y ⟨x, _, hy⟩, hy ▸ x.2

@[simp] lemma Inf_empty : Inf (∅ : set ℝ≥0) = 0 :=
by rw [← nnreal.coe_eq_zero, coe_Inf, set.image_empty, real.Inf_empty]

@[norm_cast] lemma coe_infi {ι : Sort*} (s : ι → ℝ≥0) : (↑(⨅ i, s i) : ℝ) = ⨅ i, (s i) :=
by rw [infi, infi, coe_Inf, set.range_comp]

Expand Down
2 changes: 2 additions & 0 deletions src/order/conditionally_complete_lattice.lean
Original file line number Diff line number Diff line change
Expand Up @@ -667,6 +667,8 @@ by rw [supr_of_empty', cSup_empty]

@[simp] lemma csupr_false (f : false → α) : (⨆ i, f i) = ⊥ := csupr_of_empty f

@[simp] lemma cInf_univ : Inf (univ : set α) = ⊥ := is_least_univ.cInf_eq

lemma is_lub_cSup' {s : set α} (hs : bdd_above s) : is_lub s (Sup s) :=
begin
rcases eq_empty_or_nonempty s with (rfl|hne),
Expand Down

0 comments on commit 85fffda

Please sign in to comment.