Lm1:
now for S, T, x1, x2 being set st x1 in S & x2 in T holds
<:(pr2 (S,T)),(pr1 (S,T)):> . (x1,x2) = [x2,x1]
let S,
T,
x1,
x2 be
set ;
( x1 in S & x2 in T implies <:(pr2 (S,T)),(pr1 (S,T)):> . (x1,x2) = [x2,x1] )assume A1:
(
x1 in S &
x2 in T )
;
<:(pr2 (S,T)),(pr1 (S,T)):> . (x1,x2) = [x2,x1]A2:
dom <:(pr2 (S,T)),(pr1 (S,T)):> =
(dom (pr2 (S,T))) /\ (dom (pr1 (S,T)))
by FUNCT_3:def 7
.=
(dom (pr2 (S,T))) /\ [:S,T:]
by FUNCT_3:def 4
.=
[:S,T:] /\ [:S,T:]
by FUNCT_3:def 5
.=
[:S,T:]
;
[x1,x2] in [:S,T:]
by A1, ZFMISC_1:87;
hence <:(pr2 (S,T)),(pr1 (S,T)):> . (
x1,
x2) =
[((pr2 (S,T)) . (x1,x2)),((pr1 (S,T)) . (x1,x2))]
by A2, FUNCT_3:def 7
.=
[x2,((pr1 (S,T)) . (x1,x2))]
by A1, FUNCT_3:def 5
.=
[x2,x1]
by A1, FUNCT_3:def 4
;
verum
end;
theorem Th48:
for
S1,
S2,
T1,
T2 being non
empty TopSpace for
R being
Refinement of
[:S1,T1:],
[:S2,T2:] st the
carrier of
S1 = the
carrier of
S2 & the
carrier of
T1 = the
carrier of
T2 holds
{ ([:U1,V1:] /\ [:U2,V2:]) where U1 is Subset of S1, U2 is Subset of S2, V1 is Subset of T1, V2 is Subset of T2 : ( U1 is open & U2 is open & V1 is open & V2 is open ) } is
Basis of
R
theorem Th49:
for
S1,
S2,
T1,
T2 being non
empty TopSpace for
R being
Refinement of
[:S1,T1:],
[:S2,T2:] for
R1 being
Refinement of
S1,
S2 for
R2 being
Refinement of
T1,
T2 st the
carrier of
S1 = the
carrier of
S2 & the
carrier of
T1 = the
carrier of
T2 holds
( the
carrier of
[:R1,R2:] = the
carrier of
R & the
topology of
[:R1,R2:] = the
topology of
R )