]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/library/nat/orders.ma
Move to OCaml 3.10. Requires debian packages from unstable (soon in testing).
[helm.git] / matita / library / nat / orders.ma
index 8053d50de55bfe8afc7d434243b17ceca34b9536..42454393ca45cc08676ef8205d878a437a1266f2 100644 (file)
@@ -100,6 +100,12 @@ theorem lt_S_S_to_lt: \forall n,m.
 intros. apply le_S_S_to_le. assumption.
 qed.
 
+theorem lt_to_lt_S_S: ∀n,m. n < m → S n < S m.
+intros;
+unfold lt in H;
+apply (le_S_S ? ? H).
+qed.
+
 theorem leS_to_not_zero : \forall n,m:nat. S n \leq m \to not_zero m.
 intros.elim H.exact I.exact I.
 qed.