src/ZF/OrderType.thy
changeset 32960 69916a850301
parent 26056 6a0801279f4c
child 46820 c656222c4dc1
--- a/src/ZF/OrderType.thy	Sat Oct 17 01:05:59 2009 +0200
+++ b/src/ZF/OrderType.thy	Sat Oct 17 14:43:18 2009 +0200
@@ -1,8 +1,6 @@
 (*  Title:      ZF/OrderType.thy
-    ID:         $Id$
     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     Copyright   1994  University of Cambridge
-
 *)
 
 header{*Order Types and Ordinal Arithmetic*}
@@ -161,7 +159,7 @@
 apply (rule OrdI [OF _ Ord_is_Transset])
 apply (unfold pred_def Transset_def)
 apply (blast intro: trans_onD
-	     dest!: ordermap_unfold [THEN equalityD1])+ 
+             dest!: ordermap_unfold [THEN equalityD1])+ 
 done
 
 lemma Ord_ordertype: 
@@ -172,7 +170,7 @@
 prefer 2 apply (blast intro: Ord_ordermap)
 apply (unfold Transset_def well_ord_def)
 apply (blast intro: trans_onD
-	     dest!: ordermap_unfold [THEN equalityD1])
+             dest!: ordermap_unfold [THEN equalityD1])
 done