We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
1 parent 663964d commit 12364fcCopy full SHA for 12364fc
Mathlib/NumberTheory/NumberField/Units/Regulator.lean
@@ -77,7 +77,7 @@ theorem abs_det_eq_abs_det (u : Fin (rank K) → (𝓞 K)ˣ)
77
-- And `g` corresponds to the restriction of `f⁻¹` to `{w // w ≠ w₂}`
78
let g : {w // w ≠ w₂} ≃ Fin (rank K) :=
79
(Equiv.subtypeEquiv f.symm (fun _ ↦ by simp [f])).trans
80
- (finSuccAboveEquiv (f.symm w₂)).toEquiv.symm
+ (finSuccAboveEquiv (f.symm w₂)).symm
81
have h_col := congr_arg abs <| Matrix.det_permute (g.trans e₂.symm)
82
(Matrix.of fun i w : {w // w ≠ w₂} ↦ (mult w.val : ℝ) * (w.val (u (e₂ i) : K)).log)
83
rw [abs_mul, ← Int.cast_abs, Equiv.Perm.sign_abs, Int.cast_one, one_mul] at h_col
0 commit comments