src/HOL/Num.thy
changeset 47126 e980b14c347d
parent 47108 2a1953f0d20d
child 47191 ebd8c46d156b
equal deleted inserted replaced
47125:a3a64240cd98 47126:e980b14c347d
  1008 hide_const (open) One Bit0 Bit1 BitM inc pow sqr sub dbl dbl_inc dbl_dec
  1008 hide_const (open) One Bit0 Bit1 BitM inc pow sqr sub dbl dbl_inc dbl_dec
  1009 
  1009 
  1010 subsection {* code module namespace *}
  1010 subsection {* code module namespace *}
  1011 
  1011 
  1012 code_modulename SML
  1012 code_modulename SML
  1013   Numeral Arith
  1013   Num Arith
  1014 
  1014 
  1015 code_modulename OCaml
  1015 code_modulename OCaml
  1016   Numeral Arith
  1016   Num Arith
  1017 
  1017 
  1018 code_modulename Haskell
  1018 code_modulename Haskell
  1019   Numeral Arith
  1019   Num Arith
  1020 
  1020 
  1021 end
  1021 end