src/HOL/Analysis/Path_Connected.thy
changeset 69712 dc85b5b3a532
parent 69661 a03a63b81f44
child 69939 812ce526da33
--- a/src/HOL/Analysis/Path_Connected.thy	Tue Jan 22 10:50:47 2019 +0000
+++ b/src/HOL/Analysis/Path_Connected.thy	Tue Jan 22 12:00:16 2019 +0000
@@ -2851,7 +2851,7 @@
        and cc: "connected_component (- frontier s) x y"
     have "connected_component_set (- frontier s) x \<inter> frontier s \<noteq> {}"
       apply (rule connected_Int_frontier, simp)
-      apply (metis IntI cc connected_component_in connected_component_refl empty_iff interiorE mem_Collect_eq set_rev_mp x)
+      apply (metis IntI cc connected_component_in connected_component_refl empty_iff interiorE mem_Collect_eq rev_subsetD x)
       using  y cc
       by blast
     then have "bounded (connected_component_set (- frontier s) x)"