diff -r 162bd20dae23 -r b57df8eecad6 src/HOL/Fun_Def.thy --- 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]: "(\x y. (x, y) = q \ f x y = g x y) \ p = q - \ split f p = split g q" + \ case_prod f p = case_prod g q" by (auto simp: split_def) lemma comp_cong [fundef_cong]: