Compare commits

..

No commits in common. "ecdc182f2b76661be8b3aad96bf9f8769b0a712b" and "d287c24453fa6808dc88ac03037f17bbe1448587" have entirely different histories.

1 changed files with 1 additions and 20 deletions

View File

@ -27,8 +27,6 @@ noncomputable def Laplace₂
E → F := E → F :=
fun z ↦ ∑ i, iteratedFDeriv 2 f z ![v i, v i] fun z ↦ ∑ i, iteratedFDeriv 2 f z ![v i, v i]
#check ContinuousMultilinearMap.map_sum_finset
theorem LaplaceIndep theorem LaplaceIndep
[Fintype ι] [Fintype ι]
(v₁ : Basis ι E) (v₁ : Basis ι E)
@ -51,22 +49,5 @@ theorem LaplaceIndep
right right
arg 2 arg 2
intro i intro i
--rw [ContinuousMultilinearMap.map_sum_finset] rw [ContinuousMultilinearMap.map_sum_finset]
have v : E := by sorry
let t := ![∑ j, ⟪v₁ j, v⟫_ • (v₁ j), ∑ j, ⟪v₁ j, v⟫_ • (v₁ j)]
simp at t
have L : ContinuousMultilinearMap (fun (_ : Fin 2) ↦ E) F := by exact iteratedFDeriv 2 f z
--have α : Fin 2 → Type* := by exact fun _ ↦ ι
have g : (i : Fin 2) → ι → E := by exact fun _ ↦ (fun j ↦ ⟪v₁ j, v⟫_ • (v₁ j))
have A : (i : Fin 2) → Finset ι := by exact fun _ ↦ Finset.univ
let X := ContinuousMultilinearMap.map_sum
(iteratedFDeriv 2 f z)
(fun _ ↦ (fun j ↦ ⟪v₁ j, v⟫_ • (v₁ j)))
--
-- (fun _ ↦ Finset.univ)
simp at X
sorry sorry