Skip to content

Commit 856fbf8

Browse files
change name as per suggestion from Matthew
1 parent d5ce9a8 commit 856fbf8

File tree

1 file changed

+10
-9
lines changed

1 file changed

+10
-9
lines changed

src/Function/Bundles.agda

Lines changed: 10 additions & 9 deletions
Original file line numberDiff line numberDiff line change
@@ -400,15 +400,6 @@ 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-
412403
------------------------------------------------------------------------
413404
-- Bundles specialised for propositional equality
414405
------------------------------------------------------------------------
@@ -535,6 +526,16 @@ module _ {A : Set a} {B : Set b} where
535526
, strictlyInverseʳ⇒inverseʳ to invʳ
536527
)
537528

529+
------------------------------------------------------------------------
530+
-- Inline bbreviations for oft-used items
531+
-- (but one define the ones that recur)
532+
------------------------------------------------------------------------
533+
534+
-- Same convention as above, with appended ₛ (for 'S'etoid)
535+
infixr 0 _⟶ₛ_
536+
_⟶ₛ_ : Setoid a ℓ₁ Setoid b ℓ₂ Set _
537+
_⟶ₛ_ = Func
538+
538539
------------------------------------------------------------------------
539540
-- Other
540541
------------------------------------------------------------------------

0 commit comments

Comments
 (0)