Char.agda 74 B

12345678
  1. module Data.Char where
  2. postulate Char : Set
  3. {-# BUILTIN CHAR Char #-}