Documentation

Mathlib.NumberTheory.Liouville.Measure

Volume of the set of Liouville numbers #

In this file we prove that the set of Liouville numbers with exponent (irrationality measure) strictly greater than two is a set of Lebesgue measure zero, see volume_iUnion_setOf_liouvilleWith.

Since this set is a residual set, we show that the filters residual and volume.ae are disjoint. These filters correspond to two common notions of genericity on : residual sets and sets of full measure. The fact that the filters are disjoint means that two mutually exclusive properties can be “generic” at the same time (in the sense of different “genericity” filters).

Tags #

Liouville number, Lebesgue measure, residual, generic property

theorem setOf_liouvilleWith_subset_aux :
{x : | ∃ p > 2, LiouvilleWith p x} ⋃ (m : ), (fun (x : ) => x + m) ⁻¹' ⋃ (n : ), ⋃ (_ : n > 0), {x : | ∃ᶠ (b : ) in Filter.atTop, ∃ a ∈ Finset.Icc 0 b, |x - a / b| < 1 / b ^ (2 + 1 / n)}
@[simp]
theorem volume_iUnion_setOf_liouvilleWith :
MeasureTheory.volume (⋃ (p : ), ⋃ (_ : 2 < p), {x : | LiouvilleWith p x}) = 0

The set of numbers satisfying the Liouville condition with some exponent p > 2 has Lebesgue measure zero.

theorem ae_not_liouvilleWith :
∀ᵐ (x : ), p > 2, ¬LiouvilleWith p x
theorem ae_not_liouville :
∀ᵐ (x : ), ¬Liouville x
@[simp]
theorem volume_setOf_liouville :
MeasureTheory.volume {x : | Liouville x} = 0

The set of Liouville numbers has Lebesgue measure zero.

The filters residual and volume.ae are disjoint. This means that there exists a residual set of Lebesgue measure zero (e.g., the set of Liouville numbers).