File tree 1 file changed +2
-2
lines changed
1 file changed +2
-2
lines changed Original file line number Diff line number Diff line change @@ -15,7 +15,7 @@ open import Data.Sum.Base using (_⊎_; [_,_])
15
15
open import Function.Base using (_∘_; _|>_)
16
16
open import Level using (Level; _⊔_; 0ℓ; suc; Lift)
17
17
open import Relation.Nullary.Decidable.Core using (Dec; True)
18
- open import Relation.Nullary.Negation.Core as Negation using (¬_)
18
+ open import Relation.Nullary.Negation.Core as Nullary using (¬_)
19
19
open import Relation.Binary.PropositionalEquality.Core using (_≡_)
20
20
21
21
private
@@ -165,7 +165,7 @@ syntax IUniversal P = ∀[ P ]
165
165
-- Stability - instances of P are stable wrt double negation
166
166
167
167
Stable : Pred A ℓ → Set _
168
- Stable P = ∀ x → Negation .Stable (P x)
168
+ Stable P = ∀ x → Nullary .Stable (P x)
169
169
170
170
-- Decidability - it is possible to determine if an arbitrary element
171
171
-- satisfies P.
You can’t perform that action at this time.
0 commit comments