Zulip Chat Archive
Stream: new members
Topic: Ideas for proving this number theory lemma
Roshan Kohli (Dec 03 2023 at 17:14):
lemma binomial_coeff_div {n m : ℕ} (hp : Nat.gcd m p = 1) : Nat.choose (m * p ^ n) (p ^ n) ≡ m [MOD p] := by
I am trying to prove this lemma in lean. I have attempted to do it directly however I know I can prove this by considering the polynomial over the finite field of p elements. But I have no clue on to even get started in that direction. Any advice would be appreciated. Thanks!
Kevin Buzzard (Dec 03 2023 at 17:43):
Are you sure you need hp
?
I would prove it by induction on n.
Roshan Kohli (Dec 03 2023 at 17:56):
okay i'll give that a go
Joël Riou (Dec 03 2023 at 18:05):
It seems to me the formula is the particular case i = 1
for the congruence Nat.choose (m * p ^ n) (i * p ^ n) ≡ Nat.choose m i [MOD p]
. If I had to prove the particular case, I would try to prove the more general case (which itself seems to be a special case of Lucas's theorem), which I would do by studying powers of 1+X
in polynomial algebras over rings where the prime number p
vanishes (but I do not know enough of the internals of mathlib
for this area of mathematics...).
Last updated: Dec 20 2023 at 11:08 UTC