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 elements of we can find 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:
Last updated: Dec 20 2023 at 11:08 UTC