deffunc H1( set ) -> set = $1;
defpred S1[ set , set ] means $1 c= $2;
Lm3:
for r, s being Real
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 Nat 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)) ) ) ) )
definition
let r,
s be
Real;
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
;
existence
ex b1 being FinSequence of bool REAL st
( rng b1 c= F & union (rng b1) = [.r,s.] & ( for n being Nat 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 st
( r < p & p <= s & b1 . 1 = [.r,p.[ ) & ex p being Real st
( r <= p & p < s & b1 . (len b1) = ].p,s.] ) & ( for n being Nat st 1 < n & n < len b1 holds
ex p, q being Real 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
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 Nat 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 st
( r < p & p <= s & b4 . 1 = [.r,p.[ ) & ex p being Real st
( r <= p & p < s & b4 . (len b4) = ].p,s.] ) & ( for n being Nat st 1 < n & n < len b4 holds
ex p, q being Real st
( r <= p & p < q & q <= s & b4 . n = ].p,q.[ ) ) ) ) ) );