theorem Th1:
for
i being
Nat st
i > 0 holds
ex
n,
m being
Nat st
i = (2 |^ n) * ((2 * m) + 1)
definition
existence
ex b1 being Function of [:NAT,NAT:],NAT st
for n, m being Nat holds b1 . [n,m] = ((2 |^ n) * ((2 * m) + 1)) - 1
uniqueness
for b1, b2 being Function of [:NAT,NAT:],NAT st ( for n, m being Nat holds b1 . [n,m] = ((2 |^ n) * ((2 * m) + 1)) - 1 ) & ( for n, m being Nat holds b2 . [n,m] = ((2 |^ n) * ((2 * m) + 1)) - 1 ) holds
b1 = b2
end;
Lm1:
for X being non empty set
for f being Function of [:X,X:],REAL st f is_a_pseudometric_of X holds
( f is bounded_below & ( for A being non empty Subset of X
for x being Element of X holds
( not (dist (f,x)) .: A is empty & (dist (f,x)) .: A is bounded_below ) ) )
theorem Th15:
for
T being non
empty TopSpace for
s being
Real for
FS2 being
Functional_Sequence of
[: the carrier of T, the carrier of T:],
REAL st ( for
n being
Nat ex
pmet being
Function of
[: the carrier of T, the carrier of T:],
REAL st
(
FS2 . n = pmet &
pmet is_a_pseudometric_of the
carrier of
T & ( for
pq being
Element of
[: the carrier of T, the carrier of T:] holds
pmet . pq <= s ) & ( for
pmet9 being
RealMap of
[:T,T:] st
pmet = pmet9 holds
pmet9 is
continuous ) ) ) holds
for
pmet being
Function of
[: the carrier of T, the carrier of T:],
REAL st ( for
pq being
Element of
[: the carrier of T, the carrier of T:] holds
pmet . pq = Sum (((1 / 2) GeoSeq) (#) (FS2 # pq)) ) holds
(
pmet is_a_pseudometric_of the
carrier of
T & ( for
pmet9 being
RealMap of
[:T,T:] st
pmet = pmet9 holds
pmet9 is
continuous ) )
theorem Th17:
for
T being non
empty TopSpace st
T is
T_1 holds
for
s being
Real for
FS2 being
Functional_Sequence of
[: the carrier of T, the carrier of T:],
REAL st ( for
n being
Nat ex
pmet being
Function of
[: the carrier of T, the carrier of T:],
REAL st
(
FS2 . n = pmet &
pmet is_a_pseudometric_of the
carrier of
T & ( for
pq being
Element of
[: the carrier of T, the carrier of T:] holds
pmet . pq <= s ) & ( for
pmet9 being
RealMap of
[:T,T:] st
pmet = pmet9 holds
pmet9 is
continuous ) ) ) & ( for
p being
Point of
T for
A9 being non
empty Subset of
T st not
p in A9 &
A9 is
closed holds
ex
n being
Nat st
for
pmet being
Function of
[: the carrier of T, the carrier of T:],
REAL st
FS2 . n = pmet holds
(lower_bound (pmet,A9)) . p > 0 ) holds
( ex
pmet being
Function of
[: the carrier of T, the carrier of T:],
REAL st
(
pmet is_metric_of the
carrier of
T & ( for
pq being
Element of
[: the carrier of T, the carrier of T:] holds
pmet . pq = Sum (((1 / 2) GeoSeq) (#) (FS2 # pq)) ) ) &
T is
metrizable )
Lm2:
PairFunc " = PairFunc "
by Th2, TOPS_2:def 4;
reconsider jj = 1 as Real ;