src/HOL/Predicate_Compile_Examples/Predicate_Compile_Tests.thy
changeset 40137 9eabcb1bfe50
parent 40100 98d74bbe8cd8
child 40885 da4bdafeef7c
--- a/src/HOL/Predicate_Compile_Examples/Predicate_Compile_Tests.thy	Mon Oct 25 21:17:11 2010 +0200
+++ b/src/HOL/Predicate_Compile_Examples/Predicate_Compile_Tests.thy	Mon Oct 25 21:17:12 2010 +0200
@@ -974,9 +974,10 @@
 
 code_pred [new_random_dseq inductify] avl .
 thm avl.new_random_dseq_equation
+(* TODO: has highly non-deterministic execution time!
 
 values [new_random_dseq 2, 1, 7] 5 "{t:: int tree. avl t}"
-
+*)
 fun set_of
 where
 "set_of ET = {}"