theorem Th10:
for
a,
b,
c,
d being
object st
a <> b holds
(
a,
b)
--> (
c,
d)
= (
b,
a)
--> (
d,
c)
Lm1:
for f being Function st rng f = {{}} holds
product f = {}
Lm2:
for I being 2 -element set
for f being ManySortedSet of I
for i, j being Element of I
for x being object st i <> j holds
f +* (i,x) = (i,j) --> (x,(f . j))
Lm3:
for I being non empty set
for J being non-Empty TopSpace-yielding ManySortedSet of I
for P being Subset of (product (Carrier J)) st P in FinMeetCl (product_prebasis J) holds
ex X being Subset-Family of (product (Carrier J)) ex f being b1 -valued one-to-one Function st
( X c= product_prebasis J & X is finite & P = Intersect X & dom f = X & P = product ((Carrier J) +* (product_basis_selector (J,f))) )
Lm4:
for I being 1 -element set
for J being non-Empty TopSpace-yielding ManySortedSet of I
for i being Element of I
for P being Subset of (product (Carrier J)) st P in FinMeetCl (product_prebasis J) holds
ex V being Subset of (J . i) st
( V is open & P = product ({i} --> V) )
Lm5:
for I being 1 -element set
for J being non-Empty TopSpace-yielding ManySortedSet of I
for i being Element of I
for P being Subset of (product (Carrier J)) holds
( P in FinMeetCl (product_prebasis J) iff ex V being Subset of (J . i) st
( V is open & P = product ({i} --> V) ) )
Lm6:
for I being 1 -element set
for J being non-Empty TopSpace-yielding ManySortedSet of I
for i being Element of I
for P being Subset of (product (Carrier J)) holds
( P in UniCl (FinMeetCl (product_prebasis J)) iff ex V being Subset of (J . i) st
( V is open & P = product ({i} --> V) ) )
Lm7:
for I being 1 -element set
for J being non-Empty TopSpace-yielding ManySortedSet of I holds UniCl (FinMeetCl (product_prebasis J)) = product_prebasis J
Lm8:
for I being 2 -element set
for J being non-Empty TopSpace-yielding ManySortedSet of I
for i, j being Element of I
for P being Subset of (product (Carrier J)) holds
( not i <> j or not P in product_prebasis J or ex V being Subset of (J . i) st
( V is open & P = product ((i,j) --> (V,([#] (J . j)))) ) or ex W being Subset of (J . j) st
( W is open & P = product ((i,j) --> (([#] (J . i)),W)) ) )
Lm9:
for I being 2 -element set
for J being non-Empty TopSpace-yielding ManySortedSet of I
for i, j being Element of I
for P being Subset of (product (Carrier J)) st i <> j & P in FinMeetCl (product_prebasis J) holds
ex V being Subset of (J . i) ex W being Subset of (J . j) st
( V is open & W is open & P = product ((i,j) --> (V,W)) )
:: compare FUNCT_1:4