| author | wenzelm |
| Sat, 01 Apr 2000 20:21:39 +0200 | |
| changeset 8657 | b9475dad85ed |
| parent 8122 | b43ad07660b9 |
| child 9685 | 6d123a7e30bd |
| permissions | -rw-r--r-- |
(* Title: HOL/UNITY/SubstAx ID: $Id$ Author: Lawrence C Paulson, Cambridge University Computer Laboratory Copyright 1998 University of Cambridge Weak LeadsTo relation (restricted to the set of reachable states) *) SubstAx = WFair + Constrains + constdefs Ensures :: "['a set, 'a set] => 'a program set" (infixl 60) "A Ensures B == {F. F : (reachable F Int A) ensures B}" LeadsTo :: "['a set, 'a set] => 'a program set" (infixl 60) "A LeadsTo B == {F. F : (reachable F Int A) leadsTo B}" end