Zulip Chat Archive
Stream: new members
Topic: C² implies C¹
Michael Rothgang (Sep 19 2023 at 12:38):
Seems obvious, but I couldn't find this in mathlib. Minimized code:
lemma diff {E F : Type*} {r : ℕ} (hr : r ≥ 1) {w : Set E}
[NormedAddCommGroup E] [NormedSpace ℝ E] [FiniteDimensional ℝ E]
[NormedAddCommGroup F] [NormedSpace ℝ F] [FiniteDimensional ℝ F]
{f : E → F} (hf : ContDiffOn ℝ (↑r) f w) : ContDiffOn ℝ 1 f w := sorry
Kyle Miller (Sep 19 2023 at 12:40):
Is this docs#ContDiffOn.of_le applied to hr
? (Maybe you need to transform hr
)
Michael Rothgang (Sep 19 2023 at 12:41):
Looks promising, let me check...
Kyle Miller (Sep 19 2023 at 12:43):
The proof of docs#ContDiffOn.one_of_succ looks helpful to see how to transform hr
Michael Rothgang (Sep 19 2023 at 12:43):
Works like a charm, thanks! (I need to transform hr.)
Last updated: Dec 20 2023 at 11:08 UTC