src/HOL/Filter.thy
changeset 63556 36e9732988ce
parent 63540 f8652d0534fa
child 63967 2aa42596edc3
--- a/src/HOL/Filter.thy	Sun Jul 24 16:48:41 2016 +0200
+++ b/src/HOL/Filter.thy	Thu Jul 28 17:16:16 2016 +0200
@@ -618,6 +618,12 @@
   unfolding at_top_def
   by (subst eventually_INF_base) (auto simp: eventually_principal intro: max.cobounded1 max.cobounded2)
 
+lemma eventually_at_top_linorderI:
+  fixes c::"'a::linorder"
+  assumes "\<And>x. c \<le> x \<Longrightarrow> P x"
+  shows "eventually P at_top"
+  using assms by (auto simp: eventually_at_top_linorder)
+
 lemma eventually_ge_at_top:
   "eventually (\<lambda>x. (c::_::linorder) \<le> x) at_top"
   unfolding eventually_at_top_linorder by auto