@@ -12,14 +12,14 @@ open import Data.Sum.Base as Sum hiding (map)
1212open import Data.Sum.Relation.Binary.Pointwise using (_⊎ₛ_; inj₁; inj₂)
1313open import Data.Product.Base as Product hiding (map)
1414open import Data.Product.Relation.Binary.Pointwise.NonDependent using (_×ₛ_)
15- open import Data.Empty using (⊥; ⊥-elim )
15+ open import Data.Empty using (⊥)
1616open import Effect.Applicative using (RawApplicative)
1717open import Effect.Monad using (RawMonad)
1818open import Function.Base using (_∘_; id)
1919open import Function.Indexed.Relation.Binary.Equality using (≡-setoid)
2020open import Level using (Level; _⊔_; suc; Lift; lift; lower)
2121open import Relation.Nullary.Negation
22- using (¬_; ¬¬-Monad; ¬¬-map; negated-stable)
22+ using (¬_; contradiction; ¬¬-Monad; ¬¬-map; negated-stable)
2323open import Relation.Binary.Core using (Rel)
2424open import Relation.Binary.Bundles using (Setoid)
2525import Relation.Binary.Construct.Always as Always using (setoid)
@@ -123,7 +123,7 @@ private
123123 ⟦ F ⟧ (¬ ¬ P) → ¬ ¬ ⟦ F ⟧ P
124124¬¬-pull = sequence rawApplicative
125125 (λ 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 )))
127127
128128¬¬-remove : ∀ {p} (F : PropF p) {P} →
129129 ¬ ¬ ⟦ F ⟧ (¬ ¬ P) → ¬ ¬ ⟦ F ⟧ P
0 commit comments