Derivative of the Gamma function #
This file shows that the (complex) Γ
function is complex-differentiable at all s : ℂ
with
s ∉ {-n : n ∈ ℕ}
, as well as the real counterpart.
Main results #
Complex.differentiableAt_Gamma
:Γ
is complex-differentiable at alls : ℂ
withs ∉ {-n : n ∈ ℕ}
.Real.differentiableAt_Gamma
:Γ
is real-differentiable at alls : ℝ
withs ∉ {-n : n ∈ ℕ}
.
Tags #
Gamma
Now check that the Γ
function is differentiable, wherever this makes sense.
Rewrite the Gamma integral as an example of a Mellin transform.
The derivative of the Γ
integral, at any s ∈ ℂ
with 1 < re s
, is given by the Mellin
transform of log t * exp (-t)
.
theorem
Complex.tendsto_self_mul_Gamma_nhds_zero :
Filter.Tendsto (fun (z : ℂ) => z * Complex.Gamma z) (nhdsWithin 0 {0}ᶜ) (nhds 1)
At s = 0
, the Gamma function has a simple pole with residue 1.