Skip to content

Commit

Permalink
more defeq
Browse files Browse the repository at this point in the history
  • Loading branch information
xroblot committed Sep 17, 2024
1 parent 974b8c5 commit fe7db50
Showing 1 changed file with 3 additions and 3 deletions.
6 changes: 3 additions & 3 deletions Mathlib/NumberTheory/NumberField/Units/Regulator.lean
Original file line number Diff line number Diff line change
Expand Up @@ -57,11 +57,11 @@ local instance : CommGroup (𝓞 K)ˣ := inferInstance
set_option maxSynthPendingDepth 2 -- Note this is active for the remainder of the file.

theorem regulator_eq_det' (e : {w : InfinitePlace K // w ≠ w₀} ≃ Fin (rank K)) :
regulator K = |(Matrix.of fun i ↦ (logEmbedding K) (fundSystem K (e i))).det| := by
regulator K = |(Matrix.of fun i ↦
logEmbedding K (Additive.ofMul (fundSystem K (e i)))).det| := by
simp_rw [regulator, ZLattice.covolume_eq_det _
(((basisModTorsion K).map (logEmbeddingEquiv K)).reindex e.symm), Basis.coe_reindex,
Function.comp_def, Basis.map_apply, ← fundSystem_mk, Equiv.symm_symm]
rfl
Function.comp_def, Basis.map_apply, ← fundSystem_mk, Equiv.symm_symm, logEmbeddingEquiv_apply]

/-- Let `u : Fin (rank K) → (𝓞 K)ˣ` be a family of units and let `w₁` and `w₂` be two infinite
places. Then, the two square matrices with entries `(mult w * log w (u i))_i, {w ≠ w_i}`, `i = 1,2`,
Expand Down

0 comments on commit fe7db50

Please sign in to comment.