mirror of
https://github.com/luau-lang/luau.git
synced 2024-11-15 22:35:43 +08:00
c5477d522d
* First cut of strict mode Co-authored-by: Lily Brown <lily@lily.fyi>
15 lines
386 B
Agda
15 lines
386 B
Agda
module FFI.Data.Maybe where
|
|
|
|
open import Agda.Builtin.Equality using (_≡_; refl)
|
|
|
|
{-# FOREIGN GHC import qualified Data.Maybe #-}
|
|
|
|
data Maybe (A : Set) : Set where
|
|
nothing : Maybe A
|
|
just : A → Maybe A
|
|
{-# COMPILE GHC Maybe = data Data.Maybe.Maybe (Data.Maybe.Nothing|Data.Maybe.Just) #-}
|
|
|
|
just-inv : ∀ {A} {x y : A} → (just x ≡ just y) → (x ≡ y)
|
|
just-inv refl = refl
|
|
|