Well-approximable numbers and Gallagher's ergodic theorem #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
Gallagher's ergodic theorem is a result in metric number theory. It thus belongs to that branch of mathematics concerning arithmetic properties of real numbers which hold almost eveywhere with respect to the Lebesgue measure.
Gallagher's theorem concerns the approximation of real numbers by rational numbers. The input is a
sequence of distances δ₁, δ₂, ...
, and the theorem concerns the set of real numbers x
for which
there is an infinity of solutions to:
$$
|x - m/n| < δₙ,
$$
where the rational number m/n
is in lowest terms. The result is that for any δ
, this set is
either almost all x
or almost no x
.
This result was proved by Gallagher in 1959
P. Gallagher, Approximation by reduced fractions. It is formalised here as
add_circle.add_well_approximable_ae_empty_or_univ
except with x
belonging to the circle ℝ ⧸ ℤ
since this turns out to be more natural.
Given a particular δ
, the Duffin-Schaeffer conjecture (now a theorem) gives a criterion for
deciding which of the two cases in the conclusion of Gallagher's theorem actually occurs. It was
proved by Koukoulopoulos and Maynard in 2019
D. Koukoulopoulos, J. Maynard, On the Duffin-Schaeffer conjecture.
We do not include a formalisation of the Koukoulopoulos-Maynard result here.
Main definitions and results: #
approx_order_of
: in a seminormed groupA
, givenn : ℕ
andδ : ℝ
,approx_order_of A n δ
is the set of elements within a distanceδ
of a point of ordern
.well_approximable
: in a seminormed groupA
, given a sequence of distancesδ₁, δ₂, ...
,well_approximable A δ
is the limsup asn → ∞
of the setsapprox_order_of A n δₙ
. Thus, it is the set of points that lie in infinitely many of the setsapprox_order_of A n δₙ
.add_circle.add_well_approximable_ae_empty_or_univ
: Gallagher's ergodic theorem says that for for the (additive) circle𝕊
, for any sequence of distancesδ
, the setadd_well_approximable 𝕊 δ
is almost empty or almost full.
TODO: #
The hypothesis hδ
in add_circle.add_well_approximable_ae_empty_or_univ
can be dropped.
An elementary (non-measure-theoretic) argument shows that if ¬ hδ
holds then
add_well_approximable 𝕊 δ = univ
(provided δ
is non-negative).
In a seminormed additive group A
, given n : ℕ
and δ : ℝ
,
approx_add_order_of A n δ
is the set of elements within a distance δ
of a point of order n
.
Equations
- approx_add_order_of A n δ = metric.thickening δ {y : A | add_order_of y = n}
In a seminormed group A
, given n : ℕ
and δ : ℝ
, approx_order_of A n δ
is the set of
elements within a distance δ
of a point of order n
.
Equations
- approx_order_of A n δ = metric.thickening δ {y : A | order_of y = n}
In a seminormed additive group A
, given a sequence of
distances δ₁, δ₂, ...
, add_well_approximable A δ
is the limsup as n → ∞
of the sets
approx_add_order_of A n δₙ
. Thus, it is the set of points that lie in infinitely many of the sets
approx_add_order_of A n δₙ
.
Equations
- add_well_approximable A δ = filter.blimsup (λ (n : ℕ), approx_add_order_of A n (δ n)) filter.at_top (λ (n : ℕ), 0 < n)
In a seminormed group A
, given a sequence of distances δ₁, δ₂, ...
, well_approximable A δ
is the limsup as n → ∞
of the sets approx_order_of A n δₙ
. Thus, it is the set of points that
lie in infinitely many of the sets approx_order_of A n δₙ
.
Equations
- well_approximable A δ = filter.blimsup (λ (n : ℕ), approx_order_of A n (δ n)) filter.at_top (λ (n : ℕ), 0 < n)
Gallagher's ergodic theorem on Diophantine approximation.