Finish refactoring substitution lemmas

This commit is contained in:
Yiyun Liu 2025-03-03 15:22:59 -05:00
parent 896d22ac9b
commit d68adf85f4
4 changed files with 244 additions and 235 deletions

View file

@ -12,14 +12,6 @@ Require Import Autosubst2.core Autosubst2.unscoped Autosubst2.syntax common.
Require Import Btauto.
Require Import Cdcl.Itauto.
Lemma subst_scons_id (a : PTm) :
subst_PTm (scons (VarPTm 0) (funcomp VarPTm shift)) a = a.
Proof.
have E : subst_PTm VarPTm a = a by asimpl.
rewrite -{2}E.
apply ext_PTm. case => //=.
Qed.
Ltac2 spec_refl () :=
List.iter
(fun a => match a with