Base.agda 133 B

123456789101112
  1. module Logic where
  2. data True : Set where
  3. tt : True
  4. infix 10 _/\_
  5. data _/\_ (P Q : Set) : Set where
  6. <_,_> : P -> Q -> P /\ Q