diff -r 4dc65845eab3 -r d8d7d1b785af src/HOL/MicroJava/BV/Altern.thy --- a/src/HOL/MicroJava/BV/Altern.thy Wed Feb 24 11:55:52 2010 +0100 +++ b/src/HOL/MicroJava/BV/Altern.thy Mon Mar 01 13:40:23 2010 +0100 @@ -8,19 +8,18 @@ imports BVSpec begin -constdefs - check_type :: "jvm_prog \ nat \ nat \ JVMType.state \ bool" +definition check_type :: "jvm_prog \ nat \ nat \ JVMType.state \ bool" where "check_type G mxs mxr s \ s \ states G mxs mxr" - wt_instr_altern :: "[instr,jvm_prog,ty,method_type,nat,nat,p_count, - exception_table,p_count] \ bool" +definition wt_instr_altern :: "[instr,jvm_prog,ty,method_type,nat,nat,p_count, + exception_table,p_count] \ bool" where "wt_instr_altern i G rT phi mxs mxr max_pc et pc \ app i G mxs rT pc et (phi!pc) \ check_type G mxs mxr (OK (phi!pc)) \ (\(pc',s') \ set (eff i G pc et (phi!pc)). pc' < max_pc \ G \ s' <=' phi!pc')" - wt_method_altern :: "[jvm_prog,cname,ty list,ty,nat,nat,instr list, - exception_table,method_type] \ bool" +definition wt_method_altern :: "[jvm_prog,cname,ty list,ty,nat,nat,instr list, + exception_table,method_type] \ bool" where "wt_method_altern G C pTs rT mxs mxl ins et phi \ let max_pc = length ins in 0 < max_pc \