用下面的阿格達代碼的時候,我在A₂得到的B定義的錯誤: module Whatever where
module A₁ where
data B : Set where
module A₂ where
open A₁ renaming (B to B₁)
data B : Set where
的錯誤信息是: Duplicate definition of
data MinList (min : ℕ) : Set where
[] : MinList min
_∷⟪_⟫_ : (x : ℕ) -> min ≤ x -> MinList x -> MinList min
任何理想是什麼< < >>是什麼意思? 或什麼的 _∷⟪_⟫_ : (x : ℕ) -> min ≤ x -> MinList x -> MinList min
我有兩個密切相關的問題: 首先,如何能在Haskell的箭類建模/在阿格達代表? class Arrow a where
arr :: (b -> c) -> a b c
(>>>) :: a b c -> a c d -> a b d
first :: a b c -> a (b,d) (c,d)
second :: a b c -> a (d,b