--- a/src/HOL/MicroJava/BV/JVM.thy Thu Mar 27 19:05:10 2008 +0100
+++ b/src/HOL/MicroJava/BV/JVM.thy Thu Mar 27 19:22:23 2008 +0100
@@ -11,7 +11,7 @@
constdefs
kiljvm :: "jvm_prog \<Rightarrow> nat \<Rightarrow> nat \<Rightarrow> ty \<Rightarrow> exception_table \<Rightarrow>
- instr list \<Rightarrow> state list \<Rightarrow> state list"
+ instr list \<Rightarrow> JVMType.state list \<Rightarrow> JVMType.state list"
"kiljvm G maxs maxr rT et bs ==
kildall (JVMType.le G maxs maxr) (JVMType.sup G maxs maxr) (exec G maxs rT et bs)"