aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-04-28 00:02:32 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-04-28 00:05:53 +0200
commite5fe4569f3eaeaa4e1ce377989e19f1f2c176da9 (patch)
tree3edd23e7326b0240feb82c24393e617ba684342c /test-suite/success
parentcd139311ecd872301077b9db2df812a828ce2e77 (diff)
An example for cd139311e, showing a consequence of not converting
constants up to their canonical name (taken from Daniel's formalization of Puiseux theorem).
Diffstat (limited to 'test-suite/success')
-rw-r--r--test-suite/success/remember.v13
1 files changed, 13 insertions, 0 deletions
diff --git a/test-suite/success/remember.v b/test-suite/success/remember.v
index 0befe054a..b26a9ff1e 100644
--- a/test-suite/success/remember.v
+++ b/test-suite/success/remember.v
@@ -14,3 +14,16 @@ let name := fresh "fresh" in
remember (1 + 2) as x eqn:name.
rewrite fresh.
Abort.
+
+(* An example which was working in 8.4 but failing in 8.5 and 8.5pl1 *)
+
+Module A.
+Axiom N : nat.
+End A.
+Module B.
+Include A.
+End B.
+Goal id A.N = B.N.
+reflexivity.
+Qed.
+