Maybe.agda 161 B

12345678910
  1. module Lib.Maybe where
  2. data Maybe (A : Set) : Set where
  3. nothing : Maybe A
  4. just : A -> Maybe A
  5. {-# COMPILE GHC Maybe = data Maybe (Nothing | Just) #-}