src/HOL/Transitive_Closure.thy
changeset 46635 cde737f9c911
parent 46362 b2878f059f91
child 46638 fc315796794e
--- a/src/HOL/Transitive_Closure.thy	Thu Feb 23 21:16:54 2012 +0100
+++ b/src/HOL/Transitive_Closure.thy	Thu Feb 23 21:25:59 2012 +0100
@@ -6,7 +6,7 @@
 header {* Reflexive and Transitive closure of a relation *}
 
 theory Transitive_Closure
-imports Predicate
+imports Relation
 uses "~~/src/Provers/trancl.ML"
 begin