Documentation

FormalConjectures.ErdosProblems.«228»

Erdős Problem 228 #

Reference: erdosproblems.com/228

theorem erdos_228 :
(∃ (c₁ : ) (c₂ : ), ∀ᶠ (n : ) in Filter.atTop, ∃ (p : Polynomial ), p.degree = n (∀ in, p.coeff i = 1 p.coeff i = -1) ∀ (z : ), z = 1n < c₁ * Polynomial.eval z p Polynomial.eval z p < c₂ * n) True

Does there exist, for all large $n$, a polynomial $P$ of degree $n$, with coefficients $\pm1$, such that $$\sqrt n \ll |P(z)| \ll \sqrt n$$ for all $|z|=1$, with the implied constants independent of $z$ and $n$?

The answer is yes, proved by Balister, Bollobás, Morris, Sahasrabudhe, and Tiba [BBMST19].

[BBMST19] Balister, P. and Bollob'{A}s, B. and Morris, R. and Sahasrabudhe, J. and Tiba, M., Flat Littlewood Polynomials Exist. arXiv:907.09464 (2019).