Skip to content

Instantly share code, notes, and snippets.

Show Gist options
  • Star 0 You must be signed in to star a gist
  • Fork 0 You must be signed in to fork a gist
  • Save erutuf/123da543af0d6b19ae53bb7e8ccf8b81 to your computer and use it in GitHub Desktop.
Save erutuf/123da543af0d6b19ae53bb7e8ccf8b81 to your computer and use it in GitHub Desktop.
Require Import Program List.
Open Scope list_scope.
Lemma fold_right_ext : forall (A : Type)(f g : A -> A -> A) xs x0,
(forall x y, f x y = g x y) ->
fold_right f x0 xs = fold_right g x0 xs.
Proof with simpl in *.
intros.
induction xs; [auto|]...
rewrite H.
rewrite IHxs.
reflexivity.
Qed.
Lemma fold_right_rev : forall (A: Type) (f: A -> A -> A) xs x0,
(forall x y z, f x (f y z) = f (f x y) z) ->
(forall x y, f x y = f y x) ->
List.fold_right f x0 xs = List.fold_right f x0 (List.rev xs).
Proof.
intros.
rewrite (fold_right_ext _ f (fun x y => f y x)) by auto.
rewrite <- fold_symmetric; [|auto..].
rewrite fold_left_rev_right.
reflexivity.
Qed.
Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment