Zulip Chat Archive

Stream: Is there code for X?

Topic: has primitive implies holomorphic


Alex Kontorovich (Dec 25 2023 at 22:23):

What's an easy way to go from F being a primitive of f to f being holomorphic?

import Mathlib

example {f F :   } {U : Set } (U_open : IsOpen U) (F_prim :  z  U, HasDerivAt F (f z) z)
    {z : } (hz : z  U):
    DifferentiableAt  f z := by
  have F_differentiableOn : DifferentiableOn  F U := fun z hz 
   (F_prim z hz).differentiableAt.differentiableWithinAt
  have := DifferentiableOn.contDiffOn (hd := F_differentiableOn) (hs := U_open) (n := 2) z hz
  -- this : ContDiffWithinAt ℂ 2 F U z

Junyan Xu (Dec 25 2023 at 23:22):

One solution:

import Mathlib

example {f F :   } {U : Set } (U_open : IsOpen U) (F_prim :  z  U, HasDerivAt F (f z) z)
    {z : } (hz : z  U):
    DifferentiableAt  f z := by
  have : AnalyticOn  F U := DifferentiableOn.analyticOn
    (fun z hz  _, (F_prim z hz).hasDerivWithinAt⟩) U_open
  refine (AnalyticOn.differentiableOn ?_).differentiableAt (U_open.mem_nhds hz)
  exact this.deriv.congr U_open fun z hz  (F_prim z hz).deriv

Last updated: May 02 2025 at 03:31 UTC