src/HOL/Datatype_Examples/TreeFsetI.thy
changeset 58889 5b7a9633cfa8
parent 58309 a09ec6daaa19
child 63167 0909deb8059b
--- a/src/HOL/Datatype_Examples/TreeFsetI.thy	Sun Nov 02 18:21:14 2014 +0100
+++ b/src/HOL/Datatype_Examples/TreeFsetI.thy	Sun Nov 02 18:21:45 2014 +0100
@@ -6,7 +6,7 @@
 Finitely branching possibly infinite trees, with sets of children.
 *)
 
-header {* Finitely Branching Possibly Infinite Trees, with Sets of Children *}
+section {* Finitely Branching Possibly Infinite Trees, with Sets of Children *}
 
 theory TreeFsetI
 imports "~~/src/HOL/Library/FSet"