begin
:: deftheorem Def1 defines quasi_total FUNCT_2:def 1 :
for X, Y being set
for R being Relation of X,Y holds
( ( ( Y = {} implies X = {} ) implies ( R is quasi_total iff X = dom R ) ) & ( Y = {} implies X = {} ( R is quasi_total iff R = {} ) ) );
theorem
canceled;
theorem
canceled;
theorem
theorem Th4:
theorem
theorem Th6:
theorem Th7:
theorem
theorem
scheme
FuncEx1{
F1()
-> set ,
F2()
-> set ,
P1[
set ,
set ] } :
ex
f being
Function of
F1(),
F2() st
for
x being
set st
x in F1() holds
P1[
x,
f . x]
provided
A1:
for
x being
set st
x in F1() holds
ex
y being
set st
(
y in F2() &
P1[
x,
y] )
scheme
Lambda1{
F1()
-> set ,
F2()
-> set ,
F3(
set )
-> set } :
ex
f being
Function of
F1(),
F2() st
for
x being
set st
x in F1() holds
f . x = F3(
x)
provided
A1:
for
x being
set st
x in F1() holds
F3(
x)
in F2()
:: deftheorem Def2 defines Funcs FUNCT_2:def 2 :
for X, Y, b3 being set holds
( b3 = Funcs (X,Y) iff for x being set holds
( x in b3 iff ex f being Function st
( x = f & dom f = X & rng f c= Y ) ) );
theorem
canceled;
theorem Th11:
theorem
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
for
X,
Y being
set for
f being
Function of
X,
Y st ( for
y being
set st
y in Y holds
ex
x being
set st
(
x in X &
y = f . x ) ) holds
rng f = Y
theorem Th17:
theorem Th18:
for
X,
Y being
set for
f1,
f2 being
Function of
X,
Y st ( for
x being
set st
x in X holds
f1 . x = f2 . x ) holds
f1 = f2
theorem Th19:
theorem
theorem Th21:
theorem
theorem
theorem
theorem
theorem
theorem
theorem
:: deftheorem Def3 defines onto FUNCT_2:def 3 :
for Y being set
for f being b1 -valued Relation holds
( f is onto iff rng f = Y );
theorem
theorem
theorem Th31:
theorem
theorem Th33:
theorem
theorem
theorem
theorem
theorem Th38:
theorem
canceled;
theorem
theorem
theorem
canceled;
theorem
theorem
theorem
theorem
for
X,
Y,
Q being
set for
f being
Function of
X,
Y st
Y <> {} holds
for
x being
set holds
(
x in f " Q iff (
x in X &
f . x in Q ) )
theorem
theorem Th48:
theorem
theorem Th50:
theorem
theorem
canceled;
theorem
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
theorem
theorem
theorem Th62:
theorem
canceled;
theorem
theorem Th65:
theorem Th66:
theorem Th67:
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem Th73:
theorem
canceled;
theorem
theorem
theorem Th77:
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
:: deftheorem Def4 defines bijective FUNCT_2:def 4 :
for X, Y being set
for f being PartFunc of X,Y holds
( f is bijective iff ( f is one-to-one & f is onto ) );
theorem Th83:
theorem
canceled;
theorem
theorem
theorem
theorem
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem Th92:
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem Th113:
for
X,
Y being
set for
f1,
f2 being
Function of
X,
Y st ( for
x being
Element of
X holds
f1 . x = f2 . x ) holds
f1 = f2
theorem
canceled;
theorem Th115:
for
X,
Y,
P being
set for
f being
Function of
X,
Y for
y being
set st
y in f .: P holds
ex
x being
set st
(
x in X &
x in P &
y = f . x )
theorem
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
begin
theorem Th121:
scheme
Lambda1C{
F1()
-> set ,
F2()
-> set ,
P1[
set ],
F3(
set )
-> set ,
F4(
set )
-> set } :
ex
f being
Function of
F1(),
F2() st
for
x being
set st
x in F1() holds
( (
P1[
x] implies
f . x = F3(
x) ) & (
P1[
x] implies
f . x = F4(
x) ) )
provided
A1:
for
x being
set st
x in F1() holds
( (
P1[
x] implies
F3(
x)
in F2() ) & (
P1[
x] implies
F4(
x)
in F2() ) )
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
theorem
theorem
theorem Th133:
theorem
canceled;
theorem
canceled;
theorem Th136:
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
theorem Th142:
theorem
theorem
canceled;
theorem Th145:
theorem
theorem
canceled;
theorem Th148:
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
theorem
canceled;
theorem
theorem Th155:
theorem
theorem
canceled;
theorem Th158:
theorem
theorem
theorem Th161:
theorem
theorem
canceled;
theorem
theorem
theorem Th166:
theorem Th167:
theorem
begin
theorem
definition
let A,
B,
C be non
empty set ;
canceled;let f be
Function of
A,
[:B,C:];
pr1redefine func pr1 f -> Function of
A,
B means :
Def6:
for
x being
Element of
A holds
it . x = (f . x) `1 ;
coherence
pr1 f is Function of A,B
compatibility
for b1 being Function of A,B holds
( b1 = pr1 f iff for x being Element of A holds b1 . x = (f . x) `1 )
pr2redefine func pr2 f -> Function of
A,
C means :
Def7:
for
x being
Element of
A holds
it . x = (f . x) `2 ;
coherence
pr2 f is Function of A,C
compatibility
for b1 being Function of A,C holds
( b1 = pr2 f iff for x being Element of A holds b1 . x = (f . x) `2 )
end;
:: deftheorem FUNCT_2:def 5 :
canceled;
:: deftheorem Def6 defines pr1 FUNCT_2:def 6 :
for A, B, C being non empty set
for f being Function of A,[:B,C:]
for b5 being Function of A,B holds
( b5 = pr1 f iff for x being Element of A holds b5 . x = (f . x) `1 );
:: deftheorem Def7 defines pr2 FUNCT_2:def 7 :
for A, B, C being non empty set
for f being Function of A,[:B,C:]
for b5 being Function of A,C holds
( b5 = pr2 f iff for x being Element of A holds b5 . x = (f . x) `2 );
:: deftheorem defines = FUNCT_2:def 8 :
for A1 being set
for B1 being non empty set
for A2 being set
for B2 being non empty set
for f1 being Function of A1,B1
for f2 being Function of A2,B2 holds
( f1 = f2 iff ( A1 = A2 & ( for a being Element of A1 holds f1 . a = f2 . a ) ) );
:: deftheorem defines = FUNCT_2:def 9 :
for A, B being set
for f1, f2 being Function of A,B holds
( f1 = f2 iff for a being Element of A holds f1 . a = f2 . a );
theorem
theorem Th171:
theorem
theorem
theorem
theorem
theorem Th176:
theorem
theorem
:: deftheorem Def10 defines " FUNCT_2:def 10 :
for T, S being non empty set
for f being Function of T,S
for G being Subset-Family of S
for b5 being Subset-Family of T holds
( b5 = f " G iff for A being Subset of T holds
( A in b5 iff ex B being Subset of S st
( B in G & A = f " B ) ) );
theorem
:: deftheorem Def11 defines .: FUNCT_2:def 11 :
for T, S being non empty set
for f being Function of T,S
for G being Subset-Family of T
for b5 being Subset-Family of S holds
( b5 = f .: G iff for A being Subset of S holds
( A in b5 iff ex B being Subset of T st
( B in G & A = f .: B ) ) );
theorem
theorem
theorem
theorem
theorem
:: deftheorem Def12 defines /* FUNCT_2:def 12 :
for X, Y, Z being set
for f being Function of X,Y
for p being PartFunc of Y,Z st Y <> {} & rng f c= dom p holds
p /* f = p * f;
theorem Th185:
theorem Th186:
theorem
theorem
theorem
theorem Th190:
theorem
theorem
theorem
theorem Th194:
theorem
theorem
theorem
:: deftheorem Def13 defines FUNCTION_DOMAIN FUNCT_2:def 13 :
for A, B being set
for b3 being non empty set holds
( b3 is FUNCTION_DOMAIN of A,B iff for x being Element of b3 holds x is Function of A,B );
theorem
theorem Th199:
:: deftheorem defines /. FUNCT_2:def 14 :
for X, A being non empty set
for F being Function of X,A
for x being set st x in X holds
F /. x = F . x;
theorem
theorem