src/HOL/Transitive_Closure.thy
changeset 15140 322485b816ac
parent 15131 c69542757a4d
child 15531 08c8dad8e399
--- a/src/HOL/Transitive_Closure.thy	Tue Aug 17 11:00:24 2004 +0200
+++ b/src/HOL/Transitive_Closure.thy	Wed Aug 18 11:09:40 2004 +0200
@@ -7,7 +7,7 @@
 header {* Reflexive and Transitive closure of a relation *}
 
 theory Transitive_Closure
-import Inductive
+imports Inductive
 files ("../Provers/trancl.ML")
 begin