From 568df64efe54a0365855a340ea5b75a4ea1c201d Mon Sep 17 00:00:00 2001 From: letouzey Date: Thu, 5 May 2011 15:13:20 +0000 Subject: 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 --- theories/NArith/BinNat.v | 5 +++-- 1 file changed, 3 insertions(+), 2 deletions(-) (limited to 'theories/NArith') 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. -- cgit v1.2.3