src/HOL/Decision_Procs/Reflected_Multivariate_Polynomial.thy
changeset 35046 1266f04f42ec
parent 34915 7894c7dab132
child 35054 a5db9779b026
equal deleted inserted replaced
35045:a77d200e6503 35046:1266f04f42ec
     1 (*  Title:      HOL/Decision_Procs/Reflected_Multivariate_Polynomial.thy
     1 (*  Title:      HOL/Decision_Procs/Reflected_Multivariate_Polynomial.thy
     2     Author:     Amine Chaieb
     2     Author:     Amine Chaieb
     3 *)
     3 *)
     4 
     4 
     5 header {* Implementation and verification of mutivariate polynomials Library *}
     5 header {* Implementation and verification of multivariate polynomials *}
     6 
       
     7 
     6 
     8 theory Reflected_Multivariate_Polynomial
     7 theory Reflected_Multivariate_Polynomial
     9 imports Parity Abstract_Rat Efficient_Nat List Polynomial_List
     8 imports Complex_Main Abstract_Rat Polynomial_List
    10 begin
     9 begin
    11 
    10 
    12   (* Impelementation *)
    11   (* Implementation *)
    13 
    12 
    14 subsection{* Datatype of polynomial expressions *} 
    13 subsection{* Datatype of polynomial expressions *} 
    15 
    14 
    16 datatype poly = C Num| Bound nat| Add poly poly|Sub poly poly
    15 datatype poly = C Num| Bound nat| Add poly poly|Sub poly poly
    17   | Mul poly poly| Neg poly| Pw poly nat| CN poly nat poly
    16   | Mul poly poly| Neg poly| Pw poly nat| CN poly nat poly