author | nipkow |
Wed, 09 Nov 1994 19:51:09 +0100 | |
changeset 168 | 44ff2275d44f |
parent 156 | fd1be45b64bf |
child 249 | 492493334e0f |
permissions | -rw-r--r-- |
168 | 1 |
(* Title: HOL/IOA/example/Correctness.thy |
2 |
ID: $Id$ |
|
3 |
Author: Tobias Nipkow & Konrad Slind |
|
4 |
Copyright 1994 TU Muenchen |
|
5 |
||
6 |
The main correctness proof: Impl implements Spec |
|
7 |
*) |
|
8 |
||
9 |
Correctness = Solve + Impl + Spec + |
|
156 | 10 |
|
11 |
consts |
|
12 |
||
13 |
hom :: "'m impl_state => 'm list" |
|
14 |
||
168 | 15 |
defs |
156 | 16 |
|
17 |
hom_def |
|
18 |
"hom(s) == rq(rec(s)) @ if(rbit(rec(s)) = sbit(sen(s)), \ |
|
19 |
\ sq(sen(s)), \ |
|
20 |
\ ttl(sq(sen(s))))" |
|
21 |
||
22 |
end |