Documentation

FormalConjectures.ErdosProblems.«509»

Erdős Problem 509 #

Reference: erdosproblems.com/509

structure BoundedDiscCover {M : Type u} [MetricSpace M] (S : Set M) (r : ) (ι : Type v) :
Type (max u v)

An $r$-bounded disc cover of a subset of a metric space $M$ is an indexed family of closed discs whose radii sum to at most $r$.

Instances For
    noncomputable def boundedDiscCover_empty {M : Type u} [MetricSpace M] [Nonempty M] (r : ) (hr : 0 < r) :
    Equations
    Instances For
      theorem BoundedDiscCover.bound_nonneg_of_nonempty {M : Type u} [MetricSpace M] (S : Set M) (hS : S.Nonempty) (r : ) (ι : Type v) (bdc : BoundedDiscCover S r ι) :
      0 < r
      theorem erdos_509 :
      (∀ (f : Polynomial ), f.Monicf.natDegree 0∃ (ι : Type), Nonempty (BoundedDiscCover {z : | Polynomial.eval z f 1} 2 ι)) sorry

      Let $f(z) ∈ ℂ[z]$ be a monic non-constant polynomial. Can the set $\{z ∈ ℂ : |f(z)| ≤ 1\}$ be covered by a set of closed discs the sum of whose radii is $≤ 2$?

      Let $f(z) ∈ ℂ[z]$ be a monic non-constant polynomial. Can the set $\{z ∈ ℂ : |f(z)| ≤ 1\}$ be covered by a set of closed discs the sum of whose radii is ≤2e? Solution: True. This is due to Cartan. See Sur les systèmes de fonctions holomorphes à variétés linéaires lacunaires et leurs applications, Henri Cartan, http://www.numdam.org/article/ASENS_1928_3_45__255_0.pdf

      Let $f(z) ∈ ℂ[z]$ be a monic non-constant polynomial. Can the set $\{z ∈ ℂ : |f(z)| ≤ 1\}$ be covered by a set of closed discs the sum of whose radii is $≤ 2.59$? Solution: True. This is due to Pommerenke.

      Let $f(z) ∈ ℂ[z]$ be a monic non-constant polynomial. If it is connected, can the set $\{z ∈ C : |f(z)| ≤ 1\}$ be covered by a set of circles the sum of whose radii is $≤ 2$? Solution: True. This is due to Pommerenke.