File tree Expand file tree Collapse file tree 2 files changed +19
-0
lines changed Expand file tree Collapse file tree 2 files changed +19
-0
lines changed Original file line number Diff line number Diff line change @@ -3159,6 +3159,12 @@ Additions to existing modules
3159
3159
execState : State s a → s → s
3160
3160
```
3161
3161
3162
+ * Added new application operator synonym to ` Function.Bundles ` :
3163
+ ``` agda
3164
+ _⟨$⟩_ : Func From To → Carrier From → Carrier To
3165
+ _⟨$⟩_ = Func.to
3166
+ ```
3167
+
3162
3168
* Added new proofs in ` Function.Construct.Symmetry ` :
3163
3169
```
3164
3170
bijective : Bijective ≈₁ ≈₂ f → Symmetric ≈₂ → Transitive ≈₂ → Congruent ≈₁ ≈₂ f → Bijective ≈₂ ≈₁ f⁻¹
Original file line number Diff line number Diff line change @@ -66,6 +66,7 @@ module _ (From : Setoid a ℓ₁) (To : Setoid b ℓ₂) where
66
66
open IsCongruent isCongruent public
67
67
using (module Eq₁ ; module Eq₂ )
68
68
69
+
69
70
record Injection : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
70
71
field
71
72
to : A → B
@@ -472,3 +473,15 @@ module _ {A : Set a} {B : Set b} where
472
473
, strictlyInverseʳ⇒inverseʳ to invʳ
473
474
)
474
475
476
+ ------------------------------------------------------------------------
477
+ -- Other
478
+ ------------------------------------------------------------------------
479
+
480
+ -- Alternative syntax for the application of functions
481
+
482
+ module _ {From : Setoid a ℓ₁} {To : Setoid b ℓ₂} where
483
+ open Setoid
484
+
485
+ infixl 5 _⟨$⟩_
486
+ _⟨$⟩_ : Func From To → Carrier From → Carrier To
487
+ _⟨$⟩_ = Func.to
You can’t perform that action at this time.
0 commit comments