File tree 2 files changed +10
-1
lines changed
2 files changed +10
-1
lines changed Original file line number Diff line number Diff line change @@ -140,3 +140,8 @@ Additions to existing modules
140
140
141
141
* In ` Function.Bundles ` , added ` _⟶ₛ_ ` as a synonym for ` Func ` that can
142
142
be used infix.
143
+
144
+ * Added new proof in ` Relation.Nullary.Decidable ` :
145
+ ``` agda
146
+ ⌊⌋-map′ : (a? : Dec A) → ⌊ map′ t f a? ⌋ ≡ ⌊ a? ⌋
147
+ ```
Original file line number Diff line number Diff line change @@ -19,7 +19,8 @@ open import Relation.Binary.Bundles using (Setoid; module Setoid)
19
19
open import Relation.Binary.Definitions using (Decidable)
20
20
open import Relation.Nullary
21
21
open import Relation.Nullary.Reflects using (invert)
22
- open import Relation.Binary.PropositionalEquality.Core using (_≡_; refl; cong′)
22
+ open import Relation.Binary.PropositionalEquality.Core
23
+ using (_≡_; refl; sym; trans; cong′)
23
24
24
25
private
25
26
variable
@@ -80,3 +81,6 @@ dec-no (no _) _ | refl = refl
80
81
dec-yes-irr : (a? : Dec A) → Irrelevant A → (a : A) → a? ≡ yes a
81
82
dec-yes-irr a? irr a with dec-yes a? a
82
83
... | a′ , eq rewrite irr a a′ = eq
84
+
85
+ ⌊⌋-map′ : ∀ t f (a? : Dec A) → ⌊ map′ {B = B} t f a? ⌋ ≡ ⌊ a? ⌋
86
+ ⌊⌋-map′ t f a? = trans (isYes≗does (map′ t f a?)) (sym (isYes≗does a?))
You can’t perform that action at this time.
0 commit comments