begin
Lm1:
for x, X being set holds
( {x} c= X iff x in X )
Lm2:
for Y, X, x being set st Y c= X & not x in Y holds
Y c= X \ {x}
Lm3:
for Y, x being set holds
( Y c= {x} iff ( Y = {} or Y = {x} ) )
:: deftheorem Def1 defines bool ZFMISC_1:def 1 :
for X being set
for b2 being set holds
( b2 = bool X iff for Z being set holds
( Z in b2 iff Z c= X ) );
definition
let X1,
X2 be
set ;
defpred S1[
set ]
means ex
x,
y being
set st
(
x in X1 &
y in X2 & $1
= [x,y] );
func [:X1,X2:] -> set means :
Def2:
for
z being
set holds
(
z in it iff ex
x,
y being
set st
(
x in X1 &
y in X2 &
z = [x,y] ) );
existence
ex b1 being set st
for z being set holds
( z in b1 iff ex x, y being set st
( x in X1 & y in X2 & z = [x,y] ) )
uniqueness
for b1, b2 being set st ( for z being set holds
( z in b1 iff ex x, y being set st
( x in X1 & y in X2 & z = [x,y] ) ) ) & ( for z being set holds
( z in b2 iff ex x, y being set st
( x in X1 & y in X2 & z = [x,y] ) ) ) holds
b1 = b2
end;
:: deftheorem Def2 defines [: ZFMISC_1:def 2 :
for X1, X2 being set
for b3 being set holds
( b3 = [:X1,X2:] iff for z being set holds
( z in b3 iff ex x, y being set st
( x in X1 & y in X2 & z = [x,y] ) ) );
:: deftheorem defines [: ZFMISC_1:def 3 :
for X1, X2, X3 being set holds [:X1,X2,X3:] = [:[:X1,X2:],X3:];
definition
let X1,
X2,
X3,
X4 be
set ;
func [:X1,X2,X3,X4:] -> set equals
[:[:X1,X2,X3:],X4:];
coherence
[:[:X1,X2,X3:],X4:] is set
;
end;
:: deftheorem defines [: ZFMISC_1:def 4 :
for X1, X2, X3, X4 being set holds [:X1,X2,X3,X4:] = [:[:X1,X2,X3:],X4:];
begin
theorem
theorem
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem Th6:
theorem
canceled;
theorem Th8:
for
x,
y1,
y2 being
set st
{x} = {y1,y2} holds
x = y1
theorem Th9:
for
x,
y1,
y2 being
set st
{x} = {y1,y2} holds
y1 = y2
theorem Th10:
for
x1,
x2,
y1,
y2 being
set holds
( not
{x1,x2} = {y1,y2} or
x1 = y1 or
x1 = y2 )
theorem
canceled;
theorem Th12:
Lm4:
for x, X being set st {x} \/ X c= X holds
x in X
theorem
Lm5:
for x, X being set st x in X holds
{x} \/ X = X
theorem
Lm6:
for x, X being set st {x} misses X holds
not x in X
theorem
canceled;
theorem
Lm7:
for x, X being set st not x in X holds
{x} misses X
theorem Th17:
Lm8:
for X, x being set st X /\ {x} = {x} holds
x in X
theorem
Lm9:
for x, X being set st x in X holds
X /\ {x} = {x}
theorem
Lm10:
for x, X being set holds
( {x} \ X = {x} iff not x in X )
theorem
Lm11:
for x, X being set holds
( {x} \ X = {} iff x in X )
theorem
theorem
Lm12:
for x, y, X being set holds
( {x,y} \ X = {x} iff ( not x in X & ( y in X or x = y ) ) )
theorem
theorem
theorem
for
z,
x,
y being
set holds
( not
{z} c= {x,y} or
z = x or
z = y )
theorem Th26:
theorem
Lm13:
for X, x being set st X <> {x} & X <> {} holds
ex y being set st
( y in X & y <> x )
Lm14:
for Z, x1, x2 being set holds
( Z c= {x1,x2} iff ( Z = {} or Z = {x1} or Z = {x2} or Z = {x1,x2} ) )
theorem
for
x1,
x2,
y1,
y2 being
set holds
( not
{x1,x2} c= {y1,y2} or
x1 = y1 or
x1 = y2 )
theorem
theorem
Lm15:
for X, A being set st X in A holds
X c= union A
theorem
Lm16:
for X, Y being set holds union {X,Y} = X \/ Y
theorem
theorem Th33:
for
x1,
x2,
y1,
y2 being
set st
[x1,x2] = [y1,y2] holds
(
x1 = y1 &
x2 = y2 )
Lm17:
for x, y, X, Y being set holds
( [x,y] in [:X,Y:] iff ( x in X & y in Y ) )
theorem
theorem
theorem Th36:
for
x,
y,
z being
set holds
(
[:{x},{y,z}:] = {[x,y],[x,z]} &
[:{x,y},{z}:] = {[x,z],[y,z]} )
theorem
theorem Th38:
for
x1,
x2,
Z being
set holds
(
{x1,x2} c= Z iff (
x1 in Z &
x2 in Z ) )
theorem
theorem
theorem
theorem
theorem Th43:
theorem
theorem
theorem
theorem
theorem
for
x,
Z,
y being
set st
x in Z &
y in Z holds
{x,y} \/ Z = Z
theorem
theorem
theorem
theorem
theorem
theorem
theorem Th55:
theorem
theorem Th57:
theorem
theorem
for
x,
y,
X being
set holds
( not
{x,y} /\ X = {x} or not
y in X or
x = y )
theorem
for
x,
X,
y being
set st
x in X & ( not
y in X or
x = y ) holds
{x,y} /\ X = {x}
theorem
canceled;
theorem
canceled;
theorem
theorem Th64:
for
z,
X,
x being
set holds
(
z in X \ {x} iff (
z in X &
z <> x ) )
theorem Th65:
for
X,
x being
set holds
(
X \ {x} = X iff not
x in X )
theorem
theorem
theorem
theorem
theorem
for
x,
y,
X being
set holds
(
{x,y} \ X = {x} iff ( not
x in X & (
y in X or
x = y ) ) )
by Lm12;
theorem
canceled;
theorem Th72:
for
x,
y,
X being
set holds
(
{x,y} \ X = {x,y} iff ( not
x in X & not
y in X ) )
theorem Th73:
for
x,
y,
X being
set holds
(
{x,y} \ X = {} iff (
x in X &
y in X ) )
theorem
theorem
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
theorem
theorem
theorem
theorem
theorem
theorem
canceled;
theorem
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
theorem
theorem
theorem Th95:
theorem
theorem Th97:
theorem Th98:
theorem
theorem
theorem
theorem
canceled;
theorem Th103:
for
A,
X,
Y,
z being
set st
A c= [:X,Y:] &
z in A holds
ex
x,
y being
set st
(
x in X &
y in Y &
z = [x,y] )
theorem Th104:
theorem
theorem
theorem Th107:
theorem
for
X1,
Y1,
X2,
Y2 being
set st ( for
x,
y being
set holds
(
[x,y] in [:X1,Y1:] iff
[x,y] in [:X2,Y2:] ) ) holds
[:X1,Y1:] = [:X2,Y2:]
Lm18:
for A, X1, Y1, B, X2, Y2 being set st A c= [:X1,Y1:] & B c= [:X2,Y2:] & ( for x, y being set holds
( [x,y] in A iff [x,y] in B ) ) holds
A = B
Lm19:
for A, B being set st ( for z being set st z in A holds
ex x, y being set st z = [x,y] ) & ( for z being set st z in B holds
ex x, y being set st z = [x,y] ) & ( for x, y being set holds
( [x,y] in A iff [x,y] in B ) ) holds
A = B
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem Th113:
theorem
theorem
Lm20:
for z, X, Y being set st z in [:X,Y:] holds
ex x, y being set st [x,y] = z
theorem
theorem
theorem Th118:
theorem Th119:
theorem Th120:
theorem
theorem
theorem Th123:
theorem
theorem Th125:
theorem
theorem Th127:
theorem Th128:
theorem Th129:
theorem
theorem
theorem
for
x,
y,
X being
set holds
(
[:{x,y},X:] = [:{x},X:] \/ [:{y},X:] &
[:X,{x,y}:] = [:X,{x}:] \/ [:X,{y}:] )
theorem
canceled;
theorem Th134:
theorem
theorem
theorem
begin
theorem Th138:
theorem
theorem
theorem
theorem
for
x,
y,
z,
Z being
set holds
(
Z c= {x,y,z} iff (
Z = {} or
Z = {x} or
Z = {y} or
Z = {z} or
Z = {x,y} or
Z = {y,z} or
Z = {x,z} or
Z = {x,y,z} ) )
theorem
Lm21:
for x, y, X being set st not x in X & not y in X holds
{x,y} misses X
theorem Th144:
for
x,
y,
X being
set st not
x in X & not
y in X holds
X = X \ {x,y}
theorem
for
x,
y,
X being
set st not
x in X & not
y in X holds
X = (X \/ {x,y}) \ {x,y}
:: deftheorem defines are_mutually_different ZFMISC_1:def 5 :
for x1, x2, x3 being set holds
( x1,x2,x3 are_mutually_different iff ( x1 <> x2 & x1 <> x3 & x2 <> x3 ) );
:: deftheorem defines are_mutually_different ZFMISC_1:def 6 :
for x1, x2, x3, x4 being set holds
( x1,x2,x3,x4 are_mutually_different iff ( x1 <> x2 & x1 <> x3 & x1 <> x4 & x2 <> x3 & x2 <> x4 & x3 <> x4 ) );
:: deftheorem defines are_mutually_different ZFMISC_1:def 7 :
for x1, x2, x3, x4, x5 being set holds
( x1,x2,x3,x4,x5 are_mutually_different iff ( x1 <> x2 & x1 <> x3 & x1 <> x4 & x1 <> x5 & x2 <> x3 & x2 <> x4 & x2 <> x5 & x3 <> x4 & x3 <> x5 & x4 <> x5 ) );
definition
let x1,
x2,
x3,
x4,
x5,
x6 be
set ;
pred x1,
x2,
x3,
x4,
x5,
x6 are_mutually_different means
(
x1 <> x2 &
x1 <> x3 &
x1 <> x4 &
x1 <> x5 &
x1 <> x6 &
x2 <> x3 &
x2 <> x4 &
x2 <> x5 &
x2 <> x6 &
x3 <> x4 &
x3 <> x5 &
x3 <> x6 &
x4 <> x5 &
x4 <> x6 &
x5 <> x6 );
end;
:: deftheorem defines are_mutually_different ZFMISC_1:def 8 :
for x1, x2, x3, x4, x5, x6 being set holds
( x1,x2,x3,x4,x5,x6 are_mutually_different iff ( x1 <> x2 & x1 <> x3 & x1 <> x4 & x1 <> x5 & x1 <> x6 & x2 <> x3 & x2 <> x4 & x2 <> x5 & x2 <> x6 & x3 <> x4 & x3 <> x5 & x3 <> x6 & x4 <> x5 & x4 <> x6 & x5 <> x6 ) );
definition
let x1,
x2,
x3,
x4,
x5,
x6,
x7 be
set ;
pred x1,
x2,
x3,
x4,
x5,
x6,
x7 are_mutually_different means
(
x1 <> x2 &
x1 <> x3 &
x1 <> x4 &
x1 <> x5 &
x1 <> x6 &
x1 <> x7 &
x2 <> x3 &
x2 <> x4 &
x2 <> x5 &
x2 <> x6 &
x2 <> x7 &
x3 <> x4 &
x3 <> x5 &
x3 <> x6 &
x3 <> x7 &
x4 <> x5 &
x4 <> x6 &
x4 <> x7 &
x5 <> x6 &
x5 <> x7 &
x6 <> x7 );
end;
:: deftheorem defines are_mutually_different ZFMISC_1:def 9 :
for x1, x2, x3, x4, x5, x6, x7 being set holds
( x1,x2,x3,x4,x5,x6,x7 are_mutually_different iff ( x1 <> x2 & x1 <> x3 & x1 <> x4 & x1 <> x5 & x1 <> x6 & x1 <> x7 & x2 <> x3 & x2 <> x4 & x2 <> x5 & x2 <> x6 & x2 <> x7 & x3 <> x4 & x3 <> x5 & x3 <> x6 & x3 <> x7 & x4 <> x5 & x4 <> x6 & x4 <> x7 & x5 <> x6 & x5 <> x7 & x6 <> x7 ) );
theorem
for
x1,
x2,
y1,
y2 being
set holds
[:{x1,x2},{y1,y2}:] = {[x1,y1],[x1,y2],[x2,y1],[x2,y2]}
theorem
:: deftheorem defines trivial ZFMISC_1:def 10 :
for X being set holds
( X is trivial iff for x, y being set st x in X & y in X holds
x = y );
theorem
theorem
theorem
canceled;
theorem
theorem
theorem
theorem