Compare commits

..

No commits in common. "0c15de05b88bf3408878fd8fc284260247537547" and "b2f04c1dfa59f079808d46722663294ea434b23e" have entirely different histories.

3 changed files with 4 additions and 43 deletions

View File

@ -1,39 +0,0 @@
import Mathlib.Analysis.Complex.Basic
import Mathlib.Analysis.Calculus.LineDeriv.Basic
import Mathlib.Analysis.Calculus.ContDiff.Defs
import Mathlib.Analysis.Calculus.FDeriv.Basic
noncomputable def Real.laplace : ( × ) → ( × ) := by
intro f
let f₁ := fun x ↦ lineDeriv f x ⟨1,0⟩
let f₁₁ := fun x ↦ lineDeriv f₁ x ⟨1,0⟩
let f₂ := fun x ↦ lineDeriv f x ⟨0,1⟩
let f₂₂ := fun x ↦ lineDeriv f₂ x ⟨0,1⟩
exact f₁₁ + f₂₂
noncomputable def Complex.laplace : () → () := by
intro f
let f₁ := fun x ↦ lineDeriv f x 1
let f₁₁ := fun x ↦ lineDeriv f₁ x 1
let f₂ := fun x ↦ lineDeriv f x Complex.I
let f₂₂ := fun x ↦ lineDeriv f₂ x Complex.I
exact f₁₁ + f₂₂
theorem xx : ∀ f : → , f = 0 := by
intro f
let f₁ := fun x ↦ lineDeriv f x 1
let f₂ := fun x ↦ lineDeriv f x Complex.I
have : ∀ z, fderiv f z = 0 := by
sorry
have : (fun x ↦ lineDeriv f x 1) = (fun x ↦ lineDeriv f x Complex.I) := by
unfold lineDeriv
sorry
sorry

View File

@ -11,6 +11,6 @@ noncomputable def Real.laplace : ( × ) → ( × ) :
exact f₁₁ + f₂₂
def Harmonic (f : × ) : Prop :=
(ContDiff 2 f) ∧ (∀ x, Real.laplace f x = 0)
structure Harmonic (f : × ) : Prop where
ker_Laplace : ∀ x, Real.laplace f x = 0
cont_Diff : ContDiff 2 f