File tree 2 files changed +17
-0
lines changed
src/Data/List/Relation/Binary/Permutation/Propositional
2 files changed +17
-0
lines changed Original file line number Diff line number Diff line change @@ -3037,3 +3037,8 @@ This is a full list of proofs that have changed form to use irrelevant instance
3037
3037
``` agda
3038
3038
<-weakInduction-startingFrom : P i → (∀ j → P (inject₁ j) → P (suc j)) → ∀ {j} → j ≥ i → P j
3039
3039
```
3040
+
3041
+ * Added new function to ` Data.List.Relation.Binary.Permutation.Propositional.Properties `
3042
+ ``` agda
3043
+ ↭-reverse : (xs : List A) → reverse xs ↭ xs
3044
+ ```
Original file line number Diff line number Diff line change @@ -324,6 +324,18 @@ drop-∷ = drop-mid [] []
324
324
++↭ʳ++ [] ys = ↭-refl
325
325
++↭ʳ++ (x ∷ xs) ys = ↭-trans (↭-sym (shift x xs ys)) (++↭ʳ++ xs (x ∷ ys))
326
326
327
+ ------------------------------------------------------------------------
328
+ -- reverse
329
+
330
+ ↭-reverse : (xs : List A) → reverse xs ↭ xs
331
+ ↭-reverse [] = ↭-refl
332
+ ↭-reverse (x ∷ xs) = begin
333
+ reverse (x ∷ xs) ≡⟨ Lₚ.unfold-reverse x xs ⟩
334
+ reverse xs ∷ʳ x ↭˘⟨ ∷↭∷ʳ x (reverse xs) ⟩
335
+ x ∷ reverse xs ↭⟨ prep x (↭-reverse xs) ⟩
336
+ x ∷ xs ∎
337
+ where open PermutationReasoning
338
+
327
339
------------------------------------------------------------------------
328
340
-- merge
329
341
You can’t perform that action at this time.
0 commit comments