src/ZF/IMP/Evalc0.thy
author paulson
Tue, 23 May 2000 12:44:03 +0200
changeset 8934 39d0cc787d47
parent 482 3a4e092ba69c
permissions -rw-r--r--
theory file NatSum.thy no longer needed new files for the Allocator: AllocBase.{thy,ML}

(*  Title: 	ZF/IMP/Evalc0.thy
    ID:         $Id$
    Author: 	Heiko Loetzbeyer & Robert Sandner, TUM
    Copyright   1994 TUM
*)

Evalc0 = Evalb + Com + Assign +

consts
       evalc    :: "i"
       "@evalc" :: "[i,i,i] => o"   ("<_,_>/ -c-> _")

translations
       "<ce,sig> -c-> s" == "<ce,sig,s> : evalc"
end