Skip to content

Commit

Permalink
Fix compilation error
Browse files Browse the repository at this point in the history
  • Loading branch information
kyoDralliam committed Nov 13, 2023
1 parent 894b77c commit 611e031
Show file tree
Hide file tree
Showing 3 changed files with 7 additions and 2 deletions.
2 changes: 1 addition & 1 deletion _CoqProject
Original file line number Diff line number Diff line change
Expand Up @@ -25,7 +25,7 @@ theories/DirectedDirections.v
theories/DirectedContext.v
theories/DirectedDirectioning.v
theories/DirectedSemantics.v

theories/DirectedDeclarativeTyping.v

theories/LogicalRelation.v
theories/LogicalRelation/Induction.v
Expand Down
4 changes: 3 additions & 1 deletion theories/DirectedSemantics.v
Original file line number Diff line number Diff line change
Expand Up @@ -3,8 +3,8 @@ From Coq Require Import ssreflect.
From Equations Require Import Equations.
From smpl Require Import Smpl.
From LogRel.AutoSubst Require Import core unscoped Ast Extra.
From LogRel Require Import DirectedDirections DirectedContext DirectedDirectioning DirectedDeclarativeTyping.
From LogRel Require Import Utils BasicAst.
From LogRel Require Import DirectedDirections DirectedContext DirectedDirectioning.

Reserved Notation "[ Δ |- w : t -( d )- u : A ]" (at level 0, Δ, d, t, u, A, w at level 50).
Reserved Notation "[ Δ |- ϕ : σ -( )- τ : Θ ]" (at level 0, Δ, Θ, σ, τ, ϕ at level 50).
Expand Down Expand Up @@ -113,6 +113,8 @@ Section MorphismDefinition.

where "[ Δ |- w : t -( d )- u : A ]" := (TermRel Δ t u d A w).

Close Scope typing_scope.

Context (type_act : forall (γ : list direction) (dA : direction) (A : term) (wdA : [γ |- A ◃ dA]) (σ τ : nat -> term) (φ : list term), term).

(* Given a context of directions γ coming from Θ,
Expand Down
3 changes: 3 additions & 0 deletions theories/DirectedTyping.v
Original file line number Diff line number Diff line change
Expand Up @@ -284,6 +284,9 @@ Module Examples.

Definition ctx := εᵈ ,, Fun \ U @ Discr ,, Cofun \ tProd (tRel 0) U @ Cofun.

[ Θ |-(Fun) A ]
[ Θ ,, Discr \ A @ Fun |-(Cofun) B ]

Definition sup_ctx
(* tW should bind one variable in its second argument *)
(tW : term -> term -> term) :=
Expand Down

0 comments on commit 611e031

Please sign in to comment.