src/HOL/Algebra/UnivPoly.thy
changeset 19582 a669c98b9c24
parent 17094 7a3c2efecffe
child 19783 82f365a14960
--- a/src/HOL/Algebra/UnivPoly.thy	Fri May 05 21:59:49 2006 +0200
+++ b/src/HOL/Algebra/UnivPoly.thy	Fri May 05 22:11:19 2006 +0200
@@ -297,7 +297,7 @@
     then have "k <= n ==>
       (\<Oplus>j \<in> {..k}. (\<Oplus>i \<in> {..j}. a i \<otimes> b (j-i)) \<otimes> c (n-j)) =
       (\<Oplus>j \<in> {..k}. a j \<otimes> (\<Oplus>i \<in> {..k-j}. b i \<otimes> c (n-j-i)))"
-      (concl is "?eq k")
+      (is "_ \<Longrightarrow> ?eq k")
     proof (induct k)
       case 0 then show ?case by (simp add: Pi_def m_assoc)
     next
@@ -344,7 +344,7 @@
     then have "k <= n ==>
       (\<Oplus>i \<in> {..k}. a i \<otimes> b (n-i)) =
       (\<Oplus>i \<in> {..k}. a (k-i) \<otimes> b (i+n-k))"
-      (concl is "?eq k")
+      (is "_ \<Longrightarrow> ?eq k")
     proof (induct k)
       case 0 then show ?case by (simp add: Pi_def)
     next