Lm1:
for n being Nat
for V being Subset of (TopSpaceMetr (Euclid n)) st V is open holds
for e being Point of (Euclid n) st e in V holds
ex r being Real st
( r > 0 & OpenHypercube (e,r) c= V )
Lm2:
for n being Nat
for p being Point of (TOP-REAL n)
for r being Real st r > 0 holds
( not cl_Ball (p,r) is boundary & cl_Ball (p,r) is compact )
theorem Th1:
for
N being non
zero Nat for
F being
Element of
N -tuples_on (Funcs ( the carrier of (TOP-REAL (N + 1)), the carrier of R^1)) st ( for
i being
Nat st
i in dom F holds
F . i = PROJ (
(N + 1),
i) ) holds
( ( for
t being
Point of
(TOP-REAL (N + 1)) holds
<:F:> . t = t | N ) & ( for
Sp,
Sn being
Subset of
(TOP-REAL (N + 1)) st
Sp = { u where u is Point of (TOP-REAL (N + 1)) : ( u . (N + 1) >= 0 & |.u.| = 1 ) } &
Sn = { t where t is Point of (TOP-REAL (N + 1)) : ( t . (N + 1) <= 0 & |.t.| = 1 ) } holds
(
<:F:> .: Sp = cl_Ball (
(0. (TOP-REAL N)),1) &
<:F:> .: Sn = cl_Ball (
(0. (TOP-REAL N)),1) &
<:F:> .: (Sp /\ Sn) = Sphere (
(0. (TOP-REAL N)),1) & ( for
H being
Function of
((TOP-REAL (N + 1)) | Sp),
(Tdisk ((0. (TOP-REAL N)),1)) st
H = <:F:> | Sp holds
H is
being_homeomorphism ) & ( for
H being
Function of
((TOP-REAL (N + 1)) | Sn),
(Tdisk ((0. (TOP-REAL N)),1)) st
H = <:F:> | Sn holds
H is
being_homeomorphism ) ) ) )
Lm3:
for n being Nat
for A, B being Subset of (TOP-REAL n) st n = 0 holds
for h being Function of ((TOP-REAL n) | A),((TOP-REAL n) | B) st h is being_homeomorphism holds
for p being Point of (TOP-REAL n) holds
( ( p in Fr A implies h . p in Fr B ) & ( p in Int A implies h . p in Int B ) )
theorem Th15:
for
n being
Nat for
p,
q being
Point of
(TOP-REAL n) for
r being
Real holds
(
(transl (p,(TOP-REAL n))) .: (Ball (q,r)) = Ball (
(q + p),
r) &
(transl (p,(TOP-REAL n))) .: (cl_Ball (q,r)) = cl_Ball (
(q + p),
r) &
(transl (p,(TOP-REAL n))) .: (Sphere (q,r)) = Sphere (
(q + p),
r) )
theorem Th16:
for
n being
Nat for
p being
Point of
(TOP-REAL n) for
r,
s being
Real st
s > 0 holds
(
(mlt (s,(TOP-REAL n))) .: (Ball (p,r)) = Ball (
(s * p),
(r * s)) &
(mlt (s,(TOP-REAL n))) .: (cl_Ball (p,r)) = cl_Ball (
(s * p),
(r * s)) &
(mlt (s,(TOP-REAL n))) .: (Sphere (p,r)) = Sphere (
(s * p),
(r * s)) )
Lm4:
for r being Real
for n being non zero Element of NAT
for p being Point of (TOP-REAL (n + 1)) st r <= 1 & |.p.| >= 1 & |.p.| < 1 + r & p . (n + 1) > 0 & p | n = 0* n holds
ex c being Real ex h being Function of ((TOP-REAL (n + 1)) | ((Sphere ((0. (TOP-REAL (n + 1))),1)) /\ (cl_Ball (p,r)))),(Tdisk ((0. (TOP-REAL n)),c)) st
( c > 0 & h is being_homeomorphism & h .: ((Sphere ((0. (TOP-REAL (n + 1))),1)) /\ (Sphere (p,r))) = Sphere ((0. (TOP-REAL n)),c) )