Fixed theory name
authorchaieb
Fri, 30 Jan 2009 13:41:45 +0000
changeset 29698 91feea8e41e4
parent 29697 e8785144719d
child 29699 987ed08d82cd
child 29700 22faf21db3df
Fixed theory name
src/HOL/ex/Formal_Power_Series_Examples.thy
--- a/src/HOL/ex/Formal_Power_Series_Examples.thy	Fri Jan 30 13:24:23 2009 +0000
+++ b/src/HOL/ex/Formal_Power_Series_Examples.thy	Fri Jan 30 13:41:45 2009 +0000
@@ -5,7 +5,7 @@
 
 header{* Some applications of formal power series and some properties over complex numbers*}
 
-theory Formal_Ppower_Series_Examples
+theory Formal_Power_Series_Examples
   imports Formal_Power_Series Binomial Complex
 begin