Skip to content
Snippets Groups Projects
Commit fe271b0a authored by Daniël Louwrink's avatar Daniël Louwrink
Browse files

add/clean up some TODOs for copying

parent 1311132f
No related branches found
No related tags found
No related merge requests found
......@@ -23,6 +23,11 @@ Section copying.
copy A <: A.
Proof. by iIntros (v) "!> #H". Qed.
(* TODO(COPY): have A <: copy- A rule *)
(* TODO(COPY): Show derived rules about copyability of products, sums, etc. *)
(* TODO(COPY): Commuting rule for μ, allowing `copy` to move outside the μ *)
(* TODO(COPY) *)
Lemma coreP_desired_lemma (P : iProp Σ) :
(P -∗ P) -∗ coreP P -∗ P.
Proof.
......@@ -102,7 +107,7 @@ Section copying.
iExists A; repeat iModIntro; iApply "Hv".
Qed.
(* TODO: Do the forall type former, once we have the value restriction *)
(* TODO(COPY) TODO(VALUERES): Do the forall type former, once we have the value restriction *)
(* Copyability of recursive types *)
Lemma lty_rec_copy C `{!Contractive C} :
......
......@@ -472,7 +472,7 @@ Section properties.
by iModIntro.
Qed.
(* FIXME: copy *)
(* TODO(COPY) *)
(* Lemma ltyped_load_copy A {copyA : LTyCopy A} : *)
(* ⊢ ∅ ⊨ load : ref_mut A → A * ref_mut A. *)
(* Proof. *)
......@@ -526,7 +526,7 @@ Section properties.
by iExists m.
Qed.
(* FIXME: copy *)
(* TODO(COPY) *)
(* Lemma ltyped_ref_shr_load (A : lty Σ) {copyA : LTyCopy A} : *)
(* ⊢ ∅ ⊨ load : ref_shr A → (A * ref_shr A). *)
(* Proof. *)
......
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