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 8
8
9
9
module Data.Nat.InfinitelyOften where
10
10
11
- open import Effect.Monad using (RawMonad)
12
- open import Level using (Level; 0ℓ)
13
11
open import Data.Nat.Base using (ℕ; _≤_; _⊔_; _+_; suc; zero; s≤s)
14
12
open import Data.Nat.Properties
15
13
open import Data.Product.Base as Prod hiding (map)
16
14
open import Data.Sum.Base using (inj₁; inj₂; _⊎_)
15
+ open import Effect.Monad using (RawMonad)
17
16
open import Function.Base using (_∘_; id)
17
+ open import Level using (Level; 0ℓ)
18
18
open import Relation.Binary.PropositionalEquality.Core using (_≢_)
19
19
open import Relation.Nullary.Negation using (¬¬-Monad; call/cc)
20
20
open import Relation.Nullary.Negation.Core using (¬_; contradiction)
21
21
open import Relation.Unary using (Pred; _∪_; _⊆_)
22
+ open import Relation.Nullary.Negation.Core using (contradiction)
22
23
23
24
open RawMonad (¬¬-Monad {a = 0ℓ})
24
25
You can’t perform that action at this time.
0 commit comments