src/HOL/Library/Fundamental_Theorem_Algebra.thy
changeset 32456 341c83339aeb
parent 31337 a9ed5fcc5e39
child 32960 69916a850301
equal deleted inserted replaced
32450:375db037f4d2 32456:341c83339aeb
   575 proof(induct p)
   575 proof(induct p)
   576   case 0 thus ?case by simp
   576   case 0 thus ?case by simp
   577 next
   577 next
   578   case (pCons c cs)
   578   case (pCons c cs)
   579   {assume c0: "c = 0"
   579   {assume c0: "c = 0"
   580     from pCons.hyps pCons.prems c0 have ?case apply auto
   580     from pCons.hyps pCons.prems c0 have ?case
       
   581       apply (auto)
   581       apply (rule_tac x="k+1" in exI)
   582       apply (rule_tac x="k+1" in exI)
   582       apply (rule_tac x="a" in exI, clarsimp)
   583       apply (rule_tac x="a" in exI, clarsimp)
   583       apply (rule_tac x="q" in exI)
   584       apply (rule_tac x="q" in exI)
   584       by (auto simp add: power_Suc)}
   585       by (auto)}
   585   moreover
   586   moreover
   586   {assume c0: "c\<noteq>0"
   587   {assume c0: "c\<noteq>0"
   587     hence ?case apply-
   588     hence ?case apply-
   588       apply (rule exI[where x=0])
   589       apply (rule exI[where x=0])
   589       apply (rule exI[where x=c], clarsimp)
   590       apply (rule exI[where x=c], clarsimp)