| author | wenzelm |
| Sun, 22 May 2005 16:51:13 +0200 | |
| changeset 16025 | fa2d7364d359 |
| parent 14981 | e73f8140af78 |
| child 17244 | 0b2ff9541727 |
| permissions | -rw-r--r-- |
(* Title: HOL/IOA/NTP/Correctness.thy ID: $Id$ Author: Tobias Nipkow & Konrad Slind The main correctness proof: Impl implements Spec. *) Correctness = Impl + Spec + constdefs hom :: 'm impl_state => 'm list "hom(s) == rq(rec(s)) @ (if rbit(rec s) = sbit(sen s) then sq(sen s) else tl(sq(sen s)))" end