Documentation

Mathlib.MeasureTheory.Integral.Gamma

Integrals involving the Gamma function #

In this file, we collect several integrals over or that evaluate in terms of the Real.Gamma function.

theorem integral_rpow_mul_exp_neg_rpow {p : } {q : } (hp : 0 < p) (hq : -1 < q) :
∫ (x : ) in Set.Ioi 0, x ^ q * (-x ^ p).exp = 1 / p * ((q + 1) / p).Gamma
theorem integral_rpow_mul_exp_neg_mul_rpow {p : } {q : } {b : } (hp : 0 < p) (hq : -1 < q) (hb : 0 < b) :
∫ (x : ) in Set.Ioi 0, x ^ q * (-b * x ^ p).exp = b ^ (-(q + 1) / p) * (1 / p) * ((q + 1) / p).Gamma
theorem integral_exp_neg_rpow {p : } (hp : 0 < p) :
∫ (x : ) in Set.Ioi 0, (-x ^ p).exp = (1 / p + 1).Gamma
theorem integral_exp_neg_mul_rpow {p : } {b : } (hp : 0 < p) (hb : 0 < b) :
∫ (x : ) in Set.Ioi 0, (-b * x ^ p).exp = b ^ (-1 / p) * (1 / p + 1).Gamma
theorem Complex.integral_rpow_mul_exp_neg_rpow {p : } {q : } (hp : 1 p) (hq : -2 < q) :
∫ (x : ), x ^ q * (-x ^ p).exp = 2 * Real.pi / p * ((q + 2) / p).Gamma
theorem Complex.integral_rpow_mul_exp_neg_mul_rpow {p : } {q : } {b : } (hp : 1 p) (hq : -2 < q) (hb : 0 < b) :
∫ (x : ), x ^ q * (-b * x ^ p).exp = 2 * Real.pi / p * b ^ (-(q + 2) / p) * ((q + 2) / p).Gamma
theorem Complex.integral_exp_neg_rpow {p : } (hp : 1 p) :
∫ (x : ), (-x ^ p).exp = Real.pi * (2 / p + 1).Gamma
theorem Complex.integral_exp_neg_mul_rpow {p : } {b : } (hp : 1 p) (hb : 0 < b) :
∫ (x : ), (-b * x ^ p).exp = Real.pi * b ^ (-2 / p) * (2 / p + 1).Gamma