Finish the soundness proof completely
This commit is contained in:
parent
d24991e994
commit
bdba6f50e5
3 changed files with 119 additions and 5 deletions
|
@ -91,3 +91,7 @@ Proof. case : a => //=. Qed.
|
|||
Definition ispair_ren n m (a : PTm n) (ξ : fin n -> fin m) :
|
||||
ispair (ren_PTm ξ a) = ispair a.
|
||||
Proof. case : a => //=. Qed.
|
||||
|
||||
Definition ishne_ren n m (a : PTm n) (ξ : fin n -> fin m) :
|
||||
ishne (ren_PTm ξ a) = ishne a.
|
||||
Proof. move : m ξ. elim : n / a => //=. Qed.
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue