Skip to content

Commit d5ce9a8

Browse files
Bring back a convenient short-cut for infix Func
1 parent 660d983 commit d5ce9a8

File tree

2 files changed

+12
-0
lines changed

2 files changed

+12
-0
lines changed

CHANGELOG.md

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -85,3 +85,6 @@ Additions to existing modules
8585
```agda
8686
map : (Char → Char) → String → String
8787
```
88+
89+
* In `Function.Bundles`, added `_➙_` as a synonym for `Func` that can
90+
be used infix.

src/Function/Bundles.agda

Lines changed: 9 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -400,6 +400,15 @@ module _ (From : Setoid a ℓ₁) (To : Setoid b ℓ₂) where
400400
module SplitSurjection (splitSurjection : SplitSurjection) =
401401
LeftInverse splitSurjection
402402

403+
------------------------------------------------------------------------
404+
-- Inline bbreviations for oft-used items
405+
------------------------------------------------------------------------
406+
407+
-- Since ⟶ is taken below, use a thick arrow instead
408+
infixr 0 _➙_
409+
_➙_ : Setoid a ℓ₁ Setoid b ℓ₂ Set _
410+
_➙_ = Func
411+
403412
------------------------------------------------------------------------
404413
-- Bundles specialised for propositional equality
405414
------------------------------------------------------------------------

0 commit comments

Comments
 (0)