src/HOL/Record.thy
changeset 15131 c69542757a4d
parent 14701 62a724ce51c7
child 15140 322485b816ac
--- a/src/HOL/Record.thy	Mon Aug 16 14:21:54 2004 +0200
+++ b/src/HOL/Record.thy	Mon Aug 16 14:22:27 2004 +0200
@@ -3,8 +3,10 @@
     Author:     Wolfgang Naraschewski, Norbert Schirmer  and Markus Wenzel, TU Muenchen
 *)
 
-theory Record = Product_Type
-files ("Tools/record_package.ML"):
+theory Record
+import Product_Type
+files ("Tools/record_package.ML")
+begin
 
 ML {*
 val [h1, h2] = Goal "PROP Goal (\<And>x. PROP P x) \<Longrightarrow> (PROP P x \<Longrightarrow> PROP Q) \<Longrightarrow> PROP Q";