Pair Reduction #
The goal of this file is to prove the theorem pair_reduction
. This is essentially Lemma 6.1 in
[KU23] which is an extension of Lemma B.2.7. in [Tal14].
Given pseudometric spaces T
and E
, c ≥ 0
, and a finite subset J
of T
such that
|J| ≤ aⁿ
for some a ≥ 0
and n : ℕ
, pair_reduction
states that there exists a set K ⊆ J²
such that for any function f : T → E
:
|K| ≤ a|J|
∀ (s, t) ∈ K, d(s, t) ≤ cn
sup_{s, t ∈ J : d(s, t) ≤ c} d(f(s), f(t)) ≤ 2 sup_{(s, t) ∈ K} d(f(s), f(t))
When applying the chaining technique for bounding the supremum of the incremements of stochastic
processes, pair_reduction
is used to reduce the order of the dependence of the bound on the
covering numbers of the pseudometric space. As a simple example of how it could be used, suppose
T
has an ε
-covering number N
and suppose J
is an ε
-covering of T
with |J| = N
.
Let f : Ω → T → E
be any stochastic process such that 𝔼 d(f(s), f(t)) ≤ d (s, t)
for all
s, t ∈ T
. Then naively
𝔼[sup_{(s, t) ∈ J} : d(s, t) ≤ c} d(f(s), f(t))]
≤ ∑_{(s, t) ∈ J² : d(s, t) ≤ c} 𝔼[d(f(s), f(t))]
≤ |J|² c
= c N²
but applying pair_reduction
with n = log |J|
we get
𝔼[sup_{(s, t) ∈ J : d(s, t) ≤ c} d(f(s), f(t))]
≤ 2 𝔼[sup_{(s, t) ∈ K} d(f(s), f(t))]
≤ 2 ∑_{(s, t) ∈ K} 𝔼[d(f(s), f(t))]
≤ 2 a |J| c log |J|
≤ 2 a c N log N
pair_reduction
is used in [KU23] to prove a form of the Kolmogorov-Chentsov
theorem that applies to stochastic processses which satisfy the Kolmogorov condition but works
on very general metric spaces.
Implementation #
In this section we sketch a proof of pair_reduction
with references to the corresponding steps
in the lean code.
For any V : Finset T
and t : T
we define the log-size radius of t
in V
to be the smallest
natural number k
greater than zero such that |{x ∈ V | d(t, x) ≤ kc}| ≤ aᵏ
.
(see logSizeRadius
)
We construct a sequence Vᵢ
of subsets of J
, a sequence tᵢ ∈ Vᵢ
and a sequence of rᵢ : ℕ
inductively as follows (see logSizeBallSeq
):
V₀ = J
,tₒ
is chosen arbitarily inJ
,r₀
is the log-size radius oft₀
inV₀
Vᵢ₊ᵢ = Vᵢ \ Bᵢ
whereBᵢ := {x ∈ V | d(t, x) ≤ (rᵢ - 1) c}
,tᵢ₊₁
is chosen arbitarily inVᵢ₊₁
(if it is nonempty),rᵢ₊₁
is the log-size radius oftᵢ₊₁
inVᵢ₊ᵢ
.
Then Vᵢ
is a strictly decreasing sequence (see card_finset_logSizeBallSeq_add_one_lt
) until
Vᵢ
is empty. In particular Vᵢ = ∅
for i ≥ |J|
(see card_finset_logSizeBallSeq_card_eq_zero
).
We will show that K = ⋃_{i=1}^|J| {tᵢ} × {x ∈ Vᵢ | d(tᵢ, x) ≤ crᵢ}
suffices
(see pairSet
and pairSetSeq
).
To prove (1) we have that
|K| ≤ ∑_{i=0}^|J| |{x ∈ Vᵢ : d(t, x) ≤ crᵢ}|
≤ ∑_{i=0}^|J| a ^ rᵢ (by definition of `rᵢ`)
= a ∑_{i=0}^|J| a ^ (rᵢ - 1)
≤ a ∑_{i=0}^|J| |Bᵢ| (by definition of `rᵢ`)
≤ a |J| (since the `Bᵢ` are disjoint (see `disjoint_smallBall_logSizeBallSeq`))
(see card_pairSet_le
).
(2) follows easily from the definition of K and the fact that rᵢ ≤ n
for each i
(see edist_le_of_mem_pairSet
and radius_logSizeBallSeq_le
)
Finally we prove (3). Let s, t ∈ J
such that d(s, t) ≤ c
. Let i
be the largest integer
such that both s, t ∈ Vᵢ
. WLOG suppose s ∉ Vᵢ₊₁
so that in particular s ∈ Bᵢ
which means
by definition that d(tᵢ, s) ≤ (rᵢ - 1)c
. Then we also have
d(tᵢ, t) ≤ d(tᵢ, s) + d(s, t) ≤ (rᵢ - 1)c + c = rᵢc
hence (tᵢ, s), (tᵢ, t) ∈ K
. Furthermore
d(f(s), f(t)) ≤ d(f(tᵢ), f(s)) + d(f(tᵢ), f(t))
taking supremums completes the proof (see iSup_edist_pairSet
).
References #
The log-size radius of t
in V
is the smallest natural number n greater than zero such that
|{x ∈ V | d(t, x) ≤ nc}| ≤ aⁿ
.
Equations
- PairReduction.logSizeRadius t V a c = if h : 1 < a then Nat.find ⋯ else 0
Instances For
A structure for carrying the data of logSizeBallSeq
- finset : Finset T
The underlying finite set of a
logSizeBallStruct
- point : T
The underlying point of a
logSizeBallStruct
(typically a point in the underlying finite set) - radius : ℕ
The underlying radius of a
logSizeBallStruct
(typically the log-size radius of the underlying point in the underlying finite set)
Instances For
If (V, t, r)
is a logSizeBallStruct
then logSizeBallStruct.smallBall
is {x ∈ V | d(t, x) ≤ (r - 1)c}
.
Instances For
If (V, t, r)
is a logSizeBallStruct
then logSizeBallStruct.ball
is {x ∈ V | d(t, x) ≤ rc}
.
Instances For
We recursively define a log-size ball sequence (Vᵢ, tᵢ, rᵢ)
by
V₀ = J
,tₒ
is chosen arbitarily inJ
,r₀
is the log-size radius oft₀
inV₀
Vᵢ₊ᵢ = Vᵢ \ {x ∈ V | d(t, x) ≤ (rᵢ - 1)c}
,tᵢ₊₁
is chosen arbitarily inVᵢ₊₁, rᵢ₊₁
is the log-size radius oftᵢ₊₁
inVᵢ₊ᵢ
.
Equations
- One or more equations did not get rendered due to their size.
- PairReduction.logSizeBallSeq J hJ a c 0 = { finset := J, point := Exists.choose hJ, radius := PairReduction.logSizeRadius (Exists.choose hJ) J a c }
Instances For
Given a log-size ball sequence (Vᵢ, tᵢ, rᵢ)
, we define the pair set sequence by
Kᵢ = {tᵢ} × {x ∈ Vᵢ | dist(tᵢ, x) ≤ rᵢc}
.
Equations
- PairReduction.pairSetSeq J a c n = if hJ : J.Nonempty then {(PairReduction.logSizeBallSeq J hJ a c n).point}.product ((PairReduction.logSizeBallSeq J hJ a c n).ball c) else ∅
Instances For
Given the pair set sequence Kᵢ we define the pair set K
by K = ⋃ i, Kᵢ
.
Equations
- PairReduction.pairSet J a c = (Finset.range J.card).biUnion (PairReduction.pairSetSeq J a c)
Instances For
Pair Reduction: Given pseudometric spaces T
and E
, c ≥ 0
, and a finite subset J
of
T
such that |J| ≤ aⁿ
for some a ≥ 0
and n : ℕ
, pair_reduction
states that there exists a
set K ⊆ J²
such that for any function f : T → E
:
|K| ≤ a|J|
∀ (s, t) ∈ K, d(s, t) ≤ cn
sup_{s, t ∈ J : d(s, t) ≤ c} d(f(s), f(t)) ≤ 2 sup_{(s, t) ∈ K} d(f(s), f(t))