src/HOL/ex/Numeral.thy
changeset 39499 0b61951d2682
parent 39393 917b4b6ba3d2
child 41494 e1fce873b814
equal deleted inserted replaced
39498:436554f1beaa 39499:0b61951d2682
  1084   (Eval "Integer.div'_mod/ (abs _)/ (abs _)")
  1084   (Eval "Integer.div'_mod/ (abs _)/ (abs _)")
  1085 
  1085 
  1086 code_const "HOL.equal \<Colon> int \<Rightarrow> int \<Rightarrow> bool"
  1086 code_const "HOL.equal \<Colon> int \<Rightarrow> int \<Rightarrow> bool"
  1087   (SML "!((_ : IntInf.int) = _)")
  1087   (SML "!((_ : IntInf.int) = _)")
  1088   (OCaml "Big'_int.eq'_big'_int")
  1088   (OCaml "Big'_int.eq'_big'_int")
  1089   (Haskell infixl 4 "==")
  1089   (Haskell infix 4 "==")
  1090   (Scala infixl 5 "==")
  1090   (Scala infixl 5 "==")
  1091   (Eval infixl 6 "=")
  1091   (Eval infixl 6 "=")
  1092 
  1092 
  1093 code_const "op \<le> \<Colon> int \<Rightarrow> int \<Rightarrow> bool"
  1093 code_const "op \<le> \<Colon> int \<Rightarrow> int \<Rightarrow> bool"
  1094   (SML "IntInf.<= ((_), (_))")
  1094   (SML "IntInf.<= ((_), (_))")