# HG changeset patch # User paulson # Date 1464190747 -3600 # Node ID 1aa23fe79b9761914f68bfb26da701f2ee29260a # Parent 82df5181d69988f3df7987cff1104ba7e112dd16 moved two theorems diff -r 82df5181d699 -r 1aa23fe79b97 src/HOL/Multivariate_Analysis/Conformal_Mappings.thy --- a/src/HOL/Multivariate_Analysis/Conformal_Mappings.thy Wed May 25 16:38:35 2016 +0100 +++ b/src/HOL/Multivariate_Analysis/Conformal_Mappings.thy Wed May 25 16:39:07 2016 +0100 @@ -9,33 +9,6 @@ begin -lemma finite_ball_avoid: - assumes "open S" "finite X" "p \ S" - shows "\e>0. \w\ball p e. w\S \ (w\p \ w\X)" -proof - - obtain e1 where "0 < e1" and e1_b:"ball p e1 \ S" - using open_contains_ball_eq[OF \open S\] assms by auto - obtain e2 where "0x\X. x \ p \ e2 \ dist p x" - using finite_set_avoid[OF \finite X\,of p] by auto - hence "\w\ball p (min e1 e2). w\S \ (w\p \ w\X)" using e1_b by auto - thus "\e>0. \w\ball p e. w \ S \ (w \ p \ w \ X)" using \e2>0\ \e1>0\ - apply (rule_tac x="min e1 e2" in exI) - by auto -qed - -lemma finite_cball_avoid: - fixes S :: "'a :: euclidean_space set" - assumes "open S" "finite X" "p \ S" - shows "\e>0. \w\cball p e. w\S \ (w\p \ w\X)" -proof - - obtain e1 where "e1>0" and e1: "\w\ball p e1. w\S \ (w\p \ w\X)" - using finite_ball_avoid[OF assms] by auto - define e2 where "e2 \ e1/2" - have "e2>0" and "e2e1>0\ by auto - then have "cball p e2 \ ball p e1" by (subst cball_subset_ball_iff,auto) - then show "\e>0. \w\cball p e. w \ S \ (w \ p \ w \ X)" using \e2>0\ e1 by auto -qed - subsection\Cauchy's inequality and more versions of Liouville\ lemma Cauchy_higher_deriv_bound: