File tree 1 file changed +3
-3
lines changed
src/Relation/Nullary/Decidable
1 file changed +3
-3
lines changed Original file line number Diff line number Diff line change @@ -170,11 +170,11 @@ proof (map′ A→B B→A (false because [¬a])) = of (invert [¬a] ∘ B→A)
170
170
-- Decidable predicates are stable.
171
171
172
172
decidable-stable : Dec A → Stable A
173
- decidable-stable (yes a ) ¬¬a = a
174
- decidable-stable (no ¬a ) ¬¬a = contradiction ¬a ¬¬a
173
+ decidable-stable (true because [a] ) ¬¬a = invert [a]
174
+ decidable-stable (false because [¬a] ) ¬¬a = contradiction (invert [¬a]) ¬¬a
175
175
176
176
¬-drop-Dec : Dec (¬ ¬ A) → Dec (¬ A)
177
- ¬-drop-Dec ¬¬a? = map′ negated-stable ( λ ¬a ¬¬a → contradiction ¬a ¬¬a) (¬? ¬¬a?)
177
+ ¬-drop-Dec ¬¬a? = map′ negated-stable contradiction (¬? ¬¬a?)
178
178
179
179
-- A double-negation-translated variant of excluded middle (or: every
180
180
-- nullary relation is decidable in the double-negation monad).
You can’t perform that action at this time.
0 commit comments