Seems to work but takes a million years to type check
This commit is contained in:
parent
6c11f5560d
commit
7503dea251
5 changed files with 580 additions and 572 deletions
|
@ -4,6 +4,7 @@ Import Ltac2.Notations.
|
|||
Import Ltac2.Control.
|
||||
From Hammer Require Import Tactics.
|
||||
|
||||
|
||||
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