src/HOL/MicroJava/JVM/JVMInstructions.thy
changeset 9550 19a6d1289f5e
parent 9376 c32c5696ec2a
child 10057 8c8d2d0d3ef8
--- a/src/HOL/MicroJava/JVM/JVMInstructions.thy	Mon Aug 07 14:32:56 2000 +0200
+++ b/src/HOL/MicroJava/JVM/JVMInstructions.thy	Mon Aug 07 14:34:03 2000 +0200
@@ -8,6 +8,7 @@
 
 JVMInstructions = JVMState +
 
+
 datatype 
   instr = Load nat                  (* load from local variable *)
         | Store nat                 (* store into local variable *)
@@ -17,7 +18,7 @@
         | Getfield vname cname	  	(* Fetch field from object *)
         | Putfield vname cname		  (* Set field in object     *)
         | Checkcast cname	          (* Check whether object is of given type *)
-        | Invoke mname "(ty list)"  (* inv. instance meth of an object *)
+        | Invoke cname mname "(ty list)"  (* inv. instance meth of an object *)
         | Return
         | Pop
         | Dup