Prove.thy
changeset 183 6acf9e001038
parent 83 e8f352546ad8
child 319 0ae9d9e66cb7
--- a/Prove.thy	Sun Oct 25 00:14:40 2009 +0200
+++ b/Prove.thy	Sun Oct 25 01:15:03 2009 +0200
@@ -3,7 +3,7 @@
 begin
 
 ML {*
-val r = ref (NONE:(unit -> term) option)
+val r = Unsynchronized.ref (NONE:(unit -> term) option)
 *}
 
 ML {*