File tree Expand file tree Collapse file tree 1 file changed +7
-7
lines changed Expand file tree Collapse file tree 1 file changed +7
-7
lines changed Original file line number Diff line number Diff line change @@ -1240,13 +1240,6 @@ Other minor changes
1240
1240
record IsRingWithoutOneIsoMorphism (⟦_⟧ : A → B) : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂)
1241
1241
```
1242
1242
1243
- * Added new functions in ` Category.Monad.State ` :
1244
- ```
1245
- runState : State s a → s → a × s
1246
- evalState : State s a → s → a
1247
- execState : State s a → s → s
1248
- ```
1249
-
1250
1243
* Added new proofs in ` Data.Bool.Properties ` :
1251
1244
``` agda
1252
1245
<-wellFounded : WellFounded _<_
@@ -1697,6 +1690,13 @@ Other minor changes
1697
1690
++-assoc : (xs ++ ys) ++ zs ≋ xs ++ (ys ++ zs)
1698
1691
```
1699
1692
1693
+ * Added new functions in ` Effect.Monad.State ` :
1694
+ ```
1695
+ runState : State s a → s → a × s
1696
+ evalState : State s a → s → a
1697
+ execState : State s a → s → s
1698
+ ```
1699
+
1700
1700
* Added new proofs in ` Function.Construct.Symmetry ` :
1701
1701
```
1702
1702
bijective : Bijective ≈₁ ≈₂ f → Symmetric ≈₂ → Transitive ≈₂ → Congruent ≈₁ ≈₂ f → Bijective ≈₂ ≈₁ f⁻¹
You can’t perform that action at this time.
0 commit comments