]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/matita/library/nat/compare.ma
added a function to reorder the metasenv.
[helm.git] / helm / matita / library / nat / compare.ma
index 194b38d84f255e3924a3273919f01bb96d320ca5..443c6657f9085642d307a9f1b123a22546e11074 100644 (file)
@@ -14,9 +14,9 @@
 
 set "baseuri" "cic:/matita/nat/compare".
 
-include "nat/orders.ma".
 include "datatypes/bool.ma".
 include "datatypes/compare.ma".
+include "nat/orders.ma".
 
 let rec eqb n m \def 
 match n with 
@@ -154,8 +154,8 @@ simplify.apply le_S_S.apply le_O_n.
 intro.simplify.apply le_S_S. apply le_O_n.
 intros 2.simplify.elim (nat_compare n1 m1).
 simplify. apply le_S_S.apply H.
-simplify. apply le_S_S.apply H.
 simplify. apply eq_f. apply H.
+simplify. apply le_S_S.apply H.
 qed.
 
 theorem nat_compare_n_m_m_n: \forall n,m:nat. 
@@ -181,6 +181,6 @@ cut match (nat_compare n m) with
 apply Hcut.apply nat_compare_to_Prop.
 elim (nat_compare n m).
 apply (H H3).
-apply (H2 H3).
 apply (H1 H3).
+apply (H2 H3).
 qed.