Subst/AList.thy
changeset 194 b93cc55cb7ab
parent 106 d27056ec0a5a
--- a/Subst/AList.thy	Fri Dec 02 10:26:59 1994 +0100
+++ b/Subst/AList.thy	Fri Dec 02 11:43:20 1994 +0100
@@ -14,7 +14,7 @@
 
 rules
 
-  alist_rec_def "alist_rec(al,b,c) == list_rec(al, b, split(c))"
+  alist_rec_def "alist_rec(al,b,c) == list_rec(b, split(c), al)"
 
   assoc_def     "assoc(v,d,al) == alist_rec(al,d,%x y xs g.if(v=x,y,g))"