src/HOL/Analysis/Path_Connected.thy
changeset 64394 141e1ed8d5a0
parent 64267 b9a1486e79be
child 64788 19f3d4af7a7d
equal deleted inserted replaced
64390:ad2c5f37f659 64394:141e1ed8d5a0
  1202 lemma simple_path_linepath[intro]: "a \<noteq> b \<Longrightarrow> simple_path (linepath a b)"
  1202 lemma simple_path_linepath[intro]: "a \<noteq> b \<Longrightarrow> simple_path (linepath a b)"
  1203   by (simp add: arc_imp_simple_path arc_linepath)
  1203   by (simp add: arc_imp_simple_path arc_linepath)
  1204 
  1204 
  1205 lemma linepath_trivial [simp]: "linepath a a x = a"
  1205 lemma linepath_trivial [simp]: "linepath a a x = a"
  1206   by (simp add: linepath_def real_vector.scale_left_diff_distrib)
  1206   by (simp add: linepath_def real_vector.scale_left_diff_distrib)
       
  1207 
       
  1208 lemma linepath_refl: "linepath a a = (\<lambda>x. a)"
       
  1209   by auto
  1207 
  1210 
  1208 lemma subpath_refl: "subpath a a g = linepath (g a) (g a)"
  1211 lemma subpath_refl: "subpath a a g = linepath (g a) (g a)"
  1209   by (simp add: subpath_def linepath_def algebra_simps)
  1212   by (simp add: subpath_def linepath_def algebra_simps)
  1210 
  1213 
  1211 lemma linepath_of_real: "(linepath (of_real a) (of_real b) x) = of_real ((1 - x)*a + x*b)"
  1214 lemma linepath_of_real: "(linepath (of_real a) (of_real b) x) = of_real ((1 - x)*a + x*b)"
  4359       done
  4362       done
  4360   qed
  4363   qed
  4361   with assms show ?thesis
  4364   with assms show ?thesis
  4362     by (simp add: simply_connected_eq_contractible_loop_any pathfinish_def pathstart_def)
  4365     by (simp add: simply_connected_eq_contractible_loop_any pathfinish_def pathstart_def)
  4363 qed
  4366 qed
       
  4367 
  4364 
  4368 
  4365 subsection\<open>Contractible sets\<close>
  4369 subsection\<open>Contractible sets\<close>
  4366 
  4370 
  4367 definition contractible where
  4371 definition contractible where
  4368  "contractible S \<equiv> \<exists>a. homotopic_with (\<lambda>x. True) S S id (\<lambda>x. a)"
  4372  "contractible S \<equiv> \<exists>a. homotopic_with (\<lambda>x. True) S S id (\<lambda>x. a)"