Zulip Chat Archive

Stream: Is there code for X?

Topic: isolated zeros


Vincent Beffara (May 17 2022 at 07:30):

Is one of these somewhere?

import analysis.analytic.basic
import analysis.complex.basic

open filter

lemma isolated_zeros {f :   } (hf : analytic_at  f 0) :
  (∀ᶠ z in nhds 0, f z = 0)  (∀ᶠ z in nhds_within 0 {0}, f z  0) :=
sorry

lemma isolated_zeros' {f :   } (hf : analytic_at  f 0) :
  (∃ᶠ z in nhds_within 0 {0}, f z = 0)  (∀ᶠ z in nhds 0, f z = 0) :=
sorry

Vincent Beffara (May 19 2022 at 23:15):

... it will be soon :grinning:

https://gist.github.com/vbeffara/0ddc2b65f5553162c448e2596e0d254d

(pending a lot of refactoring)


Last updated: Dec 20 2023 at 11:08 UTC