File tree Expand file tree Collapse file tree 2 files changed +12
-0
lines changed
src/Data/List/Relation/Binary/Permutation/Propositional Expand file tree Collapse file tree 2 files changed +12
-0
lines changed Original file line number Diff line number Diff line change @@ -111,6 +111,9 @@ New modules
111
111
112
112
* ` Data.List.Relation.Binary.Disjoint.Propositional.Properties ` :
113
113
Propositional counterpart to ` Data.List.Relation.Binary.Disjoint.Setoid.Properties `
114
+ ``` agda
115
+ sum-↭ : sum Preserves _↭_ ⟶ _≡_
116
+ ```
114
117
115
118
* ` Data.List.Relation.Binary.Permutation.Propositional.Properties.WithK `
116
119
Original file line number Diff line number Diff line change @@ -372,6 +372,15 @@ module _ {ℓ} {R : Rel A ℓ} (R? : Decidable R) where
372
372
x ∷ xs ++ y ∷ ys ∎
373
373
where open PermutationReasoning
374
374
375
+ ------------------------------------------------------------------------
376
+ -- sum
377
+
378
+ sum-↭ : sum Preserves _↭_ ⟶ _≡_
379
+ sum-↭ p = foldr-commMonoid ℕ-+-0.isCommutativeMonoid (↭⇒↭ₛ p)
380
+ where
381
+ module ℕ-+-0 = CommutativeMonoid ℕ.+-0-commutativeMonoid
382
+ open Permutation ℕ-+-0.setoid
383
+
375
384
------------------------------------------------------------------------
376
385
-- product
377
386
You can’t perform that action at this time.
0 commit comments