diff -r 29800666e526 -r 842917225d56 src/HOL/HOLCF/IOA/RefCorrectness.thy --- a/src/HOL/HOLCF/IOA/RefCorrectness.thy Tue Feb 23 15:37:18 2016 +0100 +++ b/src/HOL/HOLCF/IOA/RefCorrectness.thy Tue Feb 23 16:25:08 2016 +0100 @@ -182,14 +182,14 @@ "is_ref_map f C A \ ext C = ext A \ \s. reachable C s \ is_exec_frag C (s, xs) \ mk_trace C $ xs = mk_trace A $ (snd (corresp_ex A f (s, xs)))" - supply split_if [split del] + supply if_split [split del] apply (unfold corresp_ex_def) apply (pair_induct xs simp: is_exec_frag_def) text \cons case\ apply (auto simp add: mk_traceConc) apply (frule reachable.reachable_n) apply assumption - apply (auto simp add: move_subprop4 split add: split_if) + apply (auto simp add: move_subprop4 split add: if_split) done