| author | wenzelm |
| Sun, 28 Aug 2005 16:04:44 +0200 | |
| changeset 17160 | fb65eda72fc7 |
| parent 14981 | e73f8140af78 |
| child 17244 | 0b2ff9541727 |
| permissions | -rw-r--r-- |
| 6008 | 1 |
(* Title: HOL/IOA/example/Correctness.thy |
2 |
ID: $Id$ |
|
| 12218 | 3 |
Author: Olaf Müller |
| 6008 | 4 |
|
| 12218 | 5 |
Correctness Proof. |
| 6008 | 6 |
*) |
7 |
||
8 |
Correctness = SimCorrectness + Spec + Impl + |
|
9 |
||
|
12338
de0f4a63baa5
renamed class "term" to "type" (actually "HOL.type");
wenzelm
parents:
12218
diff
changeset
|
10 |
default type |
| 6008 | 11 |
|
12 |
consts |
|
13 |
||
14 |
sim_relation :: "((nat * bool) * (nat set * bool)) set" |
|
15 |
||
16 |
defs |
|
17 |
||
18 |
sim_relation_def |
|
19 |
"sim_relation == {qua. let c = fst qua; a = snd qua ;
|
|
20 |
k = fst c; b = snd c; |
|
21 |
used = fst a; c = snd a |
|
22 |
in |
|
23 |
(! l:used. l < k) & b=c }" |
|
24 |
||
25 |
end |