File tree 2 files changed +9
-0
lines changed
2 files changed +9
-0
lines changed Original file line number Diff line number Diff line change @@ -1237,6 +1237,10 @@ Other minor changes
1237
1237
≤-isDecTotalOrder-≈ : IsDecTotalOrder _≈_ _≤_
1238
1238
≤-decTotalOrder-≈ : DecTotalOrder _ _ _
1239
1239
```
1240
+ * Added new definitions in ` Data.Sum.Properties ` :
1241
+ ```
1242
+ swap-↔ : (A ⊎ B) ↔ (B ⊎ A)
1243
+ ```
1240
1244
1241
1245
* Added new proofs in ` Data.Sum.Properties ` :
1242
1246
```
Original file line number Diff line number Diff line change @@ -11,11 +11,13 @@ module Data.Sum.Properties where
11
11
open import Level
12
12
open import Data.Sum.Base
13
13
open import Function
14
+ open import Function.Bundles using (mk↔′)
14
15
open import Relation.Binary using (Decidable)
15
16
open import Relation.Binary.PropositionalEquality
16
17
open import Relation.Nullary using (yes; no)
17
18
open import Relation.Nullary.Decidable using (map′)
18
19
20
+
19
21
private
20
22
variable
21
23
a b c d e f : Level
@@ -44,6 +46,9 @@ module _ (dec₁ : Decidable {A = A} {B = A} _≡_)
44
46
swap-involutive : swap {A = A} {B = B} ∘ swap ≗ id
45
47
swap-involutive = [ (λ _ → refl) , (λ _ → refl) ]
46
48
49
+ swap-↔ : (A ⊎ B) ↔ (B ⊎ A)
50
+ swap-↔ = mk↔′ swap swap swap-involutive swap-involutive
51
+
47
52
map-id : map {A = A} {B = B} id id ≗ id
48
53
map-id (inj₁ _) = refl
49
54
map-id (inj₂ _) = refl
You can’t perform that action at this time.
0 commit comments