diff options
| author | coqbot-app[bot] | 2020-11-18 22:00:25 +0000 |
|---|---|---|
| committer | GitHub | 2020-11-18 22:00:25 +0000 |
| commit | 7ebdf6bdbca2be4fc4ecddff0ac97bbb41c80cd0 (patch) | |
| tree | b12b82d14a9249a671b27e84caf12cda999531c6 /test-suite/success/attribute_syntax.v | |
| parent | fea83b040f285e4316fd9d63d4c940d9fe444d91 (diff) | |
| parent | efa6673158f5eaa3fc11c0b3d1e3285c4acc129a (diff) | |
Merge PR #13312: [attributes] Allow boolean, single-value attributes.
Reviewed-by: Zimmi48
Reviewed-by: SkySkimmer
Ack-by: gares
Diffstat (limited to 'test-suite/success/attribute_syntax.v')
| -rw-r--r-- | test-suite/success/attribute_syntax.v | 18 |
1 files changed, 17 insertions, 1 deletions
diff --git a/test-suite/success/attribute_syntax.v b/test-suite/success/attribute_syntax.v index b403fc120c..b866c4b074 100644 --- a/test-suite/success/attribute_syntax.v +++ b/test-suite/success/attribute_syntax.v @@ -16,11 +16,16 @@ Definition ι T (x: T) := x. Check ι _ ι. +#[universes(polymorphic=no)] +Definition ιι T (x: T) := x. + +Fail Check ιι _ ιι. + #[program] Fixpoint f (n: nat) {wf lt n} : nat := _. Reset f. -#[program(true)] +#[program=yes] Fixpoint f (n: nat) {wf lt n} : nat := _. Reset f. @@ -43,3 +48,14 @@ Export Set Foo. Fail #[ export ] Export Foo. (* Attribute for Locality specified twice *) + +(* Tests for deprecated attribute syntax *) +Set Warnings "-deprecated-attribute-syntax". + +#[program(true)] +Fixpoint f (n: nat) {wf lt n} : nat := _. +Reset f. + +#[universes(monomorphic)] +Definition ιιι T (x: T) := x. +Fail Check ιιι _ ιιι. |
