File tree 1 file changed +2
-2
lines changed
Mathlib/Analysis/Calculus/Deriv
1 file changed +2
-2
lines changed Original file line number Diff line number Diff line change @@ -710,7 +710,7 @@ theorem deriv_one [One F] : deriv (1 : 𝕜 → F) = 0 := funext fun _ => deriv_
710
710
711
711
theorem deriv_natCast [NatCast F] (n : ℕ) : deriv (n : 𝕜 → F) = 0 := funext fun _ => deriv_const _ _
712
712
713
- @[simp]
713
+ @[simp low ]
714
714
theorem deriv_ofNat (n : ℕ) [OfNat F n] : deriv (ofNat(n) : 𝕜 → F) = 0 :=
715
715
funext fun _ => deriv_const _ _
716
716
@@ -727,7 +727,7 @@ theorem derivWithin_one [One F] : derivWithin (1 : 𝕜 → F) s = 0 := derivWit
727
727
theorem derivWithin_natCast [NatCast F] (n : ℕ) : derivWithin (n : 𝕜 → F) s = 0 :=
728
728
derivWithin_const _ _
729
729
730
- @[simp]
730
+ @[simp low ]
731
731
theorem derivWithin_ofNat (n : ℕ) [OfNat F n] : derivWithin (ofNat(n) : 𝕜 → F) s = 0 :=
732
732
derivWithin_const _ _
733
733
You can’t perform that action at this time.
0 commit comments