src/HOL/ex/Records.thy
changeset 16417 9bc16273c2d4
parent 15010 72fbe711e414
child 19736 d8d0f8f51d69
--- a/src/HOL/ex/Records.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/HOL/ex/Records.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -6,7 +6,7 @@
 
 header {* Using extensible records in HOL -- points and coloured points *}
 
-theory Records = Main:
+theory Records imports Main begin
 
 subsection {* Points *}