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

Commit 9d0fd52

Browse files
committed
feat(measure_theory/function/lp_space): use has_measurable_add2 instead of second_countable_topology (#11202)
Use the weaker assumption `[has_measurable_add₂ E]` instead of `[second_countable_topology E]` in 4 lemmas.
1 parent 7249895 commit 9d0fd52

File tree

1 file changed

+6
-6
lines changed

1 file changed

+6
-6
lines changed

src/measure_theory/function/lp_space.lean

Lines changed: 6 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -971,23 +971,23 @@ begin
971971
exact snorm'_lt_top_of_snorm'_lt_top_of_exponent_le hfq_m hfq_lt_top (le_of_lt hp_pos) hpq_real,
972972
end
973973

974-
lemma snorm'_sum_le [second_countable_topology E] {ι} {f : ι → α → E} {s : finset ι}
974+
section has_measurable_add
975+
variable [has_measurable_add₂ E]
976+
977+
lemma snorm'_sum_le {ι} {f : ι → α → E} {s : finset ι}
975978
(hfs : ∀ i, i ∈ s → ae_measurable (f i) μ) (hq1 : 1 ≤ q) :
976979
snorm' (∑ i in s, f i) q μ ≤ ∑ i in s, snorm' (f i) q μ :=
977980
finset.le_sum_of_subadditive_on_pred (λ (f : α → E), snorm' f q μ)
978981
(λ f, ae_measurable f μ) (snorm'_zero (zero_lt_one.trans_le hq1))
979982
(λ f g hf hg, snorm'_add_le hf hg hq1) (λ x y, ae_measurable.add) _ hfs
980983

981-
lemma snorm_sum_le [second_countable_topology E] {ι} {f : ι → α → E} {s : finset ι}
984+
lemma snorm_sum_le {ι} {f : ι → α → E} {s : finset ι}
982985
(hfs : ∀ i, i ∈ s → ae_measurable (f i) μ) (hp1 : 1 ≤ p) :
983986
snorm (∑ i in s, f i) p μ ≤ ∑ i in s, snorm (f i) p μ :=
984987
finset.le_sum_of_subadditive_on_pred (λ (f : α → E), snorm f p μ)
985988
(λ f, ae_measurable f μ) snorm_zero (λ f g hf hg, snorm_add_le hf hg hp1)
986989
(λ x y, ae_measurable.add) _ hfs
987990

988-
section second_countable_topology
989-
variable [second_countable_topology E]
990-
991991
lemma mem_ℒp.add {f g : α → E} (hf : mem_ℒp f p μ) (hg : mem_ℒp g p μ) : mem_ℒp (f + g) p μ :=
992992
⟨ae_measurable.add hf.1 hg.1, snorm_add_lt_top hf hg⟩
993993

@@ -1006,7 +1006,7 @@ begin
10061006
exact (hf i (s.mem_insert_self i)).add (ih (λ j hj, hf j (finset.mem_insert_of_mem hj))), },
10071007
end
10081008

1009-
end second_countable_topology
1009+
end has_measurable_add
10101010

10111011
end borel_space
10121012

0 commit comments

Comments
 (0)