Finish soundness for subtyping

This commit is contained in:
Yiyun Liu 2025-02-17 18:34:48 -05:00
parent ef3de3af3d
commit 067ae89b1d
2 changed files with 52 additions and 0 deletions

View file

@ -2780,3 +2780,7 @@ Module Sub.
hauto ctrs:rtc use:REReds.cong', Sub1.substing.
Qed.
End Sub.
Module ESub.
Definition R {n} (a b : PTm n) := exists c0 c1, rtc ERed.R a c0 /\ rtc ERed.R b c1 /\ Sub1.R c0 c1.
End ESub.