src/ZF/Coind/Types.thy
changeset 13339 0f89104dd377
parent 12595 0480d02221b8
child 16417 9bc16273c2d4
--- a/src/ZF/Coind/Types.thy	Wed Jul 10 16:07:52 2002 +0200
+++ b/src/ZF/Coind/Types.thy	Wed Jul 10 16:54:07 2002 +0200
@@ -54,8 +54,7 @@
 lemma te_appI:
      "[| te \<in> TyEnv; x \<in> ExVar; x \<in> te_dom(te) |] ==> te_app(te,x) \<in> Ty"
 apply (erule_tac P = "x \<in> te_dom (te) " in rev_mp)
-apply (erule TyEnv.induct)
-apply auto
+apply (erule TyEnv.induct, auto)
 done