diff -r 6a131df8e3d9 -r 82df5181d699 src/HOL/Multivariate_Analysis/Path_Connected.thy --- a/src/HOL/Multivariate_Analysis/Path_Connected.thy Wed May 25 13:13:35 2016 +0200 +++ b/src/HOL/Multivariate_Analysis/Path_Connected.thy Wed May 25 16:38:35 2016 +0100 @@ -2073,10 +2073,26 @@ "2 \ DIM('N::euclidean_space) \ path_connected(ball a r - {a::'N})" by (simp add: path_connected_open_delete) -lemma connected_punctured_ball: +corollary connected_punctured_ball: "2 \ DIM('N::euclidean_space) \ connected(ball a r - {a::'N})" by (simp add: connected_open_delete) +corollary connected_open_delete_finite: + fixes S T::"'a::euclidean_space set" + assumes S: "open S" "connected S" and 2: "2 \ DIM('a)" and "finite T" + shows "connected(S - T)" + using \finite T\ S +proof (induct T) + case empty + show ?case using \connected S\ by simp +next + case (insert x F) + then have "connected (S-F)" by auto + moreover have "open (S - F)" using finite_imp_closed[OF \finite F\] \open S\ by auto + ultimately have "connected (S - F - {x})" using connected_open_delete[OF _ _ 2] by auto + thus ?case by (metis Diff_insert) +qed + subsection\Relations between components and path components\ lemma open_connected_component: