theorem Th2:
for
r1,
r2,
r3,
r4,
r5,
r6 being
Real st
r1 < r2 &
r3 <= r4 &
r5 < r6 holds
(L[01] (r1,r2,r3,r4)) * (L[01] (r5,r6,r1,r2)) = L[01] (
r5,
r6,
r3,
r4)
theorem Th6:
for
T being non
empty TopSpace for
S being non
empty SubSpace of
T for
t1,
t2 being
Point of
T for
s1,
s2 being
Point of
S for
A,
B being
Path of
t1,
t2 for
C,
D being
Path of
s1,
s2 st
s1,
s2 are_connected &
t1,
t2 are_connected &
A = C &
B = D &
C,
D are_homotopic holds
A,
B are_homotopic
theorem
for
T being non
empty TopSpace for
S being non
empty SubSpace of
T for
t1,
t2 being
Point of
T for
s1,
s2 being
Point of
S for
A,
B being
Path of
t1,
t2 for
C,
D being
Path of
s1,
s2 st
s1,
s2 are_connected &
t1,
t2 are_connected &
A = C &
B = D &
Class (
(EqRel (S,s1,s2)),
C)
= Class (
(EqRel (S,s1,s2)),
D) holds
Class (
(EqRel (T,t1,t2)),
A)
= Class (
(EqRel (T,t1,t2)),
B)
theorem Th12:
for
T being non
empty TopSpace holds
(
T is
simply_connected iff for
t1,
t2 being
Point of
T holds
(
t1,
t2 are_connected & ( for
P,
Q being
Path of
t1,
t2 holds
Class (
(EqRel (T,t1,t2)),
P)
= Class (
(EqRel (T,t1,t2)),
Q) ) ) )
Lm1:
for T being TopStruct
for f being PartFunc of R^1,T st f = {} holds
f is parametrized-curve
definition
let T be non
empty TopStruct ;
let c1,
c2 be
with_endpoints Curve of
T;
pred c1,
c2 are_homotopic means
ex
a,
b being
Point of
T ex
p1,
p2 being
Path of
a,
b st
(
p1 = c1 * (L[01] (0,1,(inf (dom c1)),(sup (dom c1)))) &
p2 = c2 * (L[01] (0,1,(inf (dom c2)),(sup (dom c2)))) &
p1,
p2 are_homotopic );
symmetry
for c1, c2 being with_endpoints Curve of T st ex a, b being Point of T ex p1, p2 being Path of a,b st
( p1 = c1 * (L[01] (0,1,(inf (dom c1)),(sup (dom c1)))) & p2 = c2 * (L[01] (0,1,(inf (dom c2)),(sup (dom c2)))) & p1,p2 are_homotopic ) holds
ex a, b being Point of T ex p1, p2 being Path of a,b st
( p1 = c2 * (L[01] (0,1,(inf (dom c2)),(sup (dom c2)))) & p2 = c1 * (L[01] (0,1,(inf (dom c1)),(sup (dom c1)))) & p1,p2 are_homotopic )
;
end;
::
deftheorem defines
are_homotopic TOPALG_6:def 11 :
for T being non empty TopStruct
for c1, c2 being with_endpoints Curve of T holds
( c1,c2 are_homotopic iff ex a, b being Point of T ex p1, p2 being Path of a,b st
( p1 = c1 * (L[01] (0,1,(inf (dom c1)),(sup (dom c1)))) & p2 = c2 * (L[01] (0,1,(inf (dom c2)),(sup (dom c2)))) & p1,p2 are_homotopic ) );
Lm2:
for T being non empty TopStruct
for f1, f2 being FinSequence of Curves T holds (Partial_Sums (f1 ^ f2)) . (len f1) = (Partial_Sums f1) . (len f1)
Lm3:
for n being Nat
for t being Point of (TUnitSphere n)
for f being Loop of t st rng f <> the carrier of (TUnitSphere n) holds
f is nullhomotopic
Lm4:
for n being Nat
for t being Point of (TUnitSphere n)
for f being Loop of t st n >= 2 & rng f = the carrier of (TUnitSphere n) holds
ex g being Loop of t st
( g,f are_homotopic & rng g <> the carrier of (TUnitSphere n) )