changeset 61032 | b57df8eecad6 |
parent 60758 | d8d85a8172b5 |
child 61799 | 4cf66f21b764 |
--- a/src/HOL/Fun_Def.thy Thu Aug 27 13:07:45 2015 +0200 +++ b/src/HOL/Fun_Def.thy Thu Aug 27 21:19:48 2015 +0200 @@ -143,7 +143,7 @@ lemma split_cong [fundef_cong]: "(\<And>x y. (x, y) = q \<Longrightarrow> f x y = g x y) \<Longrightarrow> p = q - \<Longrightarrow> split f p = split g q" + \<Longrightarrow> case_prod f p = case_prod g q" by (auto simp: split_def) lemma comp_cong [fundef_cong]: