src/HOL/Induct/LList.thy
changeset 3842 b55686a7b22c
parent 3120 c58423c20740
child 5977 9f0c8869cf71
--- a/src/HOL/Induct/LList.thy	Fri Oct 10 18:37:49 1997 +0200
+++ b/src/HOL/Induct/LList.thy	Fri Oct 10 19:02:28 1997 +0200
@@ -11,7 +11,7 @@
 bounds on the amount of lookahead required.
 
 Could try (but would it work for the gfp analogue of term?)
-  LListD_Fun_def "LListD_Fun(A) == (%Z.diag({Numb(0)}) <++> diag(A) <**> Z)"
+  LListD_Fun_def "LListD_Fun(A) == (%Z. diag({Numb(0)}) <++> diag(A) <**> Z)"
 
 A nice but complex example would be [ML for the Working Programmer, page 176]
   from(1) = enumerate (Lmap (Lmap(pack), makeqq(from(1),from(1))))
@@ -74,7 +74,7 @@
             |] ==> (CONS a M, CONS b N) : LListD(r)"
 
 translations
-  "case p of LNil => a | LCons x l => b" == "llist_case a (%x l.b) p"
+  "case p of LNil => a | LCons x l => b" == "llist_case a (%x l. b) p"
 
 
 defs
@@ -108,7 +108,7 @@
   llist_corec_def
    "llist_corec a f == 
        Abs_llist(LList_corec a 
-                 (%z.case f z of Inl x    => Inl(x)
+                 (%z. case f z of Inl x    => Inl(x)
                                | Inr(v,w) => Inr(Leaf(v), w)))"
 
   llistD_Fun_def