Skip to content

Commit

Permalink
Update Mathlib/LinearAlgebra/Matrix/FixedDetMatrices.lean
Browse files Browse the repository at this point in the history
Co-authored-by: Ruben Van de Velde <[email protected]>
  • Loading branch information
CBirkbeck and Ruben-VandeVelde authored Oct 13, 2024
1 parent b0d1950 commit e63df39
Showing 1 changed file with 2 additions and 6 deletions.
8 changes: 2 additions & 6 deletions Mathlib/LinearAlgebra/Matrix/FixedDetMatrices.lean
Original file line number Diff line number Diff line change
Expand Up @@ -43,12 +43,8 @@ lemma smul_def (m : R) (g : SpecialLinearGroup n R) (A : (FixedDetMatrix n R m))
rfl

instance (m : R) : MulAction (SpecialLinearGroup n R) (FixedDetMatrix n R m) where
smul := fun g A => g • A
one_smul := by intro b; rw [smul_def]; simp only [coe_one, one_mul, Subtype.coe_eta]
mul_smul := by
intro x y b
simp_rw [smul_def, ← mul_assoc]
rfl
one_smul b := by rw [smul_def]; simp only [coe_one, one_mul, Subtype.coe_eta]
mul_smul x y b := by simp_rw [smul_def, ← mul_assoc, coe_mul]

lemma smul_coe (m : R) (g : SpecialLinearGroup n R) (A : FixedDetMatrix n R m) :
(g • A).1 = g * A.1 := by
Expand Down

0 comments on commit e63df39

Please sign in to comment.