src/HOL/MicroJava/JVM/JVMExec.thy
changeset 10057 8c8d2d0d3ef8
parent 10042 7164dc0d24d8
child 10060 4522e59b7d84
--- a/src/HOL/MicroJava/JVM/JVMExec.thy	Thu Sep 21 19:25:57 2000 +0200
+++ b/src/HOL/MicroJava/JVM/JVMExec.thy	Fri Sep 22 13:12:19 2000 +0200
@@ -2,30 +2,38 @@
     ID:         $Id$
     Author:     Cornelia Pusch
     Copyright   1999 Technische Universitaet Muenchen
-
-Execution of the JVM
 *)
 
-JVMExec = JVMExecInstr + 
+header {* Program Execution in the JVM *}
+
+theory JVMExec = JVMExecInstr :
+
 
 consts
- exec :: "jvm_prog \\<times> jvm_state => jvm_state option"
+  exec :: "jvm_prog \<times> jvm_state => jvm_state option"
+
 
 (** exec is not recursive. recdef is just used for pattern matching **)
 recdef exec "{}"
- "exec (G, xp, hp, []) = None"
+  "exec (G, xp, hp, []) = None"
 
- "exec (G, None, hp, (stk,loc,C,sig,pc)#frs) =
+  "exec (G, None, hp, (stk,loc,C,sig,pc)#frs) =
   (let 
      i = snd(snd(snd(the(method (G,C) sig)))) ! pc
    in
      Some (exec_instr i G hp stk loc C sig pc frs))"
 
- "exec (G, Some xp, hp, frs) = None" 
+  "exec (G, Some xp, hp, frs) = None" 
 
 
 constdefs
- exec_all :: "[jvm_prog,jvm_state,jvm_state] => bool"  ("_ \\<turnstile> _ -jvm-> _" [61,61,61]60)
- "G \\<turnstile> s -jvm-> t == (s,t) \\<in> {(s,t). exec(G,s) = Some t}^*"
+  exec_all :: "[jvm_prog,jvm_state,jvm_state] => bool"  
+              ("_ \<turnstile> _ -jvm-> _" [61,61,61]60)
+  "G \<turnstile> s -jvm-> t == (s,t) \<in> {(s,t). exec(G,s) = Some t}^*"
+
+
+syntax (HTML output)
+  exec_all :: "[jvm_prog,jvm_state,jvm_state] => bool"  
+              ("_ |- _ -jvm-> _" [61,61,61]60)
 
 end