begin
theorem Th1:
theorem
theorem Th3:
theorem
:: deftheorem defines sup RINFSUP2:def 1 :
for seq being ExtREAL_sequence holds sup seq = sup (rng seq);
:: deftheorem defines inf RINFSUP2:def 2 :
for seq being ExtREAL_sequence holds inf seq = inf (rng seq);
:: deftheorem Def3 defines bounded_below RINFSUP2:def 3 :
for seq being ExtREAL_sequence holds
( seq is bounded_below iff rng seq is bounded_below );
:: deftheorem Def4 defines bounded_above RINFSUP2:def 4 :
for seq being ExtREAL_sequence holds
( seq is bounded_above iff rng seq is bounded_above );
:: deftheorem Def5 defines bounded RINFSUP2:def 5 :
for seq being ExtREAL_sequence holds
( seq is bounded iff ( seq is bounded_above & seq is bounded_below ) );
theorem Th5:
:: deftheorem Def6 defines inferior_realsequence RINFSUP2:def 6 :
for seq, b2 being ExtREAL_sequence holds
( b2 = inferior_realsequence seq iff for n being Element of NAT ex Y being non empty Subset of ExtREAL st
( Y = { (seq . k) where k is Element of NAT : n <= k } & b2 . n = inf Y ) );
:: deftheorem Def7 defines superior_realsequence RINFSUP2:def 7 :
for seq, b2 being ExtREAL_sequence holds
( b2 = superior_realsequence seq iff for n being Element of NAT ex Y being non empty Subset of ExtREAL st
( Y = { (seq . k) where k is Element of NAT : n <= k } & b2 . n = sup Y ) );
theorem
theorem Th7:
theorem Th8:
Lm1:
for seq being ExtREAL_sequence holds superior_realsequence seq is non-increasing
Lm2:
for seq being ExtREAL_sequence holds inferior_realsequence seq is non-decreasing
:: deftheorem RINFSUP2:def 8 :
canceled;
:: deftheorem RINFSUP2:def 9 :
canceled;
:: deftheorem RINFSUP2:def 10 :
canceled;
:: deftheorem RINFSUP2:def 11 :
canceled;
:: deftheorem defines lim_sup RINFSUP2:def 12 :
for seq being ExtREAL_sequence holds lim_sup seq = inf (superior_realsequence seq);
:: deftheorem defines lim_inf RINFSUP2:def 13 :
for seq being ExtREAL_sequence holds lim_inf seq = sup (inferior_realsequence seq);
theorem Th9:
theorem Th10:
theorem Th11:
theorem Th12:
theorem Th13:
theorem Th14:
theorem Th15:
theorem Th16:
theorem Th17:
theorem Th18:
theorem Th19:
theorem Th20:
theorem
theorem
theorem Th23:
theorem Th24:
theorem Th25:
theorem Th26:
theorem
theorem Th28:
theorem Th29:
theorem Th30:
theorem Th31:
Lm3:
for seq being ExtREAL_sequence st seq is bounded & seq is non-increasing holds
( seq is convergent_to_finite_number & seq is convergent & lim seq = inf seq )
Lm4:
for seq being ExtREAL_sequence st seq is bounded & seq is non-decreasing holds
( seq is convergent_to_finite_number & seq is convergent & lim seq = sup seq )
theorem Th32:
theorem Th33:
theorem Th34:
theorem Th35:
theorem Th36:
theorem Th37:
theorem Th38:
theorem
Lm5:
for seq being ExtREAL_sequence st lim_inf seq = lim_sup seq & lim_inf seq = +infty holds
( seq is convergent & lim seq = lim_inf seq & lim seq = lim_sup seq )
Lm6:
for seq being ExtREAL_sequence st lim_inf seq = lim_sup seq & lim_inf seq = -infty holds
( seq is convergent & lim seq = lim_inf seq & lim seq = lim_sup seq )
Lm7:
for seq being ExtREAL_sequence st lim_inf seq = lim_sup seq & lim_inf seq in REAL holds
( seq is convergent & lim seq = lim_inf seq & lim seq = lim_sup seq )
theorem Th40:
theorem