Skip to content
Merged
Show file tree
Hide file tree
Changes from 1 commit
Commits
File filter

Filter by extension

Filter by extension

Conversations
Failed to load comments.
Loading
Jump to
Jump to file
Failed to load files.
Loading
Diff view
Diff view
3 changes: 3 additions & 0 deletions CHANGELOG.md
Original file line number Diff line number Diff line change
Expand Up @@ -85,3 +85,6 @@ Additions to existing modules
```agda
map : (Char → Char) → String → String
```

* In `Function.Bundles`, added `_➙_` as a synonym for `Func` that can
be used infix.
9 changes: 9 additions & 0 deletions src/Function/Bundles.agda
Original file line number Diff line number Diff line change
Expand Up @@ -400,6 +400,15 @@ module _ (From : Setoid a ℓ₁) (To : Setoid b ℓ₂) where
module SplitSurjection (splitSurjection : SplitSurjection) =
LeftInverse splitSurjection

------------------------------------------------------------------------
-- Inline bbreviations for oft-used items
------------------------------------------------------------------------

-- Since ⟶ is taken below, use a thick arrow instead
infixr 0 _➙_
_➙_ : Setoid a ℓ₁ → Setoid b ℓ₂ → Set _
_➙_ = Func

------------------------------------------------------------------------
-- Bundles specialised for propositional equality
------------------------------------------------------------------------
Expand Down