Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit ef78b32

Browse files
committed
feat(measure_theory/function/lp_space): add lemmas about snorm and mem_Lp (#9146)
Also move lemma `snorm_add_le` (and related others) out of the borel space section, since `opens_measurable_space` is a sufficient hypothesis.
1 parent 5aaa5fa commit ef78b32

File tree

2 files changed

+228
-84
lines changed

2 files changed

+228
-84
lines changed

src/measure_theory/function/ess_sup.lean

Lines changed: 10 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -118,6 +118,16 @@ begin
118118
all_goals { is_bounded_default, },
119119
end
120120

121+
lemma ess_sup_smul_measure {f : α → β} {c : ℝ≥0∞} (hc : c ≠ 0) :
122+
ess_sup f (c • μ) = ess_sup f μ :=
123+
begin
124+
simp_rw ess_sup,
125+
suffices h_smul : (c • μ).ae = μ.ae, by rw h_smul,
126+
ext1,
127+
simp_rw mem_ae_iff,
128+
simp [hc],
129+
end
130+
121131
end complete_lattice
122132

123133
section complete_linear_order

0 commit comments

Comments
 (0)