mathlib documentation

ring_theory.matrix_algebra

We show matrix n n A ≃ₐ[R] (A ⊗[R] matrix n n R).

def matrix_equiv_tensor.to_fun_bilinear (R : Type u) [comm_semiring R] (A : Type v) [semiring A] [algebra R A] (n : Type w) :
A →ₗ[R] matrix n n R →ₗ[R] matrix n n A

(Implementation detail). The function underlying (A ⊗[R] matrix n n R) →ₐ[R] matrix n n A, as an R-bilinear map.

Equations
@[simp]
theorem matrix_equiv_tensor.to_fun_bilinear_apply (R : Type u) [comm_semiring R] (A : Type v) [semiring A] [algebra R A] (n : Type w) (a : A) (m : matrix n n R) :
def matrix_equiv_tensor.to_fun_linear (R : Type u) [comm_semiring R] (A : Type v) [semiring A] [algebra R A] (n : Type w) :

(Implementation detail). The function underlying (A ⊗[R] matrix n n R) →ₐ[R] matrix n n A, as an R-linear map.

Equations
def matrix_equiv_tensor.to_fun_alg_hom (R : Type u) [comm_semiring R] (A : Type v) [semiring A] [algebra R A] (n : Type w) [decidable_eq n] [fintype n] :

The function (A ⊗[R] matrix n n R) →ₐ[R] matrix n n A, as an algebra homomorphism.

Equations
@[simp]
theorem matrix_equiv_tensor.to_fun_alg_hom_apply (R : Type u) [comm_semiring R] (A : Type v) [semiring A] [algebra R A] (n : Type w) [decidable_eq n] [fintype n] (a : A) (m : matrix n n R) :
def matrix_equiv_tensor.inv_fun (R : Type u) [comm_semiring R] (A : Type v) [semiring A] [algebra R A] (n : Type w) [decidable_eq n] [fintype n] (M : matrix n n A) :

(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
@[simp]
theorem matrix_equiv_tensor.inv_fun_zero (R : Type u) [comm_semiring R] (A : Type v) [semiring A] [algebra R A] (n : Type w) [decidable_eq n] [fintype n] :
@[simp]
theorem matrix_equiv_tensor.inv_fun_add (R : Type u) [comm_semiring R] (A : Type v) [semiring A] [algebra R A] (n : Type w) [decidable_eq n] [fintype n] (M N : matrix n n A) :
@[simp]
theorem matrix_equiv_tensor.inv_fun_smul (R : Type u) [comm_semiring R] (A : Type v) [semiring A] [algebra R A] (n : Type w) [decidable_eq n] [fintype n] (a : A) (M : matrix n n A) :
@[simp]
theorem matrix_equiv_tensor.inv_fun_algebra_map (R : Type u) [comm_semiring R] (A : Type v) [semiring A] [algebra R A] (n : Type w) [decidable_eq n] [fintype n] (M : matrix n n R) :
theorem matrix_equiv_tensor.right_inv (R : Type u) [comm_semiring R] (A : Type v) [semiring A] [algebra R A] (n : Type w) [decidable_eq n] [fintype n] (M : matrix n n A) :
theorem matrix_equiv_tensor.left_inv (R : Type u) [comm_semiring R] (A : Type v) [semiring A] [algebra R A] (n : Type w) [decidable_eq n] [fintype n] (M : tensor_product R A (matrix n n R)) :
def matrix_equiv_tensor.equiv (R : Type u) [comm_semiring R] (A : Type v) [semiring A] [algebra R A] (n : Type w) [decidable_eq n] [fintype n] :
tensor_product R A (matrix n n R) matrix n n A

(Implementation detail)

The equivalence, ignoring the algebra structure, (A ⊗[R] matrix n n R) ≃ matrix n n A.

Equations
def matrix_equiv_tensor (R : Type u) [comm_semiring R] (A : Type v) [semiring A] [algebra R A] (n : Type w) [fintype n] [decidable_eq n] :

The R-algebra isomorphism matrix n n A ≃ₐ[R] (A ⊗[R] matrix n n R).

Equations
@[simp]
theorem matrix_equiv_tensor_apply (R : Type u) [comm_semiring R] (A : Type v) [semiring A] [algebra R A] (n : Type w) [fintype n] [decidable_eq n] (M : matrix n n A) :
@[simp]
theorem matrix_equiv_tensor_apply_std_basis (R : Type u) [comm_semiring R] (A : Type v) [semiring A] [algebra R A] (n : Type w) [fintype n] [decidable_eq n] (i j : n) (x : A) :
@[simp]
theorem matrix_equiv_tensor_apply_symm (R : Type u) [comm_semiring R] (A : Type v) [semiring A] [algebra R A] (n : Type w) [fintype n] [decidable_eq n] (a : A) (M : matrix n n R) :
((matrix_equiv_tensor R A n).symm) (a ⊗ₜ[R] M) = M.map (λ (x : R), a * (algebra_map R A) x)