Non integrable functions #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we prove that the derivative of a function that tends to infinity is not interval
integrable, see interval_integral.not_integrable_has_deriv_at_of_tendsto_norm_at_top_filter
and
interval_integral.not_integrable_has_deriv_at_of_tendsto_norm_at_top_punctured
. Then we apply the
latter lemma to prove that the function λ x, x⁻¹
is integrable on a..b
if and only if a = b
or
0 ∉ [a, b]
.
Main results #
-
not_interval_integrable_of_tendsto_norm_at_top_of_deriv_is_O_punctured
: iff
tends to infinity along𝓝[≠] c
andf' = O(g)
along the same filter, theng
is not interval integrable on any nontrivial integrala..b
,c ∈ [a, b]
. -
not_interval_integrable_of_tendsto_norm_at_top_of_deriv_is_O_filter
: a version ofnot_interval_integrable_of_tendsto_norm_at_top_of_deriv_is_O_punctured
that works for one-sided neighborhoods; -
not_interval_integrable_of_sub_inv_is_O_punctured
: if1 / (x - c) = O(f)
asx → c
,x ≠ c
, thenf
is not interval integrable on any nontrivial intervala..b
,c ∈ [a, b]
; -
interval_integrable_sub_inv_iff
,interval_integrable_inv_iff
: integrability conditions for(x - c)⁻¹
andx⁻¹
.
Tags #
integrable function
If f
is eventually differentiable along a nontrivial filter l : filter ℝ
that is generated
by convex sets, the norm of f
tends to infinity along l
, and f' = O(g)
along l
, where f'
is the derivative of f
, then g
is not integrable on any interval a..b
such that
[a, b] ∈ l
.
If a ≠ b
, c ∈ [a, b]
, f
is differentiable in the neighborhood of c
within
[a, b] \ {c}
, ‖f x‖ → ∞
as x → c
within [a, b] \ {c}
, and f' = O(g)
along
𝓝[[a, b] \ {c}] c
, where f'
is the derivative of f
, then g
is not interval integrable on
a..b
.
If f
is differentiable in a punctured neighborhood of c
, ‖f x‖ → ∞
as x → c
(more
formally, along the filter 𝓝[≠] c
), and f' = O(g)
along 𝓝[≠] c
, where f'
is the derivative
of f
, then g
is not interval integrable on any nontrivial interval a..b
such that
c ∈ [a, b]
.
If f
grows in the punctured neighborhood of c : ℝ
at least as fast as 1 / (x - c)
,
then it is not interval integrable on any nontrivial interval a..b
, c ∈ [a, b]
.
The function λ x, (x - c)⁻¹
is integrable on a..b
if and only if a = b
or c ∉ [a, b]
.
The function λ x, x⁻¹
is integrable on a..b
if and only if a = b
or 0 ∉ [a, b]
.