XX:
for b being Real holds [.b,+infty.] c= ].(b - 1),+infty.]
Lemma2:
for b being Real
for n being Nat st n > 0 holds
[.b,+infty.] c= ].(b - (1 / n)),+infty.]
theorem PP:
for
r being
Real st
r > 0 holds
ex
n being
Nat st
( 1
/ n < r &
n > 0 )
definition
let Omega be non
empty set ;
let Sigma be
SigmaField of
Omega;
let r be
Real;
let I be
TheEvent of
r;
let MyFunc be
Filtration of
I,
Sigma;
let tau be
StoppingTime_Func of
MyFunc;
let A be
SetSequence of
Omega;
let t be
Element of
I;
existence
ex b1 being SetSequence of El_Filtration (t,MyFunc) st
for n being Nat holds b1 . n = Sigma_tauhelp2 (tau,A,n,t)
uniqueness
for b1, b2 being SetSequence of El_Filtration (t,MyFunc) st ( for n being Nat holds b1 . n = Sigma_tauhelp2 (tau,A,n,t) ) & ( for n being Nat holds b2 . n = Sigma_tauhelp2 (tau,A,n,t) ) holds
b1 = b2
end;
definition
let Omega be non
empty set ;
let Sigma be
SigmaField of
Omega;
let S be non
empty Subset of
REAL;
let MyFunc be
Filtration of
S,
Sigma;
let tau be
StoppingTime_Func of
Sigma,
MyFunc;
let A1 be
SetSequence of
Omega;
let t be
Element of
S;
existence
ex b1 being SetSequence of El_Filtration (t,MyFunc) st
for n being Nat holds b1 . n = Sigma_tauhelp2 (MyFunc,tau,A1,n,t)
uniqueness
for b1, b2 being SetSequence of El_Filtration (t,MyFunc) st ( for n being Nat holds b1 . n = Sigma_tauhelp2 (MyFunc,tau,A1,n,t) ) & ( for n being Nat holds b2 . n = Sigma_tauhelp2 (MyFunc,tau,A1,n,t) ) holds
b1 = b2
end;
::
deftheorem Def8868 defines
Sigma_tauhelp3 FINANCE5:def 22 :
for Omega being non empty set
for Sigma being SigmaField of Omega
for S being non empty Subset of REAL
for MyFunc being Filtration of S,Sigma
for tau being StoppingTime_Func of Sigma,MyFunc
for A1 being SetSequence of Omega
for t being Element of S
for b8 being SetSequence of El_Filtration (t,MyFunc) holds
( b8 = Sigma_tauhelp3 (MyFunc,tau,A1,t) iff for n being Nat holds b8 . n = Sigma_tauhelp2 (MyFunc,tau,A1,n,t) );