Lm1:
for A, B being finite set
for f being Function of A,B st card A = card B & f is onto holds
f is one-to-one
Lemacik:
for A, B being finite set
for f being Function of A,B st card A = card B & f is one-to-one holds
f is onto
::
deftheorem defines
<* FINSEQ_4:def 8 :
for x1, x2, x3, x4, x5 being object holds <*x1,x2,x3,x4,x5*> = <*x1,x2,x3*> ^ <*x4,x5*>;
registration
let x1,
x2,
x3,
x4 be
object ;
coherence
( not <*x1,x2,x3,x4*> is empty & <*x1,x2,x3,x4*> is Function-like & <*x1,x2,x3,x4*> is Relation-like )
;
let x5 be
object ;
coherence
( not <*x1,x2,x3,x4,x5*> is empty & <*x1,x2,x3,x4,x5*> is Function-like & <*x1,x2,x3,x4,x5*> is Relation-like )
;
end;
registration
let x1,
x2,
x3,
x4 be
object ;
coherence
<*x1,x2,x3,x4*> is FinSequence-like
;
let x5 be
object ;
coherence
<*x1,x2,x3,x4,x5*> is FinSequence-like
;
end;
definition
let D be non
empty set ;
let x1,
x2,
x3,
x4,
x5 be
Element of
D;
<*redefine func <*x1,x2,x3,x4,x5*> -> FinSequence of
D;
coherence
<*x1,x2,x3,x4,x5*> is FinSequence of D
end;
theorem Th74:
for
x1,
x2,
x3,
x4 being
object holds
(
<*x1,x2,x3,x4*> = <*x1,x2,x3*> ^ <*x4*> &
<*x1,x2,x3,x4*> = <*x1,x2*> ^ <*x3,x4*> &
<*x1,x2,x3,x4*> = <*x1*> ^ <*x2,x3,x4*> &
<*x1,x2,x3,x4*> = ((<*x1*> ^ <*x2*>) ^ <*x3*>) ^ <*x4*> )
theorem Th75:
for
x1,
x2,
x3,
x4,
x5 being
object holds
(
<*x1,x2,x3,x4,x5*> = <*x1,x2,x3*> ^ <*x4,x5*> &
<*x1,x2,x3,x4,x5*> = <*x1,x2,x3,x4*> ^ <*x5*> &
<*x1,x2,x3,x4,x5*> = (((<*x1*> ^ <*x2*>) ^ <*x3*>) ^ <*x4*>) ^ <*x5*> &
<*x1,x2,x3,x4,x5*> = <*x1,x2*> ^ <*x3,x4,x5*> &
<*x1,x2,x3,x4,x5*> = <*x1*> ^ <*x2,x3,x4,x5*> )
theorem
for
ND being non
empty set for
y1,
y2,
y3,
y4 being
Element of
ND holds
(
<*y1,y2,y3,y4*> /. 1
= y1 &
<*y1,y2,y3,y4*> /. 2
= y2 &
<*y1,y2,y3,y4*> /. 3
= y3 &
<*y1,y2,y3,y4*> /. 4
= y4 )
theorem
for
ND being non
empty set for
y1,
y2,
y3,
y4,
y5 being
Element of
ND holds
(
<*y1,y2,y3,y4,y5*> /. 1
= y1 &
<*y1,y2,y3,y4,y5*> /. 2
= y2 &
<*y1,y2,y3,y4,y5*> /. 3
= y3 &
<*y1,y2,y3,y4,y5*> /. 4
= y4 &
<*y1,y2,y3,y4,y5*> /. 5
= y5 )
registration
let x1,
x2,
x3,
x4 be
object ;
coherence
<*x1,x2,x3,x4*> is 4 -element
;
let x5 be
object ;
coherence
<*x1,x2,x3,x4,x5*> is 5 -element
;
end;
:: Dirichlet Principle
:: Pigeon Hole Principle