src/HOL/SetInterval.thy
changeset 15131 c69542757a4d
parent 15056 b75073d90bff
child 15140 322485b816ac
--- a/src/HOL/SetInterval.thy	Mon Aug 16 14:21:54 2004 +0200
+++ b/src/HOL/SetInterval.thy	Mon Aug 16 14:22:27 2004 +0200
@@ -9,7 +9,9 @@
 
 header {* Set intervals *}
 
-theory SetInterval = IntArith:
+theory SetInterval
+import IntArith
+begin
 
 constdefs
   lessThan    :: "('a::ord) => 'a set"	("(1{..<_})")