Skip to content

Commit

Permalink
fix hom issues
Browse files Browse the repository at this point in the history
  • Loading branch information
Dan committed Jun 23, 2024
1 parent 63af674 commit b91709c
Show file tree
Hide file tree
Showing 5 changed files with 10 additions and 14 deletions.
5 changes: 5 additions & 0 deletions theories/examples/delim_lang/hom.v
Original file line number Diff line number Diff line change
Expand Up @@ -16,6 +16,11 @@ Section hom.
Notation IT := (IT F R).
Notation ITV := (ITV F R).

Program Definition 𝒫_HOM : HOM (A:=natO) := exist _ 𝒫 _.
Next Obligation.
apply _.
Qed.

Program Definition AppContRSCtx_HOM {S : Set}
(α : @interp_scope F R _ S -n> IT)
(env : @interp_scope F R _ S)
Expand Down
5 changes: 0 additions & 5 deletions theories/examples/delim_lang/logpred.v
Original file line number Diff line number Diff line change
Expand Up @@ -213,11 +213,6 @@ Section logrel.
iApply "H".
Qed.

Program Definition 𝒫_HOM : @HOM sz CtxDep R _ rs := exist _ 𝒫 _.
Next Obligation.
apply _.
Qed.

Lemma compat_shift {S : Set} (Γ : S -> ty) e σ α τ β :
⊢ valid (Γ ▹ (Tcont τ α)) e σ σ β -∗ valid Γ (interp_shift _ e) τ α β.
Proof.
Expand Down
5 changes: 0 additions & 5 deletions theories/examples/delim_lang/logrel.v
Original file line number Diff line number Diff line change
Expand Up @@ -314,11 +314,6 @@ Section logrel.
assumption.
Qed.

Program Definition 𝒫_HOM : @HOM sz CtxDep R _ rs := exist _ 𝒫 _.
Next Obligation.
apply _.
Qed.

Lemma compat_shift {S : Set} (Γ : S -> ty) e (e' : exprO (inc S)) σ α τ β :
⊢ valid (Γ ▹ (τ ⤑ α)) e e' σ σ β -∗ valid Γ (interp_shift _ e) (shift/cc e') τ α β.
Proof.
Expand Down
7 changes: 3 additions & 4 deletions theories/examples/input_lang_callcc/hom.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,4 @@
(** In this module, we package up IT homomorphism in a sigma type, and
we will use it as a domain for logical relations on continuations *)
(** Particular homomorphisms for the call/cc lang *)
From gitrees Require Import gitree lang_generic.
From gitrees Require Export hom.
From gitrees.examples.input_lang_callcc Require Import lang interp.
Expand Down Expand Up @@ -74,8 +73,8 @@ Section hom.
Qed.

Program Definition OutputSCtx_HOM {S : Set}
(env : @interp_scope F A _ S)
: @HOM _ _ A _ _ := exist _ ((interp_outputk rs (λne env, idfun) env)) _.
(env : @interp_scope F A _ S) : HOM (A:=natO)
:= exist _ ((interp_outputk rs (λne env, idfun) env)) _.
Next Obligation.
intros; simpl.
apply _.
Expand Down
2 changes: 2 additions & 0 deletions theories/hom.v
Original file line number Diff line number Diff line change
@@ -1,3 +1,5 @@
(** In this module, we package up IT homomorphism in a sigma type, and
we will use it as a domain for logical relations on continuations *)
From gitrees Require Import gitree lang_generic.
Require Import Binding.Lib Binding.Set Binding.Env.

Expand Down

0 comments on commit b91709c

Please sign in to comment.