Skip to content

Commit

Permalink
analysis.calculus.uniformlimitsderiv
Browse files Browse the repository at this point in the history
  • Loading branch information
hrmacbeth committed Oct 2, 2024
1 parent ecc94ee commit a796333
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions Mathlib/Analysis/Calculus/UniformLimitsDeriv.lean
Original file line number Diff line number Diff line change
Expand Up @@ -356,8 +356,8 @@ theorem hasFDerivAt_of_tendstoUniformlyOnFilter [NeBot l]
apply ((this ε hε).filter_mono curry_le_prod).mono
intro n hn
rw [dist_eq_norm] at hn ⊢
rw [← smul_sub] at hn
rwa [sub_zero]
convert hn using 2
module
· -- (Almost) the definition of the derivatives
rw [Metric.tendsto_nhds]
intro ε hε
Expand Down

0 comments on commit a796333

Please sign in to comment.