File tree Expand file tree Collapse file tree 2 files changed +12
-0
lines changed Expand file tree Collapse file tree 2 files changed +12
-0
lines changed Original file line number Diff line number Diff line change @@ -85,3 +85,6 @@ Additions to existing modules
85
85
``` agda
86
86
map : (Char → Char) → String → String
87
87
```
88
+
89
+ * In ` Function.Bundles ` , added ` _➙_ ` as a synonym for ` Func ` that can
90
+ be used infix.
Original file line number Diff line number Diff line change @@ -400,6 +400,15 @@ module _ (From : Setoid a ℓ₁) (To : Setoid b ℓ₂) where
400
400
module SplitSurjection (splitSurjection : SplitSurjection) =
401
401
LeftInverse splitSurjection
402
402
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
+
403
412
------------------------------------------------------------------------
404
413
-- Bundles specialised for propositional equality
405
414
------------------------------------------------------------------------
You can’t perform that action at this time.
0 commit comments