begin
:: deftheorem Def1 defines Cardinal-yielding CARD_3:def 1 :
for IT being Function holds
( IT is Cardinal-yielding iff for x being set st x in dom IT holds
IT . x is Cardinal );
theorem
canceled;
theorem
canceled;
theorem
canceled;
:: deftheorem Def2 defines Card CARD_3:def 2 :
for f being Function
for b2 being Cardinal-Function holds
( b2 = Card f iff ( dom b2 = dom f & ( for x being set st x in dom f holds
b2 . x = card (f . x) ) ) );
:: deftheorem Def3 defines disjoin CARD_3:def 3 :
for f, b2 being Function holds
( b2 = disjoin f iff ( dom b2 = dom f & ( for x being set st x in dom f holds
b2 . x = [:(f . x),{x}:] ) ) );
:: deftheorem defines Union CARD_3:def 4 :
for f being Function holds Union f = union (rng f);
:: deftheorem Def5 defines product CARD_3:def 5 :
for f being Function
for b2 being set holds
( b2 = product f iff for x being set holds
( x in b2 iff ex g being Function st
( x = g & dom g = dom f & ( for y being set st y in dom f holds
g . y in f . y ) ) ) );
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem Th8:
theorem
canceled;
theorem
theorem
theorem Th12:
theorem
theorem
canceled;
theorem Th15:
theorem Th16:
theorem
theorem Th18:
theorem Th19:
theorem Th20:
defpred S1[ set ] means $1 is Function;
:: deftheorem Def6 defines pi CARD_3:def 6 :
for x, X, b3 being set holds
( b3 = pi (X,x) iff for y being set holds
( y in b3 iff ex f being Function st
( f in X & y = f . x ) ) );
theorem
canceled;
theorem
theorem
canceled;
theorem
theorem
theorem
theorem Th27:
for
X,
Y,
x being
set holds
pi (
(X \/ Y),
x)
= (pi (X,x)) \/ (pi (Y,x))
theorem
theorem Th29:
for
X,
x,
Y being
set holds
(pi (X,x)) \ (pi (Y,x)) c= pi (
(X \ Y),
x)
theorem
theorem Th31:
theorem Th32:
theorem Th33:
theorem Th34:
theorem Th35:
theorem Th36:
theorem Th37:
theorem Th38:
theorem
theorem Th40:
:: deftheorem defines Sum CARD_3:def 7 :
for F being Cardinal-Function holds Sum F = card (Union (disjoin F));
:: deftheorem defines Product CARD_3:def 8 :
for F being Cardinal-Function holds Product F = card (product F);
theorem
canceled;
theorem
canceled;
theorem Th43:
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem Th54:
theorem
theorem
scheme
FinRegularity{
F1()
-> finite set ,
P1[
set ,
set ] } :
ex
x being
set st
(
x in F1() & ( for
y being
set st
y in F1() &
y <> x holds
not
P1[
y,
x] ) )
provided
A1:
F1()
<> {}
and A2:
for
x,
y being
set st
P1[
x,
y] &
P1[
y,
x] holds
x = y
and A3:
for
x,
y,
z being
set st
P1[
x,
y] &
P1[
y,
z] holds
P1[
x,
z]
scheme
MaxFinSetElem{
F1()
-> finite set ,
P1[
set ,
set ] } :
ex
x being
set st
(
x in F1() & ( for
y being
set st
y in F1() holds
P1[
x,
y] ) )
provided
A1:
F1()
<> {}
and A2:
for
x,
y being
set holds
(
P1[
x,
y] or
P1[
y,
x] )
and A3:
for
x,
y,
z being
set st
P1[
x,
y] &
P1[
y,
z] holds
P1[
x,
z]
Lm1:
for n being Element of NAT st Rank n is finite holds
Rank (n + 1) is finite
theorem
Lm2:
for x being set
for R being Relation st x in field R holds
ex y being set st
( [x,y] in R or [y,x] in R )
theorem Th58:
theorem Th59:
theorem Th60:
theorem Th61:
theorem
begin
theorem
theorem
begin
:: deftheorem Def9 defines sproduct CARD_3:def 9 :
for f being Function
for b2 being set holds
( b2 = sproduct f iff for x being set holds
( x in b2 iff ex g being Function st
( x = g & dom g c= dom f & ( for x being set st x in dom g holds
g . x in f . x ) ) ) );
theorem Th65:
theorem Th66:
theorem Th67:
theorem Th68:
theorem Th69:
theorem
theorem Th71:
theorem Th72:
theorem Th73:
theorem
theorem
theorem Th76:
theorem
theorem Th78:
theorem
theorem Th80:
theorem Th81:
theorem Th82:
theorem
theorem Th84:
theorem
theorem Th86:
theorem
begin
:: deftheorem Def10 defines with_common_domain CARD_3:def 10 :
for IT being set holds
( IT is with_common_domain iff for f, g being Function st f in IT & g in IT holds
dom f = dom g );
theorem
:: deftheorem CARD_3:def 11 :
canceled;
:: deftheorem Def12 defines DOM CARD_3:def 12 :
for X being functional with_common_domain set
for b2 being set holds
( ( X <> {} implies ( b2 = DOM X iff for x being Function st x in X holds
b2 = dom x ) ) & ( not X <> {} implies ( b2 = DOM X iff b2 = {} ) ) );
theorem
begin
:: deftheorem Def13 defines product" CARD_3:def 13 :
for S being functional set
for b2 being Function holds
( ( not S is empty implies ( b2 = product" S iff ( ( for x being set holds
( x in dom b2 iff for f being Function st f in S holds
x in dom f ) ) & ( for i being set st i in dom b2 holds
b2 . i = pi (S,i) ) ) ) ) & ( S is empty implies ( b2 = product" S iff b2 = {} ) ) );
theorem Th89:
theorem Th90:
:: deftheorem Def14 defines product-like CARD_3:def 14 :
for S being set holds
( S is product-like iff ex f being Function st S = product f );
theorem Th92:
theorem
theorem Th94:
theorem
theorem
theorem
theorem Th98:
theorem
theorem
theorem
theorem Th102:
theorem Th103:
theorem
theorem Th105:
theorem
theorem Th107:
theorem
Lm3:
1 = card 1
by CARD_1:def 5;
Lm4:
2 = card 2
by CARD_1:def 5;
theorem
theorem
theorem Th111:
theorem Th112:
theorem Th113:
theorem Th114:
theorem Th115:
Lm5:
omega is limit_ordinal
by ORDINAL1:def 12;
theorem Th116:
theorem Th117:
theorem Th118:
theorem
theorem
theorem
theorem
theorem
theorem
theorem Th125:
theorem
:: deftheorem Def15 defines countable CARD_3:def 15 :
for X being set holds
( X is countable iff card X c= omega );
:: deftheorem defines denumerable CARD_3:def 16 :
for X being set holds
( X is denumerable iff card X = omega );
theorem Th127:
Lm6:
for Y, X being set st Y c= X & X is countable holds
Y is countable
;
theorem Th128:
theorem
theorem
theorem
theorem Th132:
theorem
theorem Th134:
theorem
theorem Th136:
theorem
theorem Th138:
for
K,
L,
M,
N being
Cardinal holds
( ( not (
K in L &
M in N ) & not (
K c= L &
M in N ) & not (
K in L &
M c= N ) & not (
K c= L &
M c= N ) ) or
K = 0 or
exp (
K,
M)
c= exp (
L,
N) )
theorem
theorem Th140:
theorem
theorem Th142:
theorem
theorem
theorem
theorem
theorem
theorem
theorem
theorem Th150:
theorem Th151:
theorem
:: deftheorem Def17 defines proj CARD_3:def 17 :
for f being Function
for x being set
for b3 being Function holds
( b3 = proj (f,x) iff ( dom b3 = product f & ( for y being Function st y in dom b3 holds
b3 . y = y . x ) ) );
theorem Th153:
theorem
theorem
theorem