src/HOL/MicroJava/BV/JVM.thy
changeset 11299 1d3d110c456e
parent 11298 acd83fa66e92
child 11701 3d51fbf81c17
--- a/src/HOL/MicroJava/BV/JVM.thy	Mon May 14 09:58:22 2001 +0200
+++ b/src/HOL/MicroJava/BV/JVM.thy	Wed May 16 12:31:25 2001 +0200
@@ -208,13 +208,13 @@
   have 
     "\<exists>ts\<in>list (length bs) (states G maxs maxr).
          ?start <=[JVMType.le G maxs maxr] ts \<and>
-         welltyping (JVMType.le G maxs maxr) Err (exec G maxs rT bs) (\<lambda>pc. succs (bs ! pc) pc) ts"
+         wt_step (JVMType.le G maxs maxr) Err (exec G maxs rT bs) (\<lambda>pc. succs (bs ! pc) pc) ts"
     by (unfold is_bcv_def) auto
 
   then obtain phi' where
     l: "phi' \<in> list (length bs) (states G maxs maxr)" and
     s: "?start <=[JVMType.le G maxs maxr] phi'" and
-    w: "welltyping (JVMType.le G maxs maxr) Err (exec G maxs rT bs) (\<lambda>pc. succs (bs ! pc) pc) phi'"
+    w: "wt_step (JVMType.le G maxs maxr) Err (exec G maxs rT bs) (\<lambda>pc. succs (bs ! pc) pc) phi'"
     by blast
    
   hence dynamic:
@@ -231,7 +231,7 @@
   
   with instrs w
   have "phi' ! 0 \<noteq> Err"
-    by (unfold welltyping_def) simp
+    by (unfold wt_step_def) simp
 
   with instrs l
   have phi0: "OK (map ok_val phi' ! 0) = phi' ! 0"
@@ -380,7 +380,7 @@
   qed         
 
   from dynamic
-  have "welltyping (le G maxs ?maxr) Err (exec G maxs rT bs) ?succs ?phi"
+  have "wt_step (le G maxs ?maxr) Err (exec G maxs rT bs) ?succs ?phi"
     by (simp add: dynamic_wt_def JVM_le_Err_conv)
   
   with start 1 2 is_bcv