From 461a5a2093f8e46708e01a27993f80919e20d4aa Mon Sep 17 00:00:00 2001 From: pboutill Date: Thu, 10 Feb 2011 14:11:14 +0000 Subject: Vectors fully use implicit arguments and take disavantages for maximal insertion git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13827 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/NArith/Ndigits.v | 2 +- 1 file changed, 1 insertion(+), 1 deletion(-) (limited to 'theories/NArith') diff --git a/theories/NArith/Ndigits.v b/theories/NArith/Ndigits.v index 1f95b1cf7..94432a7cf 100644 --- a/theories/NArith/Ndigits.v +++ b/theories/NArith/Ndigits.v @@ -1053,7 +1053,7 @@ Qed. Lemma Nand_BVand : forall n (bv bv' : Bvector n), Bv2N _ (BVand _ bv bv') = Nand (Bv2N _ bv) (Bv2N _ bv'). Proof. -refine (Vector.rect2 _ _ _); simpl; intros; auto. +refine (@Vector.rect2 _ _ _ _ _); simpl; intros; auto. rewrite H. destruct a, b, (Bv2N n v1), (Bv2N n v2); simpl; auto. -- cgit v1.2.3