Skip to content

Commit

Permalink
cleanup
Browse files Browse the repository at this point in the history
  • Loading branch information
Kaptch committed Feb 1, 2024
1 parent ddddc3f commit 12c70c5
Show file tree
Hide file tree
Showing 21 changed files with 777 additions and 728 deletions.
2 changes: 2 additions & 0 deletions _CoqProject
Original file line number Diff line number Diff line change
Expand Up @@ -48,3 +48,5 @@ theories/lib/pairs.v
theories/lib/while.v
theories/lib/factorial.v
theories/lib/iter.v

theories/utils/finite_sets.v
3 changes: 1 addition & 2 deletions theories/effects/store.v
Original file line number Diff line number Diff line change
Expand Up @@ -125,14 +125,13 @@ Section constructors.
(λne _, Next (Ret ())).
End constructors.


Section wp.
Context {n : nat}.
Variable (rs : gReifiers NotCtxDep n).
Context {R} `{!Cofe R}.
Context `{!SubOfe unitO R}.

Notation F := (gReifiers_ops NotCtxDep rs).
Notation F := (gReifiers_ops rs).
Notation IT := (IT F R).
Notation ITV := (ITV F R).
Notation stateO := (stateF ♯ IT).
Expand Down
7 changes: 3 additions & 4 deletions theories/examples/affine_lang/lang.v
Original file line number Diff line number Diff line change
Expand Up @@ -10,9 +10,8 @@ Module io_lang.
Definition expr := input_lang.lang.expr.
Definition tyctx {S : Set} := S → ty.
Definition typed {S : Set} := input_lang.lang.typed (S:=S).
Program Definition ı_scope {sz} (rs : gReifiers NotCtxDep sz) `{!subReifier reify_io rs} {R} `{!Cofe R} : @interp_scope (gReifiers_ops NotCtxDep rs) R _ Empty_set := λne (x : ∅), match x with end.
Definition interp_closed {sz} (rs : gReifiers NotCtxDep sz) `{!subReifier reify_io rs} (e : expr ∅) {R} `{!Cofe R, !SubOfe natO R} : IT (gReifiers_ops NotCtxDep rs) R :=
input_lang.interp.interp_expr rs e (ı_scope rs).
Definition interp_closed {sz} (rs : gReifiers NotCtxDep sz) `{!subReifier reify_io rs} (e : expr ∅) {R} `{!Cofe R, !SubOfe natO R} : IT (gReifiers_ops rs) R :=
input_lang.interp.interp_expr rs e ı_scope.
End io_lang.

Require Import Binding.Resolver Binding.Lib Binding.Set Binding.Auto Binding.Env.
Expand Down Expand Up @@ -51,7 +50,7 @@ Section affine.
Variable rs : gReifiers NotCtxDep sz.
Context `{!subReifier reify_store rs}.
Context `{!subReifier reify_io rs}.
Notation F := (gReifiers_ops NotCtxDep rs).
Notation F := (gReifiers_ops rs).
Context {R : ofe}.
Context `{!Cofe R, !SubOfe unitO R, !SubOfe natO R, !SubOfe locO R}.
Notation IT := (IT F R).
Expand Down
Loading

0 comments on commit 12c70c5

Please sign in to comment.