Prove the fundamental theorem

This commit is contained in:
Yiyun Liu 2025-02-06 18:09:19 -05:00
parent 399c97fa82
commit 6daa275ac8
2 changed files with 17 additions and 0 deletions

11
theories/soundness.v Normal file
View file

@ -0,0 +1,11 @@
Require Import Autosubst2.fintype Autosubst2.syntax.
Require Import fp_red logrel typing.
From Hammer Require Import Tactics.
Theorem fundamental_theorem :
(forall n (Γ : fin n -> PTm n), Γ -> Γ) /\
(forall n Γ (a A : PTm n), Γ a A -> Γ a A) /\
(forall n Γ (a b A : PTm n), Γ a b A -> Γ a b A).
apply wt_mutual; eauto with sem;[idtac].
hauto l:on use:SE_Pair.
Qed.