nevanlinna/nevanlinna/realHarmonic.lean

17 lines
573 B
Plaintext
Raw Normal View History

2024-04-26 21:18:06 +02:00
import Mathlib.Analysis.Calculus.LineDeriv.Basic
2024-04-28 21:09:38 +02:00
import Mathlib.Analysis.Calculus.ContDiff.Defs
2024-04-26 21:18:06 +02:00
2024-04-28 21:09:38 +02:00
noncomputable def Real.laplace : ( × ) → ( × ) := by
2024-04-26 21:18:06 +02:00
intro f
2024-04-28 21:09:38 +02:00
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⟩
2024-04-26 21:18:06 +02:00
exact f₁₁ + f₂₂
2024-04-28 21:09:38 +02:00
structure Harmonic (f : × ) : Prop where
ker_Laplace : ∀ x, Real.laplace f x = 0
cont_Diff : ContDiff 2 f