Documentation

FormalConjectures.ErdosProblems.«480»

Erdős Problem 480 #

Reference: erdosproblems.com/480

theorem erdos_480 :
(∀ (x : ), (∀ (n : ), x n Set.Icc 0 1){x_1 : × | ∃ (m : ) (n : ) (_ : m 0) (_ : |x (m + n) - x n| 1 / (5 * n)), (m, n) = x_1}.Infinite) True

Let $x_1,x_2,...∈[0, 1]$ be an infinite sequence. Is it true that there are infinitely many $m, n$ such that $|x_{m+n} - x_n| ≤ \frac 1 {\sqrt 5 n}$?

This was proved Chung and Graham.

theorem erdos_480.variants.chung_graham :
let c := 1 + ∑' (k : ℕ+), 1 / (Nat.fib (2 * k)); IsGreatest {C : | C > 0 ∀ (x : ), (∀ (n : ), x n Set.Icc 0 1)εSet.Ioo 0 C, ∃ (n : ), {m : | m 0 |x (n + m) - x m| < 1 / ((C - ε) * n)}.Infinite} c

For any $ϵ>0$ there must exist some $n$ such that there are infinitely many $m$ for which $|x_{m+n} - x_m| < \frac 1 {(c−ϵ)n}$, where $c= 1 + \sum_{k≥1} \frac 1 {F_{2k}} =2.535370508...$ and $F_m$ is the $m$th Fibonacci number. This constant is best possible.