Base.agda 617 B

1234567891011121314151617181920212223242526272829303132333435363738
  1. module Base where
  2. postulate String : Set
  3. Char : Set
  4. {-# BUILTIN STRING String #-}
  5. {-# BUILTIN CHAR Char #-}
  6. data Unit : Set where
  7. unit : Unit
  8. {-# COMPILED_DATA Unit () #-}
  9. data Bool : Set where
  10. true : Bool
  11. false : Bool
  12. data False : Set where
  13. record True : Set where
  14. IsTrue : Bool -> Set
  15. IsTrue true = True
  16. IsTrue false = False
  17. {-# COMPILED_DATA Bool True False #-}
  18. infixr 40 _::_
  19. data List (A : Set) : Set where
  20. [] : List A
  21. _::_ : A -> List A -> List A
  22. {-# COMPILED_DATA List [] (:) #-}
  23. data _×_ (A B : Set) : Set where
  24. _,_ : A -> B -> A × B
  25. {-# COMPILED_DATA _×_ (,) #-}