src/HOL/Record.thy
changeset 43311 1efdcb579b6c
parent 42695 a94ad372b2f5
child 44922 14f7da460ce8
--- a/src/HOL/Record.thy	Thu Jun 09 08:32:15 2011 +0200
+++ b/src/HOL/Record.thy	Thu Jun 09 08:32:16 2011 +0200
@@ -9,7 +9,7 @@
 header {* Extensible records with structural subtyping *}
 
 theory Record
-imports Plain Quickcheck_Exhaustive
+imports Plain Quickcheck_Narrowing
 uses ("Tools/record.ML")
 begin