Lemacik:
for a, b, c being set st ( a = 1 or a = 2 or a = 3 or a = 4 ) & ( b = 1 or b = 2 or b = 3 or b = 4 ) & ( c = 1 or c = 2 or c = 3 or c = 4 ) holds
{a,b,c} c= {1,2,3,4}
Lemacik2:
for a, b being set st ( a = 1 or a = 2 or a = 3 or a = 4 ) & ( b = 1 or b = 2 or b = 3 or b = 4 ) holds
{a,b} c= {1,2,3,4}
Lemacik3:
for a being set st ( a = 1 or a = 2 or a = 3 or a = 4 ) holds
{a} c= {1,2,3,4}
The1:
for A1 being SetSequence of {1,2,3,4} st ex n being Nat st A1 . n = {} holds
Intersection A1 = {}
EnLm1:
{1} c= {1,2,3,4}
by Lemacik3;
EnLm2:
{2} c= {1,2,3,4}
by Lemacik3;
EnLm3:
{3} c= {1,2,3,4}
by Lemacik3;
EnLm4:
{4} c= {1,2,3,4}
by Lemacik3;
Lm1:
{3,4} c= {1,2,3,4}
by Lemacik2;
Lm2:
{1,2} c= {1,2,3,4}
by Lemacik2;
Lm3:
{1,2} /\ {3,4} = {}
Lem1:
{1,2,3,4} \ {1,2} = {3,4}
Lem2:
{1,2,3,4} \ {3,4} = {1,2}
B13:
{1,3} in bool {1,2,3,4}
B14:
{1,4} in bool {1,2,3,4}
B124:
{1,2,4} in bool {1,2,3,4}
B134:
{1,3,4} in bool {1,2,3,4}
B234:
{2,3,4} in bool {1,2,3,4}
B123:
{1,2,3} in bool {1,2,3,4}
B23:
{2,3} in bool {1,2,3,4}
B24:
{2,4} in bool {1,2,3,4}
B25:
{1,2} in bool {1,2,3,4}
B26:
{3,4} in bool {1,2,3,4}
WW1:
{1,2,3} <> {3,4}
The0:
{{},{1,2},{3,4},{1,2,3,4}} <> bool {1,2,3,4}
set Omega3 = {1,2,3};
set Omega4 = {1,2,3,4};
ATh102:
{1,2,3} c< {1,2,3,4}
set Omega2 = {1,2};
ATh101:
{1,2} c< {1,2,3}
definition
let Omega be non
empty set ;
let F be
SigmaField of
Omega;
let X be non
empty set ;
let G be
sequence of
X;
let phi be
Real_Sequence;
let d be
Nat;
existence
ex b1 being Function of Omega,REAL st
for w being Element of Omega holds b1 . w = PortfolioValueFutExt (d,phi,F,G,w)
uniqueness
for b1, b2 being Function of Omega,REAL st ( for w being Element of Omega holds b1 . w = PortfolioValueFutExt (d,phi,F,G,w) ) & ( for w being Element of Omega holds b2 . w = PortfolioValueFutExt (d,phi,F,G,w) ) holds
b1 = b2
end;
definition
let d be
Nat;
let phi be
Real_Sequence;
let Omega be non
empty set ;
let F be
SigmaField of
Omega;
let X be non
empty set ;
let G be
sequence of
X;
let w be
Element of
Omega;
correctness
coherence
PortfolioValueFut (d,phi,F,G,w) is Real;
compatibility
for b1 being Real holds
( b1 = PortfolioValueFut (d,phi,F,G,w) iff b1 = (Partial_Sums ((RVPortfolioValueFutExt_El (phi,F,G,w)) ^\ 1)) . (d - 1) );
end;
definition
let Omega be non
empty set ;
let F be
SigmaField of
Omega;
let X be non
empty set ;
let G be
sequence of
X;
let phi be
Real_Sequence;
let d be
Nat;
existence
ex b1 being Function of Omega,REAL st
for w being Element of Omega holds b1 . w = PortfolioValueFut ((d + 1),phi,F,G,w)
uniqueness
for b1, b2 being Function of Omega,REAL st ( for w being Element of Omega holds b1 . w = PortfolioValueFut ((d + 1),phi,F,G,w) ) & ( for w being Element of Omega holds b2 . w = PortfolioValueFut ((d + 1),phi,F,G,w) ) holds
b1 = b2
end;
theorem
for
d being
Nat for
phi being
Real_Sequence for
Omega being non
empty set for
F being
SigmaField of
Omega for
X being non
empty set for
G being
sequence of
X for
w being
Element of
Omega holds
(
PortfolioValueFut (
(d + 1),
phi,
F,
G,
w)
= (RVPortfolioValueFut (phi,F,G,d)) . w &
{(PortfolioValueFut ((d + 1),phi,F,G,w))} is
Event of
Borel_Sets )
by Def4, FINANCE2:5;
Lm1B:
for Omega, Omega2 being non empty set
for F being Function of Omega,Omega2
for y being non empty set holds { z where z is Element of Omega : F . z is Element of y } = F " y
theorem
for
MySigmaField,
A1,
A2 being
set st
MySigmaField = {{},{1,2,3,4}} &
A1 in MySigmaField &
A2 in MySigmaField holds
A1 /\ A2 in MySigmaField
theorem Lm700000:
for
A1 being
SetSequence of
{1,2,3,4} st ( for
n,
k being
Nat holds not
(A1 . n) /\ (A1 . k) = {} ) &
rng A1 c= {{},{1,2},{3,4},{1,2,3,4}} & not
Intersection A1 = {} & not
Intersection A1 = {1,2} & not
Intersection A1 = {3,4} holds
Intersection A1 = {1,2,3,4}
theorem
for
A1 being
SetSequence of
{1,2,3,4} for
MyOmega being
set st
MyOmega = {{},{1,2},{3,4},{1,2,3,4}} &
Intersection A1 = {1,2,3,4} holds
Intersection A1 in MyOmega by ENUMSET1:def 2;
theorem
for
A1 being
SetSequence of
{1,2,3,4} for
MyOmega being
set st
MyOmega = {{},{1,2},{3,4},{1,2,3,4}} &
Intersection A1 = {3,4} holds
Intersection A1 in MyOmega by ENUMSET1:def 2;
theorem
for
A1 being
SetSequence of
{1,2,3,4} for
MyOmega being
set st
MyOmega = {{},{1,2},{3,4},{1,2,3,4}} &
Intersection A1 = {1,2} holds
Intersection A1 in MyOmega by ENUMSET1:def 2;
theorem
for
A1 being
SetSequence of
{1,2,3,4} for
MyOmega being
set st
MyOmega = {{},{1,2},{3,4},{1,2,3,4}} &
Intersection A1 = {} holds
Intersection A1 in MyOmega by ENUMSET1:def 2;
theorem Lm8:
for
MyOmega being
set for
A1 being
SetSequence of
{1,2,3,4} st
rng A1 c= MyOmega &
MyOmega = {{},{1,2},{3,4},{1,2,3,4}} holds
Intersection A1 in MyOmega
theorem
for
MySigmaField,
MySet being
set for
A1 being
SetSequence of
MySet st
MySet = {1,2,3,4} &
rng A1 c= MySigmaField &
MySigmaField = {{},{1,2,3,4}} holds
for
k1,
k2 being
Nat holds
(A1 . k1) /\ (A1 . k2) in MySigmaField
definition
func Special_SigmaField2 -> SigmaField of
{1,2,3,4} equals
{{},{1,2},{3,4},{1,2,3,4}};
correctness
coherence
{{},{1,2},{3,4},{1,2,3,4}} is SigmaField of {1,2,3,4};
end;
theorem
for
Omega being
set st
Omega = {1,2,3,4} holds
(
Omega in Special_SigmaField1 &
{} in Special_SigmaField1 &
{1,2} in Special_SigmaField2 &
{3,4} in Special_SigmaField2 &
Omega in Special_SigmaField2 &
{} in Special_SigmaField2 &
Omega in Trivial-SigmaField {1,2,3,4} &
{} in Trivial-SigmaField {1,2,3,4} &
{1} in Trivial-SigmaField {1,2,3,4} &
{2} in Trivial-SigmaField {1,2,3,4} &
{3} in Trivial-SigmaField {1,2,3,4} &
{4} in Trivial-SigmaField {1,2,3,4} )
by EnLm1, EnLm2, EnLm3, PROB_1:5, EnLm4, PROB_1:4, ENUMSET1:def 2;
XX1:
{{},{1,2,3,4}} c< {{},{1,2},{3,4},{1,2,3,4}}
XX2:
{{},{1,2},{3,4},{1,2,3,4}} c< bool {1,2,3,4}
definition
let k be
Element of
{1,2,3};
correctness
coherence
( ( k = 1 implies Special_SigmaField1 is Subset of (bool {1,2,3,4}) ) & ( not k = 1 implies Special_SigmaField2 is Subset of (bool {1,2,3,4}) ) );
consistency
for b1 being Subset of (bool {1,2,3,4}) holds verum;
;
end;
definition
let k be
Element of
{1,2,3};
correctness
coherence
( ( k <= 2 implies Set1_of_SigmaField3 k is Subset of (bool {1,2,3,4}) ) & ( not k <= 2 implies Trivial-SigmaField {1,2,3,4} is Subset of (bool {1,2,3,4}) ) );
consistency
for b1 being Subset of (bool {1,2,3,4}) holds verum;
;
end;
Th3:
for Sigma being SigmaField of {1,2,3,4}
for I being set st I = {1,2,3} & Sigma = bool {1,2,3,4} holds
ex MyFunc being ManySortedSigmaField of I,Sigma st
( MyFunc . 1 = Special_SigmaField1 & MyFunc . 2 = Special_SigmaField2 & MyFunc . 3 = Trivial-SigmaField {1,2,3,4} )
theorem MyNeed:
for
Omega being non
empty set for
Sigma being
SigmaField of
Omega for
I being non
empty real-membered set st
I = {1,2,3} &
Sigma = bool {1,2,3,4} &
Omega = {1,2,3,4} holds
ex
MyFunc being
Filtration of
I,
Sigma st
(
MyFunc . 1
= Special_SigmaField1 &
MyFunc . 2
= Special_SigmaField2 &
MyFunc . 3
= Trivial-SigmaField {1,2,3,4} )
Lm1A:
for Omega, Omega2 being non empty set
for F being Function of Omega,Omega2
for y being non empty set holds { z where z is Element of Omega : F . z is Element of y } = F " y
Lm2A:
for Omega being non empty set
for Sigma4 being SigmaField of Omega
for Sigma5 being SigmaField of {1} holds Omega --> 1 is random_variable of Sigma4,Sigma5
theorem THJ1:
for
Omega being non
empty set for
Sigma being
SigmaField of
Omega for
Sigma2 being
SigmaField of
{1} st
Omega = {1,2,3,4} holds
ex
X1 being
Function of
Omega,
{1} st
(
X1 is
random_variable of
Special_SigmaField1 ,
Sigma2 &
X1 is
random_variable of
Special_SigmaField2 ,
Sigma2 &
X1 is
random_variable of
Trivial-SigmaField {1,2,3,4},
Sigma2 )
theorem
for
Omega being non
empty set for
Sigma,
Sigma2 being
SigmaField of
Omega st
Sigma2 c= Sigma holds
for
E2 being
Event of
Sigma2 holds
E2 is
Event of
Sigma ;
definition
let Omega,
Omega2 be non
empty set ;
let Sigma be
SigmaField of
Omega;
let Sigma2 be
SigmaField of
Omega2;
let I,
J be non
empty Subset of
NAT;
let Stoch be
Stochastic_Process of
In (
J,
(bool REAL)),
Sigma,
Sigma2;
mode Predictable_Stochastic_Process of
I,
J,
Sigma,
Sigma2,
Stoch -> Function of
J,
(set_of_random_variables_on (Sigma,Sigma2)) means
ex
k being
Filtration of
In (
I,
(bool REAL)),
Sigma st
for
j being
Element of
In (
J,
(bool REAL))
for
i being
Element of
In (
I,
(bool REAL)) st
j - 1
= i holds
RVProcess (
Stoch,
j) is
El_Filtration (
i,
k),
Sigma2 -random_variable-like ;
existence
ex b1 being Function of J,(set_of_random_variables_on (Sigma,Sigma2)) ex k being Filtration of In (I,(bool REAL)),Sigma st
for j being Element of In (J,(bool REAL))
for i being Element of In (I,(bool REAL)) st j - 1 = i holds
RVProcess (Stoch,j) is El_Filtration (i,k),Sigma2 -random_variable-like
end;
::
deftheorem defines
Predictable_Stochastic_Process FINANCE3:def 16 :
for Omega, Omega2 being non empty set
for Sigma being SigmaField of Omega
for Sigma2 being SigmaField of Omega2
for I, J being non empty Subset of NAT
for Stoch being Stochastic_Process of In (J,(bool REAL)),Sigma,Sigma2
for b8 being Function of J,(set_of_random_variables_on (Sigma,Sigma2)) holds
( b8 is Predictable_Stochastic_Process of I,J,Sigma,Sigma2,Stoch iff ex k being Filtration of In (I,(bool REAL)),Sigma st
for j being Element of In (J,(bool REAL))
for i being Element of In (I,(bool REAL)) st j - 1 = i holds
RVProcess (Stoch,j) is El_Filtration (i,k),Sigma2 -random_variable-like );
::
deftheorem Def78 defines
Set3_for_RandomVariable FINANCE3:def 20 :
for k2, k3, k4 being Element of REAL
for Omega being non empty set
for k being Element of Omega holds
( ( k = 2 implies Set3_for_RandomVariable (k2,k3,k4,k) = k2 ) & ( not k = 2 implies Set3_for_RandomVariable (k2,k3,k4,k) = Set4_for_RandomVariable (k3,k4,k) ) );
::
deftheorem Def77 defines
Set2_for_RandomVariable FINANCE3:def 21 :
for k1, k2, k3, k4 being Element of REAL
for Omega being non empty set
for k being Element of Omega holds
( ( k = 1 implies Set2_for_RandomVariable (k1,k2,k3,k4,k) = k1 ) & ( not k = 1 implies Set2_for_RandomVariable (k1,k2,k3,k4,k) = Set3_for_RandomVariable (k2,k3,k4,k) ) );
theorem MyFunc5:
for
k1,
k2,
k3,
k4 being
Element of
REAL for
Omega being non
empty set st
Omega = {1,2,3,4} holds
for
Sigma being
SigmaField of
Omega for
I being non
empty real-membered set for
MyFunc being
ManySortedSigmaField of
I,
Sigma st
MyFunc . 1
= Special_SigmaField1 &
MyFunc . 2
= Special_SigmaField2 &
MyFunc . 3
= Trivial-SigmaField {1,2,3,4} holds
for
eli being
Element of
I st
eli = 3 holds
ex
f being
Function of
Omega,
REAL st
(
f . 1
= k1 &
f . 2
= k2 &
f . 3
= k3 &
f . 4
= k4 &
f is
El_Filtration (
eli,
MyFunc),
Borel_Sets -random_variable-like )
theorem MyFunc6:
for
k1,
k2 being
Element of
REAL for
Omega being non
empty set st
Omega = {1,2,3,4} holds
for
Sigma being
SigmaField of
Omega for
I being non
empty real-membered set for
MyFunc being
ManySortedSigmaField of
I,
Sigma st
MyFunc . 1
= Special_SigmaField1 &
MyFunc . 2
= Special_SigmaField2 &
MyFunc . 3
= Trivial-SigmaField {1,2,3,4} holds
for
eli being
Element of
I st
eli = 2 holds
ex
f being
Function of
Omega,
REAL st
(
f . 1
= k1 &
f . 2
= k1 &
f . 3
= k2 &
f . 4
= k2 &
f is
El_Filtration (
eli,
MyFunc),
Borel_Sets -random_variable-like )
theorem MyFunc7:
for
k1 being
Element of
REAL for
Omega being non
empty set st
Omega = {1,2,3,4} holds
for
Sigma being
SigmaField of
Omega for
I being non
empty real-membered set for
MyFunc being
ManySortedSigmaField of
I,
Sigma st
MyFunc . 1
= Special_SigmaField1 &
MyFunc . 2
= Special_SigmaField2 &
MyFunc . 3
= Trivial-SigmaField {1,2,3,4} holds
for
eli being
Element of
I st
eli = 1 holds
ex
f being
Function of
Omega,
REAL st
(
f . 1
= k1 &
f . 2
= k1 &
f . 3
= k1 &
f . 4
= k1 &
f is
El_Filtration (
eli,
MyFunc),
Borel_Sets -random_variable-like )
theorem
for
Omega being non
empty set st
Omega = {1,2,3,4} holds
for
Sigma being
SigmaField of
Omega for
I being non
empty real-membered set st
I = {1,2,3} &
Sigma = bool {1,2,3,4} holds
for
MyFunc being
ManySortedSigmaField of
I,
Sigma st
MyFunc . 1
= Special_SigmaField1 &
MyFunc . 2
= Special_SigmaField2 &
MyFunc . 3
= Trivial-SigmaField {1,2,3,4} holds
for
Prob being
Function of
Sigma,
REAL for
i being
Element of
I ex
RV being
Function of
Omega,
REAL st
RV is
El_Filtration (
i,
MyFunc),
Borel_Sets -random_variable-like
definition
let I be non
empty real-membered set ;
assume A0000:
I = {1,2,3}
;
let i be
Element of
I;
assume MyI:
(
i = 2 or
i = 3 )
;
let Omega be non
empty set ;
assume A000:
Omega = {1,2,3,4}
;
let Sigma be
SigmaField of
Omega;
assume A00:
Sigma = bool Omega
;
let f1 be
Function of
Omega,
REAL;
assume A0:
(
f1 . 1
= 60 &
f1 . 2
= 80 &
f1 . 3
= 100 &
f1 . 4
= 120 )
;
let f2 be
Function of
Omega,
REAL;
assume A1:
(
f2 . 1
= 80 &
f2 . 2
= 80 &
f2 . 3
= 120 &
f2 . 4
= 120 )
;
let f3 be
Function of
Omega,
REAL;
correctness
coherence
( ( i = 2 implies f2 is Element of set_of_random_variables_on (Sigma,Borel_Sets) ) & ( not i = 2 implies f1 is Element of set_of_random_variables_on (Sigma,Borel_Sets) ) );
consistency
for b1 being Element of set_of_random_variables_on (Sigma,Borel_Sets) holds verum;
end;
::
deftheorem Def1211 defines
FunctionRV1 FINANCE3:def 22 :
for I being non empty real-membered set st I = {1,2,3} holds
for i being Element of I st ( i = 2 or i = 3 ) holds
for Omega being non empty set st Omega = {1,2,3,4} holds
for Sigma being SigmaField of Omega st Sigma = bool Omega holds
for f1 being Function of Omega,REAL st f1 . 1 = 60 & f1 . 2 = 80 & f1 . 3 = 100 & f1 . 4 = 120 holds
for f2 being Function of Omega,REAL st f2 . 1 = 80 & f2 . 2 = 80 & f2 . 3 = 120 & f2 . 4 = 120 holds
for f3 being Function of Omega,REAL holds
( ( i = 2 implies FunctionRV1 (i,Sigma,f1,f2,f3) = f2 ) & ( not i = 2 implies FunctionRV1 (i,Sigma,f1,f2,f3) = f1 ) );
definition
let I be non
empty real-membered set ;
assume A0000:
I = {1,2,3}
;
let i be
Element of
I;
let Omega be non
empty set ;
assume A000:
Omega = {1,2,3,4}
;
let Sigma be
SigmaField of
Omega;
assume A00:
Sigma = bool Omega
;
let f1,
f2 be
Function of
Omega,
REAL;
let f3 be
Function of
Omega,
REAL;
assume A2:
(
f3 . 1
= 100 &
f3 . 2
= 100 &
f3 . 3
= 100 &
f3 . 4
= 100 )
;
correctness
coherence
( ( ( i = 2 or i = 3 ) implies FunctionRV1 (i,Sigma,f1,f2,f3) is Element of set_of_random_variables_on (Sigma,Borel_Sets) ) & ( i = 2 or i = 3 or f3 is Element of set_of_random_variables_on (Sigma,Borel_Sets) ) );
consistency
for b1 being Element of set_of_random_variables_on (Sigma,Borel_Sets) holds verum;
end;
::
deftheorem Def1212 defines
FunctionRV2 FINANCE3:def 23 :
for I being non empty real-membered set st I = {1,2,3} holds
for i being Element of I
for Omega being non empty set st Omega = {1,2,3,4} holds
for Sigma being SigmaField of Omega st Sigma = bool Omega holds
for f1, f2, f3 being Function of Omega,REAL st f3 . 1 = 100 & f3 . 2 = 100 & f3 . 3 = 100 & f3 . 4 = 100 holds
( ( ( i = 2 or i = 3 ) implies FunctionRV2 (i,Sigma,f1,f2,f3) = FunctionRV1 (i,Sigma,f1,f2,f3) ) & ( i = 2 or i = 3 or FunctionRV2 (i,Sigma,f1,f2,f3) = f3 ) );
theorem
for
Omega,
Omega2 being non
empty set st
Omega = {1,2,3,4} holds
for
Sigma being
SigmaField of
Omega for
I being non
empty real-membered set st
I = {1,2,3} &
Sigma = bool {1,2,3,4} holds
for
MyFunc being
Filtration of
I,
Sigma st
MyFunc . 1
= Special_SigmaField1 &
MyFunc . 2
= Special_SigmaField2 &
MyFunc . 3
= Trivial-SigmaField {1,2,3,4} holds
ex
Stoch being
Stochastic_Process of
I,
Sigma,
Borel_Sets st
( ( for
k being
Element of
I holds
( ex
RV being
Function of
Omega,
REAL st
(
Stoch . k = RV &
RV is
Sigma,
Borel_Sets -random_variable-like &
RV is
El_Filtration (
k,
MyFunc),
Borel_Sets -random_variable-like ) & ex
f being
Function of
Omega,
REAL st
(
k = 1 implies (
f . 1
= 100 &
f . 2
= 100 &
f . 3
= 100 &
f . 4
= 100 &
Stoch . k = f ) ) & ex
f being
Function of
Omega,
REAL st
(
k = 2 implies (
f . 1
= 80 &
f . 2
= 80 &
f . 3
= 120 &
f . 4
= 120 &
Stoch . k = f ) ) & ex
f being
Function of
Omega,
REAL st
(
k = 3 implies (
f . 1
= 60 &
f . 2
= 80 &
f . 3
= 100 &
f . 4
= 120 &
Stoch . k = f ) ) &
Stoch is
MyFunc -stoch_proc_wrt_to_Filtration ) ) &
Stoch is
Adapted_Stochastic_Process of
Stoch )