begin
Lm1:
for D1, D2 being set
for f being Function holds
( f is Functional_Sequence of D1,D2 iff ( dom f = NAT & ( for x being set st x in NAT holds
f . x is PartFunc of D1,D2 ) ) )
theorem
:: deftheorem SEQFUNC:def 1 :
canceled;
:: deftheorem Def2 defines (#) SEQFUNC:def 2 :
for D being non empty set
for H being Functional_Sequence of D,REAL
for r being real number
for b4 being Functional_Sequence of D,REAL holds
( b4 = r (#) H iff for n being Nat holds b4 . n = r (#) (H . n) );
definition
let D be non
empty set ;
let H be
Functional_Sequence of
D,
REAL;
func H " -> Functional_Sequence of
D,
REAL means :
Def3:
for
n being
Nat holds
it . n = (H . n) ^ ;
existence
ex b1 being Functional_Sequence of D,REAL st
for n being Nat holds b1 . n = (H . n) ^
uniqueness
for b1, b2 being Functional_Sequence of D,REAL st ( for n being Nat holds b1 . n = (H . n) ^ ) & ( for n being Nat holds b2 . n = (H . n) ^ ) holds
b1 = b2
func - H -> Functional_Sequence of
D,
REAL means :
Def4:
for
n being
Nat holds
it . n = - (H . n);
existence
ex b1 being Functional_Sequence of D,REAL st
for n being Nat holds b1 . n = - (H . n)
uniqueness
for b1, b2 being Functional_Sequence of D,REAL st ( for n being Nat holds b1 . n = - (H . n) ) & ( for n being Nat holds b2 . n = - (H . n) ) holds
b1 = b2
func abs H -> Functional_Sequence of
D,
REAL means :
Def5:
for
n being
Nat holds
it . n = abs (H . n);
existence
ex b1 being Functional_Sequence of D,REAL st
for n being Nat holds b1 . n = abs (H . n)
uniqueness
for b1, b2 being Functional_Sequence of D,REAL st ( for n being Nat holds b1 . n = abs (H . n) ) & ( for n being Nat holds b2 . n = abs (H . n) ) holds
b1 = b2
end;
:: deftheorem Def3 defines " SEQFUNC:def 3 :
for D being non empty set
for H, b3 being Functional_Sequence of D,REAL holds
( b3 = H " iff for n being Nat holds b3 . n = (H . n) ^ );
:: deftheorem Def4 defines - SEQFUNC:def 4 :
for D being non empty set
for H, b3 being Functional_Sequence of D,REAL holds
( b3 = - H iff for n being Nat holds b3 . n = - (H . n) );
:: deftheorem Def5 defines abs SEQFUNC:def 5 :
for D being non empty set
for H, b3 being Functional_Sequence of D,REAL holds
( b3 = abs H iff for n being Nat holds b3 . n = abs (H . n) );
:: deftheorem Def6 defines + SEQFUNC:def 6 :
for D being non empty set
for G, H, b4 being Functional_Sequence of D,REAL holds
( b4 = G + H iff for n being Nat holds b4 . n = (G . n) + (H . n) );
:: deftheorem defines - SEQFUNC:def 7 :
for D being non empty set
for G, H being Functional_Sequence of D,REAL holds G - H = G + (- H);
:: deftheorem Def8 defines (#) SEQFUNC:def 8 :
for D being non empty set
for G, H, b4 being Functional_Sequence of D,REAL holds
( b4 = G (#) H iff for n being Nat holds b4 . n = (G . n) (#) (H . n) );
:: deftheorem defines / SEQFUNC:def 9 :
for D being non empty set
for H, G being Functional_Sequence of D,REAL holds G / H = G (#) (H ");
theorem
canceled;
theorem
theorem Th4:
theorem
theorem Th6:
theorem
theorem Th8:
theorem
theorem
theorem Th11:
theorem Th12:
theorem
theorem
theorem
theorem Th16:
theorem Th17:
theorem
theorem
:: deftheorem Def10 defines common_on_dom SEQFUNC:def 10 :
for D1, D2 being set
for F being Functional_Sequence of D1,D2
for X being set holds
( X common_on_dom F iff ( X <> {} & ( for n being Element of NAT holds X c= dom (F . n) ) ) );
:: deftheorem Def11 defines # SEQFUNC:def 11 :
for D being non empty set
for H being Functional_Sequence of D,REAL
for x being Element of D
for b4 being Real_Sequence holds
( b4 = H # x iff for n being Element of NAT holds b4 . n = (H . n) . x );
:: deftheorem Def12 defines is_point_conv_on SEQFUNC:def 12 :
for D being non empty set
for H being Functional_Sequence of D,REAL
for X being set holds
( H is_point_conv_on X iff ( X common_on_dom H & ex f being PartFunc of D,REAL st
( X = dom f & ( for x being Element of D st x in X holds
for p being Real st p > 0 holds
ex k being Element of NAT st
for n being Element of NAT st n >= k holds
abs (((H . n) . x) - (f . x)) < p ) ) ) );
theorem Th20:
theorem Th21:
:: deftheorem Def13 defines is_unif_conv_on SEQFUNC:def 13 :
for D being non empty set
for H being Functional_Sequence of D,REAL
for X being set holds
( H is_unif_conv_on X iff ( X common_on_dom H & ex f being PartFunc of D,REAL st
( X = dom f & ( for p being Real st p > 0 holds
ex k being Element of NAT st
for n being Element of NAT
for x being Element of D st n >= k & x in X holds
abs (((H . n) . x) - (f . x)) < p ) ) ) );
:: deftheorem Def14 defines lim SEQFUNC:def 14 :
for D being non empty set
for H being Functional_Sequence of D,REAL
for X being set st H is_point_conv_on X holds
for b4 being PartFunc of D,REAL holds
( b4 = lim (H,X) iff ( dom b4 = X & ( for x being Element of D st x in dom b4 holds
b4 . x = lim (H # x) ) ) );
theorem Th22:
theorem Th23:
theorem Th24:
theorem
theorem
theorem Th27:
theorem
theorem Th29:
theorem Th30:
theorem Th31:
theorem Th32:
theorem Th33:
theorem Th34:
theorem Th35:
theorem
theorem
theorem Th38:
theorem Th39:
theorem Th40:
theorem
for
D being non
empty set for
H1,
H2 being
Functional_Sequence of
D,
REAL for
X being
set st
H1 is_point_conv_on X &
H2 is_point_conv_on X holds
(
H1 + H2 is_point_conv_on X &
lim (
(H1 + H2),
X)
= (lim (H1,X)) + (lim (H2,X)) &
H1 - H2 is_point_conv_on X &
lim (
(H1 - H2),
X)
= (lim (H1,X)) - (lim (H2,X)) &
H1 (#) H2 is_point_conv_on X &
lim (
(H1 (#) H2),
X)
= (lim (H1,X)) (#) (lim (H2,X)) )
theorem
theorem
theorem Th44:
theorem