Prove join univ pi contra

This commit is contained in:
Yiyun Liu 2024-12-25 21:11:58 -05:00
parent e2702ed277
commit 80d8b13e49
4 changed files with 202 additions and 8 deletions

4
theories/logrel.v Normal file
View file

@ -0,0 +1,4 @@
Require Import Autosubst2.core Autosubst2.fintype Autosubst2.syntax.
Definition ProdSpace {n} (PA : Tm n -> Prop)
(PF : Tm n -> (Tm n -> Prop) -> Prop) : Tm n -> Prop :=
fun b => forall a PB, PA a -> PF a PB -> PB (App b a).