Skip to content

Commit

Permalink
feat(analysis/seminorm): add lemmas for inequalities and finset.sup (
Browse files Browse the repository at this point in the history
…#12650)

These lemmas are not lean-trivial since seminorms map to the `real` and not to `nnreal`.

Co-authored-by: Eric Wieser <wieser.eric@gmail.com>
  • Loading branch information
mcdoll and eric-wieser committed Mar 14, 2022
1 parent 0f3bfda commit 520f204
Showing 1 changed file with 17 additions and 0 deletions.
17 changes: 17 additions & 0 deletions src/analysis/seminorm.lean
Expand Up @@ -310,6 +310,23 @@ begin
exact bot_le,
end

lemma finset_sup_apply_le {p : ι → seminorm 𝕜 E} {s : finset ι} {x : E} {a : ℝ} (ha : 0 ≤ a)
(h : ∀ i, i ∈ s → p i x ≤ a) : s.sup p x ≤ a :=
begin
lift a to ℝ≥0 using ha,
rw [finset_sup_apply, nnreal.coe_le_coe],
exact finset.sup_le h,
end

lemma finset_sup_apply_lt {p : ι → seminorm 𝕜 E} {s : finset ι} {x : E} {a : ℝ} (ha : 0 < a)
(h : ∀ i, i ∈ s → p i x < a) : s.sup p x < a :=
begin
lift a to ℝ≥0 using ha.le,
rw [finset_sup_apply, nnreal.coe_lt_coe, finset.sup_lt_iff],
{ exact h },
{ exact nnreal.coe_pos.mpr ha },
end

end norm_one_class
end module
end semi_normed_ring
Expand Down

0 comments on commit 520f204

Please sign in to comment.