]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/contribs/dama/dama/supremum.ma
ordered_set simplified
[helm.git] / helm / software / matita / contribs / dama / dama / supremum.ma
index e3a83a09a4f5d2d72646ee2a360b65ef82c03f90..ca422597d5a9c7a98c8b5b18d9080294ab5c1eb9 100644 (file)
@@ -202,10 +202,10 @@ record segment (O : Type) : Type â‰ {
    seg_u_ : O
 }.
 
-notation > "𝕦_term 90 s" non associative with precedence 45 for @{'upp $s}.
-notation "𝕦 \sub term 90 s" non associative with precedence 45 for @{'upp $s}. 
-notation > "𝕝_term 90 s" non associative with precedence 45 for @{'low $s}.
-notation "𝕝 \sub term 90 s" non associative with precedence 45 for @{'low $s}. 
+notation > "𝕦_term 90 s" non associative with precedence 90 for @{'upp $s}.
+notation "𝕦 \sub term 90 s" non associative with precedence 90 for @{'upp $s}. 
+notation > "𝕝_term 90 s" non associative with precedence 90 for @{'low $s}.
+notation "𝕝 \sub term 90 s" non associative with precedence 90 for @{'low $s}. 
  
 definition seg_u â‰
  ÎťO:half_ordered_set.Îťs:segment O.
@@ -340,6 +340,18 @@ whd in âŠ˘ (? (% ? ?) ?? ? ? ? â†’ ?); simplify in âŠ˘ (% â†’ ?);
 cases (wloss_prop O) (E E); do 2 rewrite < E; intros; assumption;
 qed.
 
+lemma l2sl:
+  âˆ€C,s.∀x,y:half_segment_ordered_set C s. \fst x â‰¤â‰¤ \fst y â†’ x â‰¤â‰¤ y.
+intros; intro; apply H; apply sx2x; apply H1;
+qed.
+
+
+lemma sl2l:
+  âˆ€C,s.∀x,y:half_segment_ordered_set C s. x â‰¤â‰¤ y â†’ \fst x â‰¤â‰¤ \fst y.
+intros; intro; apply H; apply x2sx; apply H1;
+qed.
+
+
 lemma h_segment_preserves_supremum:
   âˆ€O:half_ordered_set.∀s:segment O.
    âˆ€a:sequence (half_segment_ordered_set ? s).