Skip to content

Commit

Permalink
move and generalize
Browse files Browse the repository at this point in the history
  • Loading branch information
benjamindavidson committed Apr 6, 2021
1 parent 0e55f81 commit 375aa86
Show file tree
Hide file tree
Showing 2 changed files with 10 additions and 5 deletions.
5 changes: 0 additions & 5 deletions src/analysis/special_functions/integrals.lean
Original file line number Diff line number Diff line change
Expand Up @@ -79,11 +79,6 @@ lemma interval_integrable_inv (h : ∀ x : ℝ, x ∈ interval a b → f x ≠ 0
interval_integrable (λ x, (f x)⁻¹) μ a b :=
by simpa only [one_div] using interval_integrable_one_div h hf

@[simp]
lemma interval_integrable.comp (hf : continuous f) (hg : continuous g) :
interval_integrable (λ x, (f ∘ g) x) μ a b :=
(hf.comp hg).interval_integrable a b

@[simp]
lemma interval_integrable_exp : interval_integrable exp μ a b :=
continuous_exp.interval_integrable a b
Expand Down
10 changes: 10 additions & 0 deletions src/measure_theory/interval_integral.lean
Original file line number Diff line number Diff line change
Expand Up @@ -222,6 +222,16 @@ hu.continuous_on.interval_integrable

end

namespace interval_integrable

@[simp]
lemma comp [borel_space E] {μ : measure ℝ} [locally_finite_measure μ] {a b : ℝ}
{f : ℝ → E} {g : ℝ → ℝ} (hf : continuous f) (hg : continuous g) :
interval_integrable (λ x, (f ∘ g) x) μ a b :=
(hf.comp hg).interval_integrable a b

end interval_integrable

/-- Let `l'` be a measurably generated filter; let `l` be a of filter such that each `s ∈ l'`
eventually includes `Ioc u v` as both `u` and `v` tend to `l`. Let `μ` be a measure finite at `l'`.
Expand Down

0 comments on commit 375aa86

Please sign in to comment.