src/HOLCF/ex/Loop.thy
changeset 21404 eb85850d3eb7
parent 19763 ec18656a2c10
child 25895 0eaadfa8889e
--- a/src/HOLCF/ex/Loop.thy	Fri Nov 17 02:19:55 2006 +0100
+++ b/src/HOLCF/ex/Loop.thy	Fri Nov 17 02:20:03 2006 +0100
@@ -10,10 +10,11 @@
 begin
 
 definition
-  step  :: "('a -> tr)->('a -> 'a)->'a->'a"
+  step  :: "('a -> tr)->('a -> 'a)->'a->'a" where
   "step = (LAM b g x. If b$x then g$x else x fi)"
 
-  while :: "('a -> tr)->('a -> 'a)->'a->'a"
+definition
+  while :: "('a -> tr)->('a -> 'a)->'a->'a" where
   "while = (LAM b g. fix$(LAM f x. If b$x then f$(g$x) else x fi))"
 
 (* ------------------------------------------------------------------------- *)