The Cauchy-Davenport theorem #
This file proves a generalisation of the Cauchy-Davenport theorem to arbitrary groups.
Cauchy-Davenport provides a lower bound on the size of s + t
in terms of the sizes of s
and t
,
where s
and t
are nonempty finite sets in a monoid. Precisely, it says that
|s + t| ≥ |s| + |t| - 1
unless the RHS is bigger than the size of the smallest nontrivial subgroup
(in which case taking s
and t
to be that subgroup would yield a counterexample). The motivating
example is s = {0, ..., m}
, t = {0, ..., n}
in the integers, which gives
s + t = {0, ..., m + n}
and |s + t| = m + n + 1 = |s| + |t| - 1
.
There are two kinds of proof of Cauchy-Davenport:
- The first one works in linear orders by writing
a₁ < ... < aₖ
the elements ofs
,b₁ < ... < bₗ
the elements oft
, and arguing thata₁ + b₁ < ... < aₖ + b₁ < ... < aₖ + bₗ
are distinct elements ofs + t
. - The second one works in groups by performing an "e-transform". In an abelian group, the
e-transform replaces
s
andt
bys ∩ g • s
andt ∪ g⁻¹ • t
. For a suitably choseng
, this decreases|s + t|
and keeps|s| + |t|
the same. In a general group, we use a trickier e-transform (in fact, a pair of e-transforms), but the idea is the same.
Main declarations #
cauchy_davenport_minOrder_mul
: A generalisation of the Cauchy-Davenport theorem to arbitrary groups.cauchy_davenport_of_isTorsionFree
: The Cauchy-Davenport theorem in torsion-free groups.ZMod.cauchy_davenport
: The Cauchy-Davenport theorem forZMod p
.cauchy_davenport_mul_of_linearOrder_isCancelMul
: The Cauchy-Davenport theorem in linear ordered cancellative semigroups.
TODO #
Version for circle
.
References #
- Matt DeVos, On a generalization of the Cauchy-Davenport theorem
Tags #
additive combinatorics, number theory, sumset, cauchy-davenport
General case #
A generalisation of the Cauchy-Davenport theorem to arbitrary groups. The size of s * t
is
lower-bounded by |s| + |t| - 1
unless this quantity is greater than the size of the smallest
subgroup.
A generalisation of the Cauchy-Davenport theorem to arbitrary groups. The size of
s + t
is lower-bounded by |s| + |t| - 1
unless this quantity is greater than the size of the
smallest subgroup.
The Cauchy-Davenport Theorem for torsion-free groups. The size of s * t
is lower-bounded
by |s| + |t| - 1
.
The Cauchy-Davenport theorem for torsion-free groups. The size of s + t
is lower-bounded
by |s| + |t| - 1
.
$$ℤ/nℤ$$ #
The Cauchy-Davenport Theorem. If s
, t
are nonempty sets in $$ℤ/pℤ$$, then the size of
s + t
is lower-bounded by |s| + |t| - 1
, unless this quantity is greater than p
.
Linearly ordered cancellative semigroups #
The Cauchy-Davenport Theorem for linearly ordered cancellative semigroups. The size of
s * t
is lower-bounded by |s| + |t| - 1
.
The Cauchy-Davenport theorem for linearly ordered additive cancellative semigroups. The size of
s + t
is lower-bounded by |s| + |t| - 1
.