[Agda] A question on Setoid in the standard library

David Leduc david.leduc6 at googlemail.com
Wed Sep 22 17:34:34 CEST 2010


I do not understand why the following code results in a parsing error.
Please someone, help me.

{-# OPTIONS --universe-polymorphism #-}

module test where

open import Level
open import Relation.Binary
open import Data.Bool

f : (c l : Level)(A : DecSetoid c l) ->
    DecSetoid.Carrier A -> DecSetoid.Carrier A -> Bool
f c l A X Y with DecSetoid._≟_ A X Y
... | yes _ = true
... | no _ = true


More information about the Agda mailing list