Logic.agda 80 B

123456789
  1. module Logic where
  2. data True : Set where
  3. tt : True
  4. data False : Set where