src/ZF/Finite.thy
changeset 32960 69916a850301
parent 26056 6a0801279f4c
child 45602 2a858377c3d2
--- a/src/ZF/Finite.thy	Sat Oct 17 01:05:59 2009 +0200
+++ b/src/ZF/Finite.thy	Sat Oct 17 14:43:18 2009 +0200
@@ -1,5 +1,4 @@
 (*  Title:      ZF/Finite.thy
-    ID:         $Id$
     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     Copyright   1994  University of Cambridge
 
@@ -13,8 +12,8 @@
 (*The natural numbers as a datatype*)
 rep_datatype
   elimination    natE
-  induction	 nat_induct
-  case_eqns	 nat_case_0 nat_case_succ
+  induction      nat_induct
+  case_eqns      nat_case_0 nat_case_succ
   recursor_eqns  recursor_0 recursor_succ