| changeset 55419 | 8b7c7157fa11 |
| parent 46359 | 9bc43dc49d0a |
| child 56922 | d411a81b8356 |
--- 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