mirror of
https://github.com/Smaug123/agdaproofs
synced 2025-10-13 07:38:40 +00:00
N-ary expansions (#113)
This commit is contained in:
@@ -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)
|
||||
|
||||
|
Reference in New Issue
Block a user