Make progress on wt_unique
This commit is contained in:
parent
fbbce90304
commit
5eb1f9df0b
6 changed files with 145 additions and 31 deletions
theories
|
@ -39,7 +39,7 @@ Inductive Wt : list Tm -> Tm -> Tm -> Prop :=
|
|||
| T_Abs Γ a A B i :
|
||||
Γ ⊢ TBind TPi A B ∈ (Univ i) ->
|
||||
(cons A Γ) ⊢ a ∈ B ->
|
||||
Γ ⊢ Abs a ∈ TBind TPi A B
|
||||
Γ ⊢ Abs A a ∈ TBind TPi A B
|
||||
|
||||
| T_App Γ b a A B :
|
||||
Γ ⊢ b ∈ TBind TPi A B ->
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue