aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/NArith
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-05-05 15:13:20 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-05-05 15:13:20 +0000
commit568df64efe54a0365855a340ea5b75a4ea1c201d (patch)
treee971103e55de70173cecd3c2dda22cc3c07c2caa /theories/NArith
parentf440fd9b2d0f3e1bb5cd0b86df4676a46be781db (diff)
Peano recursion for positive: integration of Daniel Schepler's code
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@14110 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/NArith')
-rw-r--r--theories/NArith/BinNat.v5
1 files changed, 3 insertions, 2 deletions
diff --git a/theories/NArith/BinNat.v b/theories/NArith/BinNat.v
index 779391ed1..a63eabe5a 100644
--- a/theories/NArith/BinNat.v
+++ b/theories/NArith/BinNat.v
@@ -126,8 +126,9 @@ Qed.
Theorem peano_rect_succ P a f n :
peano_rect P a f (succ n) = f n (peano_rect P a f n).
Proof.
-destruct n; simpl;
-[rewrite Pos.peano_rect_base | rewrite Pos.peano_rect_succ]; reflexivity.
+destruct n; simpl.
+trivial.
+now rewrite Pos.peano_rect_succ.
Qed.
Definition peano_ind (P : N -> Prop) := peano_rect P.