diff options
author | herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2007-05-10 15:31:46 +0000 |
---|---|---|
committer | herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2007-05-10 15:31:46 +0000 |
commit | de6e0fdd9f3078b9b0ccf87ba8a7dcc9cc47c9aa (patch) | |
tree | 33bc723ec517a6ad737b7ca52a7e71f643ed3158 /test-suite | |
parent | afaa5d6ee5c27329423c152362e0969dc2d9afdd (diff) |
Prise en compte réversibilité des notations de la forme "Notation Nil := @nil".
Ajout @ref au niveau constr pour allègement syntaxe.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9819 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite')
-rw-r--r-- | test-suite/output/Notations.out | 4 | ||||
-rw-r--r-- | test-suite/output/Notations.v | 10 |
2 files changed, 14 insertions, 0 deletions
diff --git a/test-suite/output/Notations.out b/test-suite/output/Notations.out index be4cd4fae..2066a7ef3 100644 --- a/test-suite/output/Notations.out +++ b/test-suite/output/Notations.out @@ -46,3 +46,7 @@ fun x : nat => ifn x is succ n then n else 0 : bool -4 : Z +Nil + : forall A : Type, list A +NIL:list nat + : list nat diff --git a/test-suite/output/Notations.v b/test-suite/output/Notations.v index 3cc0a189d..6e637aca3 100644 --- a/test-suite/output/Notations.v +++ b/test-suite/output/Notations.v @@ -119,3 +119,13 @@ Require Import ZArith. Open Scope Z_scope. Notation "- 4" := (-2 + -2). Check -4. + +(**********************************************************************) +(* Check notations for references with activated or deactivated *) +(* implicit arguments *) + +Notation Nil := @nil. +Check Nil. + +Notation NIL := nil. +Check NIL : list nat. |