diff -r 29800666e526 -r 842917225d56 src/HOL/Bali/AxExample.thy --- a/src/HOL/Bali/AxExample.thy Tue Feb 23 15:37:18 2016 +0100 +++ b/src/HOL/Bali/AxExample.thy Tue Feb 23 16:25:08 2016 +0100 @@ -37,7 +37,7 @@ done -declare split_if_asm [split del] +declare if_split_asm [split del] declare lvar_def [simp] ML \ @@ -202,7 +202,7 @@ apply (tactic "ax_tac @{context} 2" (* StatRef *)) apply (rule ax_derivs.Done [THEN conseq1]) apply (tactic \inst1_tac @{context} "Q" "\vf. Normal ((\Y s Z. vf=lvar (VName e) (snd s)) \. heap_free four \. initd Base \. initd Ext)" []\) -apply (clarsimp split del: split_if) +apply (clarsimp split del: if_split) apply (frule atleast_free_weaken [THEN atleast_free_weaken]) apply (drule initedD) apply (clarsimp elim!: atleast_free_SucD simp add: arr_inv_def)