src/HOL/Groebner_Basis.thy
changeset 30079 293b896b9c25
parent 30042 31039ee583fa
child 30242 aea5d7fa7ef5
equal deleted inserted replaced
30078:beee83623cc9 30079:293b896b9c25
   145 next show "mul (pwr x q) x = pwr x (Suc q)" using pwr_Suc mul_c by simp
   145 next show "mul (pwr x q) x = pwr x (Suc q)" using pwr_Suc mul_c by simp
   146 next show "mul x x = pwr x 2" by (simp add: nat_number pwr_Suc pwr_0 mul_1 mul_c)
   146 next show "mul x x = pwr x 2" by (simp add: nat_number pwr_Suc pwr_0 mul_1 mul_c)
   147 next show "pwr (mul x y) q = mul (pwr x q) (pwr y q)" by (rule pwr_mul)
   147 next show "pwr (mul x y) q = mul (pwr x q) (pwr y q)" by (rule pwr_mul)
   148 next show "pwr (pwr x p) q = pwr x (p * q)" by (rule pwr_pwr)
   148 next show "pwr (pwr x p) q = pwr x (p * q)" by (rule pwr_pwr)
   149 next show "pwr x 0 = r1" using pwr_0 .
   149 next show "pwr x 0 = r1" using pwr_0 .
   150 next show "pwr x 1 = x" by (simp add: nat_number pwr_Suc pwr_0 mul_1 mul_c)
   150 next show "pwr x 1 = x" unfolding One_nat_def by (simp add: nat_number pwr_Suc pwr_0 mul_1 mul_c)
   151 next show "mul x (add y z) = add (mul x y) (mul x z)" using mul_d by simp
   151 next show "mul x (add y z) = add (mul x y) (mul x z)" using mul_d by simp
   152 next show "pwr x (Suc q) = mul x (pwr x q)" using pwr_Suc by simp
   152 next show "pwr x (Suc q) = mul x (pwr x q)" using pwr_Suc by simp
   153 next show "pwr x (2 * n) = mul (pwr x n) (pwr x n)" by (simp add: nat_number mul_pwr)
   153 next show "pwr x (2 * n) = mul (pwr x n) (pwr x n)" by (simp add: nat_number mul_pwr)
   154 next show "pwr x (Suc (2 * n)) = mul x (mul (pwr x n) (pwr x n))"
   154 next show "pwr x (Suc (2 * n)) = mul x (mul (pwr x n) (pwr x n))"
   155     by (simp add: nat_number pwr_Suc mul_pwr)
   155     by (simp add: nat_number pwr_Suc mul_pwr)