src/HOL/Library/Eval_Witness.thy
changeset 32740 9dd0a2f83429
parent 30970 3fe2e418a071
child 34028 1e6206763036
--- a/src/HOL/Library/Eval_Witness.thy	Tue Sep 29 14:59:24 2009 +0200
+++ b/src/HOL/Library/Eval_Witness.thy	Tue Sep 29 16:24:36 2009 +0200
@@ -48,7 +48,7 @@
 structure Eval_Witness_Method =
 struct
 
-val eval_ref : (unit -> bool) option ref = ref NONE;
+val eval_ref : (unit -> bool) option Unsynchronized.ref = Unsynchronized.ref NONE;
 
 end;
 *}