begin
:: deftheorem Def1 defines complex-valued VALUED_0:def 1 :
for f being Relation holds
( f is complex-valued iff rng f c= COMPLEX );
:: deftheorem Def2 defines ext-real-valued VALUED_0:def 2 :
for f being Relation holds
( f is ext-real-valued iff rng f c= ExtREAL );
:: deftheorem Def3 defines real-valued VALUED_0:def 3 :
for f being Relation holds
( f is real-valued iff rng f c= REAL );
:: deftheorem Def4 defines rational-valued VALUED_0:def 4 :
for f being Relation holds
( f is rational-valued iff rng f c= RAT );
:: deftheorem Def5 defines integer-valued VALUED_0:def 5 :
for f being Relation holds
( f is integer-valued iff rng f c= INT );
:: deftheorem Def6 defines natural-valued VALUED_0:def 6 :
for f being Relation holds
( f is natural-valued iff rng f c= NAT );
theorem Th1:
theorem Th2:
theorem Th3:
theorem Th4:
theorem Th5:
theorem Th6:
:: deftheorem Def7 defines complex-valued VALUED_0:def 7 :
for f being Function holds
( f is complex-valued iff for x being set st x in dom f holds
f . x is complex );
:: deftheorem Def8 defines ext-real-valued VALUED_0:def 8 :
for f being Function holds
( f is ext-real-valued iff for x being set st x in dom f holds
f . x is ext-real );
:: deftheorem Def9 defines real-valued VALUED_0:def 9 :
for f being Function holds
( f is real-valued iff for x being set st x in dom f holds
f . x is real );
:: deftheorem Def10 defines rational-valued VALUED_0:def 10 :
for f being Function holds
( f is rational-valued iff for x being set st x in dom f holds
f . x is rational );
:: deftheorem Def11 defines integer-valued VALUED_0:def 11 :
for f being Function holds
( f is integer-valued iff for x being set st x in dom f holds
f . x is integer );
:: deftheorem Def12 defines natural-valued VALUED_0:def 12 :
for f being Function holds
( f is natural-valued iff for x being set st x in dom f holds
f . x is natural );
theorem Th7:
theorem Th8:
theorem Th9:
theorem Th10:
theorem Th11:
theorem Th12:
theorem
theorem
theorem
theorem
theorem
theorem
begin
:: deftheorem Def13 defines increasing VALUED_0:def 13 :
for f being ext-real-valued Function holds
( f is increasing iff for e1, e2 being ext-real number st e1 in dom f & e2 in dom f & e1 < e2 holds
f . e1 < f . e2 );
:: deftheorem Def14 defines decreasing VALUED_0:def 14 :
for f being ext-real-valued Function holds
( f is decreasing iff for e1, e2 being ext-real number st e1 in dom f & e2 in dom f & e1 < e2 holds
f . e1 > f . e2 );
:: deftheorem Def15 defines non-decreasing VALUED_0:def 15 :
for f being ext-real-valued Function holds
( f is non-decreasing iff for e1, e2 being ext-real number st e1 in dom f & e2 in dom f & e1 <= e2 holds
f . e1 <= f . e2 );
:: deftheorem Def16 defines non-increasing VALUED_0:def 16 :
for f being ext-real-valued Function holds
( f is non-increasing iff for e1, e2 being ext-real number st e1 in dom f & e2 in dom f & e1 <= e2 holds
f . e1 >= f . e2 );
:: deftheorem Def17 defines subsequence VALUED_0:def 17 :
for X being set
for s, b3 being sequence of X holds
( b3 is subsequence of s iff ex N being increasing sequence of NAT st b3 = s * N );
theorem
theorem
theorem Th21:
theorem
:: deftheorem defines constant VALUED_0:def 18 :
for X being non empty set
for s being sequence of X holds
( s is constant iff ex x being Element of X st
for n being Nat holds s . n = x );
theorem Th23:
theorem Th24:
theorem
theorem
theorem Th27:
theorem Th28:
theorem
theorem Th30:
theorem
:: deftheorem defines zeroed VALUED_0:def 19 :
for f being ext-real-valued Function holds
( f is zeroed iff f . {} = 0 );