src/HOL/Quickcheck_Exhaustive.thy
changeset 65956 639eb3617a86
parent 64670 f77b946d18aa
child 67076 fc877448602e
--- a/src/HOL/Quickcheck_Exhaustive.thy	Sun May 28 15:46:26 2017 +0200
+++ b/src/HOL/Quickcheck_Exhaustive.thy	Mon May 29 09:14:15 2017 +0200
@@ -388,7 +388,7 @@
 
 definition enum_term_of_set :: "'a set itself \<Rightarrow> unit \<Rightarrow> term list"
   where "enum_term_of_set _ _ =
-    map (setify (TYPE('a))) (sublists (Quickcheck_Exhaustive.enum_term_of (TYPE('a)) ()))"
+    map (setify (TYPE('a))) (subseqs (Quickcheck_Exhaustive.enum_term_of (TYPE('a)) ()))"
 
 instance ..