Compare commits

..

2 Commits

Author SHA1 Message Date
Stefan Kebekus 0c15de05b8 Merge branch 'main' of git.cplx.vm.uni-freiburg.de:kebekus/nevanlinna 2024-04-30 06:52:41 +02:00
Stefan Kebekus ef75cb4579 working... 2024-04-28 21:17:45 +02:00
3 changed files with 43 additions and 4 deletions

View File

@ -0,0 +1,39 @@
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₂₂
structure Harmonic (f : × ) : Prop where
ker_Laplace : ∀ x, Real.laplace f x = 0
cont_Diff : ContDiff 2 f
def Harmonic (f : × ) : Prop :=
(ContDiff 2 f) ∧ (∀ x, Real.laplace f x = 0)