src/HOL/Library/Formal_Power_Series.thy
changeset 60017 b785d6d06430
parent 59867 58043346ca64
child 60162 645058aa9d6f
equal deleted inserted replaced
59991:09be0495dcc2 60017:b785d6d06430
   622     }
   622     }
   623     then have "\<exists>n0. \<forall> n \<ge> n0. dist (?s n) a < r"
   623     then have "\<exists>n0. \<forall> n \<ge> n0. dist (?s n) a < r"
   624       by blast
   624       by blast
   625   }
   625   }
   626   then show ?thesis
   626   then show ?thesis
   627     unfolding LIMSEQ_def by blast
   627     unfolding lim_sequentially by blast
   628 qed
   628 qed
   629 
   629 
   630 
   630 
   631 subsection{* Inverses of formal power series *}
   631 subsection{* Inverses of formal power series *}
   632 
   632