]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/contribs/dama/dama/nat_ordered_set.ma
bla bla bla
[helm.git] / helm / software / matita / contribs / dama / dama / nat_ordered_set.ma
index e7dfec46152d1ef9cb32951cc9e7a4df2bfc8f4e..6ecbe5424fc8810ab201dce248fd45520e96c90d 100644 (file)
@@ -15,7 +15,7 @@
 include "ordered_set.ma".
 
 include "nat/compare.ma".
-include "cprop_connectives.ma".
+include "cprop_connectives.ma". 
 
 definition nat_excess : nat → nat → CProp ≝ λn,m. m<n.
 
@@ -49,3 +49,15 @@ apply (mk_ordered_set ? nat_excess);
 [1: intro x; intro; apply (not_le_Sn_n ? H);
 |2: apply nat_excess_cotransitive]
 qed.
+
+alias id "le" = "cic:/matita/dama/ordered_set/le.con".
+lemma os_le_to_nat_le:
+  ∀a,b:nat_ordered_set.le nat_ordered_set a b → a ≤ b.
+intros; normalize in H; apply (not_lt_to_le ?? H);
+qed.
+lemma nat_le_to_os_le:
+  ∀a,b:nat_ordered_set.a ≤ b → le nat_ordered_set a b.
+intros 3; apply (le_to_not_lt a b);assumption;
+qed.
+  
\ No newline at end of file