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