Skip to content

Commit a162410

Browse files
committed
feat(Analysis/Calculus/TangentCone): add results about uniqueDiff (#26993)
Split from #26992 Co-authored-by: Paul Lezeau <paul.lezeau@gmail.com>
1 parent b7f38ac commit a162410

File tree

1 file changed

+6
-0
lines changed

1 file changed

+6
-0
lines changed

Mathlib/Analysis/Calculus/TangentCone.lean

Lines changed: 6 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -658,6 +658,12 @@ theorem uniqueDiffWithinAt_Ioi (a : ℝ) : UniqueDiffWithinAt ℝ (Ioi a) a :=
658658
theorem 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
662668
iff it is an accumulation point of the set. -/
663669
theorem uniqueDiffWithinAt_iff_accPt {s : Set 𝕜} {x : 𝕜} :

0 commit comments

Comments
 (0)