src/HOL/Analysis/Path_Connected.thy
changeset 69661 a03a63b81f44
parent 69620 19d8a59481db
child 69712 dc85b5b3a532
--- a/src/HOL/Analysis/Path_Connected.thy	Mon Jan 14 18:33:53 2019 +0000
+++ b/src/HOL/Analysis/Path_Connected.thy	Mon Jan 14 18:35:03 2019 +0000
@@ -767,10 +767,7 @@
 lemma path_image_subpath_gen:
   fixes g :: "_ \<Rightarrow> 'a::real_normed_vector"
   shows "path_image(subpath u v g) = g ` (closed_segment u v)"
-  apply (simp add: closed_segment_real_eq path_image_def subpath_def)
-  apply (subst o_def [of g, symmetric])
-  apply (simp add: image_comp [symmetric])
-  done
+  by (auto simp add: closed_segment_real_eq path_image_def subpath_def)
 
 lemma path_image_subpath:
   fixes g :: "real \<Rightarrow> 'a::real_normed_vector"