Hölder continuous functions #
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 #
HolderOnWith:f : X → Yis said to be Hölder continuous with constantC : ℝ≥0and exponentr : ℝ≥0on a sets, ifedist (f x) (f y) ≤ C * edist x y ^ rfor allx y ∈ s;HolderWith:f : X → Yis said to be Hölder continuous with constantC : ℝ≥0and exponentr : ℝ≥0, ifedist (f x) (f y) ≤ C * edist x y ^ rfor 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 PseudoEMetricSpaces 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.
Instances For
A function f : X → Y between two PseudoEMetricSpaces 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.
Instances For
Alias of the reverse direction of holderOnWith_one.
Alias of the reverse direction of holderWith_one.
A Hölder continuous function is uniformly continuous
If a function is (C₁, r)-Hölder and (C₂, s)-Hölder, then it is
(C₁ ^ t₁ * C₂ ^ t₂, r * t₁ + s * t₂)-Hölder for all t₁ t₂ : ℝ≥0 such that
t₁ + t₂ = 1.
If a function is Hölder over a bounded set, then it is bounded.
If a function is r-Hölder over a bounded set, then it is also s-Hölder when s ≤ r.
If a function is (C, r)-Hölder and (C, s)-Hölder,
then it is (C, r * t₁ + s * t₂)-Hölder for all t₁ t₂ : ℝ≥0 such that
t₁ + t₂ = 1.
For fixed f : X → Y, A : Set X and C : ℝ≥0, the set of all parameters r : ℝ≥0 such that
f is (C, r)-Hölder on A is convex.
Alias of the reverse direction of HolderWith.restrict_iff.
A Hölder continuous function is uniformly continuous
If a function is (C₁, r)-Hölder and (C₂, s)-Hölder, then it is
(C₁ ^ t₁ * C₂ ^ t₂, r * t₁ + s * t₂)-Hölder for all t₁ t₂ : ℝ≥0 such that
t₁ + t₂ = 1.
If a function is Hölder over a bounded space, then it is bounded.
If a function is r-Hölder over a bounded space, then it is also s-Hölder when s ≤ r.
If a function is (C, r)-Hölder and (C, s)-Hölder,
then it is (C, r * t₁ + s * t₂)-Hölder for all t₁ t₂ : ℝ≥0 such that
t₁ + t₂ = 1.
For fixed f : X → Y and C : ℝ≥0, the set of all parameters r : ℝ≥0 such that
f is (C, r)-Hölder is convex.