begin
:: deftheorem Def1 defines convergent_to_0 CFDIFF_1:def 1 :
for IT being Complex_Sequence holds
( IT is convergent_to_0 iff ( IT is non-empty & IT is convergent & lim IT = 0 ) );
theorem
:: deftheorem Def2 defines InvShift CFDIFF_1:def 2 :
for r being real number
for b2 being Complex_Sequence holds
( b2 = InvShift r iff for n being Element of NAT holds b2 . n = 1 / (n + r) );
theorem Th2:
theorem Th3:
reconsider cs = NAT --> 0c as Complex_Sequence ;
theorem
theorem
:: deftheorem Def3 defines REST-like CFDIFF_1:def 3 :
for IT being PartFunc of COMPLEX,COMPLEX holds
( IT is REST-like iff for h being convergent_to_0 Complex_Sequence holds
( (h ") (#) (IT /* h) is convergent & lim ((h ") (#) (IT /* h)) = 0 ) );
reconsider cf = COMPLEX --> 0c as Function of COMPLEX,COMPLEX ;
:: deftheorem Def4 defines linear CFDIFF_1:def 4 :
for IT being PartFunc of COMPLEX,COMPLEX holds
( IT is linear iff ex a being Complex st
for z being Complex holds IT /. z = a * z );
:: deftheorem Def5 defines Neighbourhood CFDIFF_1:def 5 :
for z0 being Complex
for b2 being Subset of COMPLEX holds
( b2 is Neighbourhood of z0 iff ex g being Real st
( 0 < g & { y where y is Complex : |.(y - z0).| < g } c= b2 ) );
theorem Th6:
theorem Th7:
Lm1:
for z0 being Complex
for N1, N2 being Neighbourhood of z0 ex N being Neighbourhood of z0 st
( N c= N1 & N c= N2 )
:: deftheorem Def6 defines is_differentiable_in CFDIFF_1:def 6 :
for f being PartFunc of COMPLEX,COMPLEX
for z0 being Complex holds
( f is_differentiable_in z0 iff ex N being Neighbourhood of z0 st
( N c= dom f & ex L being C_LINEAR ex R being C_REST st
for z being Complex st z in N holds
(f /. z) - (f /. z0) = (L /. (z - z0)) + (R /. (z - z0)) ) );
:: deftheorem Def7 defines diff CFDIFF_1:def 7 :
for f being PartFunc of COMPLEX,COMPLEX
for z0 being Complex st f is_differentiable_in z0 holds
for b3 being Complex holds
( b3 = diff (f,z0) iff ex N being Neighbourhood of z0 st
( N c= dom f & ex L being C_LINEAR ex R being C_REST st
( b3 = L /. 1r & ( for z being Complex st z in N holds
(f /. z) - (f /. z0) = (L /. (z - z0)) + (R /. (z - z0)) ) ) ) );
:: deftheorem Def8 defines differentiable CFDIFF_1:def 8 :
for f being PartFunc of COMPLEX,COMPLEX holds
( f is differentiable iff for x being Complex st x in dom f holds
f is_differentiable_in x );
:: deftheorem Def9 defines is_differentiable_on CFDIFF_1:def 9 :
for f being PartFunc of COMPLEX,COMPLEX
for X being set holds
( f is_differentiable_on X iff ( X c= dom f & f | X is differentiable ) );
theorem Th8:
:: deftheorem Def10 defines closed CFDIFF_1:def 10 :
for X being Subset of COMPLEX holds
( X is closed iff for s1 being Complex_Sequence st rng s1 c= X & s1 is convergent holds
lim s1 in X );
:: deftheorem Def11 defines open CFDIFF_1:def 11 :
for X being Subset of COMPLEX holds
( X is open iff X ` is closed );
theorem Th9:
theorem
theorem Th11:
theorem
theorem Th13:
theorem
theorem Th15:
theorem
:: deftheorem Def12 defines `| CFDIFF_1:def 12 :
for f being PartFunc of COMPLEX,COMPLEX
for X being set st f is_differentiable_on X holds
for b3 being PartFunc of COMPLEX,COMPLEX holds
( b3 = f `| X iff ( dom b3 = X & ( for x being Complex st x in X holds
b3 /. x = diff (f,x) ) ) );
theorem
theorem Th18:
theorem Th19:
theorem Th20:
theorem Th21:
theorem Th22:
theorem Th23:
theorem Th24:
theorem Th25:
theorem Th26:
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem Th34:
theorem
theorem
theorem
theorem