src/HOL/Record.thy
changeset 42695 a94ad372b2f5
parent 41229 d797baa3d57c
child 43311 1efdcb579b6c
--- a/src/HOL/Record.thy	Thu May 05 10:24:12 2011 +0200
+++ b/src/HOL/Record.thy	Thu May 05 10:47:31 2011 +0200
@@ -9,7 +9,7 @@
 header {* Extensible records with structural subtyping *}
 
 theory Record
-imports Plain Quickcheck
+imports Plain Quickcheck_Exhaustive
 uses ("Tools/record.ML")
 begin