Skip to content

Commit

Permalink
feat: add Algebra.coe_trace_int (#8513)
Browse files Browse the repository at this point in the history
From flt-regular.
  • Loading branch information
Ruben-VandeVelde committed Nov 20, 2023
1 parent c21c11f commit 7275625
Showing 1 changed file with 8 additions and 4 deletions.
12 changes: 8 additions & 4 deletions Mathlib/NumberTheory/NumberField/Norm.lean
Expand Up @@ -26,13 +26,17 @@ open scoped NumberField BigOperators

open Finset NumberField Algebra FiniteDimensional

section rat
section Rat

theorem Algebra.coe_norm_int {K : Type*} [Field K] [NumberField K] (x : π“ž K) :
Algebra.norm β„€ x = Algebra.norm β„š (x : K) :=
variable {K : Type*} [Field K] [NumberField K] (x : π“ž K)

theorem Algebra.coe_norm_int : (Algebra.norm β„€ x : β„š) = Algebra.norm β„š (x : K) :=
(Algebra.norm_localization (R := β„€) (Rβ‚˜ := β„š) (S := π“ž K) (Sβ‚˜ := K) (nonZeroDivisors β„€) x).symm

end rat
theorem Algebra.coe_trace_int : (Algebra.trace β„€ _ x : β„š) = Algebra.trace β„š K x :=
(Algebra.trace_localization (R := β„€) (Rβ‚˜ := β„š) (S := π“ž K) (Sβ‚˜ := K) (nonZeroDivisors β„€) x).symm

end Rat

namespace RingOfIntegers

Expand Down

0 comments on commit 7275625

Please sign in to comment.