diff options
author | Hugo Herbelin <Hugo.Herbelin@inria.fr> | 2017-10-04 15:37:36 +0200 |
---|---|---|
committer | Hugo Herbelin <Hugo.Herbelin@inria.fr> | 2017-10-05 08:38:45 +0200 |
commit | 40260a31cd197f655e6d3e0570a88d96fc1a9cac (patch) | |
tree | 0d0618bda35573e674b55a86364a5e39bf054442 /test-suite | |
parent | 526791d917f9b0804376eae02a462a3b32dd7cba (diff) |
Fixing BZ#5769 (variable of type "_something" was named after invalid "_").
Diffstat (limited to 'test-suite')
-rw-r--r-- | test-suite/bugs/closed/5769.v | 20 |
1 files changed, 20 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/5769.v b/test-suite/bugs/closed/5769.v new file mode 100644 index 000000000..42573aad8 --- /dev/null +++ b/test-suite/bugs/closed/5769.v @@ -0,0 +1,20 @@ +(* Check a few naming heuristics based on types *) +(* was buggy for types names _something *) + +Inductive _foo :=. +Lemma bob : (sigT (fun x : nat => _foo)) -> _foo. +destruct 1. +exact _f. +Abort. + +Inductive _'Foo :=. +Lemma bob : (sigT (fun x : nat => _'Foo)) -> _'Foo. +destruct 1. +exact _'f. +Abort. + +Inductive ____ :=. +Lemma bob : (sigT (fun x : nat => ____)) -> ____. +destruct 1. +exact x0. +Abort. |