Skip to content

Commit

Permalink
feat(analysis/calculus/cont_diff): smoothness from Taylor series (#18768
Browse files Browse the repository at this point in the history
)

The proofs are basically trivial, but I think it is very nice to have the API.
  • Loading branch information
mcdoll committed Apr 10, 2023
1 parent 8cab1cd commit 0a0b3b4
Showing 1 changed file with 13 additions and 1 deletion.
14 changes: 13 additions & 1 deletion src/analysis/calculus/cont_diff_def.lean
Expand Up @@ -621,6 +621,15 @@ def cont_diff_on (n : ℕ∞) (f : E → F) (s : set E) : Prop :=

variable {𝕜}

lemma has_ftaylor_series_up_to_on.cont_diff_on {f' : E → formal_multilinear_series 𝕜 E F}
(hf : has_ftaylor_series_up_to_on n f f' s) : cont_diff_on 𝕜 n f s :=
begin
intros x hx m hm,
use s,
simp only [set.insert_eq_of_mem hx, self_mem_nhds_within, true_and],
exact ⟨f', hf.of_le hm⟩,
end

lemma cont_diff_on.cont_diff_within_at (h : cont_diff_on 𝕜 n f s) (hx : x ∈ s) :
cont_diff_within_at 𝕜 n f s x :=
h x hx
Expand Down Expand Up @@ -1326,6 +1335,10 @@ def cont_diff (n : ℕ∞) (f : E → F) : Prop :=

variable {𝕜}

/-- If `f` has a Taylor series up to `n`, then it is `C^n`. -/
lemma has_ftaylor_series_up_to.cont_diff {f' : E → formal_multilinear_series 𝕜 E F}
(hf : has_ftaylor_series_up_to n f f') : cont_diff 𝕜 n f := ⟨f', hf⟩

theorem cont_diff_on_univ : cont_diff_on 𝕜 n f univ ↔ cont_diff 𝕜 n f :=
begin
split,
Expand Down Expand Up @@ -1390,7 +1403,6 @@ lemma cont_diff_iff_forall_nat_le :
cont_diff 𝕜 n f ↔ ∀ m : ℕ, ↑m ≤ n → cont_diff 𝕜 m f :=
by { simp_rw [← cont_diff_on_univ], exact cont_diff_on_iff_forall_nat_le }


/-! ### Iterated derivative -/

variable (𝕜)
Expand Down

0 comments on commit 0a0b3b4

Please sign in to comment.