diff options
author | herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2003-06-14 06:45:20 +0000 |
---|---|---|
committer | herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2003-06-14 06:45:20 +0000 |
commit | 172ee7f67a3aa8f8888905bee3c153cae543fcd5 (patch) | |
tree | 58bc76eb477fd27a870230386c511f05f09df7a1 /theories/Arith | |
parent | a0207c0d8a09325aef2d6bda6c9e981529fa5822 (diff) |
Deplacement de le_minus de fast_integer vers Minus
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4161 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Arith')
-rwxr-xr-x | theories/Arith/Minus.v | 7 |
1 files changed, 7 insertions, 0 deletions
diff --git a/theories/Arith/Minus.v b/theories/Arith/Minus.v index 2d00f259b..8224b8535 100755 --- a/theories/Arith/Minus.v +++ b/theories/Arith/Minus.v @@ -63,6 +63,13 @@ Symmetry; Auto with arith. Qed. Hints Resolve le_plus_minus_r : arith v62. +Theorem le_minus: (i,h:nat) (le (minus i h) i). +Proof. +Intros i h;Pattern i h; Apply nat_double_ind; [ + Auto +| Auto +| Intros m n H; Simpl; Apply le_trans with m:=m; Auto ]. +Qed. Lemma minus_Sn_m : (n,m:nat)(le m n)->((S (minus n m))=(minus (S n) m)). Proof. |