src/HOL/List.thy
changeset 2512 0231e4f467f2
parent 2369 8100f00e8950
child 2608 450c9b682a92
--- a/src/HOL/List.thy	Fri Jan 17 10:04:28 1997 +0100
+++ b/src/HOL/List.thy	Fri Jan 17 10:09:46 1997 +0100
@@ -3,10 +3,7 @@
     Author:     Tobias Nipkow
     Copyright   1994 TU Muenchen
 
-Definition of type 'a list as a datatype. This allows primrec to work.
-
-TODO: delete list_all from this theory and from ex/Sorting, etc.
-      use set_of_list instead
+The datatype of finite lists.
 *)
 
 List = Arith +
@@ -35,18 +32,15 @@
   (* list Enumeration *)
   "@list"     :: args => 'a list                          ("[(_)]")
 
-  (* Special syntax for list_all and filter *)
-  "@Alls"     :: [idt, 'a list, bool] => bool             ("(2Alls _:_./ _)" 10)
+  (* Special syntax for filter *)
   "@filter"   :: [idt, 'a list, bool] => 'a list          ("(1[_:_ ./ _])")
 
 translations
   "[x, xs]"     == "x#[xs]"
   "[x]"         == "x#[]"
   "[x:xs . P]"  == "filter (%x.P) xs"
-  "Alls x:xs.P" == "list_all (%x.P) xs"
 
 syntax (symbols)
-  "op #"      :: ['a, 'a list] => 'a list                 (infixr "\\<bullet>" 65)
   "@filter"   :: [idt, 'a list, bool] => 'a list          ("(1[_\\<in>_ ./ _])")