| author | wenzelm |
| Mon, 28 Feb 2000 13:39:45 +0100 | |
| changeset 8312 | b470bc28b59d |
| parent 244 | 929fc2c63bd0 |
| permissions | -rw-r--r-- |
(* Title: HOLCF/ex/loop.thy ID: $Id$ Author: Franz Regensburger Copyright 1993 Technische Universitaet Muenchen Theory for a loop primitive like while *) Loop = Tr2 + consts step :: "('a -> tr)->('a -> 'a)->'a->'a" while :: "('a -> tr)->('a -> 'a)->'a->'a" rules step_def "step == (LAM b g x. If b[x] then g[x] else x fi)" while_def "while == (LAM b g. fix[LAM f x.\ \ If b[x] then f[g[x]] else x fi])" end