src/HOL/Topological_Spaces.thy
changeset 56289 d8d2a2b97168
parent 56231 b98813774a63
child 56329 9597a53b3429
--- a/src/HOL/Topological_Spaces.thy	Wed Mar 26 09:19:04 2014 +0100
+++ b/src/HOL/Topological_Spaces.thy	Wed Mar 26 14:00:37 2014 +0000
@@ -615,6 +615,14 @@
   "eventually (\<lambda>x. x < (c::_::unbounded_dense_linorder)) at_bot"
   unfolding eventually_at_bot_dense by auto
 
+lemma trivial_limit_at_bot_linorder: "\<not> trivial_limit (at_bot ::('a::linorder) filter)"
+  unfolding trivial_limit_def
+  by (metis eventually_at_bot_linorder order_refl)
+
+lemma trivial_limit_at_top_linorder: "\<not> trivial_limit (at_top ::('a::linorder) filter)"
+  unfolding trivial_limit_def
+  by (metis eventually_at_top_linorder order_refl)
+
 subsection {* Sequentially *}
 
 abbreviation sequentially :: "nat filter"
@@ -1034,10 +1042,17 @@
 lemma tendsto_le_const:
   fixes f :: "'a \<Rightarrow> 'b::linorder_topology"
   assumes F: "\<not> trivial_limit F"
-  assumes x: "(f ---> x) F" and a: "eventually (\<lambda>x. a \<le> f x) F"
+  assumes x: "(f ---> x) F" and a: "eventually (\<lambda>i. a \<le> f i) F"
   shows "a \<le> x"
   using F x tendsto_const a by (rule tendsto_le)
 
+lemma tendsto_ge_const:
+  fixes f :: "'a \<Rightarrow> 'b::linorder_topology"
+  assumes F: "\<not> trivial_limit F"
+  assumes x: "(f ---> x) F" and a: "eventually (\<lambda>i. a \<ge> f i) F"
+  shows "a \<ge> x"
+  by (rule tendsto_le [OF F tendsto_const x a])
+
 subsubsection {* Rules about @{const Lim} *}
 
 lemma (in t2_space) tendsto_Lim: