src/HOL/Analysis/Further_Topology.thy
changeset 64847 54f5afc9c413
parent 64846 de4e3df6693d
child 64911 f0e07600de47
equal deleted inserted replaced
64846:de4e3df6693d 64847:54f5afc9c413
  3035 lemma not_simply_connected_circle:
  3035 lemma not_simply_connected_circle:
  3036   fixes a :: complex
  3036   fixes a :: complex
  3037   shows "0 < r \<Longrightarrow> \<not> simply_connected(sphere a r)"
  3037   shows "0 < r \<Longrightarrow> \<not> simply_connected(sphere a r)"
  3038 by (simp add: simply_connected_sphere_eq)
  3038 by (simp add: simply_connected_sphere_eq)
  3039 
  3039 
  3040   
  3040 
  3041 proposition simply_connected_punctured_convex:
  3041 proposition simply_connected_punctured_convex:
  3042   fixes a :: "'a::euclidean_space"
  3042   fixes a :: "'a::euclidean_space"
  3043   assumes "convex S" and 3: "3 \<le> aff_dim S"
  3043   assumes "convex S" and 3: "3 \<le> aff_dim S"
  3044     shows "simply_connected(S - {a})"
  3044     shows "simply_connected(S - {a})"
  3045 proof (cases "a \<in> rel_interior S")
  3045 proof (cases "a \<in> rel_interior S")
  4098 qed
  4098 qed
  4099 
  4099 
  4100 
  4100 
  4101 subsection\<open>The "Borsukian" property of sets\<close>
  4101 subsection\<open>The "Borsukian" property of sets\<close>
  4102 
  4102 
  4103 text\<open>This doesn't have a standard name. Kuratowski uses "contractible with respect to [S^1]"
  4103 text\<open>This doesn't have a standard name. Kuratowski uses ``contractible with respect to $[S^1]$''
  4104  while Whyburn uses "property b". It's closely related to unicoherence.\<close>
  4104  while Whyburn uses ``property b''. It's closely related to unicoherence.\<close>
  4105 
  4105 
  4106 definition Borsukian where
  4106 definition Borsukian where
  4107     "Borsukian S \<equiv>
  4107     "Borsukian S \<equiv>
  4108         \<forall>f. continuous_on S f \<and> f ` S \<subseteq> (- {0::complex})
  4108         \<forall>f. continuous_on S f \<and> f ` S \<subseteq> (- {0::complex})
  4109             \<longrightarrow> (\<exists>a. homotopic_with (\<lambda>h. True) S (- {0}) f (\<lambda>x. a))"
  4109             \<longrightarrow> (\<exists>a. homotopic_with (\<lambda>h. True) S (- {0}) f (\<lambda>x. a))"