src/HOL/MicroJava/JVM/JVMExec.thy
changeset 10042 7164dc0d24d8
parent 9376 c32c5696ec2a
child 10057 8c8d2d0d3ef8
--- a/src/HOL/MicroJava/JVM/JVMExec.thy	Wed Sep 20 21:20:41 2000 +0200
+++ b/src/HOL/MicroJava/JVM/JVMExec.thy	Thu Sep 21 10:42:49 2000 +0200
@@ -9,7 +9,7 @@
 JVMExec = JVMExecInstr + 
 
 consts
- exec :: "jvm_prog \\<times> jvm_state \\<Rightarrow> 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 "{}"
@@ -25,7 +25,7 @@
 
 
 constdefs
- exec_all :: "[jvm_prog,jvm_state,jvm_state] \\<Rightarrow> bool"  ("_ \\<turnstile> _ -jvm\\<rightarrow> _" [61,61,61]60)
- "G \\<turnstile> s -jvm\\<rightarrow> t \\<equiv> (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}^*"
 
 end