generalize compact_path_image to topological_space
authorhoelzl
Thu, 17 Jan 2013 11:57:17 +0100
changeset 50935 cfdf19d3ca32
parent 50934 a076e01b803f
child 50936 b28f258ebc1a
generalize compact_path_image to topological_space
src/HOL/Multivariate_Analysis/Path_Connected.thy
--- a/src/HOL/Multivariate_Analysis/Path_Connected.thy	Thu Jan 17 14:15:10 2013 +0100
+++ b/src/HOL/Multivariate_Analysis/Path_Connected.thy	Thu Jan 17 11:57:17 2013 +0100
@@ -57,7 +57,7 @@
   apply (rule convex_connected, rule convex_real_interval)
   done
 
-lemma compact_path_image[intro]: "path g \<Longrightarrow> compact(path_image g :: 'a::metric_space set)"
+lemma compact_path_image[intro]: "path g \<Longrightarrow> compact(path_image g)"
   unfolding path_def path_image_def
   by (erule compact_continuous_image, rule compact_interval)