src/HOL/Topological_Spaces.thy
changeset 53374 a14d2a854c02
parent 53215 5e47c31c6f7c
child 53381 355a4cac5440
--- a/src/HOL/Topological_Spaces.thy	Tue Sep 03 00:51:08 2013 +0200
+++ b/src/HOL/Topological_Spaces.thy	Tue Sep 03 01:12:40 2013 +0200
@@ -2145,7 +2145,8 @@
       moreover obtain b where "b \<in> B" "x < b" "b < min a y"
         using cInf_less_iff[of "B \<inter> {x <..}" x "min a y"] `?z < a` `?z < y` `x < y` `y \<in> B`
         by (auto intro: less_imp_le)
-      moreover then have "?z \<le> b"
+      moreover have "?z \<le> b"
+        using `b \<in> B` `x < b`
         by (intro cInf_lower[where z=x]) auto
       moreover have "b \<in> U"
         using `x \<le> ?z` `?z \<le> b` `b < min a y`