N-ary expansions (#113)

This commit is contained in:
Patrick Stevens
2020-04-12 12:16:20 +01:00
committed by GitHub
parent 380548134d
commit 269f2aa14f
11 changed files with 156 additions and 217 deletions

View File

@@ -1,4 +1,3 @@
{-# OPTIONS --safe --warning=error --without-K --guardedness #-}
open import Agda.Primitive using (Level; lzero; lsuc; _⊔_)
@@ -53,9 +52,6 @@ StrictlyIncreasing x = (n : ) → (index x n) < (index x (succ n))
Increasing : Sequence A Set (b c)
Increasing x = (n : ) ((index x n) < (index x (succ n))) || ((index x n) (index x (succ n)))
Bounded : Sequence A Set (a c)
Bounded x = Sg A (λ K (n : ) index x n < K)
sequencePredicate : (x : Sequence A) A Set b
sequencePredicate x a = Sg (λ n index x n a)