src/ZF/IMP/Assign.thy
author paulson
Wed, 07 Nov 2001 18:12:12 +0100
changeset 12089 34e7693271a9
parent 482 3a4e092ba69c
permissions -rw-r--r--
Sidi Ehmety's port of the fold_set operator and multisets to ZF. Also, fixes to the cancellation simprocs and a few new standard lemmas.

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

Assign = Aexp +
consts 
	"assign" :: "[i,i,i] => i"	("_[_'/_]" [900,0,0] 900)

rules 
	assign_def	"sigma[m/x] == lam y:loc. if(y=x,m,sigma`y)"
end