The Ruzsa-Szemerédi problem #
This file proves the lower bound of the Ruzsa-Szemerédi problem. The problem is to find the maximum
number of edges that a graph on n
vertices can have if all edges belong to at most one triangle.
The lower bound comes from turning the big 3AP-free set from Behrend's construction into a graph that has the property that every triangle gives a (possibly trivial) arithmetic progression on the original set.
Main declarations #
ruzsaSzemerediNumberNat n
: Maximum number of edges a graph onn
vertices can have such that each edge belongs to exactly one triangle.ruzsaSzemerediNumberNat_asymptotic_lower_bound
: There exists a graph withn
vertices andΩ((n ^ 2 * exp (-4 * sqrt (log n))))
edges such that each edge belongs to exactly one triangle.
The Ruzsa-Szemerédi number #
The Ruzsa-Szemerédi number of a fintype is the maximum number of edges a locally linear graph on that type can have.
In other words, ruzsaSzemerediNumber α
is the maximum number of edges a graph on α
can have such
that each edge belongs to exactly one triangle.
Equations
- ruzsaSzemerediNumber α = Nat.findGreatest (fun (m : ℕ) => ∃ (G : SimpleGraph α) (x : DecidableRel G.Adj), (G.cliqueFinset 3).card = m ∧ G.LocallyLinear) ((Fintype.card α).choose 3)
Instances For
The n
-th Ruzsa-Szemerédi number is the maximum number of edges a locally linear graph on
n
vertices can have.
In other words, ruzsaSzemerediNumberNat n
is the maximum number of edges a graph on n
vertices
can have such that each edge belongs to exactly one triangle.
Equations
Instances For
The Ruzsa-Szemerédi construction #
Lower bound on the Ruzsa-Szemerédi problem in terms of 3AP-free sets.
If there exists a 3AP-free subset of [1, ..., (n - 3) / 6]
of size m
, then there exists a graph
with n
vertices and (n / 3 - 2) * m
edges such that each edge belongs to exactly one triangle.
Explicit lower bound on the Ruzsa-Szemerédi problem.
There exists a graph with n
vertices and
(n / 3 - 2) * (n - 3) / 6 * exp (-4 * sqrt (log ((n - 3) / 6)))
edges such that each edge belongs
to exactly one triangle.
Asymptotic lower bound on the Ruzsa-Szemerédi problem.
There exists a graph with n
vertices and Ω((n ^ 2 * exp (-4 * sqrt (log n))))
edges such that
each edge belongs to exactly one triangle.