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

move some stuff to the lib folder

parent 4156d65d
No related branches found
No related tags found
No related merge requests found
...@@ -27,9 +27,11 @@ theories/proofmode.v ...@@ -27,9 +27,11 @@ theories/proofmode.v
theories/tests/tp_tests.v theories/tests/tp_tests.v
theories/tests/proofmode_tests.v theories/tests/proofmode_tests.v
theories/examples/lock.v theories/lib/lock.v
theories/examples/counter.v theories/lib/counter.v
theories/lib/Y.v
theories/examples/bit.v theories/examples/bit.v
theories/examples/Y.v
theories/examples/or.v theories/examples/or.v
theories/examples/generative.v theories/examples/generative.v
...@@ -6,7 +6,7 @@ Those are mostly "generative ADTs". *) ...@@ -6,7 +6,7 @@ Those are mostly "generative ADTs". *)
From iris.proofmode Require Import tactics. From iris.proofmode Require Import tactics.
From iris.heap_lang.lib Require Export par. From iris.heap_lang.lib Require Export par.
From reloc Require Export proofmode prelude.bijections. From reloc Require Export proofmode prelude.bijections.
From reloc.examples Require Export counter lock. From reloc.lib Require Export counter lock.
From reloc.typing Require Export interp soundness. From reloc.typing Require Export interp soundness.
(** Using references for name generation *) (** Using references for name generation *)
......
...@@ -79,6 +79,8 @@ Section rules. ...@@ -79,6 +79,8 @@ Section rules.
rel_load_r. repeat rel_pure_r. eauto with iFrame. rel_load_r. repeat rel_pure_r. eauto with iFrame.
Qed. Qed.
Opaque or.
(** Compatibility rule *) (** Compatibility rule *)
Lemma or_compatible e1 e2 e1' e2' A : Lemma or_compatible e1 e2 e1' e2' A :
(REL e1 << e1' : () A) -∗ (REL e1 << e1' : () A) -∗
...@@ -89,7 +91,6 @@ Section rules. ...@@ -89,7 +91,6 @@ Section rules.
rel_bind_l e2. rel_bind_r e2'. rel_bind_l e2. rel_bind_r e2'.
iApply (refines_bind with "H2"). iApply (refines_bind with "H2").
iIntros (v2 v2') "#Hv2". iIntros (v2 v2') "#Hv2".
(* ^ TODO the arrow interpretation gets unfolded here *)
rel_bind_l e1. rel_bind_r e1'. rel_bind_l e1. rel_bind_r e1'.
iApply (refines_bind with "H1"). iApply (refines_bind with "H1").
iIntros (v1 v1') "#Hv1". iSimpl. iIntros (v1 v1') "#Hv1". iSimpl.
......
File moved
From reloc Require Export proofmode. From reloc Require Export proofmode.
From reloc.typing Require Export types interp. From reloc.typing Require Export types interp.
From reloc.logic Require Import compatibility. From reloc.logic Require Import compatibility.
From reloc.examples Require Import lock. From reloc.lib Require Import lock.
From reloc.typing Require Import soundness. From reloc.typing Require Import soundness.
Definition CG_increment : val := λ: "x" "l", Definition CG_increment : val := λ: "x" "l",
......
File moved
...@@ -139,7 +139,7 @@ Section semtypes. ...@@ -139,7 +139,7 @@ Section semtypes.
End semtypes. End semtypes.
(* Nice notations *) (** Nice notations *)
Notation "()" := lty2_unit : lty_scope. Notation "()" := lty2_unit : lty_scope.
Infix "→" := lty2_arr : lty_scope. Infix "→" := lty2_arr : lty_scope.
Infix "×" := lty2_prod (at level 80) : lty_scope. Infix "×" := lty2_prod (at level 80) : lty_scope.
...@@ -242,13 +242,6 @@ End related_facts. ...@@ -242,13 +242,6 @@ End related_facts.
Section monadic. Section monadic.
Context `{relocG Σ}. Context `{relocG Σ}.
(* Lemma refines_ret_expr E e1 e2 A : *)
(* interp_expr E e1 e2 A -∗ REL e1 << e2 @ E : A. *)
(* Proof. *)
(* iIntros "HA". rewrite refines_eq /refines_def. *)
(* eauto with iFrame. *)
(* Qed. *)
Lemma refines_bind K K' E A A' e e' : Lemma refines_bind K K' E A A' e e' :
(REL e << e' @ E : A) -∗ (REL e << e' @ E : A) -∗
( v v', A v v' -∗ ( v v', A v v' -∗
......
...@@ -2,7 +2,7 @@ ...@@ -2,7 +2,7 @@
(** (Syntactic) Typing for System F_mu_ref with existential types and concurrency *) (** (Syntactic) Typing for System F_mu_ref with existential types and concurrency *)
From stdpp Require Export stringmap. From stdpp Require Export stringmap.
From iris.heap_lang Require Export lang notation metatheory. From iris.heap_lang Require Export lang notation metatheory.
From Autosubst Require Import Autosubst. From Autosubst Require Export Autosubst.
(** * Types *) (** * Types *)
Inductive type := Inductive type :=
......
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