src/HOL/Decision_Procs/Reflected_Multivariate_Polynomial.thy
changeset 54220 0e6645622f22
parent 53374 a14d2a854c02
child 54489 03ff4d1e6784
equal deleted inserted replaced
54219:63fe59f64578 54220:0e6645622f22
     3 *)
     3 *)
     4 
     4 
     5 header {* Implementation and verification of multivariate polynomials *}
     5 header {* Implementation and verification of multivariate polynomials *}
     6 
     6 
     7 theory Reflected_Multivariate_Polynomial
     7 theory Reflected_Multivariate_Polynomial
     8 imports Complex_Main "~~/src/HOL/Library/Abstract_Rat" Polynomial_List
     8 imports Complex_Main Rat_Pair Polynomial_List
     9 begin
     9 begin
    10 
    10 
    11 subsection{* Datatype of polynomial expressions *}
    11 subsection{* Datatype of polynomial expressions *}
    12 
    12 
    13 datatype poly = C Num| Bound nat| Add poly poly|Sub poly poly
    13 datatype poly = C Num| Bound nat| Add poly poly|Sub poly poly