Zulip Chat Archive
Stream: Is there code for X?
Topic: cancel division in polynomials
Eric Rodriguez (Mar 02 2022 at 10:56):
I currently have this result:
lemma cyclotomic_dvd_geom_sum_of_dvd {d n : ℕ} (hdn : d ∣ n) (hd : d ≠ 1) :
cyclotomic d ℤ ∣ geom_sum X n :=
I'd like to be able to derive (hd : d ∣ n) (hd0 : d ≠ 0) (hdn : d < n) : (cyclotomic n ℤ).eval q ∣ (q ^ n - 1) / (q ^ d - 1) (or well, the polynomial version) from this easily. However, I don't see any way to do this; div_by_monic doesn't seem to have any cancellation theorems at all! Is it just worth it to prove the appropriate result for geom_sum directly, instead?
Riccardo Brasca (Mar 02 2022 at 11:10):
I would avoid using /ₘ at all, and just providing the quotient explicitly.
Riccardo Brasca (Mar 02 2022 at 11:11):
By "explicitly" I mean using some other divisibility result, not the actual formula.
Riccardo Brasca (Mar 02 2022 at 11:13):
We know that q ^ d - 1 divides q ^ n - 1?
Eric Rodriguez (Mar 02 2022 at 11:23):
amazingly, it seems not
Riccardo Brasca (Mar 02 2022 at 11:26):
It's docs#commute.geom_sum₂_mul , isn't it? Take n = d, x = q ^(n/d) and y = 1 or something like that.
Riccardo Brasca (Mar 02 2022 at 11:31):
Why docs# doesn't work?! This theorem
Kevin Buzzard (Mar 02 2022 at 18:38):
because of the \_2 I believe
Last updated: May 02 2025 at 03:31 UTC