Skip to content

Commit

Permalink
fix(LinearAlgebra/{Free,Tensor,Clifford}Algebra): remove an unused `S…
Browse files Browse the repository at this point in the history
…MulCommClass` argument (#8373)

`SMulCommClass R S A` is always true when `Algebra R A` and `Algebra S A` and `A` is commutative, since the two actions factor via multiplication in `A`. I don't think mathlib actually knows this fact yet, but in this particular case it's also true by definition.
  • Loading branch information
eric-wieser committed Nov 12, 2023
1 parent 4cb02b4 commit 30d39f9
Show file tree
Hide file tree
Showing 3 changed files with 3 additions and 4 deletions.
3 changes: 1 addition & 2 deletions Mathlib/Algebra/FreeAlgebra.lean
Expand Up @@ -281,8 +281,7 @@ instance {R S A} [CommSemiring R] [CommSemiring S] [CommSemiring A]
simp only [Algebra.algebraMap_eq_smul_one, smul_eq_mul]
rw [smul_assoc, ←smul_one_mul]

instance {R S A} [CommSemiring R] [CommSemiring S] [CommSemiring A]
[Algebra R A] [Algebra S A] [SMulCommClass R S A] :
instance {R S A} [CommSemiring R] [CommSemiring S] [CommSemiring A] [Algebra R A] [Algebra S A] :
SMulCommClass R S (FreeAlgebra A X) where
smul_comm r s x := smul_comm (algebraMap R A r) (algebraMap S A s) x

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/LinearAlgebra/CliffordAlgebra/Basic.lean
Expand Up @@ -97,7 +97,7 @@ instance instAlgebra : Algebra R (CliffordAlgebra Q) := instAlgebra' _

instance {R S A M} [CommSemiring R] [CommSemiring S] [AddCommGroup M] [CommRing A]
[Algebra R A] [Algebra S A] [Module R M] [Module S M] [Module A M] (Q : QuadraticForm A M)
[IsScalarTower R A M] [IsScalarTower S A M] [SMulCommClass R S A] :
[IsScalarTower R A M] [IsScalarTower S A M] :
SMulCommClass R S (CliffordAlgebra Q) :=
RingQuot.instSMulCommClass _

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/LinearAlgebra/TensorAlgebra/Basic.lean
Expand Up @@ -81,7 +81,7 @@ example : (algebraNat : Algebra ℕ (TensorAlgebra R M)) = instAlgebra := rfl

instance {R S A M} [CommSemiring R] [CommSemiring S] [AddCommMonoid M] [CommSemiring A]
[Algebra R A] [Algebra S A] [Module R M] [Module S M] [Module A M]
[IsScalarTower R A M] [IsScalarTower S A M] [SMulCommClass R S A] :
[IsScalarTower R A M] [IsScalarTower S A M] :
SMulCommClass R S (TensorAlgebra A M) :=
RingQuot.instSMulCommClass _

Expand Down

0 comments on commit 30d39f9

Please sign in to comment.