]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/contribs/dama/dama/lebesgue.ma
Snapshot.
[helm.git] / helm / software / matita / contribs / dama / dama / lebesgue.ma
index e1fbd0a5a75cac9f840d207833e3319214680224..d0fcae691b5acd7fe38626411d1e70b87afd1690 100644 (file)
@@ -38,7 +38,7 @@ cases (H3 j); clear H3; cases H2; cases H7; clear H2 H7;
 intro H2; cases (H10 ? H2);
 cases (H (w1+j)); apply (H11 H7);
 qed.   
-     
+          
 (* Theorem 3.10 *)
 theorem lebesgue_oc:
   ∀C:ordered_uniform_space.
@@ -65,10 +65,10 @@ split;
     [1: apply (le_transitive ???? (H8 0)); cases (Hyi 0); assumption
     |2: apply (le_transitive ????? (H4 0)); cases (Hxi 0); assumption]
 |2: intros 3 (h);
-    letin Xi ≝ (⌊n,≪xi n,Hxi n≫⌋);
-    letin Yi ≝ (⌊n,≪yi n,Hyi n≫⌋);
-    letin Ai ≝ (⌊n,≪a n,H1 n≫⌋);
-    apply (sandwich {[l,u]} ≪?,h≫ Xi Yi Ai); try assumption;
+    letin Xi ≝ (⌊n,≪xi n, Hxi n≫⌋);
+    letin Yi ≝ (⌊n,≪yi n, Hyi n≫⌋);
+    letin Ai ≝ (⌊n,≪a n, H1 n≫⌋);
+    apply (sandwich {[l,u]} ≪?, h≫ Xi Yi Ai); try assumption;
     [1: intro j; cases (Hxy j); cases H3; cases H4; split;
         [apply (H5 0);|apply (H7 0)]
     |2: cases (H l u Xi ≪?,h≫) (Ux Uy); apply Ux; cases Hx; split; [apply H3;]
@@ -108,10 +108,10 @@ split;
 |2: intros 3;
     lapply (uparrow_upperlocated ? xi x Hx)as Ux;
     lapply (downarrow_lowerlocated ? yi x Hy)as Uy;
-    letin Xi ≝ (⌊n,≪xi n,Hxi n≫⌋);
-    letin Yi ≝ (⌊n,≪yi n,Hyi n≫⌋);
-    letin Ai ≝ (⌊n,≪a n,H1 n≫⌋);
-    apply (sandwich {[l,u]} ≪x,h≫ Xi Yi Ai); try assumption;
+    letin Xi ≝ (⌊n,≪xi n, Hxi n≫⌋);
+    letin Yi ≝ (⌊n,≪yi n, Hyi n≫⌋);
+    letin Ai ≝ (⌊n,≪a n, H1 n≫⌋);
+    apply (sandwich {[l,u]} ≪?, h≫ Xi Yi Ai); try assumption;
     [1: intro j; cases (Hxy j); cases H3; cases H4; split;
         [apply (H5 0);|apply (H7 0)]
     |2: cases (restrict_uniform_convergence_uparrow ? S ?? (H l u) Xi x Hx);