diff --git a/tests/proofmode.v b/tests/proofmode.v index f27ba2444a55188b78eff58c86ba89306983084c..9ff9c88a3a6b7644c89d1791ad3881d7ef934149 100644 --- a/tests/proofmode.v +++ b/tests/proofmode.v @@ -5,9 +5,9 @@ Section tests. Context {PROP : sbi}. Implicit Types P Q R : PROP. -Lemma type_sbi_internal_eq_annot P : - P ≡@{PROP} P ∧ (≡@{PROP}) P P ∧ (P ≡.) P ∧ (.≡ P) P. -Proof. done. Qed. +Lemma test_sbi_internal_eq_annot_sections P : + ⊢@{PROP} P ≡@{PROP} P ∧ (≡@{PROP}) P P ∧ (P ≡.) P ∧ (.≡ P) P. +Proof. by iSplit. Qed. Lemma test_eauto_emp_isplit_biwand P : emp ⊢ P ∗-∗ P. Proof. eauto 6. Qed.