src/HOL/Analysis/Path_Connected.thy
changeset 68913 55b12fde48d0
parent 68721 53ad5c01be3f
child 69064 5840724b1d71
equal deleted inserted replaced
68912:ecc76fa24a32 68913:55b12fde48d0
  1410   ultimately show ?thesis
  1410   ultimately show ?thesis
  1411     by (rule_tac x="e/2" in exI) auto
  1411     by (rule_tac x="e/2" in exI) auto
  1412 qed
  1412 qed
  1413 
  1413 
  1414 
  1414 
  1415 section \<open>Path component, considered as a "joinability" relation (from Tom Hales)\<close>
  1415 section \<open>Path component, considered as a "joinability" relation\<close>
       
  1416 
       
  1417 text \<open>(by Tom Hales)\<close>
  1416 
  1418 
  1417 definition%important "path_component s x y \<longleftrightarrow>
  1419 definition%important "path_component s x y \<longleftrightarrow>
  1418   (\<exists>g. path g \<and> path_image g \<subseteq> s \<and> pathstart g = x \<and> pathfinish g = y)"
  1420   (\<exists>g. path g \<and> path_image g \<subseteq> s \<and> pathstart g = x \<and> pathfinish g = y)"
  1419 
  1421 
  1420 abbreviation%important
  1422 abbreviation%important