File tree Expand file tree Collapse file tree 1 file changed +10
-9
lines changed Expand file tree Collapse file tree 1 file changed +10
-9
lines changed Original file line number Diff line number Diff line change @@ -400,15 +400,6 @@ 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
-
412
403
------------------------------------------------------------------------
413
404
-- Bundles specialised for propositional equality
414
405
------------------------------------------------------------------------
@@ -535,6 +526,16 @@ module _ {A : Set a} {B : Set b} where
535
526
, strictlyInverseʳ⇒inverseʳ to invʳ
536
527
)
537
528
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
+
538
539
------------------------------------------------------------------------
539
540
-- Other
540
541
------------------------------------------------------------------------
You can’t perform that action at this time.
0 commit comments