src/HOL/Proofs/Lambda/WeakNorm.thy
changeset 56073 29e308b56d23
parent 51143 0a2371e7ced3
child 58382 2ee61d28c667
--- a/src/HOL/Proofs/Lambda/WeakNorm.thy	Wed Mar 12 22:57:50 2014 +0100
+++ b/src/HOL/Proofs/Lambda/WeakNorm.thy	Thu Mar 13 07:07:07 2014 +0100
@@ -93,7 +93,7 @@
         next
           case (Cons a as)
           with argsT obtain T'' Ts where Us: "Us = T'' # Ts"
-            by (cases Us) (rule FalseE, simp+, erule that)
+            by (cases Us) (rule FalseE, simp)
           from varT and Us have varT: "e\<langle>i:T\<rangle> \<turnstile> Var x : T'' \<Rightarrow> Ts \<Rrightarrow> T'"
             by simp
           from varT eq have T: "T = T'' \<Rightarrow> Ts \<Rrightarrow> T'" by cases auto