Compare commits

..

No commits in common. "2544242b136a96886c4110ab2e8abcd8dabfcb9f" and "f480ae2a0fb9a69f2a3dbe2ccc96bd65868eeb00" have entirely different histories.

1 changed files with 6 additions and 18 deletions

View File

@ -11,7 +11,6 @@ import Mathlib.Data.Complex.Exponential
import Mathlib.Analysis.RCLike.Basic import Mathlib.Analysis.RCLike.Basic
import Mathlib.Order.Filter.Basic import Mathlib.Order.Filter.Basic
import Mathlib.Topology.Algebra.InfiniteSum.Module import Mathlib.Topology.Algebra.InfiniteSum.Module
import Mathlib.Topology.Basic
import Mathlib.Topology.Instances.RealVectorSpace import Mathlib.Topology.Instances.RealVectorSpace
import Nevanlinna.cauchyRiemann import Nevanlinna.cauchyRiemann
import Nevanlinna.partialDeriv import Nevanlinna.partialDeriv
@ -80,19 +79,7 @@ theorem laplace_compContLinAt {f : → F} {l : F →L[] G} {x : } (h :
Complex.laplace (l ∘ f) x = (l ∘ (Complex.laplace f)) x := by Complex.laplace (l ∘ f) x = (l ∘ (Complex.laplace f)) x := by
have A₂ : ∃ v ∈ nhds x, (IsOpen v) ∧ (x ∈ v) ∧ (ContDiffOn 2 f v) := by have A₂ : ∃ v ∈ nhds x, (IsOpen v) ∧ (x ∈ v) ∧ (ContDiffOn 2 f v) := by
have : ∃ u ∈ nhds x, ContDiffOn 2 f u := by sorry
apply ContDiffAt.contDiffOn h
rfl
obtain ⟨u, hu₁, hu₂⟩ := this
obtain ⟨v, hv₁, hv₂, hv₃⟩ := mem_nhds_iff.1 hu₁
use v
constructor
· exact IsOpen.mem_nhds hv₂ hv₃
· constructor
exact hv₂
constructor
· exact hv₃
· exact ContDiffOn.congr_mono hu₂ (fun x => congrFun rfl) hv₁
obtain ⟨v, hv₁, hv₂, hv₃, hv₄⟩ := A₂ obtain ⟨v, hv₁, hv₂, hv₃, hv₄⟩ := A₂
have D : ∀ w : , partialDeriv w (l ∘ f) =ᶠ[nhds x] l ∘ partialDeriv w (f) := by have D : ∀ w : , partialDeriv w (l ∘ f) =ᶠ[nhds x] l ∘ partialDeriv w (f) := by
@ -119,12 +106,13 @@ theorem laplace_compContLinAt {f : → F} {l : F →L[] G} {x : } (h :
simp simp
-- DifferentiableAt (partialDeriv Complex.I f) x -- DifferentiableAt (partialDeriv Complex.I f) x
apply ContDiffAt.differentiableAt (partialDeriv_contDiffAt (ContDiffOn.contDiffAt hv₄ hv₁) Complex.I) unfold partialDeriv
rfl
sorry
-- DifferentiableAt (partialDeriv 1 f) x -- DifferentiableAt (partialDeriv 1 f) x
apply ContDiffAt.differentiableAt (partialDeriv_contDiffAt (ContDiffOn.contDiffAt hv₄ hv₁) 1)
rfl sorry
theorem laplace_compCLE {f : → F} {l : F ≃L[] G} (h : ContDiff 2 f) : theorem laplace_compCLE {f : → F} {l : F ≃L[] G} (h : ContDiff 2 f) :