Skip to content

Commit

Permalink
feat(measure_theory/integral/interval_integral): add lemma `interval_…
Browse files Browse the repository at this point in the history
…integrable.sum` (#14069)

Formalized as part of the Sphere Eversion project.
  • Loading branch information
ocfnash committed May 11, 2022
1 parent 83bc3b9 commit 483affa
Showing 1 changed file with 4 additions and 0 deletions.
4 changes: 4 additions & 0 deletions src/measure_theory/integral/interval_integral.lean
Expand Up @@ -316,6 +316,10 @@ lemma smul [normed_field 𝕜] [normed_space 𝕜 E]
interval_integrable (λ x, f x - g x) μ a b :=
⟨hf.1.sub hg.1, hf.2.sub hg.2

lemma sum (s : finset ι) {f : ι → ℝ → E} (h : ∀ i ∈ s, interval_integrable (f i) μ a b) :
interval_integrable (∑ i in s, f i) μ a b :=
⟨integrable_finset_sum' s (λ i hi, (h i hi).1), integrable_finset_sum' s (λ i hi, (h i hi).2)⟩

lemma mul_continuous_on {f g : ℝ → ℝ}
(hf : interval_integrable f μ a b) (hg : continuous_on g [a, b]) :
interval_integrable (λ x, f x * g x) μ a b :=
Expand Down

0 comments on commit 483affa

Please sign in to comment.