Zulip Chat Archive
Stream: maths
Topic: gal of cyclotomic polynomial
Eric Rodriguez (May 13 2021 at 06:56):
Hey all, I'm trying to work on the Galois group of cyclotomic polynomials. However, I'm stuck at the starting block; just defining the damn thing causes a deterministic timeout:
import field_theory.polynomial_galois_group
import ring_theory.polynomial.cyclotomic
open polynomial
variables {F : Type*} [field F] (n : ℕ)
noncomputable def cyclotomic_gal_hom : (cyclotomic n F).gal →* units (zmod n) := sorry
--timeout
anyone have any clue what I'm doing wrong, or how to get around it?
Johan Commelin (May 13 2021 at 06:59):
This is instant:
lemma cyclotomic_gal_hom : (cyclotomic n F).gal →* units (zmod n) := _
so there is something silly going on with elaboration
Eric Rodriguez (May 13 2021 at 07:04):
even specializing to ℚ doesn't lead anywhere :/ how do we usually get around elaboration issues like these?
Johan Commelin (May 13 2021 at 07:04):
Once you have filled in the definition, switching back from lemma
to def
usually works
Johan Commelin (May 13 2021 at 07:05):
It's a bit annoying...
Eric Rodriguez (May 13 2021 at 07:05):
yikes, I'll try that though and hopefully no more issues
Johan Commelin (May 13 2021 at 07:06):
it might be that Lean is trying to figure out whether you correctly marked the def
as noncomputable
Johan Commelin (May 13 2021 at 07:06):
and that is taking a long time. But it should just give up, because of the sorry
Johan Commelin (May 13 2021 at 07:06):
But I'm just guessing...
Kevin Buzzard (May 13 2021 at 08:29):
I think Johan is right but this is really hard to minimise (i.e. get an example which is independent of mathlib)
Riccardo Brasca (May 13 2021 at 08:53):
I don't if this is relevant, but maybe the definition of cyclotomic polynomial should be irreducible, or something like that (all the basic properties are in the API, but the definition is rather unnatural, using cyclotomic'
).
Last updated: Dec 20 2023 at 11:08 UTC