src/HOL/MicroJava/BV/LBVCorrect.thy
changeset 11085 b830bf10bf71
parent 10812 ead84e90bfeb
child 12389 23bd419144eb
equal deleted inserted replaced
11084:32c1deea5bcd 11085:b830bf10bf71
   280 qed
   280 qed
   281 
   281 
   282 
   282 
   283 theorem wtl_correct:
   283 theorem wtl_correct:
   284   "wtl_jvm_prog G cert ==> \<exists> Phi. wt_jvm_prog G Phi"
   284   "wtl_jvm_prog G cert ==> \<exists> Phi. wt_jvm_prog G Phi"
   285 proof -
   285 proof -  
   286   
       
   287   assume wtl: "wtl_jvm_prog G cert"
   286   assume wtl: "wtl_jvm_prog G cert"
   288 
   287 
   289   let ?Phi = "\<lambda>C sig. let (C,rT,(maxs,maxl,ins)) = the (method (G,C) sig) in 
   288   let ?Phi = "\<lambda>C sig. let (C,rT,(maxs,maxl,ins)) = the (method (G,C) sig) in 
   290               SOME phi. wt_method G C (snd sig) rT maxs maxl ins phi"
   289               SOME phi. wt_method G C (snd sig) rT maxs maxl ins phi"
   291    
   290