src/HOLCF/IOA/meta_theory/Sequence.thy
changeset 35532 60647586b173
parent 35494 45c9a8278faf
child 35642 f478d5a9d238
--- a/src/HOLCF/IOA/meta_theory/Sequence.thy	Tue Mar 02 20:19:04 2010 -0800
+++ b/src/HOLCF/IOA/meta_theory/Sequence.thy	Tue Mar 02 20:36:07 2010 -0800
@@ -163,8 +163,7 @@
 
 lemma Last_cons: "Last$(x>>xs)= (if xs=nil then Def x else Last$xs)"
 apply (simp add: Last_def Consq_def)
-apply (rule_tac x="xs" in seq.casedist)
-apply simp
+apply (cases xs)
 apply simp_all
 done
 
@@ -208,7 +207,7 @@
 lemma Zip_UU2: "x~=nil ==> Zip$x$UU =UU"
 apply (subst Zip_unfold)
 apply simp
-apply (rule_tac x="x" in seq.casedist)
+apply (cases x)
 apply simp_all
 done