Lm1:
for n being Nat holds
( the carrier of (Euclid n) = REAL n & the carrier of (TOP-REAL n) = REAL n )
theorem Th2:
for
n being
Nat for
p1,
p2 being
Point of
(TOP-REAL n) for
r1,
r2 being
Real holds
( not
((1 - r1) * p1) + (r1 * p2) = ((1 - r2) * p1) + (r2 * p2) or
r1 = r2 or
p1 = p2 )
Lm2:
for n being Nat holds TOP-REAL n is pathwise_connected
Lm3:
for X being Subset of REAL st X is open holds
X in Family_open_set RealSpace
Lm4:
for X being Subset of REAL st X in Family_open_set RealSpace holds
X is open
Lm5:
for f being one-to-one continuous Function of R^1,R^1
for g being PartFunc of REAL,REAL holds
( not f = g or g | [.0,1.] is increasing or g | [.0,1.] is decreasing )
Lm6:
for a, b, c being Real st a <= b holds
( c in the carrier of (Closed-Interval-TSpace (a,b)) iff ( a <= c & c <= b ) )
Lm7:
for a, b, c, d being Real
for f being Function of (Closed-Interval-TSpace (a,b)),(Closed-Interval-TSpace (c,d))
for x being Point of (Closed-Interval-TSpace (a,b))
for g being PartFunc of REAL,REAL
for x1 being Real st a < b & c < d & f is_continuous_at x & x <> a & x <> b & f . a = c & f . b = d & f is one-to-one & f = g & x = x1 holds
g is_continuous_in x1
theorem Th13:
for
a,
b,
c,
d,
x1 being
Real for
f being
Function of
(Closed-Interval-TSpace (a,b)),
(Closed-Interval-TSpace (c,d)) for
x being
Point of
(Closed-Interval-TSpace (a,b)) for
g being
PartFunc of
REAL,
REAL st
a < b &
c < d &
f is_continuous_at x &
f . a = c &
f . b = d &
f is
one-to-one &
f = g &
x = x1 holds
g | [.a,b.] is_continuous_in x1
theorem Th15:
for
a,
b,
c,
d being
Real for
f being
Function of
(Closed-Interval-TSpace (a,b)),
(Closed-Interval-TSpace (c,d)) st
a < b &
c < d &
f is
continuous &
f is
one-to-one &
f . a = c &
f . b = d holds
for
x,
y being
Point of
(Closed-Interval-TSpace (a,b)) for
p,
q,
fx,
fy being
Real st
x = p &
y = q &
p < q &
fx = f . x &
fy = f . y holds
fx < fy
theorem
for
a,
b,
c,
d,
e,
f,
g,
h being
Real for
F being
Function of
(Closed-Interval-TSpace (a,b)),
(Closed-Interval-TSpace (c,d)) st
a < b &
c < d &
e < f &
a <= e &
f <= b &
F is
being_homeomorphism &
F . a = c &
F . b = d &
g = F . e &
h = F . f holds
F .: [.e,f.] = [.g,h.]
Lm8:
R^1 = TopStruct(# the carrier of RealSpace,(Family_open_set RealSpace) #)
by PCOMPS_1:def 5, TOPMETR:def 6;