Skip to content
Snippets Groups Projects
Unverified Commit 96298cd0 authored by Lennard Gäher's avatar Lennard Gäher
Browse files

provide tactic for apply_update

parent 9dd74f4b
No related branches found
No related tags found
1 merge request!10Various bug fixes
......@@ -156,8 +156,8 @@ Section updateable_rules.
typed_array_access updateable_π updateable_E updateable_L l off st lt r k (λ L2 rt2 ty2 len2 iml2 rs2 k2 rte lte re,
l ◁ₗ[updateable_π, k2] #rs2 @ ArrayLtype ty2 len2 iml2 -
(l offsetst{st} off) ◁ₗ[updateable_π, k2] re @ lte -
updateable_core updateable_π updateable_E L2)) -
P.
updateable_core updateable_π updateable_E L2))
P.
Proof.
iIntros "HT".
unshelve iApply add_updateable; first apply _.
......@@ -180,6 +180,8 @@ Ltac add_updateable :=
unshelve notypeclasses refine (tac_fast_apply (add_updateable P) _);
[ apply _ | apply _ | ]
end.
Tactic Notation "apply_update" uconstr(H) :=
refine (tac_fast_apply H _).
Section test.
Context `{!typeGS Σ}.
......@@ -193,6 +195,14 @@ Section test.
unshelve iApply (updateable_typed_array_access l off st).
idtac.
Abort.
Lemma typed_s_updateable π E L s rf R ϝ (l : loc) (off : Z) (st : syn_type) :
typed_stmt π E L s rf R ϝ.
Proof.
iStartProof.
unshelve apply_update (updateable_typed_array_access l off st).
idtac.
Abort.
End test.
Lemma tac_typed_val_expr_bind' `{!typeGS Σ} π E L K e T :
......
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