src/HOL/Decision_Procs/ex/Commutative_Ring_Ex.thy
changeset 67123 3fe40ff1b921
parent 64962 bf41e1109db3
child 67341 df79ef3b3a41
equal deleted inserted replaced
67122:85b40f300fab 67123:3fe40ff1b921
     3 *)
     3 *)
     4 
     4 
     5 section \<open>Some examples demonstrating the ring and field methods\<close>
     5 section \<open>Some examples demonstrating the ring and field methods\<close>
     6 
     6 
     7 theory Commutative_Ring_Ex
     7 theory Commutative_Ring_Ex
     8 imports "../Reflective_Field"
     8   imports "../Reflective_Field"
     9 begin
     9 begin
    10 
    10 
    11 lemma "4 * (x::int) ^ 5 * y ^ 3 * x ^ 2 * 3 + x * z + 3 ^ 5 = 12 * x ^ 7 * y ^ 3 + z * x + 243"
    11 lemma "4 * (x::int) ^ 5 * y ^ 3 * x ^ 2 * 3 + x * z + 3 ^ 5 = 12 * x ^ 7 * y ^ 3 + z * x + 243"
    12   by ring
    12   by ring
    13 
    13