Skip to content

Commit

Permalink
fix
Browse files Browse the repository at this point in the history
  • Loading branch information
sgouezel committed Oct 4, 2024
1 parent f84210d commit 5acbb59
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/Analysis/Calculus/ContDiff/FaaDiBruno.lean
Original file line number Diff line number Diff line change
Expand Up @@ -663,7 +663,7 @@ def extendEquiv (n : ℕ) :
· intro j
induction i using Fin.induction with
| zero =>
simp only [cases_zero, cast_zero, coe_fin_one]
simp only [cases_zero, cast_zero, val_eq_zero]
exact (apply_eq_of_range_eq_singleton h _).symm
| succ i => simp
· dsimp only
Expand Down

0 comments on commit 5acbb59

Please sign in to comment.