File tree Expand file tree Collapse file tree 1 file changed +3
-2
lines changed
Expand file tree Collapse file tree 1 file changed +3
-2
lines changed Original file line number Diff line number Diff line change 88
99module Data.Nat.InfinitelyOften where
1010
11- open import Effect.Monad using (RawMonad)
12- open import Level using (Level; 0ℓ)
1311open import Data.Nat.Base using (ℕ; _≤_; _⊔_; _+_; suc; zero; s≤s)
1412open import Data.Nat.Properties
1513open import Data.Product.Base as Prod hiding (map)
1614open import Data.Sum.Base using (inj₁; inj₂; _⊎_)
15+ open import Effect.Monad using (RawMonad)
1716open import Function.Base using (_∘_; id)
17+ open import Level using (Level; 0ℓ)
1818open import Relation.Binary.PropositionalEquality.Core using (_≢_)
1919open import Relation.Nullary.Negation using (¬¬-Monad; call/cc)
2020open import Relation.Nullary.Negation.Core using (¬_; contradiction)
2121open import Relation.Unary using (Pred; _∪_; _⊆_)
22+ open import Relation.Nullary.Negation.Core using (contradiction)
2223
2324open RawMonad (¬¬-Monad {a = 0ℓ})
2425
You can’t perform that action at this time.
0 commit comments