aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/3736.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-07-27 10:50:04 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-07-27 14:20:44 +0200
commitcb6c3ec2e66e3019cb9ee881b1e222e6e3691463 (patch)
tree40d68c6bbc43e6794a1eb1d836d985de35eb4ffb /test-suite/bugs/closed/3736.v
parentcb145fa37d463210832c437f013231c9f028e1aa (diff)
Fixing bug #3736 (anomaly instead of error/warning/silence on
decidability scheme). Not clear to me why it is not a warning (in verbose mode) rather than silence when a scheme supposed to be built automatically cannot be built, as in: Set Decidable Equality Schemes. Inductive a := A with b := B. which could explain why a_beq and a_eq_dec as well as b_beq and b_eq_dec are not built.
Diffstat (limited to 'test-suite/bugs/closed/3736.v')
-rw-r--r--test-suite/bugs/closed/3736.v8
1 files changed, 8 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/3736.v b/test-suite/bugs/closed/3736.v
new file mode 100644
index 000000000..637b77cc5
--- /dev/null
+++ b/test-suite/bugs/closed/3736.v
@@ -0,0 +1,8 @@
+(* Check non-error failure in case of unsupported decidability scheme *)
+Local Set Decidable Equality Schemes.
+
+Inductive a := A with b := B.
+
+(* But fails with error if explicitly asked for the scheme *)
+
+Fail Scheme Equality for a.