begin
theorem Th1:
theorem Th2:
theorem Th3:
begin
theorem Th4:
theorem Th5:
theorem Th6:
theorem Th7:
begin
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem
canceled;
theorem Th20:
theorem Th21:
theorem Th22:
theorem Th23:
theorem Th24:
begin
theorem Th25:
theorem Th26:
theorem Th27:
theorem Th28:
theorem Th29:
theorem Th30:
theorem Th31:
theorem Th32:
theorem Th33:
theorem Th34:
theorem Th35:
theorem Th36:
theorem Th37:
theorem Th38:
theorem Th39:
theorem Th40:
theorem Th41:
theorem Th42:
theorem Th43:
begin
theorem Th44:
theorem
theorem Th46:
theorem Th47:
theorem
theorem
theorem Th50:
theorem Th51:
begin
theorem
canceled;
theorem
theorem Th54:
theorem Th55:
theorem Th56:
theorem Th57:
begin
deffunc H1( set ) -> set = $1;
defpred S1[ set , set ] means $1 c= $2;
theorem
canceled;
theorem Th59:
theorem Th60:
:: deftheorem Def1 defines connected RCOMP_3:def 1 :
for T being TopStruct
for F being Subset-Family of T holds
( F is connected iff for X being Subset of T st X in F holds
X is connected );
Lm3:
for r, s being real number
for F being Subset-Family of (Closed-Interval-TSpace (r,s)) st [.r,s.] in F & r <= s holds
( rng <*[.r,s.]*> c= F & union (rng <*[.r,s.]*>) = [.r,s.] & ( for n being natural number st 1 <= n holds
( ( n <= len <*[.r,s.]*> implies not <*[.r,s.]*> /. n is empty ) & ( n + 1 <= len <*[.r,s.]*> implies ( lower_bound (<*[.r,s.]*> /. n) <= lower_bound (<*[.r,s.]*> /. (n + 1)) & upper_bound (<*[.r,s.]*> /. n) <= upper_bound (<*[.r,s.]*> /. (n + 1)) & lower_bound (<*[.r,s.]*> /. (n + 1)) < upper_bound (<*[.r,s.]*> /. n) ) ) & ( n + 2 <= len <*[.r,s.]*> implies upper_bound (<*[.r,s.]*> /. n) <= lower_bound (<*[.r,s.]*> /. (n + 2)) ) ) ) )
theorem Th61:
theorem Th62:
definition
let r,
s be
real number ;
let F be
Subset-Family of
(Closed-Interval-TSpace (r,s));
assume that A1:
F is
Cover of
(Closed-Interval-TSpace (r,s))
and A2:
F is
open
and A3:
F is
connected
and A4:
r <= s
;
mode IntervalCover of
F -> FinSequence of
bool REAL means :
Def2:
(
rng it c= F &
union (rng it) = [.r,s.] & ( for
n being
natural number st 1
<= n holds
( (
n <= len it implies not
it /. n is
empty ) & (
n + 1
<= len it implies (
lower_bound (it /. n) <= lower_bound (it /. (n + 1)) &
upper_bound (it /. n) <= upper_bound (it /. (n + 1)) &
lower_bound (it /. (n + 1)) < upper_bound (it /. n) ) ) & (
n + 2
<= len it implies
upper_bound (it /. n) <= lower_bound (it /. (n + 2)) ) ) ) & (
[.r,s.] in F implies
it = <*[.r,s.]*> ) & ( not
[.r,s.] in F implies ( ex
p being
real number st
(
r < p &
p <= s &
it . 1
= [.r,p.[ ) & ex
p being
real number st
(
r <= p &
p < s &
it . (len it) = ].p,s.] ) & ( for
n being
natural number st 1
< n &
n < len it holds
ex
p,
q being
real number st
(
r <= p &
p < q &
q <= s &
it . n = ].p,q.[ ) ) ) ) );
existence
ex b1 being FinSequence of bool REAL st
( rng b1 c= F & union (rng b1) = [.r,s.] & ( for n being natural number st 1 <= n holds
( ( n <= len b1 implies not b1 /. n is empty ) & ( n + 1 <= len b1 implies ( lower_bound (b1 /. n) <= lower_bound (b1 /. (n + 1)) & upper_bound (b1 /. n) <= upper_bound (b1 /. (n + 1)) & lower_bound (b1 /. (n + 1)) < upper_bound (b1 /. n) ) ) & ( n + 2 <= len b1 implies upper_bound (b1 /. n) <= lower_bound (b1 /. (n + 2)) ) ) ) & ( [.r,s.] in F implies b1 = <*[.r,s.]*> ) & ( not [.r,s.] in F implies ( ex p being real number st
( r < p & p <= s & b1 . 1 = [.r,p.[ ) & ex p being real number st
( r <= p & p < s & b1 . (len b1) = ].p,s.] ) & ( for n being natural number st 1 < n & n < len b1 holds
ex p, q being real number st
( r <= p & p < q & q <= s & b1 . n = ].p,q.[ ) ) ) ) )
end;
:: deftheorem Def2 defines IntervalCover RCOMP_3:def 2 :
for r, s being real number
for F being Subset-Family of (Closed-Interval-TSpace (r,s)) st F is Cover of (Closed-Interval-TSpace (r,s)) & F is open & F is connected & r <= s holds
for b4 being FinSequence of bool REAL holds
( b4 is IntervalCover of F iff ( rng b4 c= F & union (rng b4) = [.r,s.] & ( for n being natural number st 1 <= n holds
( ( n <= len b4 implies not b4 /. n is empty ) & ( n + 1 <= len b4 implies ( lower_bound (b4 /. n) <= lower_bound (b4 /. (n + 1)) & upper_bound (b4 /. n) <= upper_bound (b4 /. (n + 1)) & lower_bound (b4 /. (n + 1)) < upper_bound (b4 /. n) ) ) & ( n + 2 <= len b4 implies upper_bound (b4 /. n) <= lower_bound (b4 /. (n + 2)) ) ) ) & ( [.r,s.] in F implies b4 = <*[.r,s.]*> ) & ( not [.r,s.] in F implies ( ex p being real number st
( r < p & p <= s & b4 . 1 = [.r,p.[ ) & ex p being real number st
( r <= p & p < s & b4 . (len b4) = ].p,s.] ) & ( for n being natural number st 1 < n & n < len b4 holds
ex p, q being real number st
( r <= p & p < q & q <= s & b4 . n = ].p,q.[ ) ) ) ) ) );
theorem
theorem Th64:
theorem Th65:
theorem Th66:
theorem
theorem
theorem Th69:
theorem
theorem Th71:
theorem
theorem Th73:
:: deftheorem Def3 defines IntervalCoverPts RCOMP_3:def 3 :
for r, s being real number
for F being Subset-Family of (Closed-Interval-TSpace (r,s))
for C being IntervalCover of F st F is Cover of (Closed-Interval-TSpace (r,s)) & F is open & F is connected & r <= s holds
for b5 being FinSequence of REAL holds
( b5 is IntervalCoverPts of C iff ( len b5 = (len C) + 1 & b5 . 1 = r & b5 . (len b5) = s & ( for n being natural number st 1 <= n & n + 1 < len b5 holds
b5 . (n + 1) in ].(lower_bound (C /. (n + 1))),(upper_bound (C /. n)).[ ) ) );
theorem Th74:
theorem Th75:
theorem Th76:
theorem Th77:
theorem Th78:
theorem Th79:
theorem