src/HOLCF/Cfun3.thy
changeset 3842 b55686a7b22c
parent 3327 9b8e638f8602
child 10834 a7897aebbffc
--- a/src/HOLCF/Cfun3.thy	Fri Oct 10 18:37:49 1997 +0200
+++ b/src/HOLCF/Cfun3.thy	Fri Oct 10 19:02:28 1997 +0200
@@ -20,7 +20,7 @@
 defs
 
 Istrictify_def  "Istrictify f x == if x=UU then UU else f`x"    
-strictify_def   "strictify == (LAM f x.Istrictify f x)"
+strictify_def   "strictify == (LAM f x. Istrictify f x)"
 
 consts
         ID      :: "('a::cpo) -> 'a"
@@ -32,7 +32,7 @@
 
 defs
 
-  ID_def        "ID ==(LAM x.x)"
-  oo_def        "cfcomp == (LAM f g x.f`(g`x))" 
+  ID_def        "ID ==(LAM x. x)"
+  oo_def        "cfcomp == (LAM f g x. f`(g`x))" 
 
 end