Skip to content

Commit

Permalink
perf(Matrix.SpecialLinearGroup): clean up with dsimp first (#10738)
Browse files Browse the repository at this point in the history
This reduces the number of instructions by over a third using `dsimp` to clean up an expression before starting a proof.
  • Loading branch information
mattrobball committed Feb 20, 2024
1 parent c39e9ef commit c9eb34f
Showing 1 changed file with 1 addition and 0 deletions.
1 change: 1 addition & 0 deletions Mathlib/LinearAlgebra/Matrix/SpecialLinearGroup.lean
Original file line number Diff line number Diff line change
Expand Up @@ -311,6 +311,7 @@ def center_equiv_rootsOfUnity' (i : n) :
obtain ⟨⟨a, _⟩, ha⟩ := a
refine SetCoe.ext <| Units.eq_iff.mp <| by simp
map_mul' A B := by
dsimp
ext
simp only [Submonoid.coe_mul, coe_mul, rootsOfUnity.val_mkOfPowEq_coe, Units.val_mul]
rw [← scalar_eq_coe_self_center A i, ← scalar_eq_coe_self_center B i]
Expand Down

0 comments on commit c9eb34f

Please sign in to comment.