Coinduction.agda 330 B

123456789101112131415
  1. {-# OPTIONS --universe-polymorphism #-}
  2. module Common.Coinduction where
  3. open import Common.Level
  4. postulate
  5. ∞ : ∀ {a} (A : Set a) → Set a
  6. ♯_ : ∀ {a} {A : Set a} → A → ∞ A
  7. ♭ : ∀ {a} {A : Set a} → ∞ A → A
  8. {-# BUILTIN INFINITY ∞ #-}
  9. {-# BUILTIN SHARP ♯_ #-}
  10. {-# BUILTIN FLAT ♭ #-}