begin
Lm1:
for t, p, s being real number st 0 < s & t <= p holds
( t < p + s & t - s < p )
theorem Th1:
theorem Th2:
theorem Th3:
theorem Th4:
theorem Th5:
theorem Th6:
theorem Th7:
theorem Th8:
theorem Th9:
:: deftheorem Def1 defines Partial_Intersection PROB_3:def 1 :
for X being set
for A1, b3 being SetSequence of X holds
( b3 = Partial_Intersection A1 iff ( b3 . 0 = A1 . 0 & ( for n being Nat holds b3 . (n + 1) = (b3 . n) /\ (A1 . (n + 1)) ) ) );
:: deftheorem Def2 defines Partial_Union PROB_3:def 2 :
for X being set
for A1, b3 being SetSequence of X holds
( b3 = Partial_Union A1 iff ( b3 . 0 = A1 . 0 & ( for n being Nat holds b3 . (n + 1) = (b3 . n) \/ (A1 . (n + 1)) ) ) );
theorem Th10:
theorem Th11:
theorem Th12:
theorem Th13:
theorem Th14:
theorem Th15:
theorem Th16:
theorem Th17:
theorem Th18:
:: deftheorem Def3 defines Partial_Diff_Union PROB_3:def 3 :
for X being set
for A1, b3 being SetSequence of X holds
( b3 = Partial_Diff_Union A1 iff ( b3 . 0 = A1 . 0 & ( for n being Nat holds b3 . (n + 1) = (A1 . (n + 1)) \ ((Partial_Union A1) . n) ) ) );
theorem Th19:
theorem Th20:
theorem Th21:
theorem Th22:
theorem Th23:
:: deftheorem Def4 defines disjoint_valued PROB_3:def 4 :
for X being set
for A1 being SetSequence of X holds
( A1 is disjoint_valued iff for m, n being Nat st m <> n holds
A1 . m misses A1 . n );
theorem Th24:
:: deftheorem defines @Partial_Intersection PROB_3:def 5 :
for X being set
for Si being SigmaField of X
for XSeq being SetSequence of Si holds @Partial_Intersection XSeq = Partial_Intersection XSeq;
:: deftheorem defines @Partial_Union PROB_3:def 6 :
for X being set
for Si being SigmaField of X
for XSeq being SetSequence of Si holds @Partial_Union XSeq = Partial_Union XSeq;
:: deftheorem defines @Partial_Diff_Union PROB_3:def 7 :
for X being set
for Si being SigmaField of X
for XSeq being SetSequence of Si holds @Partial_Diff_Union XSeq = Partial_Diff_Union XSeq;
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem Th42:
theorem
theorem
theorem Th45:
theorem Th46:
theorem Th47:
theorem Th48:
theorem Th49:
theorem Th50:
theorem Th51:
theorem Th52:
theorem
theorem Th54:
:: deftheorem Def8 defines Complement PROB_3:def 8 :
for X being set
for F1, b3 being FinSequence of bool X holds
( b3 = Complement F1 iff ( len b3 = len F1 & ( for n being Nat st n in dom b3 holds
b3 . n = (F1 . n) ` ) ) );
:: deftheorem Def9 defines Intersection PROB_3:def 9 :
for X being set
for F1 being FinSequence of bool X holds
( ( F1 <> {} implies Intersection F1 = (Union (Complement F1)) ` ) & ( not F1 <> {} implies Intersection F1 = {} ) );
theorem Th55:
theorem Th56:
theorem Th57:
theorem
theorem Th59:
theorem Th60:
:: deftheorem Def10 defines FinSequence PROB_3:def 10 :
for X being set
for Si being SigmaField of X
for b3 being FinSequence of bool X holds
( b3 is FinSequence of Si iff for k being Nat st k in dom b3 holds
b3 . k in Si );
theorem Th61:
theorem Th62:
:: deftheorem defines @Complement PROB_3:def 11 :
for X being set
for S being SigmaField of X
for F being FinSequence of S holds @Complement F = Complement F;
theorem
theorem Th64:
theorem Th65:
theorem Th66:
theorem Th67:
theorem Th68:
theorem Th69:
theorem
:: deftheorem Def12 defines non-decreasing-closed PROB_3:def 12 :
for X being set
for IT being Subset-Family of X holds
( IT is non-decreasing-closed iff for A1 being SetSequence of X st A1 is non-descending & rng A1 c= IT holds
Union A1 in IT );
:: deftheorem Def13 defines non-increasing-closed PROB_3:def 13 :
for X being set
for IT being Subset-Family of X holds
( IT is non-increasing-closed iff for A1 being SetSequence of X st A1 is non-ascending & rng A1 c= IT holds
Intersection A1 in IT );
theorem Th71:
theorem Th72:
theorem Th73:
theorem Th74:
theorem Th75:
theorem
theorem Th77:
:: deftheorem PROB_3:def 14 :
canceled;
:: deftheorem Def15 defines monotoneclass PROB_3:def 15 :
for Omega being non empty set
for X being Subset-Family of Omega
for b3 being MonotoneClass of Omega holds
( b3 = monotoneclass X iff ( X c= b3 & ( for Z being set st X c= Z & Z is MonotoneClass of Omega holds
b3 c= Z ) ) );
theorem Th78:
theorem