Skip to content

Commit 12364fc

Browse files
committed
fix
1 parent 663964d commit 12364fc

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

Mathlib/NumberTheory/NumberField/Units/Regulator.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -77,7 +77,7 @@ theorem abs_det_eq_abs_det (u : Fin (rank K) → (𝓞 K)ˣ)
7777
-- And `g` corresponds to the restriction of `f⁻¹` to `{w // w ≠ w₂}`
7878
let g : {w // w ≠ w₂} ≃ Fin (rank K) :=
7979
(Equiv.subtypeEquiv f.symm (fun _ ↦ by simp [f])).trans
80-
(finSuccAboveEquiv (f.symm w₂)).toEquiv.symm
80+
(finSuccAboveEquiv (f.symm w₂)).symm
8181
have h_col := congr_arg abs <| Matrix.det_permute (g.trans e₂.symm)
8282
(Matrix.of fun i w : {w // w ≠ w₂} ↦ (mult w.val : ℝ) * (w.val (u (e₂ i) : K)).log)
8383
rw [abs_mul, ← Int.cast_abs, Equiv.Perm.sign_abs, Int.cast_one, one_mul] at h_col

0 commit comments

Comments
 (0)