src/ZF/Finite.thy
changeset 46471 2289a3869c88
parent 45602 2a858377c3d2
child 46820 c656222c4dc1
--- a/src/ZF/Finite.thy	Tue Feb 14 20:57:05 2012 +0100
+++ b/src/ZF/Finite.thy	Tue Feb 14 21:19:39 2012 +0100
@@ -27,7 +27,7 @@
     emptyI:  "0 : Fin(A)"
     consI:   "[| a: A;  b: Fin(A) |] ==> cons(a,b) : Fin(A)"
   type_intros  empty_subsetI cons_subsetI PowI
-  type_elims   PowD [THEN revcut_rl]
+  type_elims   PowD [elim_format]
 
 inductive
   domains   "FiniteFun(A,B)" <= "Fin(A*B)"