src/HOL/Multivariate_Analysis/Topology_Euclidean_Space.thy
changeset 57275 0ddb5b755cdc
parent 56742 678a52e676b6
child 57276 49c51eeaa623
--- a/src/HOL/Multivariate_Analysis/Topology_Euclidean_Space.thy	Wed Jun 18 15:23:40 2014 +0200
+++ b/src/HOL/Multivariate_Analysis/Topology_Euclidean_Space.thy	Wed Jun 18 07:31:12 2014 +0200
@@ -1855,7 +1855,7 @@
     from cInf_lessD[OF _ this] False obtain y where y: "x < y" "y \<in> I" "f y < a"
       by auto
     then have "eventually (\<lambda>x. x \<in> I \<longrightarrow> f x < a) (at_right x)"
-      unfolding eventually_at_right by (metis less_imp_le le_less_trans mono)
+      unfolding eventually_at_right[OF `x < y`] by (metis less_imp_le le_less_trans mono)
     then show "eventually (\<lambda>x. f x < a) (at x within ({x<..} \<inter> I))"
       unfolding eventually_at_filter by eventually_elim simp
   qed