Skip to content

Commit

Permalink
Update syntax
Browse files Browse the repository at this point in the history
  • Loading branch information
Ailrun committed Dec 13, 2023
1 parent 2e9baff commit f4817d4
Showing 1 changed file with 5 additions and 4 deletions.
9 changes: 5 additions & 4 deletions theories/System.v
Original file line number Diff line number Diff line change
Expand Up @@ -15,9 +15,10 @@ Reserved Notation "x : T ∈! Γ" (no associativity, at level 80).

Generalizable All Variables.

#[local] Open Scope exp_scope.
Inductive ctx_lookup : nat -> Typ -> Ctx -> Prop :=
| here : `( 0 : ( {{ T[$wk] }}%exp ) ∈! (T :: Γ) )
| there : `( n : T ∈! Γ -> (S n) : {{ T[$wk] }}%exp ∈! (T' :: Γ) )
| here : `( 0 : {{ T[$wk] }} ∈! (T :: Γ) )
| there : `( n : T ∈! Γ -> (S n) : {{ T[$wk] }} ∈! (T' :: Γ) )
where "x : T ∈! Γ" := (ctx_lookup x T Γ).


Expand Down Expand Up @@ -58,14 +59,14 @@ with wf_term : Ctx -> exp -> Typ -> Prop :=
| wf_vlookup : `(
⊢ Γ ->
x : T ∈! Γ ->
Γ ⊢ {{ #x }}%exp : T
Γ ⊢ {{ #x }} : T
)
| wf_fun_e: `(
Γ ⊢ A : typ i ->
A :: Γ ⊢ B : typ i ->
Γ ⊢ M : Π A B ->
Γ ⊢ N : A ->
Γ ⊢ {{ M N }}%exp : {{ B[$id,N] }}%exp
Γ ⊢ {{ M N }} : {{ B[$id,N] }}
)
| wf_fun_i : `(
Γ ⊢ A : typ i ->
Expand Down

0 comments on commit f4817d4

Please sign in to comment.