diff -r 7fe029e818c2 -r 1f6c140f9c72 src/HOL/Transitive_Closure.thy --- a/src/HOL/Transitive_Closure.thy Fri Feb 24 22:46:16 2012 +0100 +++ b/src/HOL/Transitive_Closure.thy Fri Feb 24 22:46:44 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