src/ZF/IMP/Evalb0.thy
author paulson
Wed, 05 Nov 1997 13:14:15 +0100
changeset 4152 451104c223e2
parent 482 3a4e092ba69c
permissions -rw-r--r--
Ran expandshort, especially to introduce Safe_tac

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

Evalb0 = Evala + Bexp +

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

translations
	"<be,sig> -b-> b" == "<be,sig,b> : evalb"
end