mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-11 06:14:41 +03:00
Rename to reverseInvolutive
This commit is contained in:
parent
bc76809288
commit
e9324fcd60
@ -672,11 +672,11 @@ revAppend (v :: vs) ns
|
|||||||
|
|
||||||
||| List reverse applied twice yields the identity function.
|
||| List reverse applied twice yields the identity function.
|
||||||
export
|
export
|
||||||
reverseInvolutory : (xs : List a) -> reverse (reverse xs) = xs
|
reverseInvolutive : (xs : List a) -> reverse (reverse xs) = xs
|
||||||
reverseInvolutory [] = Refl
|
reverseInvolutive [] = Refl
|
||||||
reverseInvolutory (x :: xs) = rewrite revOnto [x] xs in
|
reverseInvolutive (x :: xs) = rewrite revOnto [x] xs in
|
||||||
rewrite sym (revAppend (reverse xs) [x]) in
|
rewrite sym (revAppend (reverse xs) [x]) in
|
||||||
cong (x ::) $ reverseInvolutory xs
|
cong (x ::) $ reverseInvolutive xs
|
||||||
|
|
||||||
export
|
export
|
||||||
dropFusion : (n, m : Nat) -> (l : List t) -> drop n (drop m l) = drop (n+m) l
|
dropFusion : (n, m : Nat) -> (l : List t) -> drop n (drop m l) = drop (n+m) l
|
||||||
|
Loading…
Reference in New Issue
Block a user