aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Div2.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-03-31 22:17:30 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-03-31 22:17:30 +0000
commit512c2c28d009cc05845e705c662908a2764e18a5 (patch)
tree6ec862a9457fc927b5c88b0743072b4781c56e1d /theories/Arith/Div2.v
parent7f97b79b6372a115070f399d8804b57baa76ca74 (diff)
Ajout double_plus
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3828 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Arith/Div2.v')
-rw-r--r--theories/Arith/Div2.v7
1 files changed, 7 insertions, 0 deletions
diff --git a/theories/Arith/Div2.v b/theories/Arith/Div2.v
index a6782c5f8..b05eaa77d 100644
--- a/theories/Arith/Div2.v
+++ b/theories/Arith/Div2.v
@@ -106,6 +106,13 @@ Proof.
Intro. Unfold double. Simpl. Auto with arith.
Qed.
+Lemma double_plus : (m,n:nat) (double (plus m n))=(plus (double m) (double n)).
+Proof.
+Intros m n. Unfold double.
+Do 2 Rewrite -> plus_assoc_r. Rewrite -> (plus_permute n).
+Reflexivity.
+Qed.
+
Hints Resolve double_S : arith.
Lemma even_odd_double : (n:nat)