nevanlinna/Nevanlinna/bilinear.lean

40 lines
817 B
Plaintext
Raw Blame History

This file contains ambiguous Unicode characters

This file contains Unicode characters that might be confused with other characters. If you think that this is intentional, you can safely ignore this warning. Use the Escape button to reveal them.

import Mathlib.Algebra.BigOperators.Basic
import Mathlib.Analysis.InnerProductSpace.Basic
import Mathlib.Analysis.InnerProductSpace.Dual
import Mathlib.Analysis.InnerProductSpace.PiL2
open BigOperators
open Finset
variable {E : Type*} [NormedAddCommGroup E] [InnerProductSpace E] [FiniteDimensional E]
variable {F : Type*} [NormedAddCommGroup F] [NormedSpace F]
open TensorProduct
example : 0 = 1 := by
let B := (sesqFormOfInner (𝕜 := ) (E := E)).flip
have e: E := by sorry
let C := B e
let α := InnerProductSpace.toDual E
let β : E →ₗ[] := by sorry
let YY := E ⊗[] E
let ZZ := TensorProduct.mapBilinear E E
let A : E × E → LinearMap.BilinForm E := by
unfold LinearMap.BilinForm
intro (e₁, e₂)
sorry
sorry