src/HOL/Analysis/Homeomorphism.thy
changeset 69508 2a4c8a2a3f8e
parent 69313 b021008c5397
child 69620 19d8a59481db
equal deleted inserted replaced
69506:7d59af98af29 69508:2a4c8a2a3f8e
   199 qed
   199 qed
   200 
   200 
   201 lemma%unimportant segment_to_rel_frontier:
   201 lemma%unimportant segment_to_rel_frontier:
   202   fixes x :: "'a::euclidean_space"
   202   fixes x :: "'a::euclidean_space"
   203   assumes S: "convex S" "bounded S" and x: "x \<in> rel_interior S"
   203   assumes S: "convex S" "bounded S" and x: "x \<in> rel_interior S"
   204       and y: "y \<in> S" and xy: "~(x = y \<and> S = {x})"
   204       and y: "y \<in> S" and xy: "\<not>(x = y \<and> S = {x})"
   205   obtains z where "z \<in> rel_frontier S" "y \<in> closed_segment x z"
   205   obtains z where "z \<in> rel_frontier S" "y \<in> closed_segment x z"
   206                   "open_segment x z \<subseteq> rel_interior S"
   206                   "open_segment x z \<subseteq> rel_interior S"
   207 proof (cases "x=y")
   207 proof (cases "x=y")
   208   case True
   208   case True
   209   with xy have "S \<noteq> {x}"
   209   with xy have "S \<noteq> {x}"