Zulip Chat Archive

Stream: Is there code for X?

Topic: ContinuousOn_derivWithin_of_deriv


Alex Kontorovich (Mar 29 2024 at 00:03):

Any suggestions for how to do something like the below, that is, replace derivWithin with deriv (given that I only care about both on the same set as "Within"...)?

import Mathlib

lemma ContinuousOn_derivWithin_of_deriv (φ :   ) (a b : )
    (h : ContinuousOn (deriv φ) (Set.uIcc a b)) :
    ContinuousOn (derivWithin φ (Set.uIcc a b)) (Set.uIcc a b) := by sorry

Vincent Beffara (Mar 29 2024 at 00:17):

Is this true without assuming differentiability? E.g. one could conceive of a function that is nowhere differentiable but right differentiable at 0 with right derivative 1, then it is differentiable within Icc 0 1 at 0, it has deriv identically 0 but derivWithin is discontinuous at 0.

Alex Kontorovich (Mar 29 2024 at 14:09):

Ok sure, let's add differentiability:

import Mathlib

lemma ContinuousOn_derivWithin_of_deriv {φ :   } {a b : }
    (φDiff : ContDiffOn  1 φ (Set.uIcc a b)) :
    ContinuousOn (derivWithin φ (Set.uIcc a b)) (Set.uIcc a b) := by sorry

Sébastien Gouëzel (Mar 29 2024 at 14:30):

@loogle ContDiffOn, ContinuousOn, derivWithin

Michael Stoll (Mar 29 2024 at 14:31):

@loogle ContDiffOn, ContinuousOn, derivWithin

loogle (Mar 29 2024 at 14:31):

:search: ContDiffOn.continuousOn_derivWithin

Sébastien Gouëzel (Mar 29 2024 at 14:32):

Loogle is amazing, and our library is also amazing :-)

Michael Stoll (Mar 29 2024 at 14:32):

 {𝕜 : Type u_1} [inst : NontriviallyNormedField 𝕜] {F : Type uF} [inst_1 : NormedAddCommGroup F]
 [inst_2 : NormedSpace 𝕜 F] {n : } {f₂ : 𝕜  F} {s₂ : Set 𝕜}, ContDiffOn 𝕜 n f₂ s₂  UniqueDiffOn 𝕜 s₂ 
 1  n  ContinuousOn (derivWithin f₂ s₂) s₂

Pretty close...

Sébastien Gouëzel (Mar 29 2024 at 14:33):

(It won't cover exactly your use case, as for a = b then uIcc a bis not a set of unique differentiability, but since any function is continuous on a singleton you should be fine)


Last updated: May 02 2025 at 03:31 UTC