src/HOL/MicroJava/JVM/Store.thy
changeset 10042 7164dc0d24d8
parent 8038 a13c3b80d3d4
child 10057 8c8d2d0d3ef8
--- a/src/HOL/MicroJava/JVM/Store.thy	Wed Sep 20 21:20:41 2000 +0200
+++ b/src/HOL/MicroJava/JVM/Store.thy	Thu Sep 21 10:42:49 2000 +0200
@@ -12,7 +12,7 @@
 Store = Conform +  
 
 constdefs
- newref :: "('a \\<leadsto> 'b) \\<Rightarrow> 'a"
- "newref s \\<equiv> \\<epsilon>v. s v = None"
+ newref :: "('a \\<leadsto> 'b) => 'a"
+ "newref s == SOME v. s v = None"
 
 end