src/HOL/HOLCF/IOA/Storage/Correctness.thy
changeset 67613 ce654b0e6d69
parent 66453 cc19f7ca2ed6
equal deleted inserted replaced
67610:4939494ed791 67613:ce654b0e6d69
    14   sim_relation :: "((nat * bool) * (nat set * bool)) set" where
    14   sim_relation :: "((nat * bool) * (nat set * bool)) set" where
    15   "sim_relation = {qua. let c = fst qua; a = snd qua ;
    15   "sim_relation = {qua. let c = fst qua; a = snd qua ;
    16                             k = fst c;   b = snd c;
    16                             k = fst c;   b = snd c;
    17                             used = fst a; c = snd a
    17                             used = fst a; c = snd a
    18                         in
    18                         in
    19                         (! l:used. l < k) & b=c}"
    19                         (\<forall>l\<in>used. l < k) \<and> b=c}"
    20 
    20 
    21 declare split_paired_Ex [simp del]
    21 declare split_paired_Ex [simp del]
    22 
    22 
    23 
    23 
    24 (* Idea: instead of impl_con_lemma do not rewrite impl_ioa, but derive
    24 (* Idea: instead of impl_con_lemma do not rewrite impl_ioa, but derive