src/HOL/Induct/Com.thy
changeset 58889 5b7a9633cfa8
parent 58310 91ea607a34d8
child 59807 22bc39064290
--- a/src/HOL/Induct/Com.thy	Sun Nov 02 18:21:14 2014 +0100
+++ b/src/HOL/Induct/Com.thy	Sun Nov 02 18:21:45 2014 +0100
@@ -5,7 +5,7 @@
 Example of Mutual Induction via Iteratived Inductive Definitions: Commands
 *)
 
-header{*Mutual Induction via Iteratived Inductive Definitions*}
+section{*Mutual Induction via Iteratived Inductive Definitions*}
 
 theory Com imports Main begin