Skip to content

Commit

Permalink
chore(measure_theory/integral): generalize `interval_integral.norm_in…
Browse files Browse the repository at this point in the history
…tegral_le_integral_norm` (#10412)

It was formulated only for functions `f : α → ℝ`; generalize to `f : α → E`.
  • Loading branch information
urkud committed Nov 23, 2021
1 parent 2817788 commit d9e40b4
Showing 1 changed file with 5 additions and 6 deletions.
11 changes: 5 additions & 6 deletions src/measure_theory/integral/interval_integral.lean
Expand Up @@ -521,6 +521,10 @@ begin
exact le_trans (norm_integral_le_integral_norm _) (le_abs_self _)
end

lemma norm_integral_le_integral_norm (h : a ≤ b) :
∥∫ x in a..b, f x ∂μ∥ ≤ ∫ x in a..b, ∥f x∥ ∂μ :=
norm_integral_le_integral_norm_Ioc.trans_eq $ by rw [interval_oc_of_le h, integral_of_le h]

lemma norm_integral_le_of_norm_le_const_ae {a b C : ℝ} {f : ℝ → E}
(h : ∀ᵐ x, x ∈ Ι a b → ∥f x∥ ≤ C) :
∥∫ x in a..b, f x∥ ≤ C * |b - a| :=
Expand Down Expand Up @@ -1176,14 +1180,9 @@ lemma integral_nonneg [topological_space α] [opens_measurable_space α] [order_
0 ≤ (∫ u in a..b, f u ∂μ) :=
integral_nonneg_of_ae_restrict hab $ (ae_restrict_iff' measurable_set_Icc).mpr $ ae_of_all μ hf

lemma norm_integral_le_integral_norm :
∥∫ x in a..b, f x ∂μ∥ ≤ ∫ x in a..b, ∥f x∥ ∂μ :=
norm_integral_le_abs_integral_norm.trans_eq $
abs_of_nonneg $ integral_nonneg_of_forall hab $ λ x, norm_nonneg _

lemma abs_integral_le_integral_abs :
|∫ x in a..b, f x ∂μ| ≤ ∫ x in a..b, |f x| ∂μ :=
norm_integral_le_integral_norm hab
by simpa only [← real.norm_eq_abs] using norm_integral_le_integral_norm hab

section mono

Expand Down

0 comments on commit d9e40b4

Please sign in to comment.