File tree Expand file tree Collapse file tree 3 files changed +23
-9
lines changed Expand file tree Collapse file tree 3 files changed +23
-9
lines changed Original file line number Diff line number Diff line change @@ -1080,12 +1080,14 @@ Deprecated names
1080
1080
``` agda
1081
1081
map-identity ↦ map-id
1082
1082
map-fusion ↦ map-∘
1083
+ drop-fusion ↦ drop-drop
1083
1084
```
1084
1085
1085
1086
* In ` Codata.Sized.Colist.Properties ` :
1086
1087
``` agda
1087
- map-identity ↦ map-id
1088
- map-map-fusion ↦ map-∘
1088
+ map-identity ↦ map-id
1089
+ map-map-fusion ↦ map-∘
1090
+ drop-drop-fusion ↦ drop-drop
1089
1091
```
1090
1092
1091
1093
* In ` Codata.Sized.Covec.Properties ` :
Original file line number Diff line number Diff line change @@ -268,9 +268,9 @@ take-zipWith (suc n) f as bs =
268
268
------------------------------------------------------------------------
269
269
-- Properties of drop
270
270
271
- drop-fusion : ∀ m n (as : Stream A) → drop n (drop m as) ≡ drop (m + n) as
272
- drop-fusion zero n as = P.refl
273
- drop-fusion (suc m) n as = drop-fusion m n (as .tail)
271
+ drop-drop : ∀ m n (as : Stream A) → drop n (drop m as) ≡ drop (m + n) as
272
+ drop-drop zero n as = P.refl
273
+ drop-drop (suc m) n as = drop-drop m n (as .tail)
274
274
275
275
drop-zipWith : ∀ n (f : A → B → C) as bs →
276
276
drop n (zipWith f as bs) ≡ zipWith f (drop n as) (drop n bs)
@@ -331,3 +331,9 @@ map-fusion = map-∘
331
331
"Warning: map-fusion was deprecated in v2.0.
332
332
Please use map-∘ instead."
333
333
#-}
334
+
335
+ drop-fusion = drop-drop
336
+ {-# WARNING_ON_USAGE drop-fusion
337
+ "Warning: drop-fusion was deprecated in v2.0.
338
+ Please use drop-drop instead."
339
+ #-}
Original file line number Diff line number Diff line change @@ -197,11 +197,11 @@ drop-nil : ∀ m → i ⊢ drop {A = A} m [] ≈ []
197
197
drop-nil zero = []
198
198
drop-nil (suc m) = []
199
199
200
- drop-drop-fusion : ∀ m n (as : Colist A ∞) →
200
+ drop-drop : ∀ m n (as : Colist A ∞) →
201
201
i ⊢ drop n (drop m as) ≈ drop (m ℕ.+ n) as
202
- drop-drop-fusion zero n as = refl
203
- drop-drop-fusion (suc m) n [] = drop-nil n
204
- drop-drop-fusion (suc m) n (a ∷ as) = drop-drop-fusion m n (as .force)
202
+ drop-drop zero n as = refl
203
+ drop-drop (suc m) n [] = drop-nil n
204
+ drop-drop (suc m) n (a ∷ as) = drop-drop m n (as .force)
205
205
206
206
map-drop : ∀ (f : A → B) m as → i ⊢ map f (drop m as) ≈ drop m (map f as)
207
207
map-drop f zero as = refl
@@ -351,3 +351,9 @@ map-map-fusion = map-∘
351
351
"Warning: map-map-fusion was deprecated in v2.0.
352
352
Please use map-∘ instead."
353
353
#-}
354
+
355
+ drop-drop-fusion = drop-drop
356
+ {-# WARNING_ON_USAGE drop-drop-fusion
357
+ "Warning: drop-drop-fusion was deprecated in v2.0.
358
+ Please use drop-drop instead."
359
+ #-}
You can’t perform that action at this time.
0 commit comments