Skip to content
Snippets Groups Projects
Commit c35476b8 authored by Robbert Krebbers's avatar Robbert Krebbers
Browse files

An additional fix for https://github.com/coq/coq/pull/10762.

parent 92ded048
No related branches found
No related tags found
No related merge requests found
...@@ -93,5 +93,5 @@ Lemma step_fupdN_soundness' `{!invPreG Σ} φ n : ...@@ -93,5 +93,5 @@ Lemma step_fupdN_soundness' `{!invPreG Σ} φ n :
Proof. Proof.
iIntros (Hiter). eapply (step_fupdN_soundness _ n). iIntros (Hiter). eapply (step_fupdN_soundness _ n).
iIntros (Hinv). iPoseProof (Hiter Hinv) as "Hiter". iIntros (Hinv). iPoseProof (Hiter Hinv) as "Hiter".
iApply (step_fupdN_wand with "Hiter"). by iApply (fupd_mask_weaken _ _ _). iApply (step_fupdN_wand with "Hiter"). by iApply fupd_mask_weaken.
Qed. Qed.
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