(**************************************************************************)
include "ordered_uniform.ma".
+include "property_sigma.ma".
(* Definition 3.7 *)
-definition exhaustivity ≝
+definition exhaustive ≝
λC:ordered_uniform_space.
∀a,b:sequence C.
(a is_increasing → a is_upper_located → a is_cauchy) ∧
(b is_decreasing → b is_lower_located → b is_cauchy).
(* Lemma 3.8 *)
+lemma xxx:
+ ∀C:ordered_uniform_space.property_sigma C →
+ ∀l,u:C.exhaustive {[l,u]} →
+ ∀a:sequence {[l,u]}.∀x:C. (λn.fst (a n)) ↑ x →
+ x∈[l,u] ∧ ∀h:x ∈ [l,u].a uniform_converges (sig_in ?? x h).
+intros; split;
+[1: (* manca fact 2.5 *)
+
+
\ No newline at end of file