src/HOL/Analysis/Starlike.thy
changeset 69516 09bb8f470959
parent 69508 2a4c8a2a3f8e
child 69518 bf88364c9e94
equal deleted inserted replaced
69515:5bbb2bd564fa 69516:09bb8f470959
  4918   shows "\<lbrakk>closedin (subtopology euclidean U) S; x \<in> U; S \<noteq> {}; x \<notin> S\<rbrakk>
  4918   shows "\<lbrakk>closedin (subtopology euclidean U) S; x \<in> U; S \<noteq> {}; x \<notin> S\<rbrakk>
  4919          \<Longrightarrow> setdist {x} S > 0"
  4919          \<Longrightarrow> setdist {x} S > 0"
  4920   using less_eq_real_def setdist_eq_0_closedin by fastforce
  4920   using less_eq_real_def setdist_eq_0_closedin by fastforce
  4921 
  4921 
  4922 subsection%unimportant\<open>Basic lemmas about hyperplanes and halfspaces\<close>
  4922 subsection%unimportant\<open>Basic lemmas about hyperplanes and halfspaces\<close>
       
  4923 
       
  4924 lemma halfspace_Int_eq:
       
  4925      "{x. a \<bullet> x \<le> b} \<inter> {x. b \<le> a \<bullet> x} = {x. a \<bullet> x = b}"
       
  4926      "{x. b \<le> a \<bullet> x} \<inter> {x. a \<bullet> x \<le> b} = {x. a \<bullet> x = b}"
       
  4927   by auto
  4923 
  4928 
  4924 lemma hyperplane_eq_Ex:
  4929 lemma hyperplane_eq_Ex:
  4925   assumes "a \<noteq> 0" obtains x where "a \<bullet> x = b"
  4930   assumes "a \<noteq> 0" obtains x where "a \<bullet> x = b"
  4926   by (rule_tac x = "(b / (a \<bullet> a)) *\<^sub>R a" in that) (simp add: assms)
  4931   by (rule_tac x = "(b / (a \<bullet> a)) *\<^sub>R a" in that) (simp add: assms)
  4927 
  4932