Maybe.agda 142 B

1234567
  1. {-# OPTIONS --without-K #-}
  2. module Common.Maybe where
  3. data Maybe {a} (A : Set a) : Set a where
  4. nothing : Maybe A
  5. just : A → Maybe A