src/HOL/Lambda/Eta.thy
changeset 32605 43ed78ee285d
parent 32235 8f9b8d14fc9f
child 34990 81e8fdfeb849
--- a/src/HOL/Lambda/Eta.thy	Fri Sep 18 09:07:51 2009 +0200
+++ b/src/HOL/Lambda/Eta.thy	Fri Sep 18 09:35:23 2009 +0200
@@ -1,5 +1,4 @@
 (*  Title:      HOL/Lambda/Eta.thy
-    ID:         $Id$
     Author:     Tobias Nipkow and Stefan Berghofer
     Copyright   1995, 2005 TU Muenchen
 *)
@@ -87,7 +86,6 @@
 lemma square_eta: "square eta eta (eta^==) (eta^==)"
   apply (unfold square_def id_def)
   apply (rule impI [THEN allI [THEN allI]])
-  apply simp
   apply (erule eta.induct)
      apply (slowsimp intro: subst_not_free eta_subst free_eta [THEN iffD1])
     apply safe