Skip to content
This repository has been archived by the owner on Feb 5, 2022. It is now read-only.

Commit

Permalink
Simplify proof of big_parallel_cong
Browse files Browse the repository at this point in the history
  • Loading branch information
javierdiaz72 committed Feb 16, 2019
1 parent 9f01230 commit c92cc19
Showing 1 changed file with 2 additions and 10 deletions.
12 changes: 2 additions & 10 deletions Isabelle/Chi_Calculus_Examples/Utilities.thy
Expand Up @@ -272,20 +272,12 @@ next
case (Cons y ys)
have "big_parallel f xs = big_parallel f (y # ys)"
by (simp add: \<open>xs = y # ys\<close>)
also have "... = foldr (\<lambda>x p. f x \<parallel> p) (y # ys) \<zero>"
by (unfold big_parallel_def) simp
also have "... = f y \<parallel> foldr (\<lambda>x p. f x \<parallel> p) ys \<zero>"
by (simp add: foldr_Cons)
also have "... = f y \<parallel> big_parallel f ys"
by (fold big_parallel_def) simp
by (simp add: big_parallel_def)
also have "... = g y \<parallel> big_parallel g ys"
by (simp add: Cons.IH Cons.prems(1-2))
also have "... = g y \<parallel> foldr (\<lambda>x p. g x \<parallel> p) ys \<zero>"
by (unfold big_parallel_def) simp
also have "... = foldr (\<lambda>x p. g x \<parallel> p) (y # ys) \<zero>"
by (simp add: foldr_Cons)
also have "... = big_parallel g (y # ys)"
by (fold big_parallel_def) simp
by (simp add: big_parallel_def)
finally show ?case
by simp
qed
Expand Down

0 comments on commit c92cc19

Please sign in to comment.