src/HOL/Analysis/Convex_Euclidean_Space.thy
changeset 71029 934e0044e94b
parent 71008 e892f7a1fd83
child 71030 b6e69c71a9f6
--- a/src/HOL/Analysis/Convex_Euclidean_Space.thy	Sun Nov 03 20:38:08 2019 +0100
+++ b/src/HOL/Analysis/Convex_Euclidean_Space.thy	Mon Nov 04 17:06:18 2019 +0000
@@ -2615,6 +2615,10 @@
     "x \<in> open_segment a b \<longleftrightarrow> a \<noteq> b \<and> (\<exists>u. 0 < u \<and> u < 1 \<and> x = (1 - u) *\<^sub>R a + u *\<^sub>R b)"
   using less_eq_real_def by (auto simp: segment algebra_simps)
 
+lemma closed_segmentI:
+  "u \<in> {0..1} \<Longrightarrow> z = (1 - u) *\<^sub>R a + u *\<^sub>R b \<Longrightarrow> z \<in> closed_segment a b"
+  by (auto simp: closed_segment_def)
+
 lemma closed_segment_linear_image:
   "closed_segment (f a) (f b) = f ` (closed_segment a b)" if "linear f"
 proof -