definition
let Omega be non
empty set ;
let Sigma be
SigmaField of
Omega;
let P be
Probability of
Sigma;
let X be
Real-Valued-Random-Variable of
Sigma;
assume A1:
(
X is_integrable_on P &
(abs X) to_power 2
is_integrable_on P2M P )
;
correctness
existence
ex b1 being Real ex Y, E being Real-Valued-Random-Variable of Sigma st
( E = Omega --> (expect (X,P)) & Y = X - E & Y is_integrable_on P & (abs Y) to_power 2 is_integrable_on P2M P & b1 = Integral ((P2M P),((abs Y) to_power 2)) );
uniqueness
for b1, b2 being Real st ex Y, E being Real-Valued-Random-Variable of Sigma st
( E = Omega --> (expect (X,P)) & Y = X - E & Y is_integrable_on P & (abs Y) to_power 2 is_integrable_on P2M P & b1 = Integral ((P2M P),((abs Y) to_power 2)) ) & ex Y, E being Real-Valued-Random-Variable of Sigma st
( E = Omega --> (expect (X,P)) & Y = X - E & Y is_integrable_on P & (abs Y) to_power 2 is_integrable_on P2M P & b2 = Integral ((P2M P),((abs Y) to_power 2)) ) holds
b1 = b2;
end;
Lm1:
for Omega1, Omega2 being non empty finite set
for P1 being Probability of Trivial-SigmaField Omega1
for P2 being Probability of Trivial-SigmaField Omega2 ex Q being Function of [:Omega1,Omega2:],REAL st
for x, y being set st x in Omega1 & y in Omega2 holds
Q . (x,y) = (P1 . {x}) * (P2 . {y})
Lm2:
for Omega1, Omega2 being non empty finite set
for P1 being Probability of Trivial-SigmaField Omega1
for P2 being Probability of Trivial-SigmaField Omega2
for Q1, Q2 being Function of [:Omega1,Omega2:],REAL st ( for x, y being set st x in Omega1 & y in Omega2 holds
Q1 . (x,y) = (P1 . {x}) * (P2 . {y}) ) & ( for x, y being set st x in Omega1 & y in Omega2 holds
Q2 . (x,y) = (P1 . {x}) * (P2 . {y}) ) holds
Q1 = Q2
Lm3:
for Omega1, Omega2 being non empty finite set
for P1 being Probability of Trivial-SigmaField Omega1
for P2 being Probability of Trivial-SigmaField Omega2
for Q being Function of [:Omega1,Omega2:],REAL ex P being Function of (bool [:Omega1,Omega2:]),REAL st
for z being finite Subset of [:Omega1,Omega2:] holds P . z = setopfunc (z,[:Omega1,Omega2:],REAL,Q,addreal)
Lm4:
for Omega1, Omega2 being non empty finite set
for P1 being Probability of Trivial-SigmaField Omega1
for P2 being Probability of Trivial-SigmaField Omega2
for Q being Function of [:Omega1,Omega2:],REAL
for P1, P2 being Function of (bool [:Omega1,Omega2:]),REAL st ( for z being finite Subset of [:Omega1,Omega2:] holds P1 . z = setopfunc (z,[:Omega1,Omega2:],REAL,Q,addreal) ) & ( for z being finite Subset of [:Omega1,Omega2:] holds P2 . z = setopfunc (z,[:Omega1,Omega2:],REAL,Q,addreal) ) holds
P1 = P2
Lm5:
for DK, DX being non empty set
for F being Function of DX,DK
for p, q being FinSequence of DX
for fp, fq being FinSequence of DK st fp = F * p & fq = F * q holds
F * (p ^ q) = fp ^ fq
Lm6:
for p being Function st dom p = Seg 1 holds
p = <*(p . 1)*>
theorem Th11:
for
DX1,
DX2 being non
empty set for
F1 being
Function of
DX1,
REAL for
F2 being
Function of
DX2,
REAL for
G being
Function of
[:DX1,DX2:],
REAL for
Y1 being non
empty finite Subset of
DX1 for
p1 being
FinSequence of
DX1 st
p1 is
one-to-one &
rng p1 = Y1 holds
for
p2 being
FinSequence of
DX2 for
p3 being
FinSequence of
[:DX1,DX2:] for
Y2 being non
empty finite Subset of
DX2 for
Y3 being
finite Subset of
[:DX1,DX2:] st
p2 is
one-to-one &
rng p2 = Y2 &
p3 is
one-to-one &
rng p3 = Y3 &
Y3 = [:Y1,Y2:] & ( for
x,
y being
set st
x in Y1 &
y in Y2 holds
G . (
x,
y)
= (F1 . x) * (F2 . y) ) holds
Sum (Func_Seq (G,p3)) = (Sum (Func_Seq (F1,p1))) * (Sum (Func_Seq (F2,p2)))
theorem Th12:
for
DX1,
DX2 being non
empty set for
F1 being
Function of
DX1,
REAL for
F2 being
Function of
DX2,
REAL for
G being
Function of
[:DX1,DX2:],
REAL for
Y1 being non
empty finite Subset of
DX1 for
Y2 being non
empty finite Subset of
DX2 for
Y3 being
finite Subset of
[:DX1,DX2:] st
Y3 = [:Y1,Y2:] & ( for
x,
y being
set st
x in Y1 &
y in Y2 holds
G . (
x,
y)
= (F1 . x) * (F2 . y) ) holds
setopfunc (
Y3,
[:DX1,DX2:],
REAL,
G,
addreal)
= (setopfunc (Y1,DX1,REAL,F1,addreal)) * (setopfunc (Y2,DX2,REAL,F2,addreal))
theorem Th14:
for
DX being non
empty set for
F being
Function of
DX,
REAL for
Y1,
Y2 being
finite Subset of
DX st
Y1 c= Y2 & ( for
x being
set st
x in Y2 holds
0 <= F . x ) holds
setopfunc (
Y1,
DX,
REAL,
F,
addreal)
<= setopfunc (
Y2,
DX,
REAL,
F,
addreal)
reconsider jj = 1 as R_eal by XXREAL_0:def 1;
Lm7:
for Omega1, Omega2 being non empty finite set
for P1 being Probability of Trivial-SigmaField Omega1
for P2 being Probability of Trivial-SigmaField Omega2
for Q being Function of [:Omega1,Omega2:],REAL
for P being Function of (bool [:Omega1,Omega2:]),REAL
for Y1 being non empty finite Subset of Omega1
for Y2 being non empty finite Subset of Omega2 st ( for x, y being set st x in Omega1 & y in Omega2 holds
Q . (x,y) = (P1 . {x}) * (P2 . {y}) ) & ( for z being finite Subset of [:Omega1,Omega2:] holds P . z = setopfunc (z,[:Omega1,Omega2:],REAL,Q,addreal) ) holds
P . [:Y1,Y2:] = (P1 . Y1) * (P2 . Y2)
Lm8:
for Omega1, Omega2 being non empty finite set
for P1 being Probability of Trivial-SigmaField Omega1
for P2 being Probability of Trivial-SigmaField Omega2
for Q being Function of [:Omega1,Omega2:],REAL
for P being Function of (bool [:Omega1,Omega2:]),REAL st ( for x, y being set st x in Omega1 & y in Omega2 holds
Q . (x,y) = (P1 . {x}) * (P2 . {y}) ) & ( for z being finite Subset of [:Omega1,Omega2:] holds P . z = setopfunc (z,[:Omega1,Omega2:],REAL,Q,addreal) ) holds
P . [:Omega1,Omega2:] = 1
Lm9:
for Omega1, Omega2 being non empty finite set
for P1 being Probability of Trivial-SigmaField Omega1
for P2 being Probability of Trivial-SigmaField Omega2
for Q being Function of [:Omega1,Omega2:],REAL
for P being Function of (bool [:Omega1,Omega2:]),REAL st ( for x, y being set st x in Omega1 & y in Omega2 holds
Q . (x,y) = (P1 . {x}) * (P2 . {y}) ) & ( for z being finite Subset of [:Omega1,Omega2:] holds P . z = setopfunc (z,[:Omega1,Omega2:],REAL,Q,addreal) ) holds
for x being set st x c= [:Omega1,Omega2:] holds
( 0 <= P . x & P . x <= 1 )
definition
let Omega1,
Omega2 be non
empty finite set ;
let P1 be
Probability of
Trivial-SigmaField Omega1;
let P2 be
Probability of
Trivial-SigmaField Omega2;
func Product-Probability (
Omega1,
Omega2,
P1,
P2)
-> Probability of
Trivial-SigmaField [:Omega1,Omega2:] means :
Def2:
ex
Q being
Function of
[:Omega1,Omega2:],
REAL st
( ( for
x,
y being
set st
x in Omega1 &
y in Omega2 holds
Q . (
x,
y)
= (P1 . {x}) * (P2 . {y}) ) & ( for
z being
finite Subset of
[:Omega1,Omega2:] holds
it . z = setopfunc (
z,
[:Omega1,Omega2:],
REAL,
Q,
addreal) ) );
existence
ex b1 being Probability of Trivial-SigmaField [:Omega1,Omega2:] ex Q being Function of [:Omega1,Omega2:],REAL st
( ( for x, y being set st x in Omega1 & y in Omega2 holds
Q . (x,y) = (P1 . {x}) * (P2 . {y}) ) & ( for z being finite Subset of [:Omega1,Omega2:] holds b1 . z = setopfunc (z,[:Omega1,Omega2:],REAL,Q,addreal) ) )
uniqueness
for b1, b2 being Probability of Trivial-SigmaField [:Omega1,Omega2:] st ex Q being Function of [:Omega1,Omega2:],REAL st
( ( for x, y being set st x in Omega1 & y in Omega2 holds
Q . (x,y) = (P1 . {x}) * (P2 . {y}) ) & ( for z being finite Subset of [:Omega1,Omega2:] holds b1 . z = setopfunc (z,[:Omega1,Omega2:],REAL,Q,addreal) ) ) & ex Q being Function of [:Omega1,Omega2:],REAL st
( ( for x, y being set st x in Omega1 & y in Omega2 holds
Q . (x,y) = (P1 . {x}) * (P2 . {y}) ) & ( for z being finite Subset of [:Omega1,Omega2:] holds b2 . z = setopfunc (z,[:Omega1,Omega2:],REAL,Q,addreal) ) ) holds
b1 = b2
end;
::
deftheorem Def2 defines
Product-Probability RANDOM_2:def 2 :
for Omega1, Omega2 being non empty finite set
for P1 being Probability of Trivial-SigmaField Omega1
for P2 being Probability of Trivial-SigmaField Omega2
for b5 being Probability of Trivial-SigmaField [:Omega1,Omega2:] holds
( b5 = Product-Probability (Omega1,Omega2,P1,P2) iff ex Q being Function of [:Omega1,Omega2:],REAL st
( ( for x, y being set st x in Omega1 & y in Omega2 holds
Q . (x,y) = (P1 . {x}) * (P2 . {y}) ) & ( for z being finite Subset of [:Omega1,Omega2:] holds b5 . z = setopfunc (z,[:Omega1,Omega2:],REAL,Q,addreal) ) ) );
Lm10:
for Omega being non empty set
for Sigma being SigmaField of Omega holds
( Real-Valued-Random-Variables-Set Sigma is additively-linearly-closed & Real-Valued-Random-Variables-Set Sigma is multiplicatively-closed )
definition
let Omega be non
empty set ;
let Sigma be
SigmaField of
Omega;
func R_Algebra_of_Real-Valued-Random-Variables Sigma -> Algebra equals
AlgebraStr(#
(Real-Valued-Random-Variables-Set Sigma),
(mult_ ((Real-Valued-Random-Variables-Set Sigma),(RAlgebra Omega))),
(Add_ ((Real-Valued-Random-Variables-Set Sigma),(RAlgebra Omega))),
(Mult_ ((Real-Valued-Random-Variables-Set Sigma),(RAlgebra Omega))),
(One_ ((Real-Valued-Random-Variables-Set Sigma),(RAlgebra Omega))),
(Zero_ ((Real-Valued-Random-Variables-Set Sigma),(RAlgebra Omega))) #);
coherence
AlgebraStr(# (Real-Valued-Random-Variables-Set Sigma),(mult_ ((Real-Valued-Random-Variables-Set Sigma),(RAlgebra Omega))),(Add_ ((Real-Valued-Random-Variables-Set Sigma),(RAlgebra Omega))),(Mult_ ((Real-Valued-Random-Variables-Set Sigma),(RAlgebra Omega))),(One_ ((Real-Valued-Random-Variables-Set Sigma),(RAlgebra Omega))),(Zero_ ((Real-Valued-Random-Variables-Set Sigma),(RAlgebra Omega))) #) is Algebra
by C0SP1:6;
end;
::
deftheorem defines
R_Algebra_of_Real-Valued-Random-Variables RANDOM_2:def 4 :
for Omega being non empty set
for Sigma being SigmaField of Omega holds R_Algebra_of_Real-Valued-Random-Variables Sigma = AlgebraStr(# (Real-Valued-Random-Variables-Set Sigma),(mult_ ((Real-Valued-Random-Variables-Set Sigma),(RAlgebra Omega))),(Add_ ((Real-Valued-Random-Variables-Set Sigma),(RAlgebra Omega))),(Mult_ ((Real-Valued-Random-Variables-Set Sigma),(RAlgebra Omega))),(One_ ((Real-Valued-Random-Variables-Set Sigma),(RAlgebra Omega))),(Zero_ ((Real-Valued-Random-Variables-Set Sigma),(RAlgebra Omega))) #);