src/HOL/UNITY/PPROD.thy
changeset 32960 69916a850301
parent 16417 9bc16273c2d4
child 35054 a5db9779b026
--- a/src/HOL/UNITY/PPROD.thy	Sat Oct 17 01:05:59 2009 +0200
+++ b/src/HOL/UNITY/PPROD.thy	Sat Oct 17 14:43:18 2009 +0200
@@ -1,5 +1,4 @@
 (*  Title:      HOL/UNITY/PPROD.thy
-    ID:         $Id$
     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     Copyright   1998  University of Cambridge
 
@@ -274,7 +273,7 @@
     done
 
     lemma const_PLam_Increasing:
-	 "[| i \<in> I;  finite I |]
+         "[| i \<in> I;  finite I |]
           ==> ((plam x \<in> I. F) \<in> Increasing (f o sub i)) = (F \<in> Increasing f)"
     apply (unfold Increasing_def)
     apply (subgoal_tac "\<forall>z. {s. z \<subseteq> (f o sub i) s} = lift_set i {s. z \<subseteq> f s}")