Coinduction.agda 264 B

123456789101112
  1. module Common.Coinduction where
  2. postulate
  3. ∞ : ∀ {a} (A : Set a) → Set a
  4. ♯_ : ∀ {a} {A : Set a} → A → ∞ A
  5. ♭ : ∀ {a} {A : Set a} → ∞ A → A
  6. {-# BUILTIN INFINITY ∞ #-}
  7. {-# BUILTIN SHARP ♯_ #-}
  8. {-# BUILTIN FLAT ♭ #-}