aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/NArith
diff options
context:
space:
mode:
authorGravatar pboutill <pboutill@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-02-10 14:11:14 +0000
committerGravatar pboutill <pboutill@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-02-10 14:11:14 +0000
commit461a5a2093f8e46708e01a27993f80919e20d4aa (patch)
tree1e66ec78daccfa700b9461dadefb34800ac598b9 /theories/NArith
parent27ab4eb203dd5d653724f7a1af61badf2916c349 (diff)
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
Diffstat (limited to 'theories/NArith')
-rw-r--r--theories/NArith/Ndigits.v2
1 files changed, 1 insertions, 1 deletions
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.