author | kleing |
Tue, 13 May 2003 08:59:21 +0200 | |
changeset 14024 | 213dcc39358f |
parent 12338 | de0f4a63baa5 |
child 14981 | e73f8140af78 |
permissions | -rw-r--r-- |
(* Title: HOL/IOA/example/Correctness.thy ID: $Id$ Author: Olaf Müller License: GPL (GNU GENERAL PUBLIC LICENSE) Correctness Proof. *) Correctness = SimCorrectness + Spec + Impl + default type consts sim_relation :: "((nat * bool) * (nat set * bool)) set" defs sim_relation_def "sim_relation == {qua. let c = fst qua; a = snd qua ; k = fst c; b = snd c; used = fst a; c = snd a in (! l:used. l < k) & b=c }" end