@@ -647,6 +647,9 @@ theorem hasDerivAtFilter_one [One F] : HasDerivAtFilter (1 : 𝕜 → F) 0 x L :
647
647
theorem hasDerivAtFilter_natCast [NatCast F] (n : ℕ) : HasDerivAtFilter (n : 𝕜 → F) 0 x L :=
648
648
hasDerivAtFilter_const _ _ _
649
649
650
+ theorem hasDerivAtFilter_intCast [IntCast F] (z : ℤ) : HasDerivAtFilter (z : 𝕜 → F) 0 x L :=
651
+ hasDerivAtFilter_const _ _ _
652
+
650
653
theorem hasDerivAtFilter_ofNat (n : ℕ) [OfNat F n] : HasDerivAtFilter (ofNat(n) : 𝕜 → F) 0 x L :=
651
654
hasDerivAtFilter_const _ _ _
652
655
@@ -662,6 +665,9 @@ theorem hasStrictDerivAt_one [One F] : HasStrictDerivAt (1 : 𝕜 → F) 0 x :=
662
665
theorem hasStrictDerivAt_natCast [NatCast F] (n : ℕ) : HasStrictDerivAt (n : 𝕜 → F) 0 x :=
663
666
hasStrictDerivAt_const _ _
664
667
668
+ theorem hasStrictDerivAt_intCast [IntCast F] (z : ℤ) : HasStrictDerivAt (z : 𝕜 → F) 0 x :=
669
+ hasStrictDerivAt_const _ _
670
+
665
671
theorem HasStrictDerivAt_ofNat (n : ℕ) [OfNat F n] : HasStrictDerivAt (ofNat(n) : 𝕜 → F) 0 x :=
666
672
hasStrictDerivAt_const _ _
667
673
@@ -677,6 +683,9 @@ theorem hasDerivWithinAt_one [One F] : HasDerivWithinAt (1 : 𝕜 → F) 0 s x :
677
683
theorem hasDerivWithinAt_natCast [NatCast F] (n : ℕ) : HasDerivWithinAt (n : 𝕜 → F) 0 s x :=
678
684
hasDerivWithinAt_const _ _ _
679
685
686
+ theorem hasDerivWithinAt_intCast [IntCast F] (z : ℤ) : HasDerivWithinAt (z : 𝕜 → F) 0 s x :=
687
+ hasDerivWithinAt_const _ _ _
688
+
680
689
theorem hasDerivWithinAt_ofNat (n : ℕ) [OfNat F n] : HasDerivWithinAt (ofNat(n) : 𝕜 → F) 0 s x :=
681
690
hasDerivWithinAt_const _ _ _
682
691
@@ -692,6 +701,9 @@ theorem hasDerivAt_one [One F] : HasDerivAt (1 : 𝕜 → F) 0 x :=
692
701
theorem hasDerivAt_natCast [NatCast F] (n : ℕ) : HasDerivAt (n : 𝕜 → F) 0 x :=
693
702
hasDerivAt_const _ _
694
703
704
+ theorem hasDerivAt_intCast [IntCast F] (z : ℤ) : HasDerivAt (z : 𝕜 → F) 0 x :=
705
+ hasDerivAt_const _ _
706
+
695
707
theorem hasDerivAt_ofNat (n : ℕ) [OfNat F n] : HasDerivAt (ofNat(n) : 𝕜 → F) 0 x :=
696
708
hasDerivAt_const _ _
697
709
@@ -710,6 +722,8 @@ theorem deriv_one [One F] : deriv (1 : 𝕜 → F) = 0 := funext fun _ => deriv_
710
722
711
723
theorem deriv_natCast [NatCast F] (n : ℕ) : deriv (n : 𝕜 → F) = 0 := funext fun _ => deriv_const _ _
712
724
725
+ theorem deriv_intCast [IntCast F] (z : ℤ) : deriv (z : 𝕜 → F) = 0 := funext fun _ => deriv_const _ _
726
+
713
727
@[simp low]
714
728
theorem deriv_ofNat (n : ℕ) [OfNat F n] : deriv (ofNat(n) : 𝕜 → F) = 0 :=
715
729
funext fun _ => deriv_const _ _
@@ -727,6 +741,9 @@ theorem derivWithin_one [One F] : derivWithin (1 : 𝕜 → F) s = 0 := derivWit
727
741
theorem derivWithin_natCast [NatCast F] (n : ℕ) : derivWithin (n : 𝕜 → F) s = 0 :=
728
742
derivWithin_const _ _
729
743
744
+ theorem derivWithin_intCast [IntCast F] (z : ℤ) : derivWithin (z : 𝕜 → F) s = 0 :=
745
+ derivWithin_const _ _
746
+
730
747
@[simp low]
731
748
theorem derivWithin_ofNat (n : ℕ) [OfNat F n] : derivWithin (ofNat(n) : 𝕜 → F) s = 0 :=
732
749
derivWithin_const _ _
0 commit comments