The Mellin transform #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
We define the Mellin transform of a locally integrable function on Ioi 0
, and show it is
differentiable in a suitable vertical strip.
Main statements #
mellin
: the Mellin transform∫ (t : ℝ) in Ioi 0, t ^ (s - 1) • f t
, wheres
is a complex number.has_mellin
: shorthand asserting that the Mellin transform exists and has a given value (analogous tohas_sum
).mellin_differentiable_at_of_is_O_rpow
: iff
isO(x ^ (-a))
at infinity, andO(x ^ (-b))
at 0, thenmellin f
is holomorphic on the domainb < re s < a
.
Predicate on f
and s
asserting that the Mellin integral is well-defined.
Equations
- mellin_convergent f s = measure_theory.integrable_on (λ (t : ℝ), ↑t ^ (s - 1) • f t) (set.Ioi 0) measure_theory.measure_space.volume
The Mellin transform of a function f
(for a complex exponent s
), defined as the integral of
t ^ (s - 1) • f
over Ioi 0
.
Predicate standing for "the Mellin transform of f
is defined at s
and equal to m
". This
shortens some arguments.
Equations
- has_mellin f s m = (mellin_convergent f s ∧ mellin f s = m)
Convergence of Mellin transform integrals #
Auxiliary lemma to reduce convergence statements from vector-valued functions to real scalar-valued functions.
If f
is a locally integrable real-valued function which is O(x ^ (-a))
at ∞
, then for any
s < a
, its Mellin transform converges on some neighbourhood of +∞
.
If f
is a locally integrable real-valued function which is O(x ^ (-b))
at 0
, then for any
b < s
, its Mellin transform converges on some right neighbourhood of 0
.
If f
is a locally integrable real-valued function on Ioi 0
which is O(x ^ (-a))
at ∞
and O(x ^ (-b))
at 0
, then its Mellin transform integral converges for b < s < a
.
If f
is O(x ^ (-a))
as x → +∞
, then log • f
is O(x ^ (-b))
for every b < a
.
If f
is O(x ^ (-a))
as x → 0
, then log • f
is O(x ^ (-b))
for every a < b
.
Suppose f
is locally integrable on (0, ∞)
, is O(x ^ (-a))
as x → ∞
, and is
O(x ^ (-b))
as x → 0
. Then its Mellin transform is differentiable on the domain b < re s < a
,
with derivative equal to the Mellin transform of log • f
.
Suppose f
is locally integrable on (0, ∞)
, is O(x ^ (-a))
as x → ∞
, and is
O(x ^ (-b))
as x → 0
. Then its Mellin transform is differentiable on the domain b < re s < a
.
If f
is locally integrable, decays exponentially at infinity, and is O(x ^ (-b))
at 0, then
its Mellin transform converges for b < s.re
.
If f
is locally integrable, decays exponentially at infinity, and is O(x ^ (-b))
at 0, then
its Mellin transform is holomorphic on b < s.re
.
Mellin transforms of functions on Ioc 0 1
#
The Mellin transform of the indicator function of Ioc 0 1
.