Load.agda 65 B

123456
  1. module Load where
  2. data Bool : Set where
  3. tt : Bool
  4. ff : Bool