src/HOL/Record.thy
changeset 56047 1f283d0a4966
parent 55066 4e5ddf3162ac
child 56048 d311c6377e08
--- a/src/HOL/Record.thy	Tue Mar 11 15:34:38 2014 +0100
+++ b/src/HOL/Record.thy	Tue Mar 11 17:18:39 2014 +0100
@@ -9,7 +9,7 @@
 header {* Extensible records with structural subtyping *}
 
 theory Record
-imports Quickcheck_Narrowing
+imports Quickcheck_Exhaustive Quickcheck_Narrowing
 keywords "record" :: thy_decl
 begin