author | blanchet |
Wed, 12 Feb 2014 08:37:28 +0100 | |
changeset 55419 | 8b7c7157fa11 |
parent 55418 | 9f25e0cca254 |
child 55420 | 4d2123c583fa |
--- a/src/HOL/Library/Transitive_Closure_Table.thy Wed Feb 12 08:37:28 2014 +0100 +++ b/src/HOL/Library/Transitive_Closure_Table.thy Wed Feb 12 08:37:28 2014 +0100 @@ -1,6 +1,6 @@ (* Author: Stefan Berghofer, Lukas Bulwahn, TU Muenchen *) -header {* A tabled implementation of the reflexive transitive closure *} +header {* A table-based implementation of the reflexive transitive closure *} theory Transitive_Closure_Table imports Main