author | wenzelm |
Wed, 20 Feb 2002 00:53:53 +0100 | |
changeset 12902 | a23dc0b7566f |
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