src/HOL/Set.thy
changeset 2965 afbda7e26f15
parent 2912 3fac3e8d5d3e
child 3222 726a9b069947
--- a/src/HOL/Set.thy	Wed Apr 16 18:25:46 1997 +0200
+++ b/src/HOL/Set.thy	Wed Apr 16 18:46:01 1997 +0200
@@ -113,8 +113,8 @@
   "*Bex"        :: [pttrn, 'a set, bool] => bool      ("(3\\<exists> _\\<in>_./ _)" [0, 0, 10] 10)
 
 translations
-  "op \\<subseteq>" => "op <="
-  "op \\<subset>" => "op <"
+  "op \\<subseteq>" => "op <= :: [_ set, _ set] => bool"
+  "op \\<subset>" => "op <  :: [_ set, _ set] => bool"