Skip to content
Snippets Groups Projects
Commit df843150 authored by Dan Frumin's avatar Dan Frumin
Browse files

move is_closed_expr' to model.v

parent a1810700
No related branches found
No related tags found
No related merge requests found
......@@ -336,18 +336,22 @@ Section related_facts.
End related_facts.
(** TODO this is a terrible hack and I should be ashamed of myself.
See iris issue 225. *)
Notation is_closed_expr' := (λ e, vs, subst_map vs e = e).
Section monadic.
Context `{relocG Σ}.
Lemma refines_ret' E Γ e1 e2 A :
is_closed_expr [] e1
is_closed_expr [] e2
is_closed_expr' e1
is_closed_expr' e2
interp_expr E e1 e2 A -∗ {E;Γ} e1 << e2 : A.
Proof.
iIntros (??) "HA".
iIntros (Hcl1 Hcl2) "HA".
rewrite refines_eq /refines_def.
iIntros (vvs ρ) "#Hs #HΓ".
rewrite !subst_map_is_closed_nil//.
by rewrite Hcl1 Hcl2.
Qed.
Lemma refines_bind K K' E Γ A A' e e' :
......
......@@ -74,9 +74,6 @@ Section rules.
by rewrite subst_map_fill.
Qed.
(* See iris issue 225 *)
Notation is_closed_expr' := (λ e, vs, subst_map vs e = e).
Lemma refines_wp_l Γ K e1 e2 A :
is_closed_expr' e1
(WP e1 {{ v,
......
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