adding quickcheck generators in some HOL-Library theories
authorbulwahn
Tue, 20 Dec 2011 17:40:18 +0100
changeset 45928 874845660119
parent 45927 e0305e4f02c9
child 45929 d7d6c8cfb6f6
adding quickcheck generators in some HOL-Library theories
src/HOL/Library/Polynomial.thy
src/HOL/Library/RBT.thy
--- a/src/HOL/Library/Polynomial.thy	Tue Dec 20 17:40:17 2011 +0100
+++ b/src/HOL/Library/Polynomial.thy	Tue Dec 20 17:40:18 2011 +0100
@@ -1503,6 +1503,8 @@
 
 code_datatype "0::'a::zero poly" pCons
 
+quickcheck_generator poly constructors: "0::'a::zero poly", pCons
+
 declare pCons_0_0 [code_post]
 
 instantiation poly :: ("{zero, equal}") equal
--- a/src/HOL/Library/RBT.thy	Tue Dec 20 17:40:17 2011 +0100
+++ b/src/HOL/Library/RBT.thy	Tue Dec 20 17:40:18 2011 +0100
@@ -169,5 +169,8 @@
   "distinct (keys t)"
   by (simp add: keys_def RBT_Impl.keys_def distinct_entries)
 
+subsection {* Quickcheck generators *}
+
+quickcheck_generator rbt constructors: empty, insert
 
 end