Subst/AList.thy
changeset 106 d27056ec0a5a
parent 0 7949f97df77a
child 194 b93cc55cb7ab
--- a/Subst/AList.thy	Thu Aug 18 11:30:27 1994 +0200
+++ b/Subst/AList.thy	Thu Aug 18 11:40:54 1994 +0200
@@ -9,14 +9,13 @@
 
 consts
 
-  alist_rec  :: "[('a*'b) list,'c,['a,'b,('a*'b) list,'c]=>'c]=>'c"
+  alist_rec  :: "[('a*'b)list, 'c, ['a, 'b, ('a*'b)list, 'c]=>'c] => 'c"
   assoc      :: "['a,'b,('a*'b) list] => 'b"
 
 rules
 
-  alist_rec_def 
-    "alist_rec(al,b,c) == list_rec(al,b,%p xs g.split(p,%x y.c(x,y,xs,g)))"
+  alist_rec_def "alist_rec(al,b,c) == list_rec(al, b, split(c))"
 
-  assoc_def    "assoc(v,d,al) == alist_rec(al,d,%x y xs g.if(v=x,y,g))"
+  assoc_def     "assoc(v,d,al) == alist_rec(al,d,%x y xs g.if(v=x,y,g))"
 
 end