begin
:: deftheorem Def1 defines is_left_inverse_of ALTCAT_3:def 1 :
for C being non empty with_units AltCatStr
for o1, o2 being object of C
for A being Morphism of o1,o2
for B being Morphism of o2,o1 holds
( A is_left_inverse_of B iff A * B = idm o2 );
:: deftheorem Def2 defines retraction ALTCAT_3:def 2 :
for C being non empty with_units AltCatStr
for o1, o2 being object of C
for A being Morphism of o1,o2 holds
( A is retraction iff ex B being Morphism of o2,o1 st B is_right_inverse_of A );
:: deftheorem Def3 defines coretraction ALTCAT_3:def 3 :
for C being non empty with_units AltCatStr
for o1, o2 being object of C
for A being Morphism of o1,o2 holds
( A is coretraction iff ex B being Morphism of o2,o1 st B is_left_inverse_of A );
theorem Th1:
:: deftheorem Def4 defines " ALTCAT_3:def 4 :
for C being category
for o1, o2 being object of C st <^o1,o2^> <> {} & <^o2,o1^> <> {} holds
for A being Morphism of o1,o2 st A is retraction & A is coretraction holds
for b5 being Morphism of o2,o1 holds
( b5 = A " iff ( b5 is_left_inverse_of A & b5 is_right_inverse_of A ) );
theorem Th2:
theorem Th3:
theorem Th4:
:: deftheorem Def5 defines iso ALTCAT_3:def 5 :
for C being category
for o1, o2 being object of C
for A being Morphism of o1,o2 holds
( A is iso iff ( A * (A ") = idm o2 & (A ") * A = idm o1 ) );
theorem Th5:
theorem Th6:
theorem Th7:
definition
let C be
category;
let o1,
o2 be
object of
C;
pred o1,
o2 are_iso means :
Def6:
(
<^o1,o2^> <> {} &
<^o2,o1^> <> {} & ex
A being
Morphism of
o1,
o2 st
A is
iso );
reflexivity
for o1 being object of C holds
( <^o1,o1^> <> {} & <^o1,o1^> <> {} & ex A being Morphism of o1,o1 st A is iso )
symmetry
for o1, o2 being object of C st <^o1,o2^> <> {} & <^o2,o1^> <> {} & ex A being Morphism of o1,o2 st A is iso holds
( <^o2,o1^> <> {} & <^o1,o2^> <> {} & ex A being Morphism of o2,o1 st A is iso )
end;
:: deftheorem Def6 defines are_iso ALTCAT_3:def 6 :
for C being category
for o1, o2 being object of C holds
( o1,o2 are_iso iff ( <^o1,o2^> <> {} & <^o2,o1^> <> {} & ex A being Morphism of o1,o2 st A is iso ) );
theorem
:: deftheorem Def7 defines mono ALTCAT_3:def 7 :
for C being non empty AltCatStr
for o1, o2 being object of C
for A being Morphism of o1,o2 holds
( A is mono iff for o being object of C st <^o,o1^> <> {} holds
for B, C being Morphism of o,o1 st A * B = A * C holds
B = C );
:: deftheorem Def8 defines epi ALTCAT_3:def 8 :
for C being non empty AltCatStr
for o1, o2 being object of C
for A being Morphism of o1,o2 holds
( A is epi iff for o being object of C st <^o2,o^> <> {} holds
for B, C being Morphism of o2,o st B * A = C * A holds
B = C );
theorem Th9:
theorem Th10:
theorem
theorem
Lm1:
now
let C be non
empty with_units AltCatStr ;
for a being object of C holds
( idm a is epi & idm a is mono )let a be
object of
C;
( idm a is epi & idm a is mono )thus
idm a is
epi
idm a is mono
proof
let o be
object of
C;
ALTCAT_3:def 8 ( <^a,o^> <> {} implies for B, C being Morphism of a,o st B * (idm a) = C * (idm a) holds
B = C )
assume A1:
<^a,o^> <> {}
;
for B, C being Morphism of a,o st B * (idm a) = C * (idm a) holds
B = C
let B,
C be
Morphism of
a,
o;
( B * (idm a) = C * (idm a) implies B = C )
assume A2:
B * (idm a) = C * (idm a)
;
B = C
thus B =
B * (idm a)
by A1, ALTCAT_1:def 19
.=
C
by A1, A2, ALTCAT_1:def 19
;
verum
end;
thus
idm a is
mono
verum
proof
let o be
object of
C;
ALTCAT_3:def 7 ( <^o,a^> <> {} implies for B, C being Morphism of o,a st (idm a) * B = (idm a) * C holds
B = C )
assume A3:
<^o,a^> <> {}
;
for B, C being Morphism of o,a st (idm a) * B = (idm a) * C holds
B = C
let B,
C be
Morphism of
o,
a;
( (idm a) * B = (idm a) * C implies B = C )
assume A4:
(idm a) * B = (idm a) * C
;
B = C
thus B =
(idm a) * B
by A3, ALTCAT_1:24
.=
C
by A3, A4, ALTCAT_1:24
;
verum
end;
end;
theorem
theorem
theorem Th15:
theorem Th16:
theorem
theorem Th18:
theorem Th19:
theorem Th20:
theorem
theorem
theorem
theorem
:: deftheorem Def9 defines initial ALTCAT_3:def 9 :
for C being AltGraph
for o being object of C holds
( o is initial iff for o1 being object of C ex M being Morphism of o,o1 st
( M in <^o,o1^> & <^o,o1^> is trivial ) );
theorem
theorem Th26:
:: deftheorem Def10 defines terminal ALTCAT_3:def 10 :
for C being AltGraph
for o being object of C holds
( o is terminal iff for o1 being object of C ex M being Morphism of o1,o st
( M in <^o1,o^> & <^o1,o^> is trivial ) );
theorem
theorem
:: deftheorem Def11 defines _zero ALTCAT_3:def 11 :
for C being AltGraph
for o being object of C holds
( o is _zero iff ( o is initial & o is terminal ) );
theorem
:: deftheorem Def12 defines _zero ALTCAT_3:def 12 :
for C being non empty AltCatStr
for o1, o2 being object of C
for M being Morphism of o1,o2 holds
( M is _zero iff for o being object of C st o is _zero holds
for A being Morphism of o1,o
for B being Morphism of o,o2 holds M = B * A );
theorem