src/HOL/Statespace/DistinctTreeProver.thy
changeset 32740 9dd0a2f83429
parent 32010 cb1a1c94b4cd
child 32960 69916a850301
--- a/src/HOL/Statespace/DistinctTreeProver.thy	Tue Sep 29 14:59:24 2009 +0200
+++ b/src/HOL/Statespace/DistinctTreeProver.thy	Tue Sep 29 16:24:36 2009 +0200
@@ -664,7 +664,7 @@
      HOLogic.Trueprop$
        (Const ("DistinctTreeProver.all_distinct",DistinctTreeProver.treeT (Type ("nat",[])) --> HOLogic.boolT)$t')
 
-val da = ref refl;
+val da = Unsynchronized.ref refl;
 
 *}