File tree Expand file tree Collapse file tree 1 file changed +6
-0
lines changed
Mathlib/Analysis/Calculus Expand file tree Collapse file tree 1 file changed +6
-0
lines changed Original file line number Diff line number Diff line change @@ -658,6 +658,12 @@ theorem uniqueDiffWithinAt_Ioi (a : ℝ) : UniqueDiffWithinAt ℝ (Ioi a) a :=
658658theorem uniqueDiffWithinAt_Iio (a : ℝ) : UniqueDiffWithinAt ℝ (Iio a) a :=
659659 uniqueDiffWithinAt_convex (convex_Iio a) (by simp) (by simp)
660660
661+ theorem uniqueDiffWithinAt_Ici (x : ℝ) : UniqueDiffWithinAt ℝ (Ici x) x :=
662+ (uniqueDiffWithinAt_Ioi x).mono Set.Ioi_subset_Ici_self
663+
664+ theorem uniqueDiffWithinAt_Iic (x : ℝ) : UniqueDiffWithinAt ℝ (Iic x) x :=
665+ (uniqueDiffWithinAt_Iio x).mono Set.Iio_subset_Iic_self
666+
661667/-- In one dimension, a point is a point of unique differentiability of a set
662668iff it is an accumulation point of the set. -/
663669theorem uniqueDiffWithinAt_iff_accPt {s : Set 𝕜} {x : 𝕜} :
You can’t perform that action at this time.
0 commit comments