src/HOL/Record.thy
changeset 51112 da97167e03f7
parent 48891 c0eafbd55de3
child 54147 97a8ff4e4ac9
--- a/src/HOL/Record.thy	Thu Feb 14 13:16:47 2013 +0100
+++ b/src/HOL/Record.thy	Thu Feb 14 12:24:42 2013 +0100
@@ -9,7 +9,7 @@
 header {* Extensible records with structural subtyping *}
 
 theory Record
-imports Plain Quickcheck_Narrowing
+imports Quickcheck_Narrowing
 keywords "record" :: thy_decl
 begin