diff options
| author | Enrico Tassi | 2020-10-12 16:52:47 +0200 |
|---|---|---|
| committer | Enrico Tassi | 2020-11-02 10:04:48 +0100 |
| commit | fd9d10f2c7eff9ff72f42e9ecd3ffd5179de4da0 (patch) | |
| tree | 2ba3cd5e6459b6acf8b6bed63786c49d5770f9dd /test-suite/success/definition_using.v | |
| parent | a464fdc040a77022dd9e6e57129f80144918ace6 (diff) | |
[stm] support #[using] attribute
Diffstat (limited to 'test-suite/success/definition_using.v')
| -rw-r--r-- | test-suite/success/definition_using.v | 22 |
1 files changed, 22 insertions, 0 deletions
diff --git a/test-suite/success/definition_using.v b/test-suite/success/definition_using.v index a8eab93404..120e62b145 100644 --- a/test-suite/success/definition_using.v +++ b/test-suite/success/definition_using.v @@ -44,3 +44,25 @@ Check c4 : bogus -> bool. Check c5 : bogus -> nat -> bool. Check c6 : bogus -> bool. Check c7 : bogus -> nat -> bool. + +Section B. + +Variable a : bogus. +Variable h : c1 a = true. + +#[using="a*"] +Definition c8 : bogus := a. + +Collection ccc := a h. + +#[using="ccc"] +Definition c9 : bogus := a. + +#[using="ccc - h"] +Definition c10 : bogus := a. + +End B. + +Check c8 : forall a, c1 a = true -> bogus. +Check c9 : forall a, c1 a = true -> bogus. +Check c10: bogus -> bogus. |
