src/HOL/Enum.thy
changeset 45119 055c6ff9c5c3
parent 45117 3911cf09899a
child 45140 339a8b3c4791
--- a/src/HOL/Enum.thy	Mon Oct 03 14:43:15 2011 +0200
+++ b/src/HOL/Enum.thy	Mon Oct 03 15:39:30 2011 +0200
@@ -766,7 +766,7 @@
 
 subsection {* An executable (reflexive) transitive closure on finite relations *}
 
-text {* Definitions could be moved to Transitive_Closure if they are of more general use. *}
+text {* Definitions could be moved to Transitive Closure theory if they are of more general use. *}
 
 definition ntrancl :: "('a * 'a => bool) => nat => ('a * 'a => bool)"
 where