aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/4969.v
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <mattam@mattam.org>2016-09-29 17:42:53 +0200
committerGravatar Matthieu Sozeau <mattam@mattam.org>2016-09-29 17:44:27 +0200
commitc694b91bba898aad1e071d91fa70b7c5574cbf98 (patch)
tree554e1dd1c0982d42510213afbd8d29ed3712a85d /test-suite/bugs/closed/4969.v
parent5348a615a484e379896deac8a6944af1f92b2d4c (diff)
Fix bug 4969, autoapply was not tagging shelved subgoals correctly as unresolvable
Diffstat (limited to 'test-suite/bugs/closed/4969.v')
-rw-r--r--test-suite/bugs/closed/4969.v11
1 files changed, 11 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/4969.v b/test-suite/bugs/closed/4969.v
new file mode 100644
index 000000000..4dee41e22
--- /dev/null
+++ b/test-suite/bugs/closed/4969.v
@@ -0,0 +1,11 @@
+Require Import Classes.Init.
+
+Class C A := c : A.
+Instance nat_C : C nat := 0.
+Instance bool_C : C bool := true.
+Lemma silly {A} `{C A} : 0 = 0 -> c = c -> True.
+Proof. auto. Qed.
+
+Goal True.
+ class_apply @silly; [reflexivity|].
+ reflexivity. Fail Qed.