Lm1:
for n being Element of NAT
for f, g being PartFunc of REAL,(REAL n) holds f - g = f + (- g)
by NDIFF_4:1;
Lm2:
for a, b, c, d being Real st a <= b & c in ['a,b'] & d in ['a,b'] holds
['(min (c,d)),(max (c,d))'] c= ['a,b']
Lm3:
for X, Y, Z being non empty set
for f being PartFunc of X,Y st Z c= dom f holds
f | Z is Function of Z,Y
theorem Th6:
for
a,
b,
c,
d,
r being
Real for
f being
PartFunc of
REAL,
REAL st
a <= c &
c <= d &
d <= b &
f is_integrable_on ['a,b'] &
f | ['a,b'] is
bounded &
['a,b'] c= dom f holds
(
r (#) f is_integrable_on ['c,d'] &
(r (#) f) | ['c,d'] is
bounded )
theorem
for
a,
b,
c,
d being
Real for
f,
g being
PartFunc of
REAL,
REAL st
a <= c &
c <= d &
d <= b &
f is_integrable_on ['a,b'] &
g is_integrable_on ['a,b'] &
f | ['a,b'] is
bounded &
g | ['a,b'] is
bounded &
['a,b'] c= dom f &
['a,b'] c= dom g holds
(
f - g is_integrable_on ['c,d'] &
(f - g) | ['c,d'] is
bounded )
Lm4:
for a, b, c, d, e being Real
for f being PartFunc of REAL,REAL st a <= b & f is_integrable_on ['a,b'] & f | ['a,b'] is bounded & ['a,b'] c= dom f & c in ['a,b'] & d in ['a,b'] & ( for x being Real st x in ['(min (c,d)),(max (c,d))'] holds
|.(f . x).| <= e ) holds
|.(integral (f,c,d)).| <= e * |.(d - c).|
Lm5:
for A being non empty closed_interval Subset of REAL
for f being PartFunc of REAL,REAL st A c= dom f holds
f | A is Function of A,REAL
by Lm3;
theorem
for
n being
Element of
NAT for
a,
b,
c being
Real for
f being
PartFunc of
REAL,
(REAL n) st
a <= b &
f is_integrable_on ['a,b'] &
f | ['a,b'] is
bounded &
['a,b'] c= dom f &
c in ['a,b'] holds
(
f is_integrable_on ['a,c'] &
f is_integrable_on ['c,b'] &
integral (
f,
a,
b)
= (integral (f,a,c)) + (integral (f,c,b)) )
theorem Th10:
for
n being
Element of
NAT for
a,
b,
c,
d being
Real for
f,
g being
PartFunc of
REAL,
(REAL n) st
a <= c &
c <= d &
d <= b &
f is_integrable_on ['a,b'] &
g is_integrable_on ['a,b'] &
f | ['a,b'] is
bounded &
g | ['a,b'] is
bounded &
['a,b'] c= dom f &
['a,b'] c= dom g holds
(
f + g is_integrable_on ['c,d'] &
(f + g) | ['c,d'] is
bounded )
theorem Th11:
for
n being
Element of
NAT for
a,
b,
c,
d,
r being
Real for
f being
PartFunc of
REAL,
(REAL n) st
a <= c &
c <= d &
d <= b &
f is_integrable_on ['a,b'] &
f | ['a,b'] is
bounded &
['a,b'] c= dom f holds
(
r (#) f is_integrable_on ['c,d'] &
(r (#) f) | ['c,d'] is
bounded )
theorem Th13:
for
n being
Element of
NAT for
a,
b,
c,
d being
Real for
f,
g being
PartFunc of
REAL,
(REAL n) st
a <= c &
c <= d &
d <= b &
f is_integrable_on ['a,b'] &
g is_integrable_on ['a,b'] &
f | ['a,b'] is
bounded &
g | ['a,b'] is
bounded &
['a,b'] c= dom f &
['a,b'] c= dom g holds
(
f - g is_integrable_on ['c,d'] &
(f - g) | ['c,d'] is
bounded )
Lm6:
for n being Element of NAT
for E being Element of REAL n
for p being FinSequence of REAL n st ( for i being Element of NAT st i in Seg n holds
ex Pi being FinSequence of REAL st
( Pi = (proj (i,n)) * p & E . i = Sum Pi ) ) holds
E = Sum p
Lm7:
for n being Element of NAT
for E being Element of REAL n
for p being FinSequence of REAL n
for q being FinSequence of REAL st len p = len q & ( for j being Nat st j in dom p holds
|.(p /. j).| <= q /. j ) & ( for i being Element of NAT st i in Seg n holds
ex Pi being FinSequence of REAL st
( Pi = (proj (i,n)) * p & E . i = Sum Pi ) ) holds
|.E.| <= Sum q
Lm8:
for A being non empty closed_interval Subset of REAL
for n being non zero Element of NAT
for h being Function of A,(REAL n)
for f being Function of A,REAL st h is bounded & h is integrable & f = |.h.| & f is integrable holds
|.(integral h).| <= integral f
Lm9:
for n being Element of NAT
for A being non empty closed_interval Subset of REAL
for h being PartFunc of REAL,(REAL n) st A c= dom h holds
h | A is Function of A,(REAL n)
by Lm3;
theorem Th21:
for
a,
b being
Real for
n being non
zero Element of
NAT for
h being
PartFunc of
REAL,
(REAL n) st
a <= b &
['a,b'] c= dom h &
h is_integrable_on ['a,b'] &
|.h.| is_integrable_on ['a,b'] &
h | ['a,b'] is
bounded holds
|.(integral (h,a,b)).| <= integral (
|.h.|,
a,
b)
Lm10:
for a, b, c, d being Real
for n being non zero Element of NAT
for f being PartFunc of REAL,(REAL n) st a <= b & c <= d & f is_integrable_on ['a,b'] & |.f.| is_integrable_on ['a,b'] & f | ['a,b'] is bounded & ['a,b'] c= dom f & c in ['a,b'] & d in ['a,b'] holds
( f is_integrable_on ['c,d'] & |.f.| is_integrable_on ['c,d'] & |.f.| | ['c,d'] is bounded & |.(integral (f,c,d)).| <= integral (|.f.|,c,d) )
theorem Th22:
for
a,
b,
c,
d being
Real for
n being non
zero Element of
NAT for
f being
PartFunc of
REAL,
(REAL n) st
a <= b &
f is_integrable_on ['a,b'] &
|.f.| is_integrable_on ['a,b'] &
f | ['a,b'] is
bounded &
['a,b'] c= dom f &
c in ['a,b'] &
d in ['a,b'] holds
(
|.f.| is_integrable_on ['(min (c,d)),(max (c,d))'] &
|.f.| | ['(min (c,d)),(max (c,d))'] is
bounded &
|.(integral (f,c,d)).| <= integral (
|.f.|,
(min (c,d)),
(max (c,d))) )
Lm11:
for a, b, c, d being Real
for n being non zero Element of NAT
for f being PartFunc of REAL,(REAL n) st a <= b & c <= d & f is_integrable_on ['a,b'] & |.f.| is_integrable_on ['a,b'] & f | ['a,b'] is bounded & ['a,b'] c= dom f & c in ['a,b'] & d in ['a,b'] holds
( |.f.| is_integrable_on ['c,d'] & |.f.| | ['c,d'] is bounded & |.(integral (f,c,d)).| <= integral (|.f.|,c,d) )
Lm12:
for a, b, c, d being Real
for n being non zero Element of NAT
for f being PartFunc of REAL,(REAL n) st a <= b & c <= d & f is_integrable_on ['a,b'] & |.f.| is_integrable_on ['a,b'] & f | ['a,b'] is bounded & ['a,b'] c= dom f & c in ['a,b'] & d in ['a,b'] holds
|.(integral (f,d,c)).| <= integral (|.f.|,c,d)
theorem
for
a,
b,
c,
d being
Real for
n being non
zero Element of
NAT for
f being
PartFunc of
REAL,
(REAL n) st
a <= b &
c <= d &
f is_integrable_on ['a,b'] &
|.f.| is_integrable_on ['a,b'] &
f | ['a,b'] is
bounded &
['a,b'] c= dom f &
c in ['a,b'] &
d in ['a,b'] holds
(
|.f.| is_integrable_on ['c,d'] &
|.f.| | ['c,d'] is
bounded &
|.(integral (f,c,d)).| <= integral (
|.f.|,
c,
d) &
|.(integral (f,d,c)).| <= integral (
|.f.|,
c,
d) )
by Lm11, Lm12;
Lm13:
for a, b, c, d, e being Real
for n being non zero Element of NAT
for f being PartFunc of REAL,(REAL n) st a <= b & f is_integrable_on ['a,b'] & |.f.| is_integrable_on ['a,b'] & f | ['a,b'] is bounded & ['a,b'] c= dom f & c in ['a,b'] & d in ['a,b'] & ( for x being Real st x in ['(min (c,d)),(max (c,d))'] holds
|.(f /. x).| <= e ) holds
|.(integral (f,c,d)).| <= e * |.(d - c).|
Lm14:
for a, b, c, d, e being Real
for n being non zero Element of NAT
for f being PartFunc of REAL,(REAL n) st a <= b & c <= d & f is_integrable_on ['a,b'] & |.f.| is_integrable_on ['a,b'] & f | ['a,b'] is bounded & ['a,b'] c= dom f & c in ['a,b'] & d in ['a,b'] & ( for x being Real st x in ['c,d'] holds
|.(f /. x).| <= e ) holds
|.(integral (f,c,d)).| <= e * (d - c)
Lm15:
for a, b, c, d, e being Real
for n being non zero Element of NAT
for f being PartFunc of REAL,(REAL n) st a <= b & c <= d & f is_integrable_on ['a,b'] & |.f.| is_integrable_on ['a,b'] & f | ['a,b'] is bounded & ['a,b'] c= dom f & c in ['a,b'] & d in ['a,b'] & ( for x being Real st x in ['c,d'] holds
|.(f /. x).| <= e ) holds
|.(integral (f,d,c)).| <= e * (d - c)
theorem
for
a,
b,
c,
d,
e being
Real for
n being non
zero Element of
NAT for
f being
PartFunc of
REAL,
(REAL n) st
a <= b &
c <= d &
f is_integrable_on ['a,b'] &
|.f.| is_integrable_on ['a,b'] &
f | ['a,b'] is
bounded &
['a,b'] c= dom f &
c in ['a,b'] &
d in ['a,b'] & ( for
x being
Real st
x in ['c,d'] holds
|.(f /. x).| <= e ) holds
(
|.(integral (f,c,d)).| <= e * (d - c) &
|.(integral (f,d,c)).| <= e * (d - c) )
by Lm14, Lm15;
theorem Th25:
for
n being
Element of
NAT for
a,
b,
c,
d,
r being
Real for
f being
PartFunc of
REAL,
(REAL n) st
a <= b &
f is_integrable_on ['a,b'] &
f | ['a,b'] is
bounded &
['a,b'] c= dom f &
c in ['a,b'] &
d in ['a,b'] holds
integral (
(r (#) f),
c,
d)
= r * (integral (f,c,d))
theorem Th26:
for
n being
Element of
NAT for
a,
b,
c,
d being
Real for
f being
PartFunc of
REAL,
(REAL n) st
a <= b &
f is_integrable_on ['a,b'] &
f | ['a,b'] is
bounded &
['a,b'] c= dom f &
c in ['a,b'] &
d in ['a,b'] holds
integral (
(- f),
c,
d)
= - (integral (f,c,d))
theorem Th27:
for
n being
Element of
NAT for
a,
b,
c,
d being
Real for
f,
g being
PartFunc of
REAL,
(REAL n) st
a <= b &
f is_integrable_on ['a,b'] &
g is_integrable_on ['a,b'] &
f | ['a,b'] is
bounded &
g | ['a,b'] is
bounded &
['a,b'] c= dom f &
['a,b'] c= dom g &
c in ['a,b'] &
d in ['a,b'] holds
integral (
(f + g),
c,
d)
= (integral (f,c,d)) + (integral (g,c,d))
theorem Th28:
for
n being
Element of
NAT for
a,
b,
c,
d being
Real for
f,
g being
PartFunc of
REAL,
(REAL n) st
a <= b &
f is_integrable_on ['a,b'] &
g is_integrable_on ['a,b'] &
f | ['a,b'] is
bounded &
g | ['a,b'] is
bounded &
['a,b'] c= dom f &
['a,b'] c= dom g &
c in ['a,b'] &
d in ['a,b'] holds
integral (
(f - g),
c,
d)
= (integral (f,c,d)) - (integral (g,c,d))
theorem Th30:
for
n being
Element of
NAT for
a,
b,
c,
d being
Real for
f being
PartFunc of
REAL,
(REAL n) for
E being
Element of
REAL n st
a <= b & ( for
x being
Real st
x in ['a,b'] holds
f . x = E ) &
['a,b'] c= dom f &
c in ['a,b'] &
d in ['a,b'] holds
integral (
f,
c,
d)
= (d - c) * E
theorem Th31:
for
n being
Element of
NAT for
a,
b,
c,
d being
Real for
f being
PartFunc of
REAL,
(REAL n) st
a <= b &
f is_integrable_on ['a,b'] &
f | ['a,b'] is
bounded &
['a,b'] c= dom f &
c in ['a,b'] &
d in ['a,b'] holds
integral (
f,
a,
d)
= (integral (f,a,c)) + (integral (f,c,d))
theorem Th32:
for
n being
Element of
NAT for
a,
b,
c,
d,
e being
Real for
f being
PartFunc of
REAL,
(REAL n) st
a <= b &
f is_integrable_on ['a,b'] &
f | ['a,b'] is
bounded &
['a,b'] c= dom f &
c in ['a,b'] &
d in ['a,b'] & ( for
x being
Real st
x in ['(min (c,d)),(max (c,d))'] holds
|.(f /. x).| <= e ) holds
|.(integral (f,c,d)).| <= (n * e) * |.(d - c).|
Lm16:
for n being Element of NAT
for p being FinSequence of REAL n
for r being Element of REAL n
for q being FinSequence of (REAL-NS n) st p = q & ( for i being Element of NAT st i in Seg n holds
ex Pi being FinSequence of REAL st
( Pi = (proj (i,n)) * p & r . i = Sum Pi ) ) holds
r = Sum q
theorem Th45:
for
n being
Element of
NAT for
a,
b being
Real for
f being
PartFunc of
REAL,
(REAL n) for
g being
PartFunc of
REAL,
(REAL-NS n) st
f = g &
a <= b &
f | ['a,b'] is
bounded &
['a,b'] c= dom f &
f is_integrable_on ['a,b'] holds
integral (
f,
a,
b)
= integral (
g,
a,
b)
theorem
for
n being
Element of
NAT for
a,
b being
Real for
f,
g being
PartFunc of
REAL,
(REAL-NS n) st
a <= b &
f is_integrable_on ['a,b'] &
g is_integrable_on ['a,b'] &
['a,b'] c= dom f &
['a,b'] c= dom g holds
(
integral (
(f + g),
a,
b)
= (integral (f,a,b)) + (integral (g,a,b)) &
integral (
(f - g),
a,
b)
= (integral (f,a,b)) - (integral (g,a,b)) )
theorem Th48:
for
n being
Element of
NAT for
a,
b,
c,
d being
Real for
f being
PartFunc of
REAL,
(REAL-NS n) for
g being
PartFunc of
REAL,
(REAL n) st
f = g &
a <= b &
['a,b'] c= dom f &
f | ['a,b'] is
bounded &
f is_integrable_on ['a,b'] &
c in ['a,b'] &
d in ['a,b'] holds
integral (
f,
c,
d)
= integral (
g,
c,
d)
theorem
for
n being
Element of
NAT for
a,
b,
c,
d being
Real for
f,
g being
PartFunc of
REAL,
(REAL-NS n) st
a <= b &
f is_integrable_on ['a,b'] &
g is_integrable_on ['a,b'] &
f | ['a,b'] is
bounded &
g | ['a,b'] is
bounded &
['a,b'] c= dom f &
['a,b'] c= dom g &
c in ['a,b'] &
d in ['a,b'] holds
integral (
(f + g),
c,
d)
= (integral (f,c,d)) + (integral (g,c,d))
theorem Th50:
for
n being
Element of
NAT for
a,
b,
c,
d being
Real for
f,
g being
PartFunc of
REAL,
(REAL-NS n) st
a <= b &
f is_integrable_on ['a,b'] &
g is_integrable_on ['a,b'] &
f | ['a,b'] is
bounded &
g | ['a,b'] is
bounded &
['a,b'] c= dom f &
['a,b'] c= dom g &
c in ['a,b'] &
d in ['a,b'] holds
integral (
(f - g),
c,
d)
= (integral (f,c,d)) - (integral (g,c,d))
theorem Th52:
for
n being
Element of
NAT for
a,
b,
c,
d being
Real for
E being
Point of
(REAL-NS n) for
f being
PartFunc of
REAL,
(REAL-NS n) st
a <= b &
['a,b'] c= dom f & ( for
x being
Real st
x in ['a,b'] holds
f . x = E ) &
c in ['a,b'] &
d in ['a,b'] holds
integral (
f,
c,
d)
= (d - c) * E
theorem Th53:
for
n being
Element of
NAT for
a,
b,
c,
d being
Real for
f being
PartFunc of
REAL,
(REAL-NS n) st
a <= b &
f is_integrable_on ['a,b'] &
f | ['a,b'] is
bounded &
['a,b'] c= dom f &
c in ['a,b'] &
d in ['a,b'] holds
integral (
f,
a,
d)
= (integral (f,a,c)) + (integral (f,c,d))
theorem Th54:
for
n being
Element of
NAT for
a,
b,
c,
d,
e being
Real for
f being
PartFunc of
REAL,
(REAL-NS n) st
a <= b &
f is_integrable_on ['a,b'] &
f | ['a,b'] is
bounded &
['a,b'] c= dom f &
c in ['a,b'] &
d in ['a,b'] & ( for
x being
Real st
x in ['(min (c,d)),(max (c,d))'] holds
||.(f /. x).|| <= e ) holds
||.(integral (f,c,d)).|| <= (n * e) * |.(d - c).|
Lm17:
for a being Real
for X being RealNormSpace
for x being Point of X holds ||.((a ") * x).|| = ||.x.|| / |.a.|
theorem Th55:
for
a,
b,
x0 being
Real for
n being non
zero Element of
NAT for
F,
f being
PartFunc of
REAL,
(REAL-NS n) st
a <= b &
f is_integrable_on ['a,b'] &
f | ['a,b'] is
bounded &
['a,b'] c= dom f &
].a,b.[ c= dom F & ( for
x being
Real st
x in ].a,b.[ holds
F . x = integral (
f,
a,
x) ) &
x0 in ].a,b.[ &
f is_continuous_in x0 holds
(
F is_differentiable_in x0 &
diff (
F,
x0)
= f /. x0 )
Lm18:
for n being Element of NAT
for a, b being Real
for f being PartFunc of REAL,(REAL-NS n) ex F being PartFunc of REAL,(REAL-NS n) st
( ].a,b.[ c= dom F & ( for x being Real st x in ].a,b.[ holds
F . x = integral (f,a,x) ) )
theorem
for
a,
b,
x0 being
Real for
n being non
zero Element of
NAT for
f being
PartFunc of
REAL,
(REAL-NS n) st
a <= b &
f is_integrable_on ['a,b'] &
f | ['a,b'] is
bounded &
['a,b'] c= dom f &
x0 in ].a,b.[ &
f is_continuous_in x0 holds
ex
F being
PartFunc of
REAL,
(REAL-NS n) st
(
].a,b.[ c= dom F & ( for
x being
Real st
x in ].a,b.[ holds
F . x = integral (
f,
a,
x) ) &
F is_differentiable_in x0 &
diff (
F,
x0)
= f /. x0 )