aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories
diff options
context:
space:
mode:
authorGravatar Tej Chajed <tchajed@mit.edu>2018-02-12 13:24:37 -0500
committerGravatar Tej Chajed <tchajed@mit.edu>2018-02-12 13:28:00 -0500
commitac7222c70266ee2b729b81e743adc7076191e6c0 (patch)
treeb5dd1739ecd5c3632c40d71b01ebdff9e0f8d89a /theories
parent52d666a7a83e4023d9f5cd7324ed81c7f7926156 (diff)
Add notation {x & P} for sigT
Analogous to existing `{x | P}` notation for `sig`, where the type of `x` is inferred instead of specified.
Diffstat (limited to 'theories')
-rw-r--r--theories/Init/Notations.v1
-rw-r--r--theories/Init/Specif.v1
2 files changed, 2 insertions, 0 deletions
diff --git a/theories/Init/Notations.v b/theories/Init/Notations.v
index 5e8d2faa5..70a6c61e7 100644
--- a/theories/Init/Notations.v
+++ b/theories/Init/Notations.v
@@ -75,6 +75,7 @@ Reserved Notation "{ x | P & Q }" (at level 0, x at level 99).
Reserved Notation "{ x : A | P }" (at level 0, x at level 99).
Reserved Notation "{ x : A | P & Q }" (at level 0, x at level 99).
+Reserved Notation "{ x & P }" (at level 0, x at level 99).
Reserved Notation "{ x : A & P }" (at level 0, x at level 99).
Reserved Notation "{ x : A & P & Q }" (at level 0, x at level 99).
diff --git a/theories/Init/Specif.v b/theories/Init/Specif.v
index 3b4f833a3..c42cc00b8 100644
--- a/theories/Init/Specif.v
+++ b/theories/Init/Specif.v
@@ -49,6 +49,7 @@ Notation "{ x | P & Q }" := (sig2 (fun x => P) (fun x => Q)) : type_scope.
Notation "{ x : A | P }" := (sig (A:=A) (fun x => P)) : type_scope.
Notation "{ x : A | P & Q }" := (sig2 (A:=A) (fun x => P) (fun x => Q)) :
type_scope.
+Notation "{ x & P }" := (sigT (fun x => P)) : type_scope.
Notation "{ x : A & P }" := (sigT (A:=A) (fun x => P)) : type_scope.
Notation "{ x : A & P & Q }" := (sigT2 (A:=A) (fun x => P) (fun x => Q)) :
type_scope.