src/HOLCF/ex/Loop.thy
author wenzelm
Mon, 06 Feb 2006 20:59:10 +0100
changeset 18943 947d3a694654
parent 17291 94f6113fe9ed
child 19742 86f21beabafc
permissions -rw-r--r--
moved no_vars to sign.ML; removed dest_def (cf. Sign.cert_def);

(*  Title:      HOLCF/ex/Loop.thy
    ID:         $Id$
    Author:     Franz Regensburger
*)

header {* Theory for a loop primitive like while *}

theory Loop
imports HOLCF
begin

constdefs
  step  :: "('a -> tr)->('a -> 'a)->'a->'a"
  "step == (LAM b g x. If b$x then g$x else x fi)"
  while :: "('a -> tr)->('a -> 'a)->'a->'a"
  "while == (LAM b g. fix$(LAM f x.
    If b$x then f$(g$x) else x fi))"

ML {* use_legacy_bindings (the_context ()) *}

end