Absolutely Continuous Functions #
This file defines absolutely continuous functions on a closed interval uIcc a b
and proves some
basic properties about absolutely continuous functions.
A function f
is absolutely continuous on uIcc a b
if for any ε > 0
, there is δ > 0
such
that for any finite disjoint collection of intervals uIoc (a i) (b i)
for i < n
where a i
,
b i
are all in uIcc a b
for i < n
, if ∑ i ∈ range n, dist (a i) (b i) < δ
, then
∑ i ∈ range n, dist (f (a i)) (f (b i)) < ε
.
We give a filter version of the definition of absolutely continuous functions in
AbsolutelyContinuousOnInterval
based on AbsolutelyContinuousOnInterval.totalLengthFilter
and AbsolutelyContinuousOnInterval.disjWithin
and prove its equivalence with the ε
-δ
definition in absolutelyContinuousOnInterval_iff
.
We use the filter version to prove that absolutely continuous functions are closed under
- addition -
AbsolutelyContinuousOnInterval.fun_add
,AbsolutelyContinuousOnInterval.add
; - negation -
AbsolutelyContinuousOnInterval.fun_neg
,AbsolutelyContinuousOnInterval.neg
; - subtraction -
AbsolutelyContinuousOnInterval.fun_sub
,AbsolutelyContinuousOnInterval.sub
; - scalar multiplication -
AbsolutelyContinuousOnInterval.const_smul
,AbsolutelyContinuousOnInterval.const_mul
; - multiplication -
AbsolutelyContinuousOnInterval.fun_smul
,AbsolutelyContinuousOnInterval.smul
,AbsolutelyContinuousOnInterval.fun_mul
,AbsolutelyContinuousOnInterval.mul
; and that absolutely continuous implies uniform continuous inAbsolutelyContinuousOnInterval.uniformlyContinuousOn
We use the the ε
-δ
definition to prove that
- Lipschitz continuous functions are absolutely continuous -
LipschitzOnWith.absolutelyContinuousOnInterval
; - absolutely continuous functions have bounded variation -
AbsolutelyContinuousOnInterval.boundedVariationOn
.
Tags #
absolutely continuous
The filter on the collection of all the finite sequences of uIoc
intervals induced by the
function that maps the finite sequence of the intervals to the total length of the intervals.
Details:
- Technically the filter is on
ℕ × (ℕ → X × X)
. A finite sequenceuIoc (a i) (b i)
,i < n
is represented by anyE : ℕ × (ℕ → X × X)
which satisfiesE.1 = n
andE.2 i = (a i, b i)
fori < n
. Its total length is∑ i ∈ Finset.range n, dist (a i) (b i)
. - For a sequence
G : ℕ → ℕ × (ℕ → X × X)
,G
convergence alongtotalLengthFilter
means that the total length ofG j
, i.e.,∑ i ∈ Finset.range (G j).1, dist ((G j).2 i).1 ((G j).2 i).2)
, tends to0
asj
tends to infinity.
Equations
- AbsolutelyContinuousOnInterval.totalLengthFilter = Filter.comap (fun (E : ℕ × (ℕ → X × X)) => ∑ i ∈ Finset.range E.1, dist (E.2 i).1 (E.2 i).2) (nhds 0)
Instances For
The subcollection of all the finite sequences of uIoc
intervals consisting of
uIoc (a i) (b i)
, i < n
where a i
, b i
are all in uIcc a b
for i < n
and
uIoc (a i) (b i)
are mutually disjoint for i < n
. Technically the finite sequence
uIoc (a i) (b i)
, i < n
is represented by any E : ℕ × (ℕ → ℝ × ℝ)
which satisfies
E.1 = n
and E.2 i = (a i, b i)
for i < n
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
AbsolutelyContinuousOnInterval f a b
: A function f
is absolutely continuous on uIcc a b
if the function which (intuitively) maps uIoc (a i) (b i)
, i < n
to
∑ i ∈ Finset.range n, dist (f (a i)) (f (b i))
tendsto 𝓝 0
wrt totalLengthFilter
restricted
to disjWithin a b
. This is equivalent to the traditional ε
-δ
definition: for any ε > 0
,
there is δ > 0
such that for any finite disjoint collection of intervals uIoc (a i) (b i)
for
i < n
where a i
, b i
are all in uIcc a b
for i < n
, if
∑ i ∈ range n, dist (a i) (b i) < δ
, then ∑ i ∈ range n, dist (f (a i)) (f (b i)) < ε
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The traditional ε
-δ
definition of absolutely continuous: A function f
is
absolutely continuous on uIcc a b
if for any ε > 0
, there is δ > 0
such that for
any finite disjoint collection of intervals uIoc (a i) (b i)
for i < n
where a i
, b i
are
all in uIcc a b
for i < n
, if ∑ i ∈ range n, dist (a i) (b i) < δ
, then
∑ i ∈ range n, dist (f (a i)) (f (b i)) < ε
.
If f
is absolutely continuous on uIcc a b
, then f
is uniformly continuous on uIcc a b
.
If f
is absolutely continuous on uIcc a b
, then f
is continuous on uIcc a b
.
If f
is absolutely continuous on uIcc a b
, then f
is bounded on uIcc a b
.
If f
and g
are absolutely continuous on uIcc a b
, then f • g
is absolutely continuous
on uIcc a b
.
If f
and g
are absolutely continuous on uIcc a b
, then f • g
is absolutely continuous
on uIcc a b
.
If f
and g
are absolutely continuous on uIcc a b
, then f * g
is absolutely continuous
on uIcc a b
.
If f
and g
are absolutely continuous on uIcc a b
, then f * g
is absolutely continuous
on uIcc a b
.
If f
is Lipschitz on uIcc a b
, then f
is absolutely continuous on uIcc a b
.
If f
is absolutely continuous on uIcc a b
, then f
has bounded variation on uIcc a b
.