aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init/Specif.v
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2014-09-09 22:39:15 +0200
committerGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2014-09-09 22:53:59 +0200
commit0dd3f0d34873dcd126be8ec48724a310214f38ac (patch)
treeccb5c83cba1db777681e8ecb7251dc486b3f2044 /theories/Init/Specif.v
parente365fb8ffbbc62352a725de13cbf864b3fbb3840 (diff)
- Fix printing and parsing of primitive projections, including the Set
Printing All cases (bug #3597). - Fix Ltac matching with primitive projections (bug #3598). - Spotted a problem with printing of constants with maximally implicit arguments due to strange "compatibility" interpretation of Arguments [X] as Arguments {X} but didn't fix it entirely yet (might cause incompatibilities).
Diffstat (limited to 'theories/Init/Specif.v')
-rw-r--r--theories/Init/Specif.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Init/Specif.v b/theories/Init/Specif.v
index 1ddb59cf4..c3edcfdfd 100644
--- a/theories/Init/Specif.v
+++ b/theories/Init/Specif.v
@@ -285,7 +285,7 @@ Section Exc.
Definition value := @Some A.
Definition error := @None A.
End Exc.
-Arguments error [A].
+Arguments error {A}.
Definition except := False_rec. (* for compatibility with previous versions *)