diff -r e125fc7a1183 -r 5750eba8820d src/CCL/ex/List.thy --- a/src/CCL/ex/List.thy Wed Jun 21 11:35:10 1995 +0200 +++ b/src/CCL/ex/List.thy Wed Jun 21 15:01:07 1995 +0200 @@ -33,12 +33,12 @@ isort_def "isort(f) == lam l.lrec(l,[],%h t g.insert(f,h,g))" partition_def - "partition(f,l) == letrec part l a b be lcase(l,,%x xs.\ -\ if f`x then part(xs,x$a,b) else part(xs,a,x$b)) \ -\ in part(l,[],[])" - qsort_def "qsort(f) == lam l. letrec qsortx l be lcase(l,[],%h t. \ -\ let p be partition(f`h,t) \ -\ in split(p,%x y.qsortx(x) @ h$qsortx(y))) \ -\ in qsortx(l)" + "partition(f,l) == letrec part l a b be lcase(l,,%x xs. + if f`x then part(xs,x$a,b) else part(xs,a,x$b)) + in part(l,[],[])" + qsort_def "qsort(f) == lam l. letrec qsortx l be lcase(l,[],%h t. + let p be partition(f`h,t) + in split(p,%x y.qsortx(x) @ h$qsortx(y))) + in qsortx(l)" end