src/HOL/MicroJava/BV/Correct.thy
author kleing
Thu, 22 Feb 2001 18:03:11 +0100
changeset 11178 0a9d14823644
parent 11085 b830bf10bf71
child 11252 71c00cb091d2
permissions -rw-r--r--
removed unused constant
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
8011
d14c4e9e9c8e *** empty log message ***
nipkow
parents:
diff changeset
     1
(*  Title:      HOL/MicroJava/BV/Correct.thy
d14c4e9e9c8e *** empty log message ***
nipkow
parents:
diff changeset
     2
    ID:         $Id$
d14c4e9e9c8e *** empty log message ***
nipkow
parents:
diff changeset
     3
    Author:     Cornelia Pusch
d14c4e9e9c8e *** empty log message ***
nipkow
parents:
diff changeset
     4
    Copyright   1999 Technische Universitaet Muenchen
d14c4e9e9c8e *** empty log message ***
nipkow
parents:
diff changeset
     5
d14c4e9e9c8e *** empty log message ***
nipkow
parents:
diff changeset
     6
The invariant for the type safety proof.
d14c4e9e9c8e *** empty log message ***
nipkow
parents:
diff changeset
     7
*)
d14c4e9e9c8e *** empty log message ***
nipkow
parents:
diff changeset
     8
10056
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
     9
header "BV Type Safety Invariant"
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    10
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    11
theory Correct = BVSpec:
8011
d14c4e9e9c8e *** empty log message ***
nipkow
parents:
diff changeset
    12
d14c4e9e9c8e *** empty log message ***
nipkow
parents:
diff changeset
    13
constdefs
10056
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
    14
  approx_val :: "[jvm_prog,aheap,val,ty err] => bool"
10496
f2d304bdf3cc BCV integration (first step)
kleing
parents: 10060
diff changeset
    15
  "approx_val G h v any == case any of Err => True | OK T => G,h\<turnstile>v::\<preceq>T"
8011
d14c4e9e9c8e *** empty log message ***
nipkow
parents:
diff changeset
    16
10056
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
    17
  approx_loc :: "[jvm_prog,aheap,val list,locvars_type] => bool"
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
    18
  "approx_loc G hp loc LT == list_all2 (approx_val G hp) loc LT"
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
    19
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
    20
  approx_stk :: "[jvm_prog,aheap,opstack,opstack_type] => bool"
10496
f2d304bdf3cc BCV integration (first step)
kleing
parents: 10060
diff changeset
    21
  "approx_stk G hp stk ST == approx_loc G hp stk (map OK ST)"
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    22
10056
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
    23
  correct_frame  :: "[jvm_prog,aheap,state_type,nat,bytecode] => frame => bool"
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
    24
  "correct_frame G hp == \<lambda>(ST,LT) maxl ins (stk,loc,C,sig,pc).
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
    25
                         approx_stk G hp stk ST  \<and> approx_loc G hp loc LT \<and> 
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
    26
                         pc < length ins \<and> length loc=length(snd sig)+maxl+1"
8011
d14c4e9e9c8e *** empty log message ***
nipkow
parents:
diff changeset
    27
d14c4e9e9c8e *** empty log message ***
nipkow
parents:
diff changeset
    28
d14c4e9e9c8e *** empty log message ***
nipkow
parents:
diff changeset
    29
consts
10042
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
    30
 correct_frames  :: "[jvm_prog,aheap,prog_type,ty,sig,frame list] => bool"
8011
d14c4e9e9c8e *** empty log message ***
nipkow
parents:
diff changeset
    31
primrec
8045
816f566c414f Fixed a problem with returning from the last frame.
nipkow
parents: 8034
diff changeset
    32
"correct_frames G hp phi rT0 sig0 [] = True"
8011
d14c4e9e9c8e *** empty log message ***
nipkow
parents:
diff changeset
    33
8045
816f566c414f Fixed a problem with returning from the last frame.
nipkow
parents: 8034
diff changeset
    34
"correct_frames G hp phi rT0 sig0 (f#frs) =
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    35
	(let (stk,loc,C,sig,pc) = f in
10592
fc0b575a2cf7 BCV Integration
kleing
parents: 10496
diff changeset
    36
  (\<exists>ST LT rT maxs maxl ins.
10625
022c6b2bcd6b strengthened invariant: current class must be defined
kleing
parents: 10612
diff changeset
    37
    phi C sig ! pc = Some (ST,LT) \<and> is_class G C \<and> 
10592
fc0b575a2cf7 BCV Integration
kleing
parents: 10496
diff changeset
    38
    method (G,C) sig = Some(C,rT,(maxs,maxl,ins)) \<and>
10625
022c6b2bcd6b strengthened invariant: current class must be defined
kleing
parents: 10612
diff changeset
    39
	(\<exists>C' mn pTs k. pc = k+1 \<and> ins!k = (Invoke C' mn pTs) \<and> 
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    40
         (mn,pTs) = sig0 \<and> 
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    41
         (\<exists>apTs D ST' LT'.
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    42
         (phi C sig)!k = Some ((rev apTs) @ (Class D) # ST', LT') \<and>
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    43
         length apTs = length pTs \<and>
10592
fc0b575a2cf7 BCV Integration
kleing
parents: 10496
diff changeset
    44
         (\<exists>D' rT' maxs' maxl' ins'.
fc0b575a2cf7 BCV Integration
kleing
parents: 10496
diff changeset
    45
           method (G,D) sig0 = Some(D',rT',(maxs',maxl',ins')) \<and>
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    46
           G \<turnstile> rT0 \<preceq> rT') \<and>
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    47
	 correct_frame G hp (tl ST, LT) maxl ins f \<and> 
8045
816f566c414f Fixed a problem with returning from the last frame.
nipkow
parents: 8034
diff changeset
    48
	 correct_frames G hp phi rT sig frs))))"
8011
d14c4e9e9c8e *** empty log message ***
nipkow
parents:
diff changeset
    49
d14c4e9e9c8e *** empty log message ***
nipkow
parents:
diff changeset
    50
d14c4e9e9c8e *** empty log message ***
nipkow
parents:
diff changeset
    51
constdefs
10042
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
    52
 correct_state :: "[jvm_prog,prog_type,jvm_state] => bool"
10060
4522e59b7d84 added HTML syntax
kleing
parents: 10056
diff changeset
    53
                  ("_,_ \<turnstile>JVM _ \<surd>"  [51,51] 50)
10042
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
    54
"correct_state G phi == \<lambda>(xp,hp,frs).
8011
d14c4e9e9c8e *** empty log message ***
nipkow
parents:
diff changeset
    55
   case xp of
10042
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
    56
     None => (case frs of
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
    57
	           [] => True
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
    58
             | (f#fs) => G\<turnstile>h hp\<surd> \<and>
8045
816f566c414f Fixed a problem with returning from the last frame.
nipkow
parents: 8034
diff changeset
    59
			(let (stk,loc,C,sig,pc) = f
8011
d14c4e9e9c8e *** empty log message ***
nipkow
parents:
diff changeset
    60
		         in
10592
fc0b575a2cf7 BCV Integration
kleing
parents: 10496
diff changeset
    61
                         \<exists>rT maxs maxl ins s.
10625
022c6b2bcd6b strengthened invariant: current class must be defined
kleing
parents: 10612
diff changeset
    62
                         is_class G C \<and>
10592
fc0b575a2cf7 BCV Integration
kleing
parents: 10496
diff changeset
    63
                         method (G,C) sig = Some(C,rT,(maxs,maxl,ins)) \<and>
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    64
                         phi C sig ! pc = Some s \<and>
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    65
			 correct_frame G hp s maxl ins f \<and> 
8045
816f566c414f Fixed a problem with returning from the last frame.
nipkow
parents: 8034
diff changeset
    66
		         correct_frames G hp phi rT sig fs))
10042
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
    67
   | Some x => True" 
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    68
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    69
10060
4522e59b7d84 added HTML syntax
kleing
parents: 10056
diff changeset
    70
syntax (HTML)
4522e59b7d84 added HTML syntax
kleing
parents: 10056
diff changeset
    71
 correct_state :: "[jvm_prog,prog_type,jvm_state] => bool"
4522e59b7d84 added HTML syntax
kleing
parents: 10056
diff changeset
    72
                  ("_,_ |-JVM _ [ok]"  [51,51] 50)
4522e59b7d84 added HTML syntax
kleing
parents: 10056
diff changeset
    73
11085
b830bf10bf71 tuned for 99-2 release
kleing
parents: 10920
diff changeset
    74
section {* approx-val *}
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    75
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    76
lemma approx_val_Err:
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    77
  "approx_val G hp x Err"
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    78
by (simp add: approx_val_def)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    79
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    80
lemma approx_val_Null:
10496
f2d304bdf3cc BCV integration (first step)
kleing
parents: 10060
diff changeset
    81
  "approx_val G hp Null (OK (RefT x))"
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    82
by (auto intro: null simp add: approx_val_def)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    83
9941
fe05af7ec816 renamed atts: rulify to rule_format, elimify to elim_format;
wenzelm
parents: 9906
diff changeset
    84
lemma approx_val_imp_approx_val_assConvertible [rule_format]: 
10496
f2d304bdf3cc BCV integration (first step)
kleing
parents: 10060
diff changeset
    85
  "wf_prog wt G ==> approx_val G hp v (OK T) --> G\<turnstile> T\<preceq>T' 
f2d304bdf3cc BCV integration (first step)
kleing
parents: 10060
diff changeset
    86
  --> approx_val G hp v (OK T')"
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    87
by (cases T) (auto intro: conf_widen simp add: approx_val_def)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    88
9941
fe05af7ec816 renamed atts: rulify to rule_format, elimify to elim_format;
wenzelm
parents: 9906
diff changeset
    89
lemma approx_val_imp_approx_val_sup_heap [rule_format]:
10042
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
    90
  "approx_val G hp v at --> hp \<le>| hp' --> approx_val G hp' v at"
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    91
apply (simp add: approx_val_def split: err.split)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    92
apply (blast intro: conf_hext)
10056
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
    93
done
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    94
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    95
lemma approx_val_imp_approx_val_heap_update:
10042
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
    96
  "[|hp a = Some obj'; G,hp\<turnstile> v::\<preceq>T; obj_ty obj = obj_ty obj'|] 
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
    97
  ==> G,hp(a\<mapsto>obj)\<turnstile> v::\<preceq>T"
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    98
by (cases v, auto simp add: obj_ty_def conf_def)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
    99
9941
fe05af7ec816 renamed atts: rulify to rule_format, elimify to elim_format;
wenzelm
parents: 9906
diff changeset
   100
lemma approx_val_imp_approx_val_sup [rule_format]:
10056
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   101
  "wf_prog wt G ==> (approx_val G h v us) --> (G \<turnstile> us <=o us') 
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   102
  --> (approx_val G h v us')"
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   103
apply (simp add: sup_PTS_eq approx_val_def split: err.split)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   104
apply (blast intro: conf_widen)
10056
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   105
done
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   106
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   107
lemma approx_loc_imp_approx_val_sup:
10056
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   108
  "[| wf_prog wt G; approx_loc G hp loc LT; idx < length LT; 
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   109
      v = loc!idx; G \<turnstile> LT!idx <=o at |]
10042
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
   110
  ==> approx_val G hp v at"
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   111
apply (unfold approx_loc_def)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   112
apply (unfold list_all2_def)
10056
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   113
apply (auto intro: approx_val_imp_approx_val_sup 
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   114
            simp add: split_def all_set_conv_all_nth)
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   115
done
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   116
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   117
11085
b830bf10bf71 tuned for 99-2 release
kleing
parents: 10920
diff changeset
   118
section {* approx-loc *}
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   119
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   120
lemma approx_loc_Cons [iff]:
10056
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   121
  "approx_loc G hp (s#xs) (l#ls) = 
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   122
  (approx_val G hp s l \<and> approx_loc G hp xs ls)"
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   123
by (simp add: approx_loc_def)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   124
9941
fe05af7ec816 renamed atts: rulify to rule_format, elimify to elim_format;
wenzelm
parents: 9906
diff changeset
   125
lemma assConv_approx_stk_imp_approx_loc [rule_format]:
10042
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
   126
  "wf_prog wt G ==> (\<forall>tt'\<in>set (zip tys_n ts). tt' \<in> widen G) 
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
   127
  --> length tys_n = length ts --> approx_stk G hp s tys_n --> 
10496
f2d304bdf3cc BCV integration (first step)
kleing
parents: 10060
diff changeset
   128
  approx_loc G hp s (map OK ts)"
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   129
apply (unfold approx_stk_def approx_loc_def list_all2_def)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   130
apply (clarsimp simp add: all_set_conv_all_nth)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   131
apply (rule approx_val_imp_approx_val_assConvertible)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   132
apply auto
10056
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   133
done
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   134
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   135
9941
fe05af7ec816 renamed atts: rulify to rule_format, elimify to elim_format;
wenzelm
parents: 9906
diff changeset
   136
lemma approx_loc_imp_approx_loc_sup_heap [rule_format]:
10056
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   137
  "\<forall>lvars. approx_loc G hp lvars lt --> hp \<le>| hp' 
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   138
  --> approx_loc G hp' lvars lt"
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   139
apply (unfold approx_loc_def list_all2_def)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   140
apply (cases lt)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   141
 apply simp
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   142
apply clarsimp
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   143
apply (rule approx_val_imp_approx_val_sup_heap)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   144
apply auto
10056
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   145
done
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   146
9941
fe05af7ec816 renamed atts: rulify to rule_format, elimify to elim_format;
wenzelm
parents: 9906
diff changeset
   147
lemma approx_loc_imp_approx_loc_sup [rule_format]:
10056
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   148
  "wf_prog wt G ==> approx_loc G hp lvars lt --> G \<turnstile> lt <=l lt' 
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   149
  --> approx_loc G hp lvars lt'"
10812
ead84e90bfeb merged semilattice orders with <=' from Convert.thy (now defined in JVMType.thy)
kleing
parents: 10625
diff changeset
   150
apply (unfold Listn.le_def lesub_def sup_loc_def approx_loc_def list_all2_def)
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   151
apply (auto simp add: all_set_conv_all_nth)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   152
apply (auto elim: approx_val_imp_approx_val_sup)
10056
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   153
done
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   154
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   155
9941
fe05af7ec816 renamed atts: rulify to rule_format, elimify to elim_format;
wenzelm
parents: 9906
diff changeset
   156
lemma approx_loc_imp_approx_loc_subst [rule_format]:
10042
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
   157
  "\<forall>loc idx x X. (approx_loc G hp loc LT) --> (approx_val G hp x X) 
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
   158
  --> (approx_loc G hp (loc[idx:=x]) (LT[idx:=X]))"
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   159
apply (unfold approx_loc_def list_all2_def)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   160
apply (auto dest: subsetD [OF set_update_subset_insert] simp add: zip_update)
10056
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   161
done
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   162
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   163
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   164
lemmas [cong] = conj_cong 
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   165
9941
fe05af7ec816 renamed atts: rulify to rule_format, elimify to elim_format;
wenzelm
parents: 9906
diff changeset
   166
lemma approx_loc_append [rule_format]:
10042
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
   167
  "\<forall>L1 l2 L2. length l1=length L1 --> 
10056
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   168
  approx_loc G hp (l1@l2) (L1@L2) = 
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   169
  (approx_loc G hp l1 L1 \<and> approx_loc G hp l2 L2)"
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   170
apply (unfold approx_loc_def list_all2_def)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   171
apply simp
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   172
apply blast
10056
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   173
done
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   174
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   175
lemmas [cong del] = conj_cong
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   176
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   177
11085
b830bf10bf71 tuned for 99-2 release
kleing
parents: 10920
diff changeset
   178
section {* approx-stk *}
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   179
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   180
lemma approx_stk_rev_lem:
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   181
  "approx_stk G hp (rev s) (rev t) = approx_stk G hp s t"
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   182
apply (unfold approx_stk_def approx_loc_def list_all2_def)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   183
apply (auto simp add: zip_rev sym [OF rev_map])
10056
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   184
done
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   185
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   186
lemma approx_stk_rev:
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   187
  "approx_stk G hp (rev s) t = approx_stk G hp s (rev t)"
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   188
by (auto intro: subst [OF approx_stk_rev_lem])
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   189
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   190
9941
fe05af7ec816 renamed atts: rulify to rule_format, elimify to elim_format;
wenzelm
parents: 9906
diff changeset
   191
lemma approx_stk_imp_approx_stk_sup_heap [rule_format]:
10056
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   192
  "\<forall>lvars. approx_stk G hp lvars lt --> hp \<le>| hp' 
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   193
  --> approx_stk G hp' lvars lt"
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   194
by (auto intro: approx_loc_imp_approx_loc_sup_heap simp add: approx_stk_def)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   195
9941
fe05af7ec816 renamed atts: rulify to rule_format, elimify to elim_format;
wenzelm
parents: 9906
diff changeset
   196
lemma approx_stk_imp_approx_stk_sup [rule_format]:
10496
f2d304bdf3cc BCV integration (first step)
kleing
parents: 10060
diff changeset
   197
  "wf_prog wt G ==> approx_stk G hp lvars st --> (G \<turnstile> map OK st <=l (map OK st')) 
10042
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
   198
  --> approx_stk G hp lvars st'" 
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   199
by (auto intro: approx_loc_imp_approx_loc_sup simp add: approx_stk_def)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   200
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   201
lemma approx_stk_Nil [iff]:
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   202
  "approx_stk G hp [] []"
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   203
by (simp add: approx_stk_def approx_loc_def)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   204
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   205
lemma approx_stk_Cons [iff]:
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   206
  "approx_stk G hp (x # stk) (S#ST) = 
10496
f2d304bdf3cc BCV integration (first step)
kleing
parents: 10060
diff changeset
   207
   (approx_val G hp x (OK S) \<and> approx_stk G hp stk ST)"
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   208
by (simp add: approx_stk_def approx_loc_def)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   209
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   210
lemma approx_stk_Cons_lemma [iff]:
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   211
  "approx_stk G hp stk (S#ST') = 
10496
f2d304bdf3cc BCV integration (first step)
kleing
parents: 10060
diff changeset
   212
  (\<exists>s stk'. stk = s#stk' \<and> approx_val G hp s (OK S) \<and> approx_stk G hp stk' ST')"
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   213
by (simp add: list_all2_Cons2 approx_stk_def approx_loc_def)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   214
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   215
lemma approx_stk_append_lemma:
10042
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
   216
  "approx_stk G hp stk (S@ST') ==>
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   217
   (\<exists>s stk'. stk = s@stk' \<and> length s = length S \<and> length stk' = length ST' \<and> 
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   218
             approx_stk G hp s S \<and> approx_stk G hp stk' ST')"
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   219
by (simp add: list_all2_append2 approx_stk_def approx_loc_def)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   220
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   221
11085
b830bf10bf71 tuned for 99-2 release
kleing
parents: 10920
diff changeset
   222
section {* oconf *}
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   223
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   224
lemma correct_init_obj:
10042
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
   225
  "[|is_class G C; wf_prog wt G|] ==> 
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   226
  G,h \<turnstile> (C, map_of (map (\<lambda>(f,fT).(f,default_val fT)) (fields(G,C)))) \<surd>"
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   227
apply (unfold oconf_def lconf_def)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   228
apply (simp add: map_of_map)
10612
779af7c58743 improved superclass entry for classes and definition status of is_class, class
oheimb
parents: 10592
diff changeset
   229
apply (force intro: defval_conf dest: map_of_SomeD fields_is_type)
10056
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   230
done
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   231
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   232
9941
fe05af7ec816 renamed atts: rulify to rule_format, elimify to elim_format;
wenzelm
parents: 9906
diff changeset
   233
lemma oconf_imp_oconf_field_update [rule_format]:
10042
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
   234
  "[|map_of (fields (G, oT)) FD = Some T; G,hp\<turnstile>v::\<preceq>T; G,hp\<turnstile>(oT,fs)\<surd> |]
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
   235
  ==> G,hp\<turnstile>(oT, fs(FD\<mapsto>v))\<surd>"
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   236
by (simp add: oconf_def lconf_def)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   237
9941
fe05af7ec816 renamed atts: rulify to rule_format, elimify to elim_format;
wenzelm
parents: 9906
diff changeset
   238
lemma oconf_imp_oconf_heap_newref [rule_format]:
10920
9b74eceea2d2 newref -> new_Addr
kleing
parents: 10812
diff changeset
   239
"hp oref = None --> G,hp\<turnstile>obj\<surd> --> G,hp\<turnstile>obj'\<surd> --> G,(hp(oref\<mapsto>obj'))\<turnstile>obj\<surd>"
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   240
apply (unfold oconf_def lconf_def)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   241
apply simp
11085
b830bf10bf71 tuned for 99-2 release
kleing
parents: 10920
diff changeset
   242
apply (fast intro: conf_hext hext_new)
10056
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   243
done
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   244
9941
fe05af7ec816 renamed atts: rulify to rule_format, elimify to elim_format;
wenzelm
parents: 9906
diff changeset
   245
lemma oconf_imp_oconf_heap_update [rule_format]:
10042
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
   246
  "hp a = Some obj' --> obj_ty obj' = obj_ty obj'' --> G,hp\<turnstile>obj\<surd> 
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
   247
  --> G,hp(a\<mapsto>obj'')\<turnstile>obj\<surd>"
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   248
apply (unfold oconf_def lconf_def)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   249
apply simp
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   250
apply (force intro: approx_val_imp_approx_val_heap_update)
10056
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   251
done
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   252
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   253
11085
b830bf10bf71 tuned for 99-2 release
kleing
parents: 10920
diff changeset
   254
section {* hconf *}
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   255
9941
fe05af7ec816 renamed atts: rulify to rule_format, elimify to elim_format;
wenzelm
parents: 9906
diff changeset
   256
lemma hconf_imp_hconf_newref [rule_format]:
10920
9b74eceea2d2 newref -> new_Addr
kleing
parents: 10812
diff changeset
   257
  "hp oref = None --> G\<turnstile>h hp\<surd> --> G,hp\<turnstile>obj\<surd> --> G\<turnstile>h hp(oref\<mapsto>obj)\<surd>"
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   258
apply (simp add: hconf_def)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   259
apply (fast intro: oconf_imp_oconf_heap_newref)
10056
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   260
done
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   261
9941
fe05af7ec816 renamed atts: rulify to rule_format, elimify to elim_format;
wenzelm
parents: 9906
diff changeset
   262
lemma hconf_imp_hconf_field_update [rule_format]:
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   263
  "map_of (fields (G, oT)) (F, D) = Some T \<and> hp oloc = Some(oT,fs) \<and> 
10042
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
   264
  G,hp\<turnstile>v::\<preceq>T \<and> G\<turnstile>h hp\<surd> --> G\<turnstile>h hp(oloc \<mapsto> (oT, fs((F,D)\<mapsto>v)))\<surd>"
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   265
apply (simp add: hconf_def)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   266
apply (force intro: oconf_imp_oconf_heap_update oconf_imp_oconf_field_update 
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   267
             simp add: obj_ty_def)
10056
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   268
done
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   269
11085
b830bf10bf71 tuned for 99-2 release
kleing
parents: 10920
diff changeset
   270
section {* correct-frames *}
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   271
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   272
lemmas [simp del] = fun_upd_apply
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   273
9941
fe05af7ec816 renamed atts: rulify to rule_format, elimify to elim_format;
wenzelm
parents: 9906
diff changeset
   274
lemma correct_frames_imp_correct_frames_field_update [rule_format]:
10042
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
   275
  "\<forall>rT C sig. correct_frames G hp phi rT sig frs --> 
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
   276
  hp a = Some (C,od) --> map_of (fields (G, C)) fl = Some fd --> 
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
   277
  G,hp\<turnstile>v::\<preceq>fd 
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
   278
  --> correct_frames G (hp(a \<mapsto> (C, od(fl\<mapsto>v)))) phi rT sig frs";
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   279
apply (induct frs)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   280
 apply simp
10920
9b74eceea2d2 newref -> new_Addr
kleing
parents: 10812
diff changeset
   281
apply clarify
9b74eceea2d2 newref -> new_Addr
kleing
parents: 10812
diff changeset
   282
apply simp
9b74eceea2d2 newref -> new_Addr
kleing
parents: 10812
diff changeset
   283
apply clarify
9b74eceea2d2 newref -> new_Addr
kleing
parents: 10812
diff changeset
   284
apply (unfold correct_frame_def)
9b74eceea2d2 newref -> new_Addr
kleing
parents: 10812
diff changeset
   285
apply (simp (no_asm_use))
9b74eceea2d2 newref -> new_Addr
kleing
parents: 10812
diff changeset
   286
apply clarsimp
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   287
apply (intro exI conjI)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   288
     apply simp
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   289
    apply simp
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   290
   apply force
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   291
  apply simp
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   292
 apply (rule approx_stk_imp_approx_stk_sup_heap)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   293
  apply simp
11085
b830bf10bf71 tuned for 99-2 release
kleing
parents: 10920
diff changeset
   294
 apply (rule hext_upd_obj)
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   295
 apply simp
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   296
apply (rule approx_loc_imp_approx_loc_sup_heap)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   297
 apply simp
11085
b830bf10bf71 tuned for 99-2 release
kleing
parents: 10920
diff changeset
   298
apply (rule hext_upd_obj)
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   299
apply simp
10056
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   300
done
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   301
9941
fe05af7ec816 renamed atts: rulify to rule_format, elimify to elim_format;
wenzelm
parents: 9906
diff changeset
   302
lemma correct_frames_imp_correct_frames_newref [rule_format]:
10042
7164dc0d24d8 unsymbolized
kleing
parents: 9941
diff changeset
   303
  "\<forall>rT C sig. hp x = None --> correct_frames G hp phi rT sig frs \<and> oconf G hp obj 
10920
9b74eceea2d2 newref -> new_Addr
kleing
parents: 10812
diff changeset
   304
  --> correct_frames G (hp(x \<mapsto> obj)) phi rT sig frs"
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   305
apply (induct frs)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   306
 apply simp
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   307
apply (clarsimp simp add: correct_frame_def)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   308
apply (intro exI conjI)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   309
     apply simp
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   310
    apply simp
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   311
   apply force
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   312
  apply simp
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   313
 apply (rule approx_stk_imp_approx_stk_sup_heap)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   314
  apply simp
11085
b830bf10bf71 tuned for 99-2 release
kleing
parents: 10920
diff changeset
   315
 apply (rule hext_new)
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   316
 apply simp
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   317
apply (rule approx_loc_imp_approx_loc_sup_heap)
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   318
 apply simp
11085
b830bf10bf71 tuned for 99-2 release
kleing
parents: 10920
diff changeset
   319
apply (rule hext_new)
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   320
apply simp
10056
9f84ffa4a8d0 tuned spacing for document generation
kleing
parents: 10042
diff changeset
   321
done
8011
d14c4e9e9c8e *** empty log message ***
nipkow
parents:
diff changeset
   322
d14c4e9e9c8e *** empty log message ***
nipkow
parents:
diff changeset
   323
end
9757
1024a2d80ac0 functional LBV style, dead code, type safety -> Isar
kleing
parents: 9549
diff changeset
   324