src/HOLCF/IOA/Storage/Correctness.thy
author wenzelm
Sat, 01 Dec 2001 18:52:32 +0100
changeset 12338 de0f4a63baa5
parent 12218 6597093b77e7
child 14981 e73f8140af78
permissions -rw-r--r--
renamed class "term" to "type" (actually "HOL.type");

(*  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