src/HOL/Complex/CLim.thy
changeset 15131 c69542757a4d
parent 15013 34264f5e4691
child 15140 322485b816ac
equal deleted inserted replaced
15130:dc6be28d7f4e 15131:c69542757a4d
     4     Conversion to Isar and new proofs by Lawrence C Paulson, 2004
     4     Conversion to Isar and new proofs by Lawrence C Paulson, 2004
     5 *)
     5 *)
     6 
     6 
     7 header{*Limits, Continuity and Differentiation for Complex Functions*}
     7 header{*Limits, Continuity and Differentiation for Complex Functions*}
     8 
     8 
     9 theory CLim = CSeries:
     9 theory CLim
       
    10 import CSeries
       
    11 begin
    10 
    12 
    11 (*not in simpset?*)
    13 (*not in simpset?*)
    12 declare hypreal_epsilon_not_zero [simp]
    14 declare hypreal_epsilon_not_zero [simp]
    13 
    15 
    14 (*??generalize*)
    16 (*??generalize*)