Documentation

FormalConjectures.ErdosProblems.«326»

Erdős Problem 326 #

Reference: erdosproblems.com/326

theorem erdos_326 :
(∀ (A : Set ), A.IsAddBasisOfOrder 2∃ (b : ), StrictMono b ∀ (n : ), b n A (Set.range b).IsAddBasis ∀ (x : ), ¬Filter.Tendsto (fun (n : ) => (b n) / n ^ 2) Filter.atTop (nhds x)) sorry

Let $A \subset \mathbb{N}$ be an additive basis of order 2.

Must there exist $B = \{b_1 < b_2 < \dots\} \subseteq A$ which is also a basis such that $\lim_{k\to\infty} \frac{b_k}{k^2}$ does not exist?

theorem erdos_326.variants.eq :
(∀ (A : Set ), A.IsAddBasisOfOrder 2∃ (a : ), StrictMono a Set.range a = A ∀ (x : ), ¬Filter.Tendsto (fun (n : ) => (a n) / n ^ 2) Filter.atTop (nhds x)) False

Erdős originally asked whether this was true with A = B, but this was disproved by Cassels.