Move projection axioms to the subtyping relation
This commit is contained in:
parent
2e2e41cbe6
commit
0e5b82b162
4 changed files with 96 additions and 21 deletions
3
theories/common.v
Normal file
3
theories/common.v
Normal file
|
@ -0,0 +1,3 @@
|
|||
Require Import Autosubst2.fintype Autosubst2.syntax.
|
||||
Definition renaming_ok {n m} (Γ : fin n -> PTm n) (Δ : fin m -> PTm m) (ξ : fin m -> fin n) :=
|
||||
forall (i : fin m), ren_PTm ξ (Δ i) = Γ (ξ i).
|
Loading…
Add table
Add a link
Reference in a new issue