src/HOL/UNITY/SubstAx.thy
author wenzelm
Tue, 27 Apr 1999 10:50:50 +0200
changeset 6522 2f6cec5c046f
parent 5648 fe887910e32e
child 6536 281d44905cab
permissions -rw-r--r--
adapted add_inductive;

(*  Title:      HOL/UNITY/SubstAx
    ID:         $Id$
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
    Copyright   1998  University of Cambridge

LeadsTo relation: restricted to the set of reachable states.
*)

SubstAx = WFair + Constrains + 

constdefs

   LeadsTo :: "['a set, 'a set] => 'a program set"
    "LeadsTo A B == {F. F : leadsTo (reachable F  Int  A)
	   	                    (reachable F  Int  B)}"
end