Skip to content

Commit e9b7abd

Browse files
[Refractor] contradiction over ⊥-elim in ¬¬-pull def (#2659)
* [Refractor] contradiction over ⊥-elim in ¬¬-pull def * remove bot/elim * Update src/Relation/Nullary/Universe.agda --------- Co-authored-by: jamesmckinna <[email protected]>
1 parent 3236742 commit e9b7abd

File tree

1 file changed

+3
-3
lines changed

1 file changed

+3
-3
lines changed

src/Relation/Nullary/Universe.agda

+3-3
Original file line numberDiff line numberDiff line change
@@ -12,14 +12,14 @@ open import Data.Sum.Base as Sum hiding (map)
1212
open import Data.Sum.Relation.Binary.Pointwise using (_⊎ₛ_; inj₁; inj₂)
1313
open import Data.Product.Base as Product hiding (map)
1414
open import Data.Product.Relation.Binary.Pointwise.NonDependent using (_×ₛ_)
15-
open import Data.Empty using (⊥; ⊥-elim)
15+
open import Data.Empty using (⊥)
1616
open import Effect.Applicative using (RawApplicative)
1717
open import Effect.Monad using (RawMonad)
1818
open import Function.Base using (_∘_; id)
1919
open import Function.Indexed.Relation.Binary.Equality using (≡-setoid)
2020
open import Level using (Level; _⊔_; suc; Lift; lift; lower)
2121
open import Relation.Nullary.Negation
22-
using (¬_; ¬¬-Monad; ¬¬-map; negated-stable)
22+
using (¬_; contradiction; ¬¬-Monad; ¬¬-map; negated-stable)
2323
open import Relation.Binary.Core using (Rel)
2424
open import Relation.Binary.Bundles using (Setoid)
2525
import 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

Comments
 (0)