Integrals with exponential decay at ∞ #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
As easy special cases of general theorems in the library, we prove the following test for integrability:
- integrable_of_is_O_exp_neg: If- fis continuous on- [a,∞), for some- a ∈ ℝ, and there exists- b > 0such that- f(x) = O(exp(-b x))as- x → ∞, then- fis integrable on- (a, ∞).
    
theorem
exp_neg_integrable_on_Ioi
    (a : ℝ)
    {b : ℝ}
    (h : 0 < b) :
measure_theory.integrable_on (λ (x : ℝ), rexp (-b * x)) (set.Ioi a) measure_theory.measure_space.volume
exp (-b * x) is integrable on (a, ∞).