------------------------------------------------------------------------ -- The Agda standard library -- -- Coinductive lists where all elements satisfy a predicate ------------------------------------------------------------------------ {-# OPTIONS --cubical-compatible --guardedness #-} module Codata.Musical.Colist.Relation.Unary.All where open import Codata.Musical.Colist.Base open import Codata.Musical.Notation open import Level using (Level; _⊔_) open import Relation.Unary using (Pred) private variable a b p : Level A : Set a B : Set b P : Pred A p data All {A : Set a} (P : Pred A p) : Pred (Colist A) (a ⊔ p) where [] : All P [] _∷_ : ∀ {x xs} (px : P x) (pxs : ∞ (All P (♭ xs))) → All P (x ∷ xs) infixr 5 _∷_
RetroSearch is an open source project built by @garambo | Open a GitHub Issue
Search and Browse the WWW like it's 1997 | Search results from DuckDuckGo
HTML:
3.2
| Encoding:
UTF-8
| Version:
0.7.4