begin
theorem Th1:
theorem Th2:
:: deftheorem Def1 defines JSum BOR_CANT:def 1 :
for s, b2 being Real_Sequence holds
( b2 = JSum s iff for d being Nat holds b2 . d = Sum ((- (s . d)) rExpSeq) );
theorem Th3:
theorem Th4:
definition
let n1,
n2 be
Element of
NAT ;
func Special_Function (
n1,
n2)
-> sequence of
NAT means :
Def2:
for
n being
Element of
NAT holds
it . n = IFGT (
n,
n1,
(n + n2),
n);
existence
ex b1 being sequence of NAT st
for n being Element of NAT holds b1 . n = IFGT (n,n1,(n + n2),n)
uniqueness
for b1, b2 being sequence of NAT st ( for n being Element of NAT holds b1 . n = IFGT (n,n1,(n + n2),n) ) & ( for n being Element of NAT holds b2 . n = IFGT (n,n1,(n + n2),n) ) holds
b1 = b2
end;
:: deftheorem Def2 defines Special_Function BOR_CANT:def 2 :
for n1, n2 being Element of NAT
for b3 being sequence of NAT holds
( b3 = Special_Function (n1,n2) iff for n being Element of NAT holds b3 . n = IFGT (n,n1,(n + n2),n) );
:: deftheorem Def3 defines Special_Function2 BOR_CANT:def 3 :
for k being Element of NAT
for b2 being sequence of NAT holds
( b2 = Special_Function2 k iff for n being Element of NAT holds b2 . n = n + k );
definition
let k be
Element of
NAT ;
func Special_Function3 k -> sequence of
NAT means :
Def4:
for
n being
Element of
NAT holds
it . n = IFGT (
n,
k,
0,1);
existence
ex b1 being sequence of NAT st
for n being Element of NAT holds b1 . n = IFGT (n,k,0,1)
uniqueness
for b1, b2 being sequence of NAT st ( for n being Element of NAT holds b1 . n = IFGT (n,k,0,1) ) & ( for n being Element of NAT holds b2 . n = IFGT (n,k,0,1) ) holds
b1 = b2
end;
:: deftheorem Def4 defines Special_Function3 BOR_CANT:def 4 :
for k being Element of NAT
for b2 being sequence of NAT holds
( b2 = Special_Function3 k iff for n being Element of NAT holds b2 . n = IFGT (n,k,0,1) );
definition
let n1,
n2 be
Element of
NAT ;
func Special_Function4 (
n1,
n2)
-> sequence of
NAT means :
Def5:
for
n being
Element of
NAT holds
it . n = IFGT (
n,
(n1 + 1),
(n + n2),
n);
existence
ex b1 being sequence of NAT st
for n being Element of NAT holds b1 . n = IFGT (n,(n1 + 1),(n + n2),n)
uniqueness
for b1, b2 being sequence of NAT st ( for n being Element of NAT holds b1 . n = IFGT (n,(n1 + 1),(n + n2),n) ) & ( for n being Element of NAT holds b2 . n = IFGT (n,(n1 + 1),(n + n2),n) ) holds
b1 = b2
end;
:: deftheorem Def5 defines Special_Function4 BOR_CANT:def 5 :
for n1, n2 being Element of NAT
for b3 being sequence of NAT holds
( b3 = Special_Function4 (n1,n2) iff for n being Element of NAT holds b3 . n = IFGT (n,(n1 + 1),(n + n2),n) );
:: deftheorem defines Shift_Seq BOR_CANT:def 6 :
for X being set
for s being Element of NAT
for A being SetSequence of X holds Shift_Seq (A,s) = A ^\ s;
:: deftheorem defines @Shift_Seq BOR_CANT:def 7 :
for Omega being non empty set
for Sigma being SigmaField of Omega
for s being Element of NAT
for A being SetSequence of Sigma holds @Shift_Seq (A,s) = Shift_Seq (A,s);
theorem Th5:
:: deftheorem Def8 defines is_all_independent_wrt BOR_CANT:def 8 :
for Omega being non empty set
for Sigma being SigmaField of Omega
for Prob being Probability of Sigma
for A being SetSequence of Sigma holds
( A is_all_independent_wrt Prob iff for B being SetSequence of Sigma st ex e being sequence of NAT st
( e is one-to-one & ( for n being Element of NAT holds A . (e . n) = B . n ) ) holds
for n being Element of NAT holds (Partial_Product (Prob * B)) . n = Prob . ((@Partial_Intersection B) . n) );
theorem Th6:
theorem Th7:
theorem Th8:
:: deftheorem Def9 defines Union_Shift_Seq BOR_CANT:def 9 :
for X being set
for A, b3 being SetSequence of X holds
( b3 = Union_Shift_Seq A iff for n being Element of NAT holds b3 . n = Union (Shift_Seq (A,n)) );
:: deftheorem defines @Union_Shift_Seq BOR_CANT:def 10 :
for Omega being non empty set
for Sigma being SigmaField of Omega
for A being SetSequence of Sigma holds @Union_Shift_Seq A = Union_Shift_Seq A;
:: deftheorem defines @lim_sup BOR_CANT:def 11 :
for Omega being non empty set
for Sigma being SigmaField of Omega
for A being SetSequence of Sigma holds @lim_sup A = @Intersection (@Union_Shift_Seq A);
:: deftheorem Def12 defines Intersect_Shift_Seq BOR_CANT:def 12 :
for X being set
for A, b3 being SetSequence of X holds
( b3 = Intersect_Shift_Seq A iff for n being Element of NAT holds b3 . n = Intersection (Shift_Seq (A,n)) );
:: deftheorem defines @Intersect_Shift_Seq BOR_CANT:def 13 :
for Omega being non empty set
for Sigma being SigmaField of Omega
for A being SetSequence of Sigma holds @Intersect_Shift_Seq A = Intersect_Shift_Seq A;
:: deftheorem defines @lim_inf BOR_CANT:def 14 :
for Omega being non empty set
for Sigma being SigmaField of Omega
for A being SetSequence of Sigma holds @lim_inf A = Union (@Intersect_Shift_Seq A);
theorem Th9:
theorem Th10:
theorem Th11:
theorem
:: deftheorem Def15 defines Sum_Shift_Seq BOR_CANT:def 15 :
for Omega being non empty set
for Sigma being SigmaField of Omega
for Prob being Probability of Sigma
for A being SetSequence of Sigma
for b5 being Real_Sequence holds
( b5 = Sum_Shift_Seq (Prob,A) iff for n being Element of NAT holds b5 . n = Sum (Prob * (@Shift_Seq (A,n))) );
theorem Th13:
theorem Th14:
theorem Th15:
theorem Th16:
theorem Th17:
theorem
theorem
theorem
theorem