src/HOL/ex/Transitive_Closure_Table_Ex.thy
changeset 58889 5b7a9633cfa8
parent 58310 91ea607a34d8
child 61343 5b5656a63bd6
--- a/src/HOL/ex/Transitive_Closure_Table_Ex.thy	Sun Nov 02 18:21:14 2014 +0100
+++ b/src/HOL/ex/Transitive_Closure_Table_Ex.thy	Sun Nov 02 18:21:45 2014 +0100
@@ -1,6 +1,6 @@
 (* Author: Stefan Berghofer, Lukas Bulwahn, TU Muenchen *)
 
-header {* Simple example for table-based implementation of the reflexive transitive closure *}
+section {* Simple example for table-based implementation of the reflexive transitive closure *}
 
 theory Transitive_Closure_Table_Ex
 imports "~~/src/HOL/Library/Transitive_Closure_Table"