aboutsummaryrefslogtreecommitdiff
path: root/test-suite/micromega
diff options
context:
space:
mode:
authorFrédéric Besson2020-08-10 15:31:58 +0200
committerFrédéric Besson2020-08-10 15:35:30 +0200
commit4da8f114155d2abb31ce8a45a2f17f21f7d97a0e (patch)
treeb271937251f65b7e454d67c2cca97687b24766fd /test-suite/micromega
parentef08abec26c2f0017d1136870f8f99144e579538 (diff)
[zify] fix for bug#12791
The elimination of let bindings is performing a convertibility check in order to deal with type aliases.
Diffstat (limited to 'test-suite/micromega')
-rw-r--r--test-suite/micromega/bug_12791.v9
1 files changed, 9 insertions, 0 deletions
diff --git a/test-suite/micromega/bug_12791.v b/test-suite/micromega/bug_12791.v
new file mode 100644
index 0000000000..8aec1904a4
--- /dev/null
+++ b/test-suite/micromega/bug_12791.v
@@ -0,0 +1,9 @@
+Require Import Lia.
+
+Definition t := nat.
+
+Goal forall (a b: t), let c := a in b = a -> b = c.
+Proof.
+ intros a b c H.
+ lia.
+Qed.