src/ZF/List.thy
changeset 1926 1957ae3f9301
parent 1806 12708740f58d
child 2539 ddd22ceee8cc
--- a/src/ZF/List.thy	Tue Aug 20 12:32:16 1996 +0200
+++ b/src/ZF/List.thy	Tue Aug 20 12:36:58 1996 +0200
@@ -49,6 +49,8 @@
   length :: i=>i
   "length(l)   == list_rec(l,  0,  %x xs r. succ(r))"
 
+  set_of_list :: i=>i
+  "set_of_list(l)   == list_rec(l,  0,  %x xs r. cons(x,r))"
 
 consts  (*Cannot use constdefs because @ is not an identifier*)
   "@"        :: [i,i]=>i                        (infixr 60)