begin
:: deftheorem defines Inter INTERVA1:def 1 :
for U being set
for X, Y being Subset of U holds Inter (X,Y) = { A where A is Subset of U : ( X c= A & A c= Y ) } ;
theorem Th1:
theorem Th2:
theorem Th3:
theorem
theorem Th5:
theorem Th6:
theorem Th7:
theorem Th8:
:: deftheorem Def2 defines IntervalSet INTERVA1:def 2 :
for U being set
for b2 being Subset-Family of U holds
( b2 is IntervalSet of U iff ex A, B being Subset of U st b2 = Inter (A,B) );
theorem
theorem Th10:
theorem Th11:
theorem Th12:
theorem Th13:
:: deftheorem defines _/\_ INTERVA1:def 3 :
for U being non empty set
for A, B being non empty IntervalSet of U holds A _/\_ B = INTERSECTION (A,B);
:: deftheorem defines _\/_ INTERVA1:def 4 :
for U being non empty set
for A, B being non empty IntervalSet of U holds A _\/_ B = UNION (A,B);
definition
let U be non
empty set ;
let A be non
empty IntervalSet of
U;
func A ``1 -> Subset of
U means :
Def5:
ex
B being
Subset of
U st
A = Inter (
it,
B);
existence
ex b1, B being Subset of U st A = Inter (b1,B)
uniqueness
for b1, b2 being Subset of U st ex B being Subset of U st A = Inter (b1,B) & ex B being Subset of U st A = Inter (b2,B) holds
b1 = b2
by Th6;
func A ``2 -> Subset of
U means :
Def6:
ex
B being
Subset of
U st
A = Inter (
B,
it);
existence
ex b1, B being Subset of U st A = Inter (B,b1)
uniqueness
for b1, b2 being Subset of U st ex B being Subset of U st A = Inter (B,b1) & ex B being Subset of U st A = Inter (B,b2) holds
b1 = b2
by Th6;
end;
:: deftheorem Def5 defines ``1 INTERVA1:def 5 :
for U being non empty set
for A being non empty IntervalSet of U
for b3 being Subset of U holds
( b3 = A ``1 iff ex B being Subset of U st A = Inter (b3,B) );
:: deftheorem Def6 defines ``2 INTERVA1:def 6 :
for U being non empty set
for A being non empty IntervalSet of U
for b3 being Subset of U holds
( b3 = A ``2 iff ex B being Subset of U st A = Inter (B,b3) );
theorem Th14:
theorem Th15:
theorem Th16:
theorem Th17:
theorem Th18:
:: deftheorem defines = INTERVA1:def 7 :
for U being non empty set
for A, B being non empty IntervalSet of U holds
( A = B iff ( A ``1 = B ``1 & A ``2 = B ``2 ) );
theorem
theorem
theorem
theorem
theorem Th23:
theorem Th24:
Lm1:
for X being set
for A, B, C being Subset-Family of X holds UNION (A,(INTERSECTION (B,C))) c= INTERSECTION ((UNION (A,B)),(UNION (A,C)))
:: deftheorem Def8 defines ordered INTERVA1:def 8 :
for X being set
for F being Subset-Family of X holds
( F is ordered iff ex A, B being set st
( A in F & B in F & ( for Y being set holds
( Y in F iff ( A c= Y & Y c= B ) ) ) ) );
theorem Th25:
theorem Th26:
Lm2:
for X being set
for F being non empty ordered Subset-Family of X
for G being set st G in F holds
( G = min F iff for Y being set st Y in F holds
G c= Y )
Lm3:
for X being set
for F being non empty ordered Subset-Family of X
for G being set st G in F holds
( G = max F iff for Y being set st Y in F holds
Y c= G )
theorem Th27:
theorem Th28:
Lm4:
for U being non empty set
for A being non empty IntervalSet of U holds A is non empty ordered Subset-Family of U
by Th26;
theorem Th29:
Lm5:
for X being set
for A, B, C being Subset-Family of X holds INTERSECTION (A,(UNION (B,C))) c= UNION ((INTERSECTION (A,B)),(INTERSECTION (A,C)))
theorem Th30:
theorem
theorem
theorem Th33:
theorem Th34:
theorem Th35:
theorem Th36:
begin
theorem Th37:
theorem Th38:
theorem Th39:
:: deftheorem defines _\_ INTERVA1:def 9 :
for U being non empty set
for A, B being non empty IntervalSet of U holds A _\_ B = DIFFERENCE (A,B);
theorem Th40:
theorem Th41:
theorem Th42:
theorem Th43:
theorem Th44:
:: deftheorem defines ^ INTERVA1:def 10 :
for U being non empty set
for A being non empty IntervalSet of U holds A ^ = (Inter (([#] U),([#] U))) _\_ A;
theorem Th45:
theorem Th46:
theorem
theorem
begin
theorem
theorem
theorem
theorem
theorem
theorem
begin
:: deftheorem Def11 defines IntervalSets INTERVA1:def 11 :
for U, b2 being non empty set holds
( b2 = IntervalSets U iff for x being set holds
( x in b2 iff x is non empty IntervalSet of U ) );
definition
let U be non
empty set ;
func InterLatt U -> non
empty strict LattStr means :
Def12:
( the
carrier of
it = IntervalSets U & ( for
a,
b being
Element of the
carrier of
it for
a9,
b9 being non
empty IntervalSet of
U st
a9 = a &
b9 = b holds
( the
L_join of
it . (
a,
b)
= a9 _\/_ b9 & the
L_meet of
it . (
a,
b)
= a9 _/\_ b9 ) ) );
existence
ex b1 being non empty strict LattStr st
( the carrier of b1 = IntervalSets U & ( for a, b being Element of the carrier of b1
for a9, b9 being non empty IntervalSet of U st a9 = a & b9 = b holds
( the L_join of b1 . (a,b) = a9 _\/_ b9 & the L_meet of b1 . (a,b) = a9 _/\_ b9 ) ) )
uniqueness
for b1, b2 being non empty strict LattStr st the carrier of b1 = IntervalSets U & ( for a, b being Element of the carrier of b1
for a9, b9 being non empty IntervalSet of U st a9 = a & b9 = b holds
( the L_join of b1 . (a,b) = a9 _\/_ b9 & the L_meet of b1 . (a,b) = a9 _/\_ b9 ) ) & the carrier of b2 = IntervalSets U & ( for a, b being Element of the carrier of b2
for a9, b9 being non empty IntervalSet of U st a9 = a & b9 = b holds
( the L_join of b2 . (a,b) = a9 _\/_ b9 & the L_meet of b2 . (a,b) = a9 _/\_ b9 ) ) holds
b1 = b2
end;
:: deftheorem Def12 defines InterLatt INTERVA1:def 12 :
for U being non empty set
for b2 being non empty strict LattStr holds
( b2 = InterLatt U iff ( the carrier of b2 = IntervalSets U & ( for a, b being Element of the carrier of b2
for a9, b9 being non empty IntervalSet of U st a9 = a & b9 = b holds
( the L_join of b2 . (a,b) = a9 _\/_ b9 & the L_meet of b2 . (a,b) = a9 _/\_ b9 ) ) ) );
:: deftheorem Def13 defines RoughSet INTERVA1:def 13 :
for X being Tolerance_Space
for b2 being Element of [:(bool the carrier of X),(bool the carrier of X):] holds
( b2 is RoughSet of X iff verum );
theorem Th55:
:: deftheorem defines RS INTERVA1:def 14 :
for X being Tolerance_Space
for A being Subset of X holds RS A = [(LAp A),(UAp A)];
:: deftheorem defines LAp INTERVA1:def 15 :
for X being Tolerance_Space
for A being RoughSet of X holds LAp A = A `1 ;
:: deftheorem defines UAp INTERVA1:def 16 :
for X being Tolerance_Space
for A being RoughSet of X holds UAp A = A `2 ;
:: deftheorem Def17 defines = INTERVA1:def 17 :
for X being Tolerance_Space
for A, B being RoughSet of X holds
( A = B iff ( LAp A = LAp B & UAp A = UAp B ) );
:: deftheorem defines _\/_ INTERVA1:def 18 :
for X being Tolerance_Space
for A, B being RoughSet of X holds A _\/_ B = [((LAp A) \/ (LAp B)),((UAp A) \/ (UAp B))];
:: deftheorem defines _/\_ INTERVA1:def 19 :
for X being Tolerance_Space
for A, B being RoughSet of X holds A _/\_ B = [((LAp A) /\ (LAp B)),((UAp A) /\ (UAp B))];
theorem Th56:
theorem Th57:
theorem Th58:
theorem Th59:
theorem
theorem Th61:
theorem
theorem
theorem Th64:
theorem Th65:
theorem Th66:
theorem Th67:
theorem
begin
:: deftheorem Def20 defines RoughSets INTERVA1:def 20 :
for X being Tolerance_Space
for b2 being set holds
( b2 = RoughSets X iff for x being set holds
( x in b2 iff x is RoughSet of X ) );
:: deftheorem defines @ INTERVA1:def 21 :
for X being Tolerance_Space
for R being Element of RoughSets X holds @ R = R;
:: deftheorem defines @ INTERVA1:def 22 :
for X being Tolerance_Space
for R being RoughSet of X holds R @ = R;
definition
let X be
Tolerance_Space;
func RSLattice X -> strict LattStr means :
Def23:
( the
carrier of
it = RoughSets X & ( for
A,
B being
Element of
RoughSets X for
A9,
B9 being
RoughSet of
X st
A = A9 &
B = B9 holds
( the
L_join of
it . (
A,
B)
= A9 _\/_ B9 & the
L_meet of
it . (
A,
B)
= A9 _/\_ B9 ) ) );
existence
ex b1 being strict LattStr st
( the carrier of b1 = RoughSets X & ( for A, B being Element of RoughSets X
for A9, B9 being RoughSet of X st A = A9 & B = B9 holds
( the L_join of b1 . (A,B) = A9 _\/_ B9 & the L_meet of b1 . (A,B) = A9 _/\_ B9 ) ) )
uniqueness
for b1, b2 being strict LattStr st the carrier of b1 = RoughSets X & ( for A, B being Element of RoughSets X
for A9, B9 being RoughSet of X st A = A9 & B = B9 holds
( the L_join of b1 . (A,B) = A9 _\/_ B9 & the L_meet of b1 . (A,B) = A9 _/\_ B9 ) ) & the carrier of b2 = RoughSets X & ( for A, B being Element of RoughSets X
for A9, B9 being RoughSet of X st A = A9 & B = B9 holds
( the L_join of b2 . (A,B) = A9 _\/_ B9 & the L_meet of b2 . (A,B) = A9 _/\_ B9 ) ) holds
b1 = b2
end;
:: deftheorem Def23 defines RSLattice INTERVA1:def 23 :
for X being Tolerance_Space
for b2 being strict LattStr holds
( b2 = RSLattice X iff ( the carrier of b2 = RoughSets X & ( for A, B being Element of RoughSets X
for A9, B9 being RoughSet of X st A = A9 & B = B9 holds
( the L_join of b2 . (A,B) = A9 _\/_ B9 & the L_meet of b2 . (A,B) = A9 _/\_ B9 ) ) ) );
Lm6:
for X being Tolerance_Space
for a, b being Element of (RSLattice X) holds a "\/" b = b "\/" a
Lm7:
for X being Tolerance_Space
for a, b, c being Element of (RSLattice X) holds a "\/" (b "\/" c) = (a "\/" b) "\/" c
Lm8:
for X being Tolerance_Space
for K, L being Element of RoughSets X holds the L_join of (RSLattice X) . (( the L_meet of (RSLattice X) . (K,L)),L) = L
Lm9:
for X being Tolerance_Space
for a, b being Element of (RSLattice X) holds (a "/\" b) "\/" b = b
Lm10:
for X being Tolerance_Space
for a, b being Element of (RSLattice X) holds a "/\" b = b "/\" a
Lm11:
for X being Tolerance_Space
for a, b, c being Element of (RSLattice X) holds a "/\" (b "/\" c) = (a "/\" b) "/\" c
Lm12:
for X being Tolerance_Space
for K, L, M being Element of RoughSets X holds the L_meet of (RSLattice X) . (K,( the L_join of (RSLattice X) . (L,M))) = the L_join of (RSLattice X) . (( the L_meet of (RSLattice X) . (K,L)),( the L_meet of (RSLattice X) . (K,M)))
Lm13:
for X being Tolerance_Space
for a, b being Element of (RSLattice X) holds a "/\" (a "\/" b) = a
:: deftheorem defines ERS INTERVA1:def 24 :
for X being Tolerance_Space holds ERS X = [{},{}];
Lm14:
for X being Tolerance_Space holds ERS X in RoughSets X
by Def20;
theorem Th69:
:: deftheorem defines TRS INTERVA1:def 25 :
for X being Tolerance_Space holds TRS X = [([#] X),([#] X)];
Lm15:
for X being Tolerance_Space holds TRS X in RoughSets X
by Def20;
theorem Th70:
theorem Th71:
Lm16:
for X being Tolerance_Space holds RSLattice X is complete