aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Vectors
diff options
context:
space:
mode:
authorGravatar pboutill <pboutill@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-02-10 14:11:12 +0000
committerGravatar pboutill <pboutill@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-02-10 14:11:12 +0000
commit27ab4eb203dd5d653724f7a1af61badf2916c349 (patch)
tree95791fafbc20e50f6341178c916e456b6e635894 /theories/Vectors
parentc5fa08bbecbc665e1d82d38d2e41f5256efcd545 (diff)
Fixpoints are traverse during implicits arguments search to toplevel
registration (& CHANGES update) git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13826 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Vectors')
-rw-r--r--theories/Vectors/VectorDef.v8
1 files changed, 0 insertions, 8 deletions
diff --git a/theories/Vectors/VectorDef.v b/theories/Vectors/VectorDef.v
index 807748edd..cff72c11b 100644
--- a/theories/Vectors/VectorDef.v
+++ b/theories/Vectors/VectorDef.v
@@ -269,14 +269,6 @@ end.
End ITERATORS.
-Implicit Arguments rectS.
-Implicit Arguments rect2.
-Implicit Arguments fold_left.
-Implicit Arguments fold_right.
-Implicit Arguments map.
-Implicit Arguments fold_left2.
-
-
Section SCANNING.
Inductive Forall {A} (P: A -> Prop): forall {n} (v: t A n), Prop :=
|Forall_nil: Forall P []