File tree Expand file tree Collapse file tree 2 files changed +11
-0
lines changed Expand file tree Collapse file tree 2 files changed +11
-0
lines changed Original file line number Diff line number Diff line change @@ -1949,6 +1949,12 @@ Other minor changes
1949
1949
from-Σ : (I : Set i) (C : I → Container s p) → ⟦ Σ I C ⟧ A → ∃ λ i → ⟦ C i ⟧ A
1950
1950
```
1951
1951
1952
+ * Added a non-dependent version of ` Function.Base.flip ` due to an issue noted in
1953
+ Pull Request #1812 :
1954
+ ``` agda
1955
+ flip′ : (A → B → C) → (B → A → C)
1956
+ ```
1957
+
1952
1958
NonZero/Positive/Negative changes
1953
1959
---------------------------------
1954
1960
Original file line number Diff line number Diff line change @@ -137,6 +137,11 @@ f ∘′ g = _∘_ f g
137
137
_∘₂′_ : (C → D) → (A → B → C) → (A → B → D)
138
138
f ∘₂′ g = _∘₂_ f g
139
139
140
+ -- Flipping order of arguments
141
+
142
+ flip′ : (A → B → C) → (B → A → C)
143
+ flip′ = flip
144
+
140
145
-- Application
141
146
142
147
_$′_ : (A → B) → (A → B)
You can’t perform that action at this time.
0 commit comments