File tree Expand file tree Collapse file tree 1 file changed +10
-2
lines changed Expand file tree Collapse file tree 1 file changed +10
-2
lines changed Original file line number Diff line number Diff line change @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
4
4
Authors: Jakob von Raumer
5
5
6
6
! This file was ported from Lean 3 source module linear_algebra.tensor_product_basis
7
- ! leanprover-community/mathlib commit 4977fd9da637b6e0a805c1cf460c3a6b8df3f556
7
+ ! leanprover-community/mathlib commit f784cc6142443d9ee623a20788c282112c322081
8
8
! Please do not edit these lines, except to modify the commit id
9
9
! if you have ported upstream changes.
10
10
-/
@@ -54,5 +54,13 @@ theorem Basis.tensorProduct_apply' (b : Basis ι R M) (c : Basis κ R N) (i : ι
54
54
Basis.tensorProduct b c i = b i.1 ⊗ₜ c i.2 := by simp [Basis.tensorProduct]
55
55
#align basis.tensor_product_apply' Basis.tensorProduct_apply'
56
56
57
- end CommRing
57
+ -- Porting note: resolved diamond
58
+ set_option synthInstance.etaExperiment true in
59
+ @[simp]
60
+ theorem Basis.tensorProduct_repr_tmul_apply (b : Basis ι R M) (c : Basis κ R N) (m : M) (n : N)
61
+ (i : ι) (j : κ) :
62
+ (Basis.tensorProduct b c).repr (m ⊗ₜ n) (i, j) = b.repr m i * c.repr n j := by
63
+ simp [Basis.tensorProduct]
64
+ #align basis.tensor_product_repr_tmul_apply Basis.tensorProduct_repr_tmul_apply
58
65
66
+ end CommRing
You can’t perform that action at this time.
0 commit comments