summaryrefslogtreecommitdiff
path: root/Examples.agda
diff options
context:
space:
mode:
authorHelmut Grohne <grohne@cs.uni-bonn.de>2014-02-10 15:49:35 +0100
committerHelmut Grohne <grohne@cs.uni-bonn.de>2014-02-10 15:49:35 +0100
commit04b7bf8fabf64a2414d64cfb385f6a397da0a0fb (patch)
tree361986e772b733b199d868a4810e6721077dee1b /Examples.agda
parent0a1558b7cb0bccbe4a8c8411ac08d11a87547eea (diff)
downloadbidiragda-04b7bf8fabf64a2414d64cfb385f6a397da0a0fb.tar.gz
add sieve to examples
Diffstat (limited to 'Examples.agda')
-rw-r--r--Examples.agda9
1 files changed, 8 insertions, 1 deletions
diff --git a/Examples.agda b/Examples.agda
index 70628a5..5971460 100644
--- a/Examples.agda
+++ b/Examples.agda
@@ -1,6 +1,6 @@
module Examples where
-open import Data.Nat using (ℕ ; zero ; suc ; _⊓_ ; _∸_)
+open import Data.Nat using (ℕ ; zero ; suc ; _⊓_ ; _∸_ ; ⌈_/2⌉)
open import Data.Vec using (Vec ; [] ; _∷_ ; reverse ; _++_)
import GetTypes
@@ -37,3 +37,10 @@ drop' n = assume-get (f n)
f zero xs = xs
f (suc n) [] = []
f (suc n) (x ∷ xs) = f n xs
+
+sieve' : Get
+sieve' = assume-get f
+ where f : {A : Set} {n : ℕ} → Vec A n → Vec A ⌈ n /2⌉
+ f [] = []
+ f (x ∷ []) = x ∷ []
+ f (x ∷ _ ∷ xs) = x ∷ f xs