Compare commits

..

2 Commits

Author SHA1 Message Date
Stefan Kebekus
ff00a0db82 Update tensor.lean 2024-07-03 11:17:47 +02:00
Stefan Kebekus
36c3d0f66b Create tensor.lean 2024-07-02 11:45:03 +02:00

47
Nevanlinna/tensor.lean Normal file
View File

@@ -0,0 +1,47 @@
import Mathlib.Analysis.InnerProductSpace.PiL2
open RCLike Real Filter
open Topology ComplexConjugate
open LinearMap (BilinForm)
open TensorProduct
open InnerProductSpace
open Inner
example
{E : Type*} [NormedAddCommGroup E] [InnerProductSpace E]
{F : Type*} [NormedAddCommGroup F] [InnerProductSpace F]
: 1 = 0 := by
let e : E [] E [] := innerₗ E
let f : F [] F [] := innerₗ F
let e₂ := TensorProduct.map₂ e f
let l := TensorProduct.lid
have : e1 e2 : E, f1 f2 : F, e₂ (e1 f1) (e2 f2) =
let X : InnerProductSpace.Core (E [] F) := {
inner := by
intro a b
exact TensorProduct.lid ((TensorProduct.map₂ (innerₗ E) (innerₗ F)) a b)
conj_symm := by
simp
intro x y
unfold innerₗ
simp
sorry
nonneg_re := _
definite := _
add_left := _
smul_left := _
}
let inner : E [𝕜] E E [𝕜] E 𝕜 :=
--let x := TensorProduct.lift
--E.inner
--TensorProduct.map₂
sorry
sorry