Skip to content

Commit fe11fa0

Browse files
Bring back a convenient short-cut for infix Func (#2239)
* Bring back a convenient short-cut for infix Func * change name as per suggestion from Matthew * propagate use of shortcut to where it increases readability * Revert "propagate use of shortcut to where it increases readability" This reverts commit debfec1. * Move definitions up. Fix comments.
1 parent f0b24be commit fe11fa0

File tree

2 files changed

+14
-0
lines changed

2 files changed

+14
-0
lines changed

CHANGELOG.md

+3
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

+11
Original file line numberDiff line numberDiff line change
@@ -400,6 +400,17 @@ module _ (From : Setoid a ℓ₁) (To : Setoid b ℓ₂) where
400400
module SplitSurjection (splitSurjection : SplitSurjection) =
401401
LeftInverse splitSurjection
402402

403+
------------------------------------------------------------------------
404+
-- Infix abbreviations for oft-used items
405+
------------------------------------------------------------------------
406+
407+
-- Same naming convention as used for propositional equality below, with
408+
-- appended ₛ (for 'S'etoid).
409+
410+
infixr 0 _⟶ₛ_
411+
_⟶ₛ_ : Setoid a ℓ₁ Setoid b ℓ₂ Set _
412+
_⟶ₛ_ = Func
413+
403414
------------------------------------------------------------------------
404415
-- Bundles specialised for propositional equality
405416
------------------------------------------------------------------------

0 commit comments

Comments
 (0)