src/ZF/IMP/Evalc0.thy
author nipkow
Fri, 04 Jul 1997 14:37:30 +0200
changeset 3499 ce1664057431
parent 482 3a4e092ba69c
permissions -rw-r--r--
Reduced priority of postfix ^* etc operators such that they are the same as application. Eg wf r^* now needs to be written wf(r^*).

(*  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