src/ZF/OrderType.thy
changeset 46841 49b91b716cbe
parent 46821 ff6b0c1087f2
child 46927 faf4a0b02b71
--- a/src/ZF/OrderType.thy	Tue Mar 06 17:01:37 2012 +0000
+++ b/src/ZF/OrderType.thy	Thu Mar 08 16:43:29 2012 +0000
@@ -74,8 +74,7 @@
   The smaller ordinal is an initial segment of the larger *)
 lemma lt_pred_Memrel:
     "j<i ==> pred(i, j, Memrel(i)) = j"
-apply (unfold pred_def lt_def)
-apply (simp (no_asm_simp))
+apply (simp add: pred_def lt_def)
 apply (blast intro: Ord_trans)
 done