begin
theorem
:: deftheorem Def1 defines non-decreasing INTEGRA2:def 1 :
for IT being FinSequence of REAL holds
( IT is non-decreasing iff for n being Element of NAT st n in dom IT & n + 1 in dom IT holds
IT . n <= IT . (n + 1) );
theorem
theorem
theorem
begin
:: deftheorem INTEGRA2:def 2 :
canceled;
theorem
theorem
theorem
theorem Th8:
theorem
theorem
theorem
theorem
theorem Th13:
theorem Th14:
theorem Th15:
theorem Th16:
begin
theorem Th17:
theorem Th18:
theorem Th19:
theorem Th20:
theorem Th21:
theorem Th22:
theorem Th23:
theorem Th24:
theorem Th25:
theorem Th26:
theorem Th27:
theorem Th28:
theorem Th29:
theorem Th30:
theorem Th31:
begin
theorem Th32:
theorem Th33:
theorem
begin
theorem
theorem
:: deftheorem INTEGRA2:def 3 :
canceled;
definition
let A be
closed-interval Subset of
REAL;
let f be
PartFunc of
A,
REAL;
let T be
DivSequence of
A;
func upper_sum (
f,
T)
-> Real_Sequence means
for
i being
Element of
NAT holds
it . i = upper_sum (
f,
(T . i));
existence
ex b1 being Real_Sequence st
for i being Element of NAT holds b1 . i = upper_sum (f,(T . i))
uniqueness
for b1, b2 being Real_Sequence st ( for i being Element of NAT holds b1 . i = upper_sum (f,(T . i)) ) & ( for i being Element of NAT holds b2 . i = upper_sum (f,(T . i)) ) holds
b1 = b2
func lower_sum (
f,
T)
-> Real_Sequence means
for
i being
Element of
NAT holds
it . i = lower_sum (
f,
(T . i));
existence
ex b1 being Real_Sequence st
for i being Element of NAT holds b1 . i = lower_sum (f,(T . i))
uniqueness
for b1, b2 being Real_Sequence st ( for i being Element of NAT holds b1 . i = lower_sum (f,(T . i)) ) & ( for i being Element of NAT holds b2 . i = lower_sum (f,(T . i)) ) holds
b1 = b2
end;
:: deftheorem defines upper_sum INTEGRA2:def 4 :
for A being closed-interval Subset of REAL
for f being PartFunc of A,REAL
for T being DivSequence of A
for b4 being Real_Sequence holds
( b4 = upper_sum (f,T) iff for i being Element of NAT holds b4 . i = upper_sum (f,(T . i)) );
:: deftheorem defines lower_sum INTEGRA2:def 5 :
for A being closed-interval Subset of REAL
for f being PartFunc of A,REAL
for T being DivSequence of A
for b4 being Real_Sequence holds
( b4 = lower_sum (f,T) iff for i being Element of NAT holds b4 . i = lower_sum (f,(T . i)) );
theorem
theorem
canceled;
theorem
canceled;
theorem
theorem
begin
theorem