Skip to content
Snippets Groups Projects
Commit aa0081c5 authored by Ralf Jung's avatar Ralf Jung
Browse files

8.16-compat

parent 73f69784
No related branches found
No related tags found
No related merge requests found
Pipeline #70822 passed
...@@ -56,7 +56,7 @@ trigger-iris.dev: ...@@ -56,7 +56,7 @@ trigger-iris.dev:
variables: variables:
STDPP_REPO: "iris/stdpp" STDPP_REPO: "iris/stdpp"
IRIS_REPO: "iris/iris" IRIS_REPO: "iris/iris"
OPAM_PINS: "coq version 8.15.dev git+https://gitlab.mpi-sws.org/$STDPP_REPO#$STDPP_REV git+https://gitlab.mpi-sws.org/$IRIS_REPO#$IRIS_REV" OPAM_PINS: "coq version 8.16.dev git+https://gitlab.mpi-sws.org/$STDPP_REPO#$STDPP_REV git+https://gitlab.mpi-sws.org/$IRIS_REPO#$IRIS_REV"
except: except:
only: only:
refs: refs:
......
...@@ -61,7 +61,7 @@ Section fixpoint. ...@@ -61,7 +61,7 @@ Section fixpoint.
{ split; (intros [H1 H2]; split; [apply H1|apply H2]). } { split; (intros [H1 H2]; split; [apply H1|apply H2]). }
apply limit_preserving_and; repeat (apply limit_preserving_forall=> ?). apply limit_preserving_and; repeat (apply limit_preserving_forall=> ?).
+ apply bi.limit_preserving_Persistent; solve_proper. + apply bi.limit_preserving_Persistent; solve_proper.
+ apply limit_preserving_impl, bi.limit_preserving_entails; + apply limit_preserving_impl', bi.limit_preserving_entails;
solve_proper_core ltac:(fun _ => eapply ty_size_ne || f_equiv). solve_proper_core ltac:(fun _ => eapply ty_size_ne || f_equiv).
Qed. Qed.
......
...@@ -209,7 +209,7 @@ Section typing. ...@@ -209,7 +209,7 @@ Section typing.
iDestruct (ty_size_eq with "Hrown") as ">Heq". iDestruct "Heq" as %Heq. iDestruct (ty_size_eq with "Hrown") as ">Heq". iDestruct "Heq" as %Heq.
(* FIXME: Changing the order of $Hr↦ $Hc'↦ breaks applying...?? *) (* FIXME: Changing the order of $Hr↦ $Hc'↦ breaks applying...?? *)
wp_apply (wp_memcpy with "[$Hr↦ $Hc'↦]"). wp_apply (wp_memcpy with "[$Hr↦ $Hc'↦]").
{ by rewrite Heq. } { rewrite Heq /= ?Nat2Z.id //. }
{ f_equal. done. } { f_equal. done. }
iIntros "[Hr↦ Hc'↦]". wp_seq. iIntros "[Hr↦ Hc'↦]". wp_seq.
iDestruct "Hx" as "[Hx↦ Hx†]". iDestruct "Hx↦" as (vx) "[Hx↦ Hxown]". iDestruct "Hx" as "[Hx↦ Hx†]". iDestruct "Hx↦" as (vx) "[Hx↦ Hxown]".
...@@ -225,7 +225,7 @@ Section typing. ...@@ -225,7 +225,7 @@ Section typing.
{ rewrite 2!tctx_interp_cons tctx_interp_singleton !tctx_hasty_val. { rewrite 2!tctx_interp_cons tctx_interp_singleton !tctx_hasty_val.
iFrame "Hc". rewrite !tctx_hasty_val' //. iSplitL "Hx↦ Hx†". iFrame "Hc". rewrite !tctx_hasty_val' //. iSplitL "Hx↦ Hx†".
- iFrame. iExists _. iFrame. iNext. iApply uninit_own. done. - iFrame. iExists _. iFrame. iNext. iApply uninit_own. done.
- iFrame. iExists _. iFrame. } - try rewrite !Nat2Z.id. iFrame. iExists _. iFrame. }
iApply type_delete; [solve_typing..|]. iApply type_delete; [solve_typing..|].
iApply type_delete; [solve_typing..|]. iApply type_delete; [solve_typing..|].
iApply type_jump; solve_typing. iApply type_jump; solve_typing.
......
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