src/CTT/CTT.thy
changeset 65338 2ffda850f844
parent 64980 7dc25cf5793e
child 65447 fae6051ec192
--- a/src/CTT/CTT.thy	Mon Mar 20 21:53:37 2017 +0100
+++ b/src/CTT/CTT.thy	Thu Mar 23 17:20:47 2017 +0100
@@ -285,11 +285,7 @@
 
 text \<open>Compare with standard version: \<open>B\<close> is applied to UNSIMPLIFIED expression!\<close>
 lemma SumIL2: "\<lbrakk>c = a : A; d = b : B(a)\<rbrakk> \<Longrightarrow> <c,d> = <a,b> : Sum(A,B)"
-  apply (rule sym_elem)
-  apply (rule SumIL)
-   apply (rule_tac [!] sym_elem)
-   apply assumption+
-  done
+  by (rule sym_elem) (rule SumIL; rule sym_elem)
 
 lemmas intrL2_rls = NI_succL ProdIL SumIL2 PlusI_inlL PlusI_inrL