src/HOL/Library/Formal_Power_Series.thy
changeset 30746 d6915b738bd9
parent 30488 5c4c3a9e9102
child 30747 b8ca7e450de3
equal deleted inserted replaced
30599:4216e9c70cfe 30746:d6915b738bd9
   386   finally have "(a*b) $ (i+j) \<noteq> 0" .
   386   finally have "(a*b) $ (i+j) \<noteq> 0" .
   387   then show "a*b \<noteq> 0" unfolding fps_nonzero_nth by blast
   387   then show "a*b \<noteq> 0" unfolding fps_nonzero_nth by blast
   388 qed
   388 qed
   389 
   389 
   390 instance fps :: (idom) idom ..
   390 instance fps :: (idom) idom ..
       
   391 
       
   392 instantiation fps :: (comm_ring_1) number_ring
       
   393 begin
       
   394 definition number_of_fps_def: "(number_of k::'a fps) = of_int k"
       
   395 
       
   396 instance 
       
   397 by (intro_classes, rule number_of_fps_def)
       
   398 end
   391 
   399 
   392 subsection{* Inverses of formal power series *}
   400 subsection{* Inverses of formal power series *}
   393 
   401 
   394 declare setsum_cong[fundef_cong]
   402 declare setsum_cong[fundef_cong]
   395 
   403