pair-eta/theories/logrel.v

5 lines
229 B
Coq
Raw Normal View History

2024-12-25 21:11:58 -05:00
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).