File tree Expand file tree Collapse file tree 2 files changed +12
-0
lines changed
src/Data/Vec/Relation/Binary/Equality Expand file tree Collapse file tree 2 files changed +12
-0
lines changed Original file line number Diff line number Diff line change @@ -716,6 +716,13 @@ Other minor changes
716
716
→ dsubst₂ C p q (f x₁ y₁) ≡ f x₂ y₂
717
717
```
718
718
719
+ * Added vector associativity proof to
720
+ ` Data/Vec/Relation/Binary/Equality/Setoid.agda ` :
721
+ ```
722
+ ++-assoc : ∀ {n m k} (xs : Vec A n) → (ys : Vec A m)
723
+ → (zs : Vec A k) → (xs ++ ys) ++ zs ≋ xs ++ (ys ++ zs)
724
+ ```
725
+
719
726
NonZero/Positive/Negative changes
720
727
---------------------------------
721
728
Original file line number Diff line number Diff line change @@ -68,6 +68,11 @@ open PW public using (++⁺ ; ++⁻ ; ++ˡ⁻; ++ʳ⁻)
68
68
++-identityʳ [] = []
69
69
++-identityʳ (x ∷ xs) = refl ∷ ++-identityʳ xs
70
70
71
+ ++-assoc : ∀ {n m k} (xs : Vec A n) (ys : Vec A m) (zs : Vec A k) →
72
+ (xs ++ ys) ++ zs ≋ xs ++ (ys ++ zs)
73
+ ++-assoc [] ys zs = ≋-refl
74
+ ++-assoc (x ∷ xs) ys zs = refl ∷ ++-assoc xs ys zs
75
+
71
76
map-++-commute : ∀ {b m n} {B : Set b}
72
77
(f : B → A) (xs : Vec B m) {ys : Vec B n} →
73
78
map f (xs ++ ys) ≋ map f xs ++ map f ys
You can’t perform that action at this time.
0 commit comments