Skip to content

Commit

Permalink
chore(analysis/calculus/cont_diff): rename and add @[simp] to `iterat…
Browse files Browse the repository at this point in the history
…ed_fderiv_within_zero_fun` (#15896)

Rename the lemma `iterated_fderiv_within_zero_fun` to `iterated_fderiv_zero_fun` because it is not stated with `iterated_fderiv_within` and add the `simp` attribute.
  • Loading branch information
mcdoll committed Aug 9, 2022
1 parent a5413b6 commit 511caf6
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions src/analysis/calculus/cont_diff.lean
Expand Up @@ -1578,7 +1578,7 @@ end

/-! ### Constants -/

lemma iterated_fderiv_within_zero_fun {n : ℕ} :
@[simp] lemma iterated_fderiv_zero_fun {n : ℕ} :
iterated_fderiv 𝕜 n (λ x : E, (0 : F)) = 0 :=
begin
induction n with n IH,
Expand All @@ -1594,7 +1594,7 @@ lemma cont_diff_zero_fun :
cont_diff 𝕜 n (λ x : E, (0 : F)) :=
begin
apply cont_diff_of_differentiable_iterated_fderiv (λm hm, _),
rw iterated_fderiv_within_zero_fun,
rw iterated_fderiv_zero_fun,
apply differentiable_const (0 : (E [×m]→L[𝕜] F))
end

Expand Down

0 comments on commit 511caf6

Please sign in to comment.