Zulip Chat Archive

Stream: maths

Topic: Erdős–Ginzburg–Ziv theorem


Yaël Dillies (Jan 04 2023 at 21:53):

As a followup to Kneser's addition theorem, I thought I would give a stab at Erdős–Ginzburg–Ziv, which says that among any 2p12p - 1 elements of Z/pZℤ/pℤ we can find pp elements of sum zero.

Yaël Dillies (Jan 04 2023 at 21:58):

And I just finished the proof! #18063

/-- The **Erdős–Ginzburg–Ziv theorem**: Any (not necessarily distinct) `2 * p - 1` elements of
`zmod p` contain `p` elements whose sum is zero. -/
lemma zmod.exists_le_sum_eq_zero {p : } [fact p.prime] {s : multiset (zmod p)} (hs : s.card = 2 * p - 1) :
    t  s, t.card = p  t.sum = 0 :=
...

#print axioms zmod.exists_le_sum_eq_zero
/-
propext
quot.sound
classical.choice
-/

Yaël Dillies (Jan 04 2023 at 21:59):

This to me is quite interesting, because I used the Chevalley-Warning proof, and AFAIK this is the first ever application of docs#char_dvd_card_solutions_family.

Yaël Dillies (Jan 04 2023 at 22:03):

Thank you, 2019 @Johan Commelin, for proving Chevalley-Warning :smile:

Johan Commelin (Jan 05 2023 at 06:45):

@Yaël Dillies Your welcome! :smiley:

Antoine Chambert-Loir (Feb 11 2024 at 14:05):

Two late comments, @Yaël Dillies :

  1. As the proof of docs#char_dvd_card_solutions_of_sum_lt indicates, the theorem for one polynomial and its version for a family are elementary equivalent.
  2. There is a version of EGZ for integers: If n>0n>0 is an integer, among 2n12n-1 integers, one can find nn of them whose sum is divisible by nn.

Yaël Dillies (Feb 11 2024 at 14:13):

  1. How is that relevant to EGZ?
  2. I am aware, and in fact I have an almost complete proof of this fact in LeanCamCombi.

Yaël Dillies (Feb 11 2024 at 14:14):

If you're interested in reviewing EGZ, I can PR it soon and tag you

Antoine Chambert-Loir (Feb 11 2024 at 14:26):

(For 1 : it is just that you say this might be the only application of the CW-theorem for several polynomials )

Yaël Dillies (Feb 11 2024 at 14:27):

Oh that's not what I meant. I meant this is the first application of CW, all versions included.

Antoine Chambert-Loir (Feb 11 2024 at 14:36):

Well, CW has a few classical applications!
One of them is the proof that all finite fields are commutative (using the reduced norm), or to the theory of quadratic forms over finite fields (which are thus automatically isotropic in dimension 3\geq3…)
There are also combinatorical applications : how many hyperplanes are needed to cover the affine space over a finite field? and if you insist that these hyperplanes avoid the origin?
And applications in code theory.
Maybe more importantly, it relates the geometric properties of an algebraic variety with the presence of rational points, and is directly a motivation to quite fundamental questions in arithmetic geometry (papers by Ax, Katz, Esnault, Fakhruddin-Rajan…)

Yaël Dillies (Feb 11 2024 at 14:38):

In mathlib! I mean first application in mathlib.

Yaël Dillies (Feb 11 2024 at 14:39):

Sorry, clearly I haven't been very clear :grinning:

Antoine Chambert-Loir (Feb 11 2024 at 16:12):

That's OK ! — I'm a bit too “milky soup” these times…


Last updated: May 02 2025 at 03:31 UTC