aboutsummaryrefslogtreecommitdiff
path: root/theories/Program/Syntax.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Program/Syntax.v')
-rw-r--r--theories/Program/Syntax.v7
1 files changed, 7 insertions, 0 deletions
diff --git a/theories/Program/Syntax.v b/theories/Program/Syntax.v
index aff2da946e..2064977fef 100644
--- a/theories/Program/Syntax.v
+++ b/theories/Program/Syntax.v
@@ -46,6 +46,13 @@ Notation " [ ] " := nil : list_scope.
Notation " [ x ] " := (cons x nil) : list_scope.
Notation " [ x ; .. ; y ] " := (cons x .. (cons y nil) ..) : list_scope.
+(** Implicit arguments for vectors. *)
+
+Require Import Bvector.
+
+Implicit Arguments Vnil [[A]].
+Implicit Arguments Vcons [[A] [n]].
+
(** Treating n-ary exists *)
Notation " 'exists' x y , p" := (ex (fun x => (ex (fun y => p))))