diff --git a/theories/tests/proofmode.v b/theories/tests/proofmode.v index c43c2f5c3a9006a75242c42593d419e7aeeaf1db..9d4f4061cb46fc0f9dd03e48ef80da7d47950ee6 100644 --- a/theories/tests/proofmode.v +++ b/theories/tests/proofmode.v @@ -78,6 +78,11 @@ Lemma test_very_fast_iIntros P : ∀ x y : nat, (⌜ x = y ⌠→ P -∗ P)%I. Proof. by iIntros. Qed. +(** Prior to 0b84351c this used to loop, now `iAssumption` instantiates `R` with +`False` and performs false elimination. *) +Lemma test_iAssumption_evar_ex_false : ∃ R, R ⊢ ∀ P, P. +Proof. eexists. iIntros "?" (P). iAssumption. Qed. + Lemma test_iAssumption_affine P Q R `{!Affine P, !Affine R} : P -∗ Q -∗ R -∗ Q. Proof. iIntros "H1 H2 H3". iAssumption. Qed.