src/HOL/Library/Parallel.thy
changeset 58249 180f1b3508ed
parent 52435 6646bb548c6b
child 58310 91ea607a34d8
--- a/src/HOL/Library/Parallel.thy	Tue Sep 09 17:51:07 2014 +0200
+++ b/src/HOL/Library/Parallel.thy	Tue Sep 09 20:51:36 2014 +0200
@@ -8,7 +8,7 @@
 
 subsection {* Futures *}
 
-datatype 'a future = fork "unit \<Rightarrow> 'a"
+datatype_new 'a future = fork "unit \<Rightarrow> 'a"
 
 primrec join :: "'a future \<Rightarrow> 'a" where
   "join (fork f) = f ()"