src/HOLCF/IOA/Storage/Correctness.thy
changeset 6008 d0e9b1619468
child 12218 6597093b77e7
equal deleted inserted replaced
6007:91070f559b4d 6008:d0e9b1619468
       
     1 (*  Title:      HOL/IOA/example/Correctness.thy
       
     2     ID:         $Id$
       
     3     Author:     Olaf Mueller
       
     4     Copyright   1997  TU Muenchen
       
     5 
       
     6 Correctness Proof
       
     7 *)
       
     8 
       
     9 Correctness = SimCorrectness + Spec + Impl + 
       
    10 
       
    11 default term
       
    12 
       
    13 consts
       
    14 
       
    15 sim_relation   :: "((nat * bool) * (nat set * bool)) set"
       
    16 
       
    17 defs
       
    18   
       
    19 sim_relation_def
       
    20   "sim_relation == {qua. let c = fst qua; a = snd qua ; 
       
    21                              k = fst c;   b = snd c;
       
    22                              used = fst a; c = snd a
       
    23                          in
       
    24                          (! l:used. l < k) & b=c }"
       
    25 
       
    26 end