Skip to content

Commit

Permalink
chore(LinearAlgebra/DirectSum/TensorProduct): missing lemma (#7399)
Browse files Browse the repository at this point in the history
We had the lemma about how the forward direction of this equivalence behaves, but not the reverse direction.
  • Loading branch information
eric-wieser committed Oct 2, 2023
1 parent 4298bf3 commit 80b890f
Showing 1 changed file with 7 additions and 0 deletions.
7 changes: 7 additions & 0 deletions Mathlib/LinearAlgebra/DirectSum/TensorProduct.lean
Expand Up @@ -155,6 +155,13 @@ theorem directSum_lof_tmul_lof (i₁ : ι₁) (m₁ : M₁ i₁) (i₂ : ι₂)
simp [TensorProduct.directSum]
#align tensor_product.direct_sum_lof_tmul_lof TensorProduct.directSum_lof_tmul_lof

@[simp]
theorem directSum_symm_lof_tmul (i₁ : ι₁) (m₁ : M₁ i₁) (i₂ : ι₂) (m₂ : M₂ i₂) :
(TensorProduct.directSum R M₁ M₂).symm
(DirectSum.lof R (ι₁ × ι₂) (fun i => M₁ i.1 ⊗[R] M₂ i.2) (i₁, i₂) (m₁ ⊗ₜ m₂)) =
(DirectSum.lof R ι₁ M₁ i₁ m₁ ⊗ₜ DirectSum.lof R ι₂ M₂ i₂ m₂) := by
rw [LinearEquiv.symm_apply_eq, directSum_lof_tmul_lof]

@[simp]
theorem directSumLeft_tmul_lof (i : ι₁) (x : M₁ i) (y : M₂') :
directSumLeft R M₁ M₂' (DirectSum.lof R _ _ i x ⊗ₜ[R] y) =
Expand Down

0 comments on commit 80b890f

Please sign in to comment.