src/HOL/MicroJava/JVM/JVMState.thy
changeset 10057 8c8d2d0d3ef8
parent 10042 7164dc0d24d8
child 10922 f1209aff9517
--- a/src/HOL/MicroJava/JVM/JVMState.thy	Thu Sep 21 19:25:57 2000 +0200
+++ b/src/HOL/MicroJava/JVM/JVMState.thy	Fri Sep 22 13:12:19 2000 +0200
@@ -2,25 +2,26 @@
     ID:         $Id$
     Author:     Cornelia Pusch
     Copyright   1999 Technische Universitaet Muenchen
-
-State of the JVM
 *)
 
-JVMState = Store +
+
+header {* State of the JVM *}
 
 
-(** frame stack **)
+theory JVMState = Store:
 
+
+text {* frame stack :*}
 types
  opstack 	 = "val list"
  locvars 	 = "val list" 
  p_count 	 = nat
 
- frame = "opstack \\<times>			
-	  locvars \\<times>		
-	  cname \\<times>			
-	  sig \\<times>			
-	  p_count"
+ frame = "opstack \<times>			
+          locvars \<times>		
+          cname \<times>			
+          sig \<times>			
+          p_count"
 
 	(* operand stack *)
 	(* local variables *)
@@ -29,22 +30,20 @@
 	(* program counter within frame *)
 
 
-(** exceptions **)
-
+text {* exceptions: *}
 constdefs
- raise_xcpt :: "bool => xcpt => xcpt option"
-"raise_xcpt c x == (if c then Some x else None)"
-
-(** runtime state **)
-
-types
- jvm_state = "xcpt option \\<times> aheap \\<times> frame list"	
+  raise_xcpt :: "bool => xcpt => xcpt option"
+  "raise_xcpt c x == (if c then Some x else None)"
 
 
+text {* runtime state: *}
+types
+  jvm_state = "xcpt option \<times> aheap \<times> frame list"	
 
-(** dynamic method lookup **)
 
+text {* dynamic method lookup: *}
 constdefs
- dyn_class	:: "'code prog \\<times> sig \\<times> cname => cname"
-"dyn_class == \\<lambda>(G,sig,C). fst(the(method(G,C) sig))"
+  dyn_class	:: "'code prog \<times> sig \<times> cname => cname"
+  "dyn_class == \<lambda>(G,sig,C). fst(the(method(G,C) sig))"
+
 end