Lm1:
for S, T being non empty MetrSpace
for f being Function of (TopSpaceMetr S),(TopSpaceMetr T) st TopSpaceMetr S is compact holds
( f is continuous iff for e being Real st 0 < e holds
ex d being Real st
( 0 < d & ( for x1, x2 being Point of S st dist (x1,x2) < d holds
dist ((In ((f /. x1),T)),(In ((f /. x2),T))) < e ) ) )
Lm2:
for S, T being non empty MetrSpace
for F being Subset of (Funcs ( the carrier of S, the carrier of T)) st TopSpaceMetr S is compact holds
( F is equicontinuous iff for x being Point of S holds F is_equicontinuous_at x )
theorem Th10:
for
S being non
empty TopSpace for
T being non
empty MetrSpace ex
F being
Function of
[:(ContinuousFunctions (S,T)),(ContinuousFunctions (S,T)):],
REAL st
for
f,
g being
Function of
S,
(TopSpaceMetr T) st
f in ContinuousFunctions (
S,
T) &
g in ContinuousFunctions (
S,
T) holds
ex
Dist being
RealMap of
S st
( ( for
x being
Point of
S holds
Dist . x = dist (
(In ((f . x),T)),
(In ((g . x),T))) ) &
F . (
f,
g)
= upper_bound (rng Dist) )
definition
let S be non
empty TopSpace;
let T be non
empty MetrSpace;
func dist_Func (
S,
T)
-> Function of
[:(ContinuousFunctions (S,T)),(ContinuousFunctions (S,T)):],
REAL means :
Def5:
for
f,
g being
Function of
S,
(TopSpaceMetr T) st
f in ContinuousFunctions (
S,
T) &
g in ContinuousFunctions (
S,
T) holds
ex
Dist being
RealMap of
S st
( ( for
x being
Point of
S holds
Dist . x = dist (
(In ((f . x),T)),
(In ((g . x),T))) ) &
it . (
f,
g)
= upper_bound (rng Dist) );
existence
ex b1 being Function of [:(ContinuousFunctions (S,T)),(ContinuousFunctions (S,T)):],REAL st
for f, g being Function of S,(TopSpaceMetr T) st f in ContinuousFunctions (S,T) & g in ContinuousFunctions (S,T) holds
ex Dist being RealMap of S st
( ( for x being Point of S holds Dist . x = dist ((In ((f . x),T)),(In ((g . x),T))) ) & b1 . (f,g) = upper_bound (rng Dist) )
by Th10;
uniqueness
for b1, b2 being Function of [:(ContinuousFunctions (S,T)),(ContinuousFunctions (S,T)):],REAL st ( for f, g being Function of S,(TopSpaceMetr T) st f in ContinuousFunctions (S,T) & g in ContinuousFunctions (S,T) holds
ex Dist being RealMap of S st
( ( for x being Point of S holds Dist . x = dist ((In ((f . x),T)),(In ((g . x),T))) ) & b1 . (f,g) = upper_bound (rng Dist) ) ) & ( for f, g being Function of S,(TopSpaceMetr T) st f in ContinuousFunctions (S,T) & g in ContinuousFunctions (S,T) holds
ex Dist being RealMap of S st
( ( for x being Point of S holds Dist . x = dist ((In ((f . x),T)),(In ((g . x),T))) ) & b2 . (f,g) = upper_bound (rng Dist) ) ) holds
b1 = b2
end;
::
deftheorem Def5 defines
dist_Func ASCOLI2:def 5 :
for S being non empty TopSpace
for T being non empty MetrSpace
for b3 being Function of [:(ContinuousFunctions (S,T)),(ContinuousFunctions (S,T)):],REAL holds
( b3 = dist_Func (S,T) iff for f, g being Function of S,(TopSpaceMetr T) st f in ContinuousFunctions (S,T) & g in ContinuousFunctions (S,T) holds
ex Dist being RealMap of S st
( ( for x being Point of S holds Dist . x = dist ((In ((f . x),T)),(In ((g . x),T))) ) & b3 . (f,g) = upper_bound (rng Dist) ) );
Lm3:
for S being non empty compact TopSpace
for T being non empty MetrSpace holds
( MetricSpace_of_ContinuousFunctions (S,T) is Reflexive & MetricSpace_of_ContinuousFunctions (S,T) is discerning & MetricSpace_of_ContinuousFunctions (S,T) is symmetric & MetricSpace_of_ContinuousFunctions (S,T) is triangle )