Coinduction.agda 194 B

123456789
  1. {-# OPTIONS --without-K --guardedness #-}
  2. module Common.Coinduction where
  3. open import Agda.Builtin.Coinduction public
  4. private
  5. my-♯ : ∀ {a} {A : Set a} → A → ∞ A
  6. my-♯ x = ♯ x