Lm1:
dom proj2 = the carrier of (TOP-REAL 2)
by FUNCT_2:def 1;
Lm2:
for r being Real
for X being Subset of (TOP-REAL 2) st r in proj2 .: X holds
ex x being Point of (TOP-REAL 2) st
( x in X & proj2 . x = r )
Lm3:
now for a, A, B, C being set holds
( not a in (A \/ B) \/ C or a in A or a in B or a in C )
end;
Lm4:
for A, B, C, D being set st A misses D & B misses D & C misses D holds
(A \/ B) \/ C misses D
theorem Th11:
for
P being
Subset of the
carrier of
(TOP-REAL 2) for
p1,
p2,
q1,
q2 being
Point of
(TOP-REAL 2) st
P is_an_arc_of p1,
p2 &
p1 <> q1 &
p2 <> q2 holds
( not
p1 in Segment (
P,
p1,
p2,
q1,
q2) & not
p2 in Segment (
P,
p1,
p2,
q1,
q2) )