src/HOL/Analysis/Arcwise_Connected.thy
changeset 71025 be8cec1abcbb
parent 70817 dd675800469d
child 71028 c2465b429e6e
--- a/src/HOL/Analysis/Arcwise_Connected.thy	Mon Nov 04 20:24:52 2019 +0100
+++ b/src/HOL/Analysis/Arcwise_Connected.thy	Mon Nov 04 17:18:25 2019 -0500
@@ -8,6 +8,11 @@
 imports Path_Connected Ordered_Euclidean_Space "HOL-Computational_Algebra.Primes"
 begin
 
+lemma path_connected_interval [simp]:
+  fixes a b::"'a::ordered_euclidean_space"
+  shows "path_connected {a..b}"
+  using is_interval_cc is_interval_path_connected by blast
+
 subsection \<open>The Brouwer reduction theorem\<close>
 
 theorem Brouwer_reduction_theorem_gen: