Skip to content

Commit

Permalink
fix
Browse files Browse the repository at this point in the history
  • Loading branch information
sgouezel committed Nov 7, 2024
1 parent a09ce0b commit 4f89185
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/Analysis/Calculus/ContDiff/FTaylorSeries.lean
Original file line number Diff line number Diff line change
Expand Up @@ -355,7 +355,7 @@ theorem hasFTaylorSeriesUpToOn_top_iff_right (hN : ∞ ≤ N) :
fun n ↦ (hasFTaylorSeriesUpToOn_succ_nat_iff_right.1 (h n)).2.2
· apply (hasFTaylorSeriesUpToOn_top_iff_add hN 1).2 (fun n ↦ ?_)
rw [hasFTaylorSeriesUpToOn_succ_nat_iff_right]
exact ⟨h.1, h.2.1, (h.2.2).of_le (m := n) (nat_le_of_infty_le hN n)⟩
exact ⟨h.1, h.2.1, (h.2.2).of_le (m := n) (nat_le_of_infty_le_withTop hN n)⟩

/-- `p` is a Taylor series of `f` up to `n+1` if and only if `p.shift` is a Taylor series up to `n`
for `p 1`, which is a derivative of `f`. Version for `n : WithTop ℕ∞`. -/
Expand Down

0 comments on commit 4f89185

Please sign in to comment.