src/HOL/Library/Formal_Power_Series.thy
changeset 58881 b9556a055632
parent 58709 efdc6c533bd3
child 59667 651ea265d568
--- a/src/HOL/Library/Formal_Power_Series.thy	Sun Nov 02 17:16:01 2014 +0100
+++ b/src/HOL/Library/Formal_Power_Series.thy	Sun Nov 02 17:20:45 2014 +0100
@@ -2,7 +2,7 @@
     Author:     Amine Chaieb, University of Cambridge
 *)
 
-header{* A formalization of formal power series *}
+section{* A formalization of formal power series *}
 
 theory Formal_Power_Series
 imports "~~/src/HOL/Number_Theory/Binomial"