src/HOL/Analysis/Retracts.thy
changeset 71193 777d673fa672
parent 71184 d62fdaafdafc
child 72490 df988eac234e
equal deleted inserted replaced
71192:a8ccea88b725 71193:777d673fa672
  2590   assumes "S homeomorphic cbox a b" "2 \<le> DIM('a)"
  2590   assumes "S homeomorphic cbox a b" "2 \<le> DIM('a)"
  2591   shows "connected(-S)"
  2591   shows "connected(-S)"
  2592   using assms path_connected_complement_homeomorphic_interval path_connected_imp_connected by blast
  2592   using assms path_connected_complement_homeomorphic_interval path_connected_imp_connected by blast
  2593 
  2593 
  2594 
  2594 
  2595 lemma path_connected_arc_complement:
       
  2596   fixes \<gamma> :: "real \<Rightarrow> 'a::euclidean_space"
       
  2597   assumes "arc \<gamma>" "2 \<le> DIM('a)"
       
  2598   shows "path_connected(- path_image \<gamma>)"
       
  2599 proof -
       
  2600   have "path_image \<gamma> homeomorphic {0..1::real}"
       
  2601     by (simp add: assms homeomorphic_arc_image_interval)
       
  2602   then
       
  2603   show ?thesis
       
  2604     apply (rule path_connected_complement_homeomorphic_convex_compact)
       
  2605       apply (auto simp: assms)
       
  2606     done
       
  2607 qed
       
  2608 
       
  2609 lemma connected_arc_complement:
       
  2610   fixes \<gamma> :: "real \<Rightarrow> 'a::euclidean_space"
       
  2611   assumes "arc \<gamma>" "2 \<le> DIM('a)"
       
  2612   shows "connected(- path_image \<gamma>)"
       
  2613   by (simp add: assms path_connected_arc_complement path_connected_imp_connected)
       
  2614 
       
  2615 lemma inside_arc_empty:
       
  2616   fixes \<gamma> :: "real \<Rightarrow> 'a::euclidean_space"
       
  2617   assumes "arc \<gamma>"
       
  2618     shows "inside(path_image \<gamma>) = {}"
       
  2619 proof (cases "DIM('a) = 1")
       
  2620   case True
       
  2621   then show ?thesis
       
  2622     using assms connected_arc_image connected_convex_1_gen inside_convex by blast
       
  2623 next
       
  2624   case False
       
  2625   show ?thesis
       
  2626   proof (rule inside_bounded_complement_connected_empty)
       
  2627     show "connected (- path_image \<gamma>)"
       
  2628       apply (rule connected_arc_complement [OF assms])
       
  2629       using False
       
  2630       by (metis DIM_ge_Suc0 One_nat_def Suc_1 not_less_eq_eq order_class.order.antisym)
       
  2631     show "bounded (path_image \<gamma>)"
       
  2632       by (simp add: assms bounded_arc_image)
       
  2633   qed
       
  2634 qed
       
  2635 
       
  2636 lemma inside_simple_curve_imp_closed:
       
  2637   fixes \<gamma> :: "real \<Rightarrow> 'a::euclidean_space"
       
  2638     shows "\<lbrakk>simple_path \<gamma>; x \<in> inside(path_image \<gamma>)\<rbrakk> \<Longrightarrow> pathfinish \<gamma> = pathstart \<gamma>"
       
  2639   using arc_simple_path  inside_arc_empty by blast
       
  2640 
       
  2641 end
  2595 end