Zulip Chat Archive

Stream: Is there code for X?

Topic: Algebra.norm ℤ


Andrew Yang (Sep 27 2023 at 07:06):

Do we have this somewhere? Is there an easy proof to it?

import Mathlib.NumberTheory.NumberField.Norm

open scoped NumberField

example {K : Type*} [Field K] [NumberField K] (x : 𝓞 K) :
  Algebra.norm  x = Algebra.norm  (x : K) := sorry

Riccardo Brasca (Sep 27 2023 at 07:52):

Not sure it is literally this, but docs#RingOfIntegers.norm_apply_coe should be very close.

Riccardo Brasca (Sep 27 2023 at 07:52):

In any case docs#RingOfIntegers.norm is there exactly to consider the norm of an element of the ring of integers

Andrew Yang (Sep 27 2023 at 08:32):

RingOfIntegers.normis defined by restricting Algebra.norm K onto 𝓞 K, but I don't think we know that it is equal to Algebra.norm (𝓞 K).

Xavier Roblot (Sep 27 2023 at 08:36):

I think what you want is docs#Algebra.norm_localization

Riccardo Brasca (Sep 27 2023 at 08:40):

(deleted)

Riccardo Brasca (Sep 27 2023 at 08:42):

Ah yes, sorry. I am always a little bit worried about Algebra.norm K, since in the relative case it is not the right notion.

Andrew Yang (Sep 27 2023 at 10:47):

Xavier Roblot said:

I think what you want is docs#Algebra.norm_localization

Thanks! Works like a charm.


Last updated: Dec 20 2023 at 11:08 UTC