diff -r 4c51ab632cda -r 2b8c2a7547ab src/ZF/ex/TF.thy --- a/src/ZF/ex/TF.thy Mon Feb 05 21:33:14 1996 +0100 +++ b/src/ZF/ex/TF.thy Tue Feb 06 12:27:17 1996 +0100 @@ -1,6 +1,6 @@ -(* Title: ZF/ex/TF.thy +(* Title: ZF/ex/TF.thy ID: $Id$ - Author: Lawrence C Paulson, Cambridge University Computer Laboratory + Author: Lawrence C Paulson, Cambridge University Computer Laboratory Copyright 1994 University of Cambridge Trees & forests, a mutually recursive type definition. @@ -24,14 +24,14 @@ defs TF_rec_def - "TF_rec(z,b,c,d) == Vrec(z, - %z r. tree_forest_case(%x f. b(x, f, r`f), - c, - %t f. d(t, f, r`t, r`f), z))" + "TF_rec(z,b,c,d) == Vrec(z, + %z r. tree_forest_case(%x f. b(x, f, r`f), + c, + %t f. d(t, f, r`t, r`f), z))" list_of_TF_def "list_of_TF(z) == TF_rec(z, %x f r. [Tcons(x,f)], [], - %t f r1 r2. Cons(t, r2))" + %t f r1 r2. Cons(t, r2))" TF_of_list_def "TF_of_list(f) == list_rec(f, Fnil, %t f r. Fcons(t,r))"