src/HOL/ex/Codegenerator.thy
changeset 21460 cda5cd8bfd16
parent 21420 8b15e5e66813
child 21511 16c62deb1adf
equal deleted inserted replaced
21459:20c2ddee8bc5 21460:cda5cd8bfd16
   177   fac
   177   fac
   178   "op div :: int \<Rightarrow> int \<Rightarrow> int"
   178   "op div :: int \<Rightarrow> int \<Rightarrow> int"
   179   "op mod :: int \<Rightarrow> int \<Rightarrow> int"  
   179   "op mod :: int \<Rightarrow> int \<Rightarrow> int"  
   180   (SML) (Haskell)
   180   (SML) (Haskell)
   181 code_gen
   181 code_gen
   182   "Code_Generator.eq :: bool \<Rightarrow> bool \<Rightarrow> bool"
   182   "op = :: bool \<Rightarrow> bool \<Rightarrow> bool"
   183   "Code_Generator.eq :: nat \<Rightarrow> nat \<Rightarrow> bool"
   183   "op = :: nat \<Rightarrow> nat \<Rightarrow> bool"
   184   "Code_Generator.eq :: int \<Rightarrow> int \<Rightarrow> bool"
   184   "op = :: int \<Rightarrow> int \<Rightarrow> bool"
   185   "Code_Generator.eq :: ('a\<Colon>eq) * ('b\<Colon>eq) \<Rightarrow> 'a * 'b \<Rightarrow> bool"
   185   "op = :: ('a\<Colon>eq) * ('b\<Colon>eq) \<Rightarrow> 'a * 'b \<Rightarrow> bool"
   186   "Code_Generator.eq :: ('a\<Colon>eq) + ('b\<Colon>eq) \<Rightarrow> 'a + 'b \<Rightarrow> bool"
   186   "op = :: ('a\<Colon>eq) + ('b\<Colon>eq) \<Rightarrow> 'a + 'b \<Rightarrow> bool"
   187   "Code_Generator.eq :: ('a\<Colon>eq) option \<Rightarrow> 'a option \<Rightarrow> bool"
   187   "op = :: ('a\<Colon>eq) option \<Rightarrow> 'a option \<Rightarrow> bool"
   188   "Code_Generator.eq :: ('a\<Colon>eq) list \<Rightarrow> 'a list \<Rightarrow> bool"
   188   "op = :: ('a\<Colon>eq) list \<Rightarrow> 'a list \<Rightarrow> bool"
   189   "Code_Generator.eq :: mut1 \<Rightarrow> mut1 \<Rightarrow> bool"
   189   "op = :: mut1 \<Rightarrow> mut1 \<Rightarrow> bool"
   190   "Code_Generator.eq :: mut2 \<Rightarrow> mut2 \<Rightarrow> bool"
   190   "op = :: mut2 \<Rightarrow> mut2 \<Rightarrow> bool"
   191   "Code_Generator.eq :: ('a\<Colon>eq) point_scheme \<Rightarrow> 'a point_scheme \<Rightarrow> bool"
   191   "op = :: ('a\<Colon>eq) point_scheme \<Rightarrow> 'a point_scheme \<Rightarrow> bool"
   192 
   192 
   193 code_gen (SML *) (Haskell -)
   193 code_gen (SML *) (Haskell -)
   194 
   194 
   195 end
   195 end