src/HOL/Limits.thy
changeset 50326 b5afeccab2db
parent 50325 5e40ad9f212a
child 50327 bbea2e82871c
--- a/src/HOL/Limits.thy	Mon Dec 03 18:19:04 2012 +0100
+++ b/src/HOL/Limits.thy	Mon Dec 03 18:19:05 2012 +0100
@@ -373,6 +373,12 @@
 definition (in topological_space) at :: "'a \<Rightarrow> 'a filter"
   where "at a = nhds a within - {a}"
 
+abbreviation at_right :: "'a\<Colon>{topological_space, order} \<Rightarrow> 'a filter" where
+  "at_right x \<equiv> at x within {x <..}"
+
+abbreviation at_left :: "'a\<Colon>{topological_space, order} \<Rightarrow> 'a filter" where
+  "at_left x \<equiv> at x within {..< x}"
+
 definition at_infinity :: "'a::real_normed_vector filter" where
   "at_infinity = Abs_filter (\<lambda>P. \<exists>r. \<forall>x. r \<le> norm x \<longrightarrow> P x)"