File tree 3 files changed +1
-74
lines changed
3 files changed +1
-74
lines changed Original file line number Diff line number Diff line change @@ -2494,7 +2494,6 @@ import Mathlib.NumberTheory.Multiplicity
2494
2494
import Mathlib.NumberTheory.NumberField.Basic
2495
2495
import Mathlib.NumberTheory.NumberField.CanonicalEmbedding
2496
2496
import Mathlib.NumberTheory.NumberField.ClassNumber
2497
- import Mathlib.NumberTheory.NumberField.Discriminant
2498
2497
import Mathlib.NumberTheory.NumberField.Embeddings
2499
2498
import Mathlib.NumberTheory.NumberField.Norm
2500
2499
import Mathlib.NumberTheory.NumberField.Units
Load Diff This file was deleted.
Original file line number Diff line number Diff line change @@ -3,9 +3,9 @@ Copyright (c) 2021 Riccardo Brasca. All rights reserved.
3
3
Released under Apache 2.0 license as described in the file LICENSE.
4
4
Authors: Riccardo Brasca
5
5
-/
6
- import Mathlib.NumberTheory.NumberField.Basic
7
6
import Mathlib.RingTheory.Trace
8
7
import Mathlib.RingTheory.Norm
8
+ import Mathlib.NumberTheory.NumberField.Basic
9
9
10
10
#align_import ring_theory.discriminant from "leanprover-community/mathlib" @"3e068ece210655b7b9a9477c3aff38a492400aa1"
11
11
@@ -376,21 +376,6 @@ end Integral
376
376
377
377
end Field
378
378
379
- section Int
380
-
381
- end Int
382
-
383
- /-- Two (finite) ℤ-basis have the same discriminant. -/
384
- theorem discr_eq_discr [Fintype ι] (b : Basis ι ℤ A) (b' : Basis ι ℤ A) :
385
- Algebra.discr ℤ b = Algebra.discr ℤ b' := by
386
- convert Algebra.discr_of_matrix_vecMul b' (b'.toMatrix b)
387
- · rw [Basis.toMatrix_map_vecMul]
388
- · suffices IsUnit (b'.toMatrix b).det by
389
- rw [Int.isUnit_iff, ← sq_eq_one_iff] at this
390
- rw [this, one_mul]
391
- rw [← LinearMap.toMatrix_id_eq_basis_toMatrix b b']
392
- exact LinearEquiv.isUnit_det (LinearEquiv.refl ℤ A) b b'
393
-
394
379
end Discr
395
380
396
381
end Algebra
You can’t perform that action at this time.
0 commit comments