| author | wenzelm |
| Fri, 31 Jul 1998 11:03:31 +0200 | |
| changeset 5228 | 66925577cefe |
| parent 5111 | 8f4b72f0c15d |
| child 5253 | 82a5ca6290aa |
| permissions | -rw-r--r-- |
| 4776 | 1 |
(* Title: HOL/UNITY/SubstAx |
2 |
ID: $Id$ |
|
3 |
Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
|
4 |
Copyright 1998 University of Cambridge |
|
5 |
||
6 |
My treatment of the Substitution Axiom -- not as an axiom! |
|
7 |
*) |
|
8 |
||
9 |
SubstAx = WFair + |
|
10 |
||
11 |
constdefs |
|
12 |
||
| 5111 | 13 |
LeadsTo :: "['a set * ('a * 'a)set set, 'a set, 'a set] => bool"
|
14 |
"LeadsTo == %(Init,Acts) A B. |
|
15 |
leadsTo Acts (reachable (Init,Acts) Int A) |
|
16 |
(reachable (Init,Acts) Int B)" |
|
| 4776 | 17 |
|
18 |
||
19 |
end |