src/HOL/Decision_Procs/Commutative_Ring_Complete.thy
changeset 60767 ad5b4771fc19
parent 60708 f425e80a3eb0
child 61586 5197a2ecb658
equal deleted inserted replaced
60766:76560ce8dead 60767:ad5b4771fc19
   210   case (7 x P2 Q2 y R)
   210   case (7 x P2 Q2 y R)
   211   consider "x = 0" | "x = 1" | d where "x = Suc (Suc d)"
   211   consider "x = 0" | "x = 1" | d where "x = Suc (Suc d)"
   212     by atomize_elim arith
   212     by atomize_elim arith
   213   then show ?case
   213   then show ?case
   214   proof cases
   214   proof cases
   215     case x: 1
   215     case 1
   216     with 7 show ?thesis
   216     with 7 show ?thesis
   217       by (auto simp add: norm_Pinj_0_False)
   217       by (auto simp add: norm_Pinj_0_False)
   218   next
   218   next
   219     case x: 2
   219     case x: 2
   220     from 7 have "isnorm R" "isnorm P2"
   220     from 7 have "isnorm R" "isnorm P2"