src/HOL/UNITY/SubstAx.thy
author wenzelm
Fri, 31 Jul 1998 11:03:31 +0200
changeset 5228 66925577cefe
parent 5111 8f4b72f0c15d
child 5253 82a5ca6290aa
permissions -rw-r--r--
isatool expandshort;

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

My treatment of the Substitution Axiom -- not as an axiom!
*)

SubstAx = WFair +

constdefs

   LeadsTo :: "['a set * ('a * 'a)set set, 'a set, 'a set] => bool"
    "LeadsTo == %(Init,Acts) A B.
		 leadsTo Acts (reachable (Init,Acts) Int A)
			      (reachable (Init,Acts) Int B)"


end