begin
theorem Th1:
:: deftheorem Def1 defines convergent_to_0 FDIFF_1:def 1 :
for IT being Real_Sequence holds
( IT is convergent_to_0 iff ( IT is non-zero & IT is convergent & lim IT = 0 ) );
reconsider cs = NAT --> 0 as Real_Sequence by FUNCOP_1:57;
:: deftheorem FDIFF_1:def 2 :
canceled;
:: deftheorem Def3 defines REST-like FDIFF_1:def 3 :
for IT being PartFunc of REAL,REAL holds
( IT is REST-like iff ( IT is total & ( for h being convergent_to_0 Real_Sequence holds
( (h ") (#) (IT /* h) is convergent & lim ((h ") (#) (IT /* h)) = 0 ) ) ) );
reconsider cf = REAL --> 0 as Function of REAL,REAL by FUNCOP_1:57;
:: deftheorem Def4 defines linear FDIFF_1:def 4 :
for IT being PartFunc of REAL,REAL holds
( IT is linear iff ( IT is total & ex r being Real st
for p being Real holds IT . p = r * p ) );
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem Th6:
theorem Th7:
theorem Th8:
theorem Th9:
theorem Th10:
theorem Th11:
:: deftheorem Def5 defines is_differentiable_in FDIFF_1:def 5 :
for f being PartFunc of REAL,REAL
for x0 being real number holds
( f is_differentiable_in x0 iff ex N being Neighbourhood of x0 st
( N c= dom f & ex L being LINEAR ex R being REST st
for x being Real st x in N holds
(f . x) - (f . x0) = (L . (x - x0)) + (R . (x - x0)) ) );
:: deftheorem Def6 defines diff FDIFF_1:def 6 :
for f being PartFunc of REAL,REAL
for x0 being real number st f is_differentiable_in x0 holds
for b3 being Real holds
( b3 = diff (f,x0) iff ex N being Neighbourhood of x0 st
( N c= dom f & ex L being LINEAR ex R being REST st
( b3 = L . 1 & ( for x being Real st x in N holds
(f . x) - (f . x0) = (L . (x - x0)) + (R . (x - x0)) ) ) ) );
:: deftheorem Def7 defines is_differentiable_on FDIFF_1:def 7 :
for f being PartFunc of REAL,REAL
for X being set holds
( f is_differentiable_on X iff ( X c= dom f & ( for x being Real st x in X holds
f | X is_differentiable_in x ) ) );
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem Th15:
theorem Th16:
theorem
:: deftheorem Def8 defines `| FDIFF_1:def 8 :
for f being PartFunc of REAL,REAL
for X being set st f is_differentiable_on X holds
for b3 being PartFunc of REAL,REAL holds
( b3 = f `| X iff ( dom b3 = X & ( for x being Real st x in X holds
b3 . x = diff (f,x) ) ) );
theorem
canceled;
theorem
theorem Th20:
theorem Th21:
theorem Th22:
theorem Th23:
theorem Th24:
theorem Th25:
theorem
theorem
theorem
theorem
theorem
theorem
theorem Th32:
theorem
theorem Th34:
theorem
:: deftheorem Def9 defines differentiable FDIFF_1:def 9 :
for f being PartFunc of REAL,REAL holds
( f is differentiable iff f is_differentiable_on dom f );
Lm1:
{} REAL is closed
Lm2:
[#] REAL is open
theorem