src/HOL/Set.thy
changeset 15131 c69542757a4d
parent 15120 f0359f75682e
child 15140 322485b816ac
--- a/src/HOL/Set.thy	Mon Aug 16 14:21:54 2004 +0200
+++ b/src/HOL/Set.thy	Mon Aug 16 14:22:27 2004 +0200
@@ -5,7 +5,9 @@
 
 header {* Set theory for higher-order logic *}
 
-theory Set = HOL:
+theory Set
+import HOL
+begin
 
 text {* A set in HOL is simply a predicate. *}