src/HOL/UNITY/SubstAx.thy
author paulson
Thu, 06 Aug 1998 15:47:26 +0200
changeset 5277 e4297d03e5d2
parent 5253 82a5ca6290aa
child 5313 1861a564d7e2
permissions -rw-r--r--
A higher-level treatment of LeadsTo, minimizing use of "reachable"

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

constdefs

   LeadsTo :: "['a program, 'a set, 'a set] => bool"
    "LeadsTo prg A B ==
		 leadsTo (Acts prg)
                         (reachable prg  Int  A)
  		         (reachable prg  Int  B)"
end