src/HOL/Transitive_Closure.thy
changeset 15131 c69542757a4d
parent 15096 be1d3b8cfbd5
child 15140 322485b816ac
--- a/src/HOL/Transitive_Closure.thy	Mon Aug 16 14:21:54 2004 +0200
+++ b/src/HOL/Transitive_Closure.thy	Mon Aug 16 14:22:27 2004 +0200
@@ -6,9 +6,10 @@
 
 header {* Reflexive and Transitive closure of a relation *}
 
-theory Transitive_Closure = Inductive
-
-files ("../Provers/trancl.ML"):
+theory Transitive_Closure
+import Inductive
+files ("../Provers/trancl.ML")
+begin
 
 text {*
   @{text rtrancl} is reflexive/transitive closure,