src/CCL/Set.thy
changeset 24825 c4f13ab78f9d
parent 20140 98acc6d0fab6
child 32153 a0e57fb1b930
--- a/src/CCL/Set.thy	Wed Oct 03 19:49:33 2007 +0200
+++ b/src/CCL/Set.thy	Wed Oct 03 21:29:05 2007 +0200
@@ -16,8 +16,8 @@
 consts
   Collect       :: "['a => o] => 'a set"                    (*comprehension*)
   Compl         :: "('a set) => 'a set"                     (*complement*)
-  Int           :: "['a set, 'a set] => 'a set"         (infixl 70)
-  Un            :: "['a set, 'a set] => 'a set"         (infixl 65)
+  Int           :: "['a set, 'a set] => 'a set"         (infixl "Int" 70)
+  Un            :: "['a set, 'a set] => 'a set"         (infixl "Un" 65)
   Union         :: "(('a set)set) => 'a set"                (*...of a set*)
   Inter         :: "(('a set)set) => 'a set"                (*...of a set*)
   UNION         :: "['a set, 'a => 'b set] => 'b set"       (*general*)
@@ -25,11 +25,10 @@
   Ball          :: "['a set, 'a => o] => o"                 (*bounded quants*)
   Bex           :: "['a set, 'a => o] => o"                 (*bounded quants*)
   mono          :: "['a set => 'b set] => o"                (*monotonicity*)
-  ":"           :: "['a, 'a set] => o"                  (infixl 50) (*membership*)
-  "<="          :: "['a set, 'a set] => o"              (infixl 50)
+  mem           :: "['a, 'a set] => o"                  (infixl ":" 50) (*membership*)
+  subset        :: "['a set, 'a set] => o"              (infixl "<=" 50)
   singleton     :: "'a => 'a set"                       ("{_}")
   empty         :: "'a set"                             ("{}")
-  "oo"          :: "['b => 'c, 'a => 'b, 'a] => 'c"     (infixr 50) (*composition*)
 
 syntax
   "@Coll"       :: "[idt, o] => 'a set"                 ("(1{_./ _})") (*collection*)