@@ -134,13 +134,13 @@ map-const : (a : A) (bs : Stream B) → map (const a) bs ≈ repeat a
134
134
map-const a bs .head = P.refl
135
135
map-const a bs .tail = map-const a (bs .tail)
136
136
137
- map-identity : (as : Stream A) → map id as ≈ as
138
- map-identity as .head = P.refl
139
- map-identity as .tail = map-identity (as .tail)
137
+ map-id : (as : Stream A) → map id as ≈ as
138
+ map-id as .head = P.refl
139
+ map-id as .tail = map-id (as .tail)
140
140
141
- map-fusion : ∀ (g : B → C) (f : A → B) as → map g (map f as) ≈ map (g ∘′ f) as
142
- map-fusion g f as .head = P.refl
143
- map-fusion g f as .tail = map-fusion g f (as .tail)
141
+ map-∘ : ∀ (g : B → C) (f : A → B) as → map g (map f as) ≈ map (g ∘′ f) as
142
+ map-∘ g f as .head = P.refl
143
+ map-∘ g f as .tail = map-∘ g f (as .tail)
144
144
145
145
map-unfold : ∀ (g : B → C) (f : A → A × B) a →
146
146
map g (unfold f a) ≈ unfold (Prod.map₂ g ∘′ f) a
@@ -309,3 +309,24 @@ interleave-evens-odds : (as : Stream A) → interleave (evens as) (odds as) ≈
309
309
interleave-evens-odds as .head = P.refl
310
310
interleave-evens-odds as .tail .head = P.refl
311
311
interleave-evens-odds as .tail .tail = interleave-evens-odds (as .tail .tail)
312
+
313
+ ------------------------------------------------------------------------
314
+ -- DEPRECATED
315
+ ------------------------------------------------------------------------
316
+ -- Please use the new names as continuing support for the old names is
317
+ -- not guaranteed.
318
+
319
+ -- Version 2.0
320
+
321
+ map-identity = map-id
322
+ {-# WARNING_ON_USAGE map-identity
323
+ "Warning: map-identity was deprecated in v2.0.
324
+ Please use map-id instead."
325
+ #-}
326
+
327
+ map-fusion = map-∘
328
+ {-# WARNING_ON_USAGE map-fusion
329
+ "Warning: map-fusion was deprecated in v2.0.
330
+ Please use map-∘ instead."
331
+ #-}
332
+
0 commit comments