Constant speed #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file defines the notion of constant (and unit) speed for a function f : ℝ → E
with
pseudo-emetric structure on E
with respect to a set s : set ℝ
and "speed" l : ℝ≥0
, and shows
that if f
has locally bounded variation on s
, it can be obtained (up to distance zero, on s
),
as a composite φ ∘ (variation_on_from_to f s a)
, where φ
has unit speed and a ∈ s
.
Main definitions #
has_constant_speed_on_with f s l
, stating that the speed off
ons
isl
.has_unit_speed_on f s
, stating that the speed off
ons
is1
.natural_parameterization f s a : ℝ → E
, the unit speed reparameterization off
ons
relative toa
.
Main statements #
unique_unit_speed_on_Icc_zero
proves that iff
andf ∘ φ
are both naturally parameterized on closed intervals starting at0
, thenφ
must be the identity on those intervals.edist_natural_parameterization_eq_zero
proves that iff
has locally bounded variation, then precomposingnatural_parameterization f s a
withvariation_on_from_to f s a
yields a function at distance zero fromf
ons
.has_unit_speed_natural_parameterization
proves that iff
has locally bounded variation, thennatural_parameterization f s a
has unit speed ons
.
Tags #
arc-length, parameterization
f
has constant speed l
on s
if the variation of f
on s ∩ Icc x y
is equal to
l * (y - x)
for any x y
in s
.
f
has unit speed on s
if it is linearly parameterized by l = 1
on s
.
Equations
- has_unit_speed_on f s = has_constant_speed_on_with f s 1
If both f
and f ∘ φ
have unit speed (on t
and s
respectively) and φ
monotonically maps s
onto t
, then φ
is just a translation (on s
).
If both f
and f ∘ φ
have unit speed (on Icc 0 t
and Icc 0 s
respectively)
and φ
monotonically maps Icc 0 s
onto Icc 0 t
, then φ
is the identity on Icc 0 s
The natural parameterization of f
on s
, which, if f
has locally bounded variation on s
,
- has unit speed on
s
(bynatural_parameterization_has_unit_speed
). - composed with
variation_on_from_to f s a
, is at distance zero fromf
(bynatural_parameterization_edist_zero
).
Equations
- natural_parameterization f s a = f ∘ function.inv_fun_on (variation_on_from_to f s a) s