@@ -12,14 +12,14 @@ open import Data.Sum.Base as Sum hiding (map)
12
12
open import Data.Sum.Relation.Binary.Pointwise using (_⊎ₛ_; inj₁; inj₂)
13
13
open import Data.Product.Base as Product hiding (map)
14
14
open import Data.Product.Relation.Binary.Pointwise.NonDependent using (_×ₛ_)
15
- open import Data.Empty using (⊥; ⊥-elim )
15
+ open import Data.Empty using (⊥)
16
16
open import Effect.Applicative using (RawApplicative)
17
17
open import Effect.Monad using (RawMonad)
18
18
open import Function.Base using (_∘_; id)
19
19
open import Function.Indexed.Relation.Binary.Equality using (≡-setoid)
20
20
open import Level using (Level; _⊔_; suc; Lift; lift; lower)
21
21
open import Relation.Nullary.Negation
22
- using (¬_; ¬¬-Monad; ¬¬-map; negated-stable)
22
+ using (¬_; contradiction; ¬¬-Monad; ¬¬-map; negated-stable)
23
23
open import Relation.Binary.Core using (Rel)
24
24
open import Relation.Binary.Bundles using (Setoid)
25
25
import Relation.Binary.Construct.Always as Always using (setoid)
@@ -123,7 +123,7 @@ private
123
123
⟦ F ⟧ (¬ ¬ P) → ¬ ¬ ⟦ F ⟧ P
124
124
¬¬-pull = sequence rawApplicative
125
125
(λ f → f lower)
126
- (λ f g → g (λ x → ⊥-elim (f x ( λ y → g (λ _ → y)))))
126
+ (λ f g → g (λ x → contradiction ( λ y → g (λ _ → y)) (f x )))
127
127
128
128
¬¬-remove : ∀ {p} (F : PropF p) {P} →
129
129
¬ ¬ ⟦ F ⟧ (¬ ¬ P) → ¬ ¬ ⟦ F ⟧ P
0 commit comments