File tree 3 files changed +15
-8
lines changed
3 files changed +15
-8
lines changed Original file line number Diff line number Diff line change @@ -407,6 +407,11 @@ Additions to existing modules
407
407
WeaklyDecidable : Set _
408
408
```
409
409
410
+ * Added new proof in ` Relation.Nullary.Decidable.Core ` :
411
+ ``` agda
412
+ recompute-irr : (a? : Dec A) (p q : A) → recompute a? p ≡ recompute a? q
413
+ ```
414
+
410
415
* Added new proof in ` Relation.Nullary.Decidable ` :
411
416
``` agda
412
417
⌊⌋-map′ : (a? : Dec A) → ⌊ map′ t f a? ⌋ ≡ ⌊ a? ⌋
@@ -419,13 +424,8 @@ Additions to existing modules
419
424
420
425
* Added new definitions in ` Relation.Nullary.Reflects ` :
421
426
``` agda
422
- recompute : Reflects A b → Recomputable A
423
- ```
424
-
425
- * Added new definitions in ` Relation.Unary `
426
- ```
427
- Stable : Pred A ℓ → Set _
428
- WeaklyDecidable : Pred A ℓ → Set _
427
+ recompute : Reflects A b → Recomputable A
428
+ recompute-irr : (r : Reflects A b) (p q : A) → recompute r p ≡ recompute r q
429
429
```
430
430
431
431
* Added new definitions in ` Relation.Unary `
Original file line number Diff line number Diff line change @@ -18,9 +18,10 @@ open import Data.Product.Base using (_×_)
18
18
open import Data.Sum.Base using (_⊎_)
19
19
open import Function.Base using (_∘_; const; _$_; flip)
20
20
open import Relation.Nullary.Recomputable
21
- open import Relation.Nullary.Reflects as Reflects hiding (recompute)
21
+ open import Relation.Nullary.Reflects as Reflects hiding (recompute; recompute-irr )
22
22
open import Relation.Nullary.Negation.Core
23
23
using (¬_; Stable; negated-stable; contradiction; DoubleNegation)
24
+ open import Agda.Builtin.Equality using (_≡_)
24
25
25
26
private
26
27
variable
@@ -73,6 +74,9 @@ module _ {A : Set a} where
73
74
recompute : Dec A → Recomputable A
74
75
recompute = Reflects.recompute ∘ proof
75
76
77
+ recompute-irr : (a? : Dec A) (p q : A) → recompute a? p ≡ recompute a? q
78
+ recompute-irr = Reflects.recompute-irr ∘ proof
79
+
76
80
------------------------------------------------------------------------
77
81
-- Interaction with negation, sum, product etc.
78
82
Original file line number Diff line number Diff line change @@ -61,6 +61,9 @@ recompute : ∀ {b} → Reflects A b → Recomputable A
61
61
recompute (ofʸ a) _ = a
62
62
recompute (ofⁿ ¬a) a = contradiction-irr a ¬a
63
63
64
+ recompute-irr : ∀ {b} (r : Reflects A b) (p q : A) → recompute r p ≡ recompute r q
65
+ recompute-irr r p q = refl
66
+
64
67
------------------------------------------------------------------------
65
68
-- Interaction with negation, product, sums etc.
66
69
You can’t perform that action at this time.
0 commit comments