Skip to content

Commit 20129f5

Browse files
authored
simp low
1 parent 8e22772 commit 20129f5

File tree

1 file changed

+2
-2
lines changed

1 file changed

+2
-2
lines changed

Mathlib/Analysis/Calculus/Deriv/Basic.lean

+2-2
Original file line numberDiff line numberDiff line change
@@ -710,7 +710,7 @@ theorem deriv_one [One F] : deriv (1 : 𝕜 → F) = 0 := funext fun _ => deriv_
710710

711711
theorem deriv_natCast [NatCast F] (n : ℕ) : deriv (n : 𝕜 → F) = 0 := funext fun _ => deriv_const _ _
712712

713-
@[simp]
713+
@[simp low]
714714
theorem deriv_ofNat (n : ℕ) [OfNat F n] : deriv (ofNat(n) : 𝕜 → F) = 0 :=
715715
funext fun _ => deriv_const _ _
716716

@@ -727,7 +727,7 @@ theorem derivWithin_one [One F] : derivWithin (1 : 𝕜 → F) s = 0 := derivWit
727727
theorem derivWithin_natCast [NatCast F] (n : ℕ) : derivWithin (n : 𝕜 → F) s = 0 :=
728728
derivWithin_const _ _
729729

730-
@[simp]
730+
@[simp low]
731731
theorem derivWithin_ofNat (n : ℕ) [OfNat F n] : derivWithin (ofNat(n) : 𝕜 → F) s = 0 :=
732732
derivWithin_const _ _
733733

0 commit comments

Comments
 (0)