Lm1:
for r being set
for I being interval Subset of REAL st r in I & I is closed_interval & not ( r = inf I & r = lower_bound I ) & not ( r = sup I & r = upper_bound I ) holds
r in ].(inf I),(sup I).[
Lm2:
for r being set
for I being interval Subset of REAL st r in I & I is right_open_interval & not ( r = inf I & r = lower_bound I ) holds
r in ].(inf I),(sup I).[
Lm3:
for r being set
for I being interval Subset of REAL st r in I & I is left_open_interval & not ( r = sup I & r = upper_bound I ) holds
r in ].(inf I),(sup I).[
Lm4:
for r being set
for I being interval Subset of REAL st r in I & I is open_interval holds
r in ].(inf I),(sup I).[
Lm5:
for I being interval Subset of REAL st inf I in I holds
inf I = lower_bound I
Lm6:
for I being interval Subset of REAL st sup I in I holds
sup I = upper_bound I
definition
let f be
PartFunc of
REAL,
REAL;
let I be non
empty interval Subset of
REAL;
assume A1:
f is_differentiable_on_interval I
;
existence
ex b1 being PartFunc of REAL,REAL st
( dom b1 = I & ( for x being Real st x in I holds
( ( x = inf I implies b1 . x = Rdiff (f,x) ) & ( x = sup I implies b1 . x = Ldiff (f,x) ) & ( x <> inf I & x <> sup I implies b1 . x = diff (f,x) ) ) ) )
uniqueness
for b1, b2 being PartFunc of REAL,REAL st dom b1 = I & ( for x being Real st x in I holds
( ( x = inf I implies b1 . x = Rdiff (f,x) ) & ( x = sup I implies b1 . x = Ldiff (f,x) ) & ( x <> inf I & x <> sup I implies b1 . x = diff (f,x) ) ) ) & dom b2 = I & ( for x being Real st x in I holds
( ( x = inf I implies b2 . x = Rdiff (f,x) ) & ( x = sup I implies b2 . x = Ldiff (f,x) ) & ( x <> inf I & x <> sup I implies b2 . x = diff (f,x) ) ) ) holds
b1 = b2
end;
theorem
for
f being
PartFunc of
REAL,
REAL for
a,
b being
Real st
a <= b &
f is_differentiable_on_interval ['a,b'] holds
(
(f `\ ['a,b']) . a = Rdiff (
f,
a) &
(f `\ ['a,b']) . b = Ldiff (
f,
b) & ( for
x being
Real st
x in ].a,b.[ holds
(f `\ ['a,b']) . x = diff (
f,
x) ) )
Lm7:
for x, r being Real
for h being non-zero 0 -convergent Real_Sequence
for c being constant Real_Sequence st r > 0 & rng c = {x} & ( for n being Nat holds h . n > 0 ) holds
ex N being Nat st
( rng ((h ^\ N) + c) c= ].x,(x + r).[ & ( for m being Nat holds ((h ^\ N) + c) . m = (h + c) . (N + m) ) & ( for m being Nat st N <= m holds
( |.(h . m).| < r & x < (h + c) . m & (h + c) . m < x + r ) ) )
Lm8:
for x, r being Real
for h being non-zero 0 -convergent Real_Sequence
for c being constant Real_Sequence st r > 0 & rng c = {x} & ( for n being Nat holds h . n < 0 ) holds
ex N being Nat st
( rng ((h ^\ N) + c) c= ].(x - r),x.[ & ( for m being Nat holds ((h ^\ N) + c) . m = (h + c) . (N + m) ) & ( for m being Nat st N <= m holds
( |.(h . m).| < r & x - r < (h + c) . m & (h + c) . m < x ) ) )
Lm9:
for I being non empty Interval
for x being Real st inf I < x & x < sup I holds
ex Z being open Subset of REAL st
( x in Z & Z c= ].(inf I),(sup I).[ )
Lm10:
for X being set st X is Subset of REAL holds
X is Subset of ExtREAL
Lm11:
for I being non empty Interval holds
( not inf I in I or I is closed_interval or I is right_open_interval )
Lm12:
for I being non empty Interval holds
( not sup I in I or I is closed_interval or I is left_open_interval )
Lm13:
for I being non empty Interval holds ].(inf I),(sup I).[ c= I
by Th2;
Lm14:
for I being non empty Interval st inf I in I & inf I < sup I holds
ex e being Real st
( e > 0 & [.(lower_bound I),((lower_bound I) + e).] c= I )
Lm15:
for I being non empty Interval st sup I in I & inf I < sup I holds
ex e being Real st
( e > 0 & [.((upper_bound I) - e),(upper_bound I).] c= I )
Lm16:
for f being PartFunc of REAL,REAL
for x0 being Real st f is_right_differentiable_in x0 holds
( 0 (#) f is_right_differentiable_in x0 & Rdiff ((0 (#) f),x0) = 0 )
Lm17:
for f being PartFunc of REAL,REAL
for x0 being Real st f is_left_differentiable_in x0 holds
( 0 (#) f is_left_differentiable_in x0 & Ldiff ((0 (#) f),x0) = 0 )
Lm18:
for f being PartFunc of REAL,REAL
for x0, r being Real st r <> 0 & f is_right_differentiable_in x0 holds
( r (#) f is_right_differentiable_in x0 & Rdiff ((r (#) f),x0) = r * (Rdiff (f,x0)) )
Lm19:
for f being PartFunc of REAL,REAL
for x0, r being Real st r <> 0 & f is_left_differentiable_in x0 holds
( r (#) f is_left_differentiable_in x0 & Ldiff ((r (#) f),x0) = r * (Ldiff (f,x0)) )
Lm20:
for x0 being Real
for f1, f2 being PartFunc of REAL,REAL st f1 is_right_differentiable_in x0 & f2 is_differentiable_in f1 . x0 holds
ex r being Real st
( r > 0 & [.x0,(x0 + r).] c= dom (f2 * f1) )
Lm21:
for x0 being Real
for f1, f2 being PartFunc of REAL,REAL st f1 is_left_differentiable_in x0 & f2 is_differentiable_in f1 . x0 holds
ex r being Real st
( r > 0 & [.(x0 - r),x0.] c= dom (f2 * f1) )
Lm22:
for I being non empty Interval holds
( I = [.(inf I),(sup I).] or I = ].(inf I),(sup I).] or I = [.(inf I),(sup I).[ or I = ].(inf I),(sup I).[ )
Lm23:
for I being non empty Interval holds
( not inf I in I or I = [.(inf I),(sup I).] or I = [.(inf I),(sup I).[ )
Lm24:
for I being non empty Interval holds
( not sup I in I or I = [.(inf I),(sup I).] or I = ].(inf I),(sup I).] )
Lm25:
for I being non empty Interval st not sup I in I & not inf I in I holds
I = ].(inf I),(sup I).[
Lm26:
for x0 being Real
for f1, f2 being PartFunc of REAL,REAL
for I, J being non empty Interval st f1 is_differentiable_on_interval I & f2 is_differentiable_on_interval J & f1 .: I c= J & x0 = inf I & x0 in I holds
( f2 * f1 is_right_differentiable_in x0 & Rdiff ((f2 * f1),x0) = (((f2 `\ J) * f1) (#) (f1 `\ I)) . x0 )
Lm27:
for x0 being Real
for f1, f2 being PartFunc of REAL,REAL
for I, J being non empty Interval st f1 is_differentiable_on_interval I & f2 is_differentiable_on_interval J & f1 .: I c= J & x0 = sup I & x0 in I holds
( f2 * f1 is_left_differentiable_in x0 & Ldiff ((f2 * f1),x0) = (((f2 `\ J) * f1) (#) (f1 `\ I)) . x0 )
Lm28:
for x0 being Real
for f1, f2 being PartFunc of REAL,REAL
for I, J being non empty Interval st f1 is_differentiable_on_interval I & f2 is_differentiable_on_interval J & f1 .: I c= J & x0 in ].(inf I),(sup I).[ & x0 in I holds
( f2 * f1 is_differentiable_in x0 & diff ((f2 * f1),x0) = (((f2 `\ J) * f1) (#) (f1 `\ I)) . x0 )