src/HOL/Analysis/Jordan_Curve.thy
changeset 69508 2a4c8a2a3f8e
parent 68651 16d98ef49a2c
child 69922 4a9167f377b0
--- a/src/HOL/Analysis/Jordan_Curve.thy	Wed Dec 26 20:57:23 2018 +0100
+++ b/src/HOL/Analysis/Jordan_Curve.thy	Thu Dec 27 19:48:28 2018 +0100
@@ -374,7 +374,7 @@
       qed
       then have "connected_component (- (path_image u \<union> path_image d \<union> path_image g)) x y"
         by (simp add: Un_ac)
-      moreover have "~(connected_component (- (path_image c)) x y)"
+      moreover have "\<not>(connected_component (- (path_image c)) x y)"
         by (metis (no_types, lifting) \<open>\<not> bounded outer\<close> \<open>bounded inner\<close> \<open>x \<in> inner\<close> \<open>y \<in> outer\<close> componentsE connected_component_eq inner mem_Collect_eq outer)
       ultimately show False
         by (auto simp: ud_Un [symmetric] connected_component_def)