Skip to content

Commit

Permalink
rm comments
Browse files Browse the repository at this point in the history
  • Loading branch information
Kaptch committed Jul 9, 2024
1 parent 1738ebc commit e54d14e
Show file tree
Hide file tree
Showing 3 changed files with 0 additions and 3 deletions.
1 change: 0 additions & 1 deletion theories/examples/delim_lang/interp.v
Original file line number Diff line number Diff line change
Expand Up @@ -159,7 +159,6 @@ Section interp.
λne env, Ret n.

(** ** CONT *)
(** XXX DF: why do we need a tick here? Seems to be necessary for soundness *)
Program Definition interp_cont_val {S} (K : S -n> (IT -n> IT)) : S -n> IT :=
λne env, (λit x, Tick $ 𝒫 (K env x)).
Solve All Obligations with solve_proper_please.
Expand Down
1 change: 0 additions & 1 deletion theories/examples/input_lang_callcc/interp.v
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,6 @@ From gitrees.effects Require Export callcc.
From gitrees.examples.input_lang_callcc Require Import lang.
Require Import Binding.Lib Binding.Set.

(* XXX TODO: this duplicates wp_input and wp_output *)
Section weakestpre.
Context {sz : nat}.
Variable (rs : gReifiers CtxDep sz).
Expand Down
1 change: 0 additions & 1 deletion theories/lib/factorial.v
Original file line number Diff line number Diff line change
Expand Up @@ -67,7 +67,6 @@ Section fact.
iNext. iNext. iIntros "Hacc".
iApply wp_val. iModIntro.
simpl. unfold NatOpRSCtx.
(* TODO: look at this with amin *)
iAssert (IT_of_V (E:=F) (RetV m) ≡ (Ret m))%I as "#Hm".
{ iPureIntro. apply (IT_of_V_Ret (B:=R)). }
iRewrite "Hm".
Expand Down

0 comments on commit e54d14e

Please sign in to comment.