如何添加兩個理性..我正在嘗試這個,但這是不正確的。因爲我無法證明這個coprime部分。 open import Data.Rational
open import Data.Integer
open import Data.Nat
_add_ : ℚ -> ℚ -> ℚ
x add y = (nx Data.Integer.* dy Data.Integer.+ dx Data.In
So類型的預期用途是什麼?音譯成阿格達: data So : Bool → Set where
oh : So true
So升降機布爾命題到邏輯一。 Oury和Swierstra的介紹性文章The Power of Pi給出了一個由表格列索引的關係代數的例子。以兩個表的產品需要,他們有不同的列,爲此,他們使用So: Schema = List (String × U) -- U i
我能夠輕易獲得密鑰列表如下: open import Relation.Binary
open import Relation.Binary.PropositionalEquality using (_≡_)
module AVL-Tree-Functions
{ k v ℓ } { Key : Set k }
(Value : Key → Set v)
{ _
這裏是一個類似於在Data.List.All一個定義: open import Data.Vec
data All {α π} {A : Set α} (P : A -> Set π) : ∀ {n} -> Vec A n -> Set π where
[]ₐ : All P []
_∷ₐ_ : ∀ {n x} {xs : Vec A n} -> P x -> All P
恢復型 比方說,我有一個數據類型: data Term : Type -> Type where
Id : Term (a -> a)
...
App : Term (a -> b) -> Term a -> Term b
有了一個證明事情是App: data So : Bool -> Type where
Oh : So True
isApp :