src/HOL/Lambda/ListOrder.thy
changeset 9906 5c027cca6262
parent 9811 39ffdb8cab03
child 9941 fe05af7ec816
--- a/src/HOL/Lambda/ListOrder.thy	Thu Sep 07 21:06:55 2000 +0200
+++ b/src/HOL/Lambda/ListOrder.thy	Thu Sep 07 21:10:11 2000 +0200
@@ -64,7 +64,7 @@
   apply (blast intro: append_eq_appendI)
   done
 
-lemma Cons_step1E [rulify_prems, elim!]:
+lemma Cons_step1E [rulified, elim!]:
   "[| (ys, x # xs) \<in> step1 r;
     \<forall>y. ys = y # xs --> (y, x) \<in> r --> R;
     \<forall>zs. ys = x # zs --> (zs, xs) \<in> step1 r --> R
@@ -87,7 +87,7 @@
   apply blast
   done
 
-lemma Cons_acc_step1I [rulify, intro!]:
+lemma Cons_acc_step1I [rulified, intro!]:
     "x \<in> acc r ==> \<forall>xs. xs \<in> acc (step1 r) --> x # xs \<in> acc (step1 r)"
   apply (erule acc_induct)
   apply (erule thin_rl)