src/HOL/Limits.thy
changeset 57275 0ddb5b755cdc
parent 56541 0e3abadbef39
child 57276 49c51eeaa623
--- a/src/HOL/Limits.thy	Wed Jun 18 15:23:40 2014 +0200
+++ b/src/HOL/Limits.thy	Wed Jun 18 07:31:12 2014 +0200
@@ -54,6 +54,11 @@
   "at_bot \<le> (at_infinity :: real filter)"
   unfolding at_infinity_eq_at_top_bot by simp
 
+lemma filterlim_at_top_imp_at_infinity:
+  fixes f :: "_ \<Rightarrow> real"
+  shows "filterlim f at_top F \<Longrightarrow> filterlim f at_infinity F"
+  by (rule filterlim_mono[OF _ at_top_le_at_infinity order_refl])
+
 subsubsection {* Boundedness *}
 
 definition Bfun :: "('a \<Rightarrow> 'b::metric_space) \<Rightarrow> 'a filter \<Rightarrow> bool" where