Zulip Chat Archive
Stream: Is there code for X?
Topic: Ramification iff divides discriminant
Gareth Ma (Nov 14 2024 at 13:56):
Does the following theorem exist?
For non-infinite primes of number fields, it seems that there is no direct notion for "a prime ramifies". Should it exist or is Mathlib happy with 0 < ramificationIdx something
?
Andrew Yang (Nov 14 2024 at 14:13):
It’s essentially docs#pow_sub_one_dvd_differentIdeal
Riccardo Brasca (Nov 14 2024 at 14:14):
In flt-regular
we have a notion of being unramified at a prime. We didn't need connection with the discriminant, but all the prerequisites are there.
Andrew Yang (Nov 14 2024 at 14:14):
Andrew Yang said:
It’s essentially docs#pow_sub_one_dvd_differentIdeal
(at least one direction of it)
Thomas Browning (Nov 14 2024 at 14:14):
Andrew Yang said:
It’s essentially docs#pow_sub_one_dvd_differentIdeal
Does that tell you that ramify implies divides discriminant, but not divides discriminant implies ramifies?
Thomas Browning (Nov 14 2024 at 14:15):
For something I'm working on, I'll need to know that every number field has at least one ramified prime, which requires the opposite direction.
Riccardo Brasca (Nov 14 2024 at 14:15):
I think it's time to have the discriminant ideal!
Riccardo Brasca (Nov 14 2024 at 14:16):
Thomas Browning said:
For something I'm working on, I'll need to know that every number field has at least one ramified prime, which requires the opposite direction.
Note that the hard part of this result, Minkowski bound, is in mathlib.
Gareth Ma (Nov 14 2024 at 14:17):
In fact there's
Mathlib/NumberTheory/NumberField/Discriminant/Basic.lean
18:* `NumberField.abs_discr_gt_two`: **Hermite-Minkowski Theorem**. A nontrivial number field has
192:theorem abs_discr_gt_two (h : 1 < finrank ℚ K) : 2 < |discr K| := by
Gareth Ma (Nov 14 2024 at 14:19):
(I saw this but nothing like "Q has no unramified extensions", hence this question.) I think the IsUnramified{At}
notion from flt-regular should be brought to Mathlib, seems natural at least to me
Riccardo Brasca (Nov 14 2024 at 14:19):
Yes, I mean we know all we need about the discriminant, we are missing the connection between the discriminant and remification.
Riccardo Brasca (Nov 14 2024 at 14:19):
If you want to PR those results please feel free to do so
Riccardo Brasca (Nov 14 2024 at 14:20):
I am in the process of moving stuff from flt-regular
to mathlib, but currently working on other results
Gareth Ma (Nov 14 2024 at 14:20):
Oh yeah I just meant even the Minkowski bound => discr > 1 part is done :D
Gareth Ma (Nov 14 2024 at 14:20):
I'm probably not free to do it myself, sorry :(
Riccardo Brasca (Nov 14 2024 at 14:20):
But I don't think we should spend too much time with the discriminant as an integer, we need the ideal
Riccardo Brasca (Nov 14 2024 at 14:21):
And this does not exist I think
Riccardo Brasca (Nov 14 2024 at 14:22):
@Andrew Yang you mentionned that someone else was working on improving the status of primeOver
or something similar. Is this done?
Andrew Yang (Nov 14 2024 at 14:39):
I belieive the mathlib counter part for primeOver
is docs#Ideal.LiesOver. And I think @Thomas Browning's frobenius element work will give a better framework for the remaining parts of galoisPrime.lean too.
Kevin Buzzard (Nov 14 2024 at 21:59):
PS the hypothesis that B is free as an A-module is not necessary. I'm guessing that Milne (incorrectly) only defines the discriminant in this situation?
Riccardo Brasca (Nov 14 2024 at 22:51):
We have a lot of places where we can remove freeness :(
David Loeffler (Nov 15 2024 at 05:16):
Kevin Buzzard said:
PS the hypothesis that B is free as an A-module is not necessary. I'm guessing that Milne (incorrectly) only defines the discriminant in this situation?
"Incorrectly" is a bit harsh; maybe his results are not maximally general, but that doesn't mean they aren't correct, and clearly the most important case is A = ZZ
.
Gareth Ma (Nov 15 2024 at 16:27):
Kevin Buzzard said:
PS the hypothesis that B is free as an A-module is not necessary. I'm guessing that Milne (incorrectly) only defines the discriminant in this situation?
Correct!
Gareth Ma (Nov 15 2024 at 16:28):
But as David said is important and PID most of the time
Gareth Ma (Nov 15 2024 at 16:31):
Ahh but I guess a subsequent question I should ask first is does anyone have an introductory reference that also removes the hypothesis?
Riccardo Brasca (Nov 15 2024 at 16:34):
In general you take all integral bases of L
as K
-vector space, and the discriminant lies in 𝓞 K
. You don't need 𝓞 L
to be free as 𝓞 K
-module.
Riccardo Brasca (Nov 15 2024 at 16:37):
It's called the "relative discriminant". Neukirch surely explains it
Riccardo Brasca (Nov 15 2024 at 16:39):
You can also look at "Local Fields", chapter II for a more abstract approach
Gareth Ma (Nov 15 2024 at 16:40):
:man_facepalming: how did I forget about Neukirch. (p.201)
Gareth Ma (Nov 15 2024 at 16:41):
Random side note, but Wikipedia has a section on it as well, but their field extension is somehow and adjacent things written a bit weirdly :/
Gareth Ma (Nov 16 2024 at 10:53):
I guess this is a Lean/Mathlib question rather than a math question, but are there better ways to write relDiscr
? And is the discr ℤ (integralBasis K)
part correct?
import Mathlib
open NumberField Algebra
-- Relative discriminant (ideal) of field extension L/K
set_option linter.unusedVariables false
def relDiscr (L K : Type*) [Field K] [Field L] [Algebra K L] : Ideal (𝓞 K) :=
Ideal.span { d |
∃ (ι : Type*) (inst₁ : DecidableEq ι) (inst₂ : Fintype ι) (b : Basis ι K L),
∀ i, IsIntegral K (b i) ∧ discr K b = d }
-- Relative discriminant of K/ℚ is just principal ideal of absolute discriminant disc(K)
example (K : Type*) [Field K] [NumberField K] :
(relDiscr K ℚ).map Rat.ringOfIntegersEquiv = Ideal.span { discr ℤ (integralBasis K) } := by
sorry
Riccardo Brasca (Nov 16 2024 at 11:34):
Note that we also have NumberField.discr
Riccardo Brasca (Nov 16 2024 at 11:36):
For the absolute discriminant you should definitely use that
Gareth Ma (Nov 16 2024 at 11:37):
Yes, sorry I didn't know that haha
Riccardo Brasca (Nov 16 2024 at 11:38):
For the relative one I am not sure. Maybe we can go via the different
Riccardo Brasca (Nov 16 2024 at 11:39):
cc @Xavier Roblot
Xavier Roblot (Nov 16 2024 at 12:45):
I would use a definition similar to the one you give for the relative discriminant but for all families, not just bases.
import Mathlib
open NumberField Algebra
open Classical in
def relDiscr (L K : Type*) [Field K] [Field L] [Algebra K L] : Ideal (𝓞 K) :=
Ideal.span { d | ∃ (ι : Type*) (_ : Fintype ι) (v : ι → 𝓞 L),
Algebra.discr K (fun i ↦ (v i : L)) = d }
Kevin Buzzard (Nov 16 2024 at 15:04):
I think differents exist in some huge generality. Aren't they used in the theory of finite flat group schemes?
Andrew Yang (Nov 16 2024 at 15:22):
What's the definition in that case? The annihilator of the sheaf of differentials?
Kevin Buzzard (Nov 16 2024 at 16:19):
I have some old notes of Conrad where he goes through all this and my instinct is to refer you to these, but they appear to be no longer on his website. When I get home later I'll see if I can dig them out.
Kevin Buzzard (Nov 16 2024 at 17:29):
Sorry for the delay -- home now. This is from Conrad--Lieblich "Galois Representations Arising from p-Divisible Groups", a mythical text which Brian seems to have removed from his website. I have no idea whether it got published.
Screenshot from 2024-11-16 17-27-41.png
Kevin Buzzard (Nov 16 2024 at 17:34):
I don't know of any published reference which works in this generality, I'm just saying I trust Brian.
Andrew Yang (Nov 16 2024 at 17:42):
I managed to find the same text at Lieblich’s website here.
Riccardo Brasca (Nov 19 2024 at 12:02):
Riccardo Brasca said:
We have a lot of places where we can remove freeness :(
See for example #19244 for a generalization of the relative norm
Antoine Chambert-Loir (Nov 19 2024 at 20:32):
The reference I would have looked at for these questions is the old paper by Mazur and Roberts (1970), “Local Euler Characteristics” , Invent. Math. 9, p. 201–234. doi:10.1007/BF01404325 The appendix should be something like that.
Andrew Yang (Feb 17 2025 at 16:02):
@Thomas Browning said:
For something I'm working on, I'll need to know that every number field has at least one ramified prime, which requires the opposite direction.
Are there any updates on this? Both divides discriminant => ramified and Q has no nontrivial unramified extensions.
Riccardo Brasca (Feb 17 2025 at 16:15):
I didn't see anything related to this recently.
Riccardo Brasca (Feb 17 2025 at 16:19):
Waiting for the PR :stuck_out_tongue:
Thomas Browning (Feb 17 2025 at 18:23):
No, I'm not aware of any progress on this. But there is progress on inertia groups with #20899 and #21770.
Andrew Yang (Feb 17 2025 at 18:24):
I’ll try to think about this then.
Last updated: May 02 2025 at 03:31 UTC