From e09064ff153ee9f909e8c2c1ee2aaa249b324a78 Mon Sep 17 00:00:00 2001 From: pboutill Date: Tue, 28 Sep 2010 16:27:26 +0000 Subject: Bvector.Vshiftin was wrong for ages git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13471 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/Bool/Bvector.v | 2 +- 1 file changed, 1 insertion(+), 1 deletion(-) (limited to 'theories/Bool') diff --git a/theories/Bool/Bvector.v b/theories/Bool/Bvector.v index 0cb3c3670..88bc15c69 100644 --- a/theories/Bool/Bvector.v +++ b/theories/Bool/Bvector.v @@ -92,7 +92,7 @@ Proof. exact (Vcons a 0 v). inversion v as [| a0 n0 H0 H1 ]. - exact (Vcons a (S n) (f a H0)). + exact (Vcons a0 (S n) (f a H0)). Defined. Lemma Vshiftrepeat : forall n:nat, vector (S n) -> vector (S (S n)). -- cgit v1.2.3