| author | wenzelm |
| Sat, 14 Jan 2006 22:25:34 +0100 | |
| changeset 18688 | abf0f018b5ec |
| parent 17244 | 0b2ff9541727 |
| child 19739 | c58ef2aa5430 |
| permissions | -rw-r--r-- |
|
3073
88366253a09a
Old NTP files now running under the IOA meta theory based on HOLCF;
mueller
parents:
diff
changeset
|
1 |
(* Title: HOL/IOA/NTP/Correctness.thy |
|
88366253a09a
Old NTP files now running under the IOA meta theory based on HOLCF;
mueller
parents:
diff
changeset
|
2 |
ID: $Id$ |
|
88366253a09a
Old NTP files now running under the IOA meta theory based on HOLCF;
mueller
parents:
diff
changeset
|
3 |
Author: Tobias Nipkow & Konrad Slind |
|
88366253a09a
Old NTP files now running under the IOA meta theory based on HOLCF;
mueller
parents:
diff
changeset
|
4 |
*) |
|
88366253a09a
Old NTP files now running under the IOA meta theory based on HOLCF;
mueller
parents:
diff
changeset
|
5 |
|
| 17244 | 6 |
header {* The main correctness proof: Impl implements Spec *}
|
7 |
||
8 |
theory Correctness |
|
9 |
imports Impl Spec |
|
10 |
begin |
|
|
3073
88366253a09a
Old NTP files now running under the IOA meta theory based on HOLCF;
mueller
parents:
diff
changeset
|
11 |
|
|
88366253a09a
Old NTP files now running under the IOA meta theory based on HOLCF;
mueller
parents:
diff
changeset
|
12 |
constdefs |
| 17244 | 13 |
hom :: "'m impl_state => 'm list" |
14 |
"hom(s) == rq(rec(s)) @ (if rbit(rec s) = sbit(sen s) then sq(sen s) |
|
| 3898 | 15 |
else tl(sq(sen s)))" |
|
3073
88366253a09a
Old NTP files now running under the IOA meta theory based on HOLCF;
mueller
parents:
diff
changeset
|
16 |
|
| 17244 | 17 |
ML {* use_legacy_bindings (the_context ()) *}
|
18 |
||
|
3073
88366253a09a
Old NTP files now running under the IOA meta theory based on HOLCF;
mueller
parents:
diff
changeset
|
19 |
end |