begin
theorem Th1:
theorem Th2:
theorem Th3:
theorem Th4:
:: deftheorem Def1 defines is_Lcontinuous_in FDIFF_3:def 1 :
for f being PartFunc of REAL,REAL
for x0 being Real holds
( f is_Lcontinuous_in x0 iff ( x0 in dom f & ( for a being Real_Sequence st rng a c= (left_open_halfline x0) /\ (dom f) & a is convergent & lim a = x0 holds
( f /* a is convergent & f . x0 = lim (f /* a) ) ) ) );
:: deftheorem Def2 defines is_Rcontinuous_in FDIFF_3:def 2 :
for f being PartFunc of REAL,REAL
for x0 being Real holds
( f is_Rcontinuous_in x0 iff ( x0 in dom f & ( for a being Real_Sequence st rng a c= (right_open_halfline x0) /\ (dom f) & a is convergent & lim a = x0 holds
( f /* a is convergent & f . x0 = lim (f /* a) ) ) ) );
:: deftheorem Def3 defines is_right_differentiable_in FDIFF_3:def 3 :
for f being PartFunc of REAL,REAL
for x0 being Real holds
( f is_right_differentiable_in x0 iff ( ex r being Real st
( r > 0 & [.x0,(x0 + r).] c= dom f ) & ( for h being convergent_to_0 Real_Sequence
for c being V8() Real_Sequence st rng c = {x0} & rng (h + c) c= dom f & ( for n being Element of NAT holds h . n > 0 ) holds
(h ") (#) ((f /* (h + c)) - (f /* c)) is convergent ) ) );
:: deftheorem Def4 defines is_left_differentiable_in FDIFF_3:def 4 :
for f being PartFunc of REAL,REAL
for x0 being Real holds
( f is_left_differentiable_in x0 iff ( ex r being Real st
( r > 0 & [.(x0 - r),x0.] c= dom f ) & ( for h being convergent_to_0 Real_Sequence
for c being V8() Real_Sequence st rng c = {x0} & rng (h + c) c= dom f & ( for n being Element of NAT holds h . n < 0 ) holds
(h ") (#) ((f /* (h + c)) - (f /* c)) is convergent ) ) );
theorem Th5:
theorem Th6:
theorem Th7:
theorem Th8:
:: deftheorem Def5 defines Ldiff FDIFF_3:def 5 :
for x0 being Real
for f being PartFunc of REAL,REAL st f is_left_differentiable_in x0 holds
for b3 being Real holds
( b3 = Ldiff (f,x0) iff for h being convergent_to_0 Real_Sequence
for c being V8() Real_Sequence st rng c = {x0} & rng (h + c) c= dom f & ( for n being Element of NAT holds h . n < 0 ) holds
b3 = lim ((h ") (#) ((f /* (h + c)) - (f /* c))) );
:: deftheorem Def6 defines Rdiff FDIFF_3:def 6 :
for x0 being Real
for f being PartFunc of REAL,REAL st f is_right_differentiable_in x0 holds
for b3 being Real holds
( b3 = Rdiff (f,x0) iff for h being convergent_to_0 Real_Sequence
for c being V8() Real_Sequence st rng c = {x0} & rng (h + c) c= dom f & ( for n being Element of NAT holds h . n > 0 ) holds
b3 = lim ((h ") (#) ((f /* (h + c)) - (f /* c))) );
theorem Th9:
theorem
theorem
theorem
Lm1:
for f1, f2 being PartFunc of REAL,REAL
for x0 being Real st f1 is_left_differentiable_in x0 & f2 is_left_differentiable_in x0 & ex r0 being Real st
( r0 > 0 & ( for g being Real st g in dom f2 & g in [.(x0 - r0),x0.] holds
f2 . g <> 0 ) ) holds
( f1 / f2 is_left_differentiable_in x0 & Ldiff ((f1 / f2),x0) = (((Ldiff (f1,x0)) * (f2 . x0)) - ((Ldiff (f2,x0)) * (f1 . x0))) / ((f2 . x0) ^2) )
theorem
Lm2:
for f being PartFunc of REAL,REAL
for x0 being Real st f is_left_differentiable_in x0 & ex r0 being Real st
( r0 > 0 & ( for g being Real st g in dom f & g in [.(x0 - r0),x0.] holds
f . g <> 0 ) ) holds
( f ^ is_left_differentiable_in x0 & Ldiff ((f ^),x0) = - ((Ldiff (f,x0)) / ((f . x0) ^2)) )
theorem
theorem Th15:
theorem
theorem
theorem
Lm3:
for f1, f2 being PartFunc of REAL,REAL
for x0 being Real st f1 is_right_differentiable_in x0 & f2 is_right_differentiable_in x0 & ex r0 being Real st
( r0 > 0 & ( for g being Real st g in dom f2 & g in [.x0,(x0 + r0).] holds
f2 . g <> 0 ) ) holds
( f1 / f2 is_right_differentiable_in x0 & Rdiff ((f1 / f2),x0) = (((Rdiff (f1,x0)) * (f2 . x0)) - ((Rdiff (f2,x0)) * (f1 . x0))) / ((f2 . x0) ^2) )
theorem
Lm4:
for f being PartFunc of REAL,REAL
for x0 being Real st f is_right_differentiable_in x0 & ex r0 being Real st
( r0 > 0 & ( for g being Real st g in dom f & g in [.x0,(x0 + r0).] holds
f . g <> 0 ) ) holds
( f ^ is_right_differentiable_in x0 & Rdiff ((f ^),x0) = - ((Rdiff (f,x0)) / ((f . x0) ^2)) )
theorem
theorem
theorem