definition
let A,
B be
AltCatStr ;
symmetry
for A, B being AltCatStr st ( for a1, a2, a3 being object holds the Comp of A . [a1,a2,a3] tolerates the Comp of B . [a1,a2,a3] ) holds
for a1, a2, a3 being object holds the Comp of B . [a1,a2,a3] tolerates the Comp of A . [a1,a2,a3]
;
end;
theorem Th10:
for
A,
B being
AltCatStr holds
(
A,
B have_the_same_composition iff for
a1,
a2,
a3,
x being
object st
x in dom ( the Comp of A . [a1,a2,a3]) &
x in dom ( the Comp of B . [a1,a2,a3]) holds
( the Comp of A . [a1,a2,a3]) . x = ( the Comp of B . [a1,a2,a3]) . x )
theorem Th11:
for
A,
B being non
empty transitive AltCatStr holds
(
A,
B have_the_same_composition iff for
a1,
a2,
a3 being
Object of
A st
<^a1,a2^> <> {} &
<^a2,a3^> <> {} holds
for
b1,
b2,
b3 being
Object of
B st
<^b1,b2^> <> {} &
<^b2,b3^> <> {} &
b1 = a1 &
b2 = a2 &
b3 = a3 holds
for
f1 being
Morphism of
a1,
a2 for
g1 being
Morphism of
b1,
b2 st
g1 = f1 holds
for
f2 being
Morphism of
a2,
a3 for
g2 being
Morphism of
b2,
b3 st
g2 = f2 holds
f2 * f1 = g2 * g1 )
theorem Th16:
for
I1,
I2 being
set for
A1,
B1 being
ManySortedSet of
I1 for
A2,
B2 being
ManySortedSet of
I2 for
A,
B being
ManySortedSet of
I1 /\ I2 st
A = Intersect (
A1,
A2) &
B = Intersect (
B1,
B2) holds
for
F being
ManySortedFunction of
A1,
B1 for
G being
ManySortedFunction of
A2,
B2 st ( for
x being
set st
x in dom F &
x in dom G holds
F . x tolerates G . x ) holds
Intersect (
F,
G) is
ManySortedFunction of
A,
B
theorem Th18:
for
I,
J being
set for
F1,
F2 being
ManySortedSet of
[:I,I:] for
G1,
G2 being
ManySortedSet of
[:J,J:] ex
H1,
H2 being
ManySortedSet of
[:(I /\ J),(I /\ J):] st
(
H1 = Intersect (
F1,
G1) &
H2 = Intersect (
F2,
G2) &
Intersect (
{|F1,F2|},
{|G1,G2|})
= {|H1,H2|} )
theorem Th23:
for
A,
B being
AltCatStr st
A,
B have_the_same_composition holds
for
a1,
a2 being
Object of
A for
b1,
b2 being
Object of
B for
o1,
o2 being
Object of
(Intersect (A,B)) st
o1 = a1 &
o1 = b1 &
o2 = a2 &
o2 = b2 &
<^a1,a2^> <> {} &
<^b1,b2^> <> {} holds
for
f being
Morphism of
a1,
a2 for
g being
Morphism of
b1,
b2 st
f = g holds
f in <^o1,o2^>
scheme
SubcategoryUniq{
F1()
-> category,
F2()
-> non
empty subcategory of
F1(),
F3()
-> non
empty subcategory of
F1(),
P1[
set ],
P2[
set ,
set ,
set ] } :
provided
A1:
for
a being
Object of
F1() holds
(
a is
Object of
F2() iff
P1[
a] )
and A2:
for
a,
b being
Object of
F1()
for
a9,
b9 being
Object of
F2() st
a9 = a &
b9 = b &
<^a,b^> <> {} holds
for
f being
Morphism of
a,
b holds
(
f in <^a9,b9^> iff
P2[
a,
b,
f] )
and A3:
for
a being
Object of
F1() holds
(
a is
Object of
F3() iff
P1[
a] )
and A4:
for
a,
b being
Object of
F1()
for
a9,
b9 being
Object of
F3() st
a9 = a &
b9 = b &
<^a,b^> <> {} holds
for
f being
Morphism of
a,
b holds
(
f in <^a9,b9^> iff
P2[
a,
b,
f] )
::
deftheorem defines
are_isomorphic_under YELLOW20:def 4 :
for A, B being category
for F being FunctorStr over A,B
for A9, B9 being category holds
( A9,B9 are_isomorphic_under F iff ( A9 is subcategory of A & B9 is subcategory of B & ex G being covariant Functor of A9,B9 st
( G is bijective & ( for a9 being Object of A9
for a being Object of A st a9 = a holds
G . a9 = F . a ) & ( for b9, c9 being Object of A9
for b, c being Object of A st <^b9,c9^> <> {} & b9 = b & c9 = c holds
for f9 being Morphism of b9,c9
for f being Morphism of b,c st f9 = f holds
G . f9 = (Morph-Map (F,b,c)) . f ) ) ) );
::
deftheorem defines
are_anti-isomorphic_under YELLOW20:def 5 :
for A, B being category
for F being FunctorStr over A,B
for A9, B9 being category holds
( A9,B9 are_anti-isomorphic_under F iff ( A9 is subcategory of A & B9 is subcategory of B & ex G being contravariant Functor of A9,B9 st
( G is bijective & ( for a9 being Object of A9
for a being Object of A st a9 = a holds
G . a9 = F . a ) & ( for b9, c9 being Object of A9
for b, c being Object of A st <^b9,c9^> <> {} & b9 = b & c9 = c holds
for f9 being Morphism of b9,c9
for f being Morphism of b,c st f9 = f holds
G . f9 = (Morph-Map (F,b,c)) . f ) ) ) );
theorem
for
A1,
A2 being
category for
F being
covariant Functor of
A1,
A2 for
B1 being non
empty subcategory of
A1 for
B2 being non
empty subcategory of
A2 st
F is
bijective & ( for
a being
Object of
A1 holds
(
a is
Object of
B1 iff
F . a is
Object of
B2 ) ) & ( for
a,
b being
Object of
A1 st
<^a,b^> <> {} holds
for
a1,
b1 being
Object of
B1 st
a1 = a &
b1 = b holds
for
a2,
b2 being
Object of
B2 st
a2 = F . a &
b2 = F . b holds
for
f being
Morphism of
a,
b holds
(
f in <^a1,b1^> iff
F . f in <^a2,b2^> ) ) holds
B1,
B2 are_isomorphic_under F
theorem
for
A1,
A2 being
category for
F being
contravariant Functor of
A1,
A2 for
B1 being non
empty subcategory of
A1 for
B2 being non
empty subcategory of
A2 st
F is
bijective & ( for
a being
Object of
A1 holds
(
a is
Object of
B1 iff
F . a is
Object of
B2 ) ) & ( for
a,
b being
Object of
A1 st
<^a,b^> <> {} holds
for
a1,
b1 being
Object of
B1 st
a1 = a &
b1 = b holds
for
a2,
b2 being
Object of
B2 st
a2 = F . a &
b2 = F . b holds
for
f being
Morphism of
a,
b holds
(
f in <^a1,b1^> iff
F . f in <^b2,a2^> ) ) holds
B1,
B2 are_anti-isomorphic_under F