Hölder continuous functions #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we define Hölder continuity on a set and on the whole space. We also prove some basic properties of Hölder continuous functions.
Main definitions #
holder_on_with
:f : X → Y
is said to be Hölder continuous with constantC : ℝ≥0
and exponentr : ℝ≥0
on a sets
, ifedist (f x) (f y) ≤ C * edist x y ^ r
for allx y ∈ s
;holder_with
:f : X → Y
is said to be Hölder continuous with constantC : ℝ≥0
and exponentr : ℝ≥0
, ifedist (f x) (f y) ≤ C * edist x y ^ r
for allx y : X
.
Implementation notes #
We use the type ℝ≥0
(a.k.a. nnreal
) for C
because this type has coercion both to ℝ
and
ℝ≥0∞
, so it can be easily used both in inequalities about dist
and edist
. We also use ℝ≥0
for r
to ensure that d ^ r
is monotone in d
. It might be a good idea to use
ℝ>0
for r
but we don't have this type in mathlib
(yet).
Tags #
Hölder continuity, Lipschitz continuity
A function f : X → Y
between two pseudo_emetric_space
s is Hölder continuous with constant
C : ℝ≥0
and exponent r : ℝ≥0
, if edist (f x) (f y) ≤ C * edist x y ^ r
for all x y : X
.
Equations
- holder_with C r f = ∀ (x y : X), has_edist.edist (f x) (f y) ≤ ↑C * has_edist.edist x y ^ ↑r
A function f : X → Y
between two pseudo_emeteric_space
s is Hölder continuous with constant
C : ℝ≥0
and exponent r : ℝ≥0
on a set s : set X
, if edist (f x) (f y) ≤ C * edist x y ^ r
for all x y ∈ s
.
Equations
- holder_on_with C r f s = ∀ (x : X), x ∈ s → ∀ (y : X), y ∈ s → has_edist.edist (f x) (f y) ≤ ↑C * has_edist.edist x y ^ ↑r
Alias of the reverse direction of holder_on_with_one
.
Alias of the reverse direction of holder_with_one
.
A Hölder continuous function is uniformly continuous
A Hölder continuous function is uniformly continuous