Skip to content
Snippets Groups Projects
Verified Commit b0141831 authored by Tej Chajed's avatar Tej Chajed
Browse files

Add back a proofmode test for issue #288

This test is incompatible with Coq 8.8 and Coq 8.9, but Iris no longer
supports those versions.
parent 832a63d6
No related branches found
No related tags found
No related merge requests found
...@@ -410,15 +410,13 @@ Proof. ...@@ -410,15 +410,13 @@ Proof.
Qed. Qed.
(* Test for issue #288 *) (* Test for issue #288 *)
(* FIXME: Restore once we drop support for Coq 8.8 and Coq 8.9. Lemma test_iExists_unused : P : PROP, x : nat, P.
Lemma test_iExists_unused : (∃ P : PROP, ∃ x : nat, P)%I.
Proof. Proof.
iExists _. iExists _.
iExists 10. iExists 10.
iAssert emp%I as "H"; first done. iAssert emp%I as "H"; first done.
iExact "H". iExact "H".
Qed. Qed.
*)
(* Check coercions *) (* Check coercions *)
Lemma test_iExist_coercion (P : Z PROP) : ( x, P x) -∗ x, P x. Lemma test_iExist_coercion (P : Z PROP) : ( x, P x) -∗ x, P x.
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Finish editing this message first!
Please register or to comment