aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Minus.v
diff options
context:
space:
mode:
authorGravatar mohring <mohring@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-04-08 17:18:57 +0000
committerGravatar mohring <mohring@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-04-08 17:18:57 +0000
commitd41db01560cb49974af197d22dabc367c71a64ed (patch)
tree75517698617653da2fd0a522cda1942421baa023 /theories/Arith/Minus.v
parent509940521cda3057455adb0f0af8b16d88b73df6 (diff)
ajout des lemmes Zimmerman
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1556 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Arith/Minus.v')
-rwxr-xr-xtheories/Arith/Minus.v13
1 files changed, 13 insertions, 0 deletions
diff --git a/theories/Arith/Minus.v b/theories/Arith/Minus.v
index 29a978070..afb5a1984 100755
--- a/theories/Arith/Minus.v
+++ b/theories/Arith/Minus.v
@@ -94,3 +94,16 @@ Intros n m; Pattern n m; Apply nat_double_ind; Simpl; Auto with arith.
Intros; Absurd (lt O O); Trivial with arith.
Qed.
Hints Immediate lt_O_minus_lt : arith v62.
+
+Theorem pred_of_minus : (x:nat)(pred x)=(minus x (S O)).
+Induction x; Auto with arith.
+Save.
+
+
+Theorem inj_minus_aux: (x,y:nat) ~(le y x) -> (minus x y) = O.
+Intros y x; Pattern y x ; Apply nat_double_ind; [
+ Simpl; Trivial with arith
+| Intros n H; Absurd (le O (S n)); [ Assumption | Apply le_O_n]
+| Simpl; Intros n m H1 H2; Apply H1;
+ Unfold not ; Intros H3; Apply H2; Apply le_n_S; Assumption].
+Save.