Zulip Chat Archive
Stream: maths
Topic: measurable derivative/integral
Yury G. Kudryashov (Aug 05 2020 at 23:00):
Is it true that fderiv
of a measurable function f : E → F
is a measurable function uncurry (fderiv f) : E × E → F
? I can prove this for the directional derivative dir_deriv f a v = deriv (λ t, f (a + t * v)) 0
, so the question is whether the set {x | differentiable_at f x}
is measurable. It is for E = \R
. What about other domains?
Heather Macbeth (Aug 05 2020 at 23:16):
Is this the same, or have I overlooked a hypothesis?
https://math.stackexchange.com/questions/905083/characterization-of-sets-of-differentiability
Yury G. Kudryashov (Aug 06 2020 at 01:03):
This answers "It is for "
Sebastien Gouezel (Aug 06 2020 at 14:40):
It is true that the derivative of a function (measurable or not) is measurable when the target space is complete, as a map from to the space of continuous linear maps from to . Let me give a proof.
Sebastien Gouezel (Aug 06 2020 at 14:44):
Let me first show that the set of differentiability points is measurable. For , let denote the set of points for which there exist a continuous linear map (a "candidate derivative") and two numbers and such that, for all , one has , and for all one has .
Sebastien Gouezel (Aug 06 2020 at 14:45):
It is clear that is open: indeed, if belongs to this set, then any nearby point also does, upon reducing a little bit and (and keeping the same ). I claim that the set of differentiability points is equal to , from which the measurability follows readily.
Sebastien Gouezel (Aug 06 2020 at 14:49):
We have two inclusions to show. Let us start with the easy one: if is a point of differentiability, then it belongs to . Fix some . Let be the derivative of at . For small enough , one has for all the inequality . Subtracting the corresponding inequality at , one obtains . This shows that whenever and are large enough, as requested.
Sebastien Gouezel (Aug 06 2020 at 14:54):
The other inclusion is a little bit harder. Take , we have to show that is differentiable at . In particular, we should exhibit in some way its derivative. The main remark is that the candidate derivative is essentially unique: if two continuous linear maps and satisfy (and the same for ) for all for some , then (take any , and apply the previous inequalities to and ).
Sebastien Gouezel (Aug 06 2020 at 14:57):
Let . The assumption that belongs to ensures that, for larger than some , then belongs to , yielding a candidate derivative . The almost uniqueness argument above shows that is within of (using the fact that both these candidate derivatives work in a ball of radius roughly ), which is itself withing of (same argument using the ball of radius ).
Sebastien Gouezel (Aug 06 2020 at 15:00):
Let . The same argument shows that and are within distance of each other when , as they are both candidate derivatives on a common ball of very small radius. It follows that is a Cauchy sequence, converging to a continuous linear operator by completeness. It follows readily that is a derivative of at .
Sebastien Gouezel (Aug 06 2020 at 15:02):
This concludes the proof of the measurability of the set of differentiability points. The measurability of the differential is proved similarly. One should show that, for any closed set in the space of continuous linear maps from to , the set of points where is differentiable with derivative in is measurable. This set can be described exactly as before, requiring additionally in the definition of that the candidate derivative belongs to .
Sebastien Gouezel (Aug 06 2020 at 15:03):
(And no, I am not going to formalize this now :-)
Yury G. Kudryashov (Aug 09 2020 at 04:06):
Why do you need both and (or and )?
Yury G. Kudryashov (Nov 10 2020 at 22:35):
@Sebastien Gouezel It seems that your construction deals with strict differentiability, not Frechet differentiability.
Yury G. Kudryashov (Nov 10 2020 at 22:36):
I can modify it to prove that any continuous function has measurable derivative.
Yury G. Kudryashov (Nov 10 2020 at 22:37):
But I can't get rid of the continuity assumption
Yury G. Kudryashov (Nov 10 2020 at 22:43):
Now I can. I'll write down details once I come back home
Sebastien Gouezel (Nov 11 2020 at 08:48):
It's funny, I am precisely working on this now! I can confirm that it's for usual differentiability (strict differentiability is much easier). I'll PR something in a few hours, hopefully.
Sebastien Gouezel (Nov 11 2020 at 08:49):
(The proof of measurability of the differentiability set is already there in the branch deriv_measurable
, I'm working on the measurability of the derivative)
Yury G. Kudryashov (Nov 11 2020 at 09:01):
Branch measurable-fderiv
has the proof
Yury G. Kudryashov (Nov 11 2020 at 09:02):
Yury G. Kudryashov (Nov 11 2020 at 09:04):
What should we do with 2 proofs?
Yury G. Kudryashov (Nov 11 2020 at 09:07):
I'm sorry for not announcing my intent to formalize this before starting to write the code.
Sebastien Gouezel (Nov 11 2020 at 09:10):
It's funny! Let me finish my proof, and then I will learn a lot by reading yours!
Yury G. Kudryashov (Nov 11 2020 at 09:22):
The first difference is that I'm using ≤ ε * ||y - x||
and shells while you're using ≤ ε * r
and balls.
Yury G. Kudryashov (Nov 11 2020 at 09:31):
Not sure which approach is simpler.
Yury G. Kudryashov (Nov 11 2020 at 09:32):
But this means that merging proofs is not an option; we'll have to choose one of them for mathlib.
Sebastien Gouezel (Nov 11 2020 at 09:40):
I think we'll go for your proof because it is already complete, and because you have been able to separate things more cleanly than I do (I have a monster proof of 170 lines, while you have been able to cut it in pieces). I'd like to eliminate the continuity requirement from your argument, though, because it doesn't show up in mine.
I have PR'ed mine at #4974 (not for merging). I'll salvage the supporting lemmas because they can be useful anyway!
Sebastien Gouezel (Nov 11 2020 at 09:42):
One thing I like better in mine, also, is the file-level docstring in which I give a high-level overview of the proof :)
Yury G. Kudryashov (Nov 11 2020 at 09:42):
I see that you have a better version of #4970
Yury G. Kudryashov (Nov 11 2020 at 09:43):
I don't think that we can avoid continuity argument in my proof without changing it from shells to balls.
Yury G. Kudryashov (Nov 11 2020 at 09:44):
Because the assumption about y ∈ B(x, R) \ B(x, r)
says nothing about x' in nhds x
.
Sebastien Gouezel (Nov 11 2020 at 09:48):
Yury G. Kudryashov said:
I see that you have a better version of #4970
Yes, you have a useless assumption. Can you remove it from #4970?
Yury G. Kudryashov (Nov 11 2020 at 09:51):
Probably I'm too sleepy. Which assumption is useless?
Yury G. Kudryashov (Nov 11 2020 at 09:51):
I saw that you have more additions to the same file but didn't pay attention to the list of assumptions.
Yury G. Kudryashov (Nov 11 2020 at 09:52):
Indeed, I'm too sleepy. We don't need 0 ≤ y
.
Yury G. Kudryashov (Nov 11 2020 at 09:55):
I can remove it once I wake up (or you can PR your diff to algebra/archimedean
)
Sebastien Gouezel (Nov 11 2020 at 09:57):
Good night! I'll review while you sleep.
Sebastien Gouezel (Nov 11 2020 at 13:39):
Comparing the two proofs, I think I like mine better because it gives a lower complexity in the Borel scale for the differentiability set (it shows that the differentiability set is a countable intersection of union of intersection of open sets, while yours give something like intersection of union of intersection of union of something which is measurable, but not open). But I like better the way you have presented the proof. I could refactor my proof based on some ideas in yours, to have the best of both worlds. What do you think?
(And apologies also for not telling you I was going to work on this. I was tired of doing boring stuff, so I took one day off to play with Lean :-)
Yury G. Kudryashov (Nov 11 2020 at 15:32):
You can do whatever you prefer. I just want the statements to be in mathlib
soon.
Yury G. Kudryashov (Nov 11 2020 at 15:33):
I am formalizing Stokes' Theorem, and need measurable (fderiv k f)
at one of the steps.
Yury G. Kudryashov (Nov 11 2020 at 15:55):
BTW, my proof can be easily modified to match complexity in the Borel scale.
Yury G. Kudryashov (Nov 11 2020 at 15:56):
You just replace continuous_at f x
with the actual inequality we use later in the proof.
Sebastien Gouezel (Nov 11 2020 at 16:08):
ok, let me do the refactoring.
Sebastien Gouezel (Nov 11 2020 at 22:16):
#4974 is ready for review. I have copied some parts from #4972.
Last updated: Dec 20 2023 at 11:08 UTC