]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambda_delta/Ground_2/arith.ma
- first properties of strongly normalizing terms
[helm.git] / matita / matita / contribs / lambda_delta / Ground_2 / arith.ma
index 418a176d5024ab7e8190c2c3220d7e45c1b3d0b2..39d28c959182d17c31fa4a851751928c3fc12b8d 100644 (file)
@@ -17,7 +17,7 @@ include "Ground_2/star.ma".
 
 (* ARITHMETICAL PROPERTIES **************************************************)
 
-(* equations ****************************************************************)
+(* Equations ****************************************************************)
 
 lemma le_plus_minus: ∀m,n,p. p ≤ n → m + n - p = m + (n - p).
 /2 by plus_minus/ qed.
@@ -69,4 +69,8 @@ qed-.
 (*
 lemma pippo: ∀x,y,z. x < z → y < z - x → x + y < z.
 /3 width=2/
+
+lemma le_or_ge: ∀m,n. m ≤ n ∨ n ≤ m.
+#m #n elim (lt_or_ge m n) /2 width=1/ /3 width=2/
+qed-.
 *)