src/HOL/Multivariate_Analysis/Ordered_Euclidean_Space.thy
changeset 61076 bdc1e2f0a86a
parent 60420 884f54e01427
child 61169 4de9ff3ea29a
--- a/src/HOL/Multivariate_Analysis/Ordered_Euclidean_Space.thy	Tue Sep 01 17:25:36 2015 +0200
+++ b/src/HOL/Multivariate_Analysis/Ordered_Euclidean_Space.thy	Tue Sep 01 22:32:58 2015 +0200
@@ -177,7 +177,7 @@
 text\<open>Instantiation for intervals on @{text ordered_euclidean_space}\<close>
 
 lemma
-  fixes a :: "'a\<Colon>ordered_euclidean_space"
+  fixes a :: "'a::ordered_euclidean_space"
   shows cbox_interval: "cbox a b = {a..b}"
     and interval_cbox: "{a..b} = cbox a b"
     and eucl_le_atMost: "{x. \<forall>i\<in>Basis. x \<bullet> i <= a \<bullet> i} = {..a}"
@@ -185,17 +185,17 @@
     by (auto simp: eucl_le[where 'a='a] eucl_less_def box_def cbox_def)
 
 lemma closed_eucl_atLeastAtMost[simp, intro]:
-  fixes a :: "'a\<Colon>ordered_euclidean_space"
+  fixes a :: "'a::ordered_euclidean_space"
   shows "closed {a..b}"
   by (simp add: cbox_interval[symmetric] closed_cbox)
 
 lemma closed_eucl_atMost[simp, intro]:
-  fixes a :: "'a\<Colon>ordered_euclidean_space"
+  fixes a :: "'a::ordered_euclidean_space"
   shows "closed {..a}"
   by (simp add: eucl_le_atMost[symmetric])
 
 lemma closed_eucl_atLeast[simp, intro]:
-  fixes a :: "'a\<Colon>ordered_euclidean_space"
+  fixes a :: "'a::ordered_euclidean_space"
   shows "closed {a..}"
   by (simp add: eucl_le_atLeast[symmetric])