THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
(Implementation detail).
The function underlying (A ⊗[R] matrix n n R) →ₐ[R] matrix n n A
,
as an R
-bilinear map.
Equations
- matrix_equiv_tensor.to_fun_bilinear R A n = (algebra.lsmul R (matrix n n A)).to_linear_map.compl₂ (algebra.linear_map R A).map_matrix
(Implementation detail).
The function underlying (A ⊗[R] matrix n n R) →ₐ[R] matrix n n A
,
as an R
-linear map.
Equations
The function (A ⊗[R] matrix n n R) →ₐ[R] matrix n n A
, as an algebra homomorphism.
(Implementation detail.)
The bare function matrix n n A → A ⊗[R] matrix n n R
.
(We don't need to show that it's an algebra map, thankfully --- just that it's an inverse.)
Equations
- matrix_equiv_tensor.inv_fun R A n M = finset.univ.sum (λ (p : n × n), M p.fst p.snd ⊗ₜ[R] matrix.std_basis_matrix p.fst p.snd 1)
(Implementation detail)
The equivalence, ignoring the algebra structure, (A ⊗[R] matrix n n R) ≃ matrix n n A
.
Equations
- matrix_equiv_tensor.equiv R A n = {to_fun := ⇑(matrix_equiv_tensor.to_fun_alg_hom R A n), inv_fun := matrix_equiv_tensor.inv_fun R A n _inst_5, left_inv := _, right_inv := _}
The R
-algebra isomorphism matrix n n A ≃ₐ[R] (A ⊗[R] matrix n n R)
.
Equations
- matrix_equiv_tensor R A n = {to_fun := (matrix_equiv_tensor.to_fun_alg_hom R A n).to_fun, inv_fun := (matrix_equiv_tensor.equiv R A n).inv_fun, left_inv := _, right_inv := _, map_mul' := _, map_add' := _, commutes' := _}.symm