aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Vectors
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2016-09-26 13:11:03 -0400
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-09-26 23:44:04 +0200
commit53ac7ca0cd74b62d47472c0dabfcc8dc1cacd86c (patch)
tree26623ffeff84941c654d68b824fe2274d29a9a04 /theories/Vectors
parentf8745b1dbc87a8fee4943a91f517dc2afcd7804b (diff)
Remove spaces from around vector notations
Diffstat (limited to 'theories/Vectors')
-rw-r--r--theories/Vectors/VectorDef.v8
1 files changed, 4 insertions, 4 deletions
diff --git a/theories/Vectors/VectorDef.v b/theories/Vectors/VectorDef.v
index 095cda398..f49b34075 100644
--- a/theories/Vectors/VectorDef.v
+++ b/theories/Vectors/VectorDef.v
@@ -30,7 +30,7 @@ Inductive t A : nat -> Type :=
|nil : t A 0
|cons : forall (h:A) (n:nat), t A n -> t A (S n).
-Local Notation " [ ] " := (nil _) (format "[ ]").
+Local Notation "[ ]" := (nil _) (format "[ ]").
Local Notation "h :: t" := (cons _ h _ t) (at level 60, right associativity).
Section SCHEMES.
@@ -294,11 +294,11 @@ End VECTORLIST.
Module VectorNotations.
Delimit Scope vector_scope with vector.
-Notation " [ ] " := [] (format "[ ]") : vector_scope.
+Notation "[ ]" := [] (format "[ ]") : vector_scope.
Notation "h :: t" := (h :: t) (at level 60, right associativity)
: vector_scope.
-Notation " [ x ] " := (x :: []) : vector_scope.
-Notation " [ x ; y ; .. ; z ] " := (cons _ x _ (cons _ y _ .. (cons _ z _ (nil _)) ..)) : vector_scope
+Notation "[ x ]" := (x :: []) : vector_scope.
+Notation "[ x ; y ; .. ; z ]" := (cons _ x _ (cons _ y _ .. (cons _ z _ (nil _)) ..)) : vector_scope
.
Notation "v [@ p ]" := (nth v p) (at level 1, format "v [@ p ]") : vector_scope.
Open Scope vector_scope.