src/HOL/Code_Numeral.thy
changeset 48431 6efff142bb54
parent 47255 30a1692557b0
child 49834 b27bbb021df1
equal deleted inserted replaced
48430:6cbfe187a0f9 48431:6efff142bb54
   296   (Eval infixl 8 "+")
   296   (Eval infixl 8 "+")
   297 
   297 
   298 code_const "minus \<Colon> code_numeral \<Rightarrow> code_numeral \<Rightarrow> code_numeral"
   298 code_const "minus \<Colon> code_numeral \<Rightarrow> code_numeral \<Rightarrow> code_numeral"
   299   (SML "Int.max/ (0 : int,/ Int.-/ ((_),/ (_)))")
   299   (SML "Int.max/ (0 : int,/ Int.-/ ((_),/ (_)))")
   300   (OCaml "Big'_int.max'_big'_int/ Big'_int.zero'_big'_int/ (Big'_int.sub'_big'_int/ _/ _)")
   300   (OCaml "Big'_int.max'_big'_int/ Big'_int.zero'_big'_int/ (Big'_int.sub'_big'_int/ _/ _)")
   301   (Haskell "max/ (0 :: Integer)/ (_/ -/ _)")
   301   (Haskell "Prelude.max/ (0 :: Integer)/ (_/ -/ _)")
   302   (Scala "!(_/ -/ _).max(0)")
   302   (Scala "!(_/ -/ _).max(0)")
   303   (Eval "Integer.max/ 0/ (_/ -/ _)")
   303   (Eval "Integer.max/ 0/ (_/ -/ _)")
   304 
   304 
   305 code_const "times \<Colon> code_numeral \<Rightarrow> code_numeral \<Rightarrow> code_numeral"
   305 code_const "times \<Colon> code_numeral \<Rightarrow> code_numeral \<Rightarrow> code_numeral"
   306   (SML "Int.*/ ((_),/ (_))")
   306   (SML "Int.*/ ((_),/ (_))")