src/HOL/Analysis/Brouwer_Fixpoint.thy
changeset 69566 c41954ee87cf
parent 69529 4ab9657b3257
child 69620 19d8a59481db
equal deleted inserted replaced
69565:1daf07b65385 69566:c41954ee87cf
   405 
   405 
   406 text \<open>Absolute retracts (AR), absolute neighbourhood retracts (ANR) and also Euclidean neighbourhood
   406 text \<open>Absolute retracts (AR), absolute neighbourhood retracts (ANR) and also Euclidean neighbourhood
   407 retracts (ENR). We define AR and ANR by specializing the standard definitions for a set to embedding
   407 retracts (ENR). We define AR and ANR by specializing the standard definitions for a set to embedding
   408 in spaces of higher dimension.
   408 in spaces of higher dimension.
   409 
   409 
   410 John Harrison writes: "This turns out to be sufficient (since any set in $\mathbb{R}^n$ can be
   410 John Harrison writes: "This turns out to be sufficient (since any set in \<open>\<real>\<^sup>n\<close> can be
   411 embedded as a closed subset of a convex subset of $\mathbb{R}^{n+1}$) to derive the usual
   411 embedded as a closed subset of a convex subset of \<open>\<real>\<^sup>n\<^sup>+\<^sup>1\<close>) to derive the usual
   412 definitions, but we need to split them into two implications because of the lack of type
   412 definitions, but we need to split them into two implications because of the lack of type
   413 quantifiers. Then ENR turns out to be equivalent to ANR plus local compactness."\<close>
   413 quantifiers. Then ENR turns out to be equivalent to ANR plus local compactness."\<close>
   414 
   414 
   415 definition%important AR :: "'a::topological_space set \<Rightarrow> bool" where
   415 definition%important AR :: "'a::topological_space set \<Rightarrow> bool" where
   416 "AR S \<equiv> \<forall>U. \<forall>S'::('a * real) set.
   416 "AR S \<equiv> \<forall>U. \<forall>S'::('a * real) set.