src/HOL/Induct/SList.thy
changeset 58889 5b7a9633cfa8
parent 58305 57752a91eec4
child 60530 44f9873d6f6f
--- a/src/HOL/Induct/SList.thy	Sun Nov 02 18:21:14 2014 +0100
+++ b/src/HOL/Induct/SList.thy	Sun Nov 02 18:21:45 2014 +0100
@@ -21,7 +21,7 @@
 datatype 'a m = Node 'a * 'a m list
 *)
 
-header {* Extended List Theory (old) *}
+section {* Extended List Theory (old) *}
 
 theory SList
 imports Sexp