src/HOL/Integ/IntDef.thy
changeset 20485 3078fd2eec7b
parent 20453 855f07fabd76
child 20595 db6bedfba498
equal deleted inserted replaced
20484:3d3d24186352 20485:3078fd2eec7b
   933            Pretty.str (IntInf.toString (HOLogic.dest_binum bin))) handle TERM _ => NONE)
   933            Pretty.str (IntInf.toString (HOLogic.dest_binum bin))) handle TERM _ => NONE)
   934   | number_of_codegen thy defs gr s thyname b (Const ("Numeral.number_of",
   934   | number_of_codegen thy defs gr s thyname b (Const ("Numeral.number_of",
   935       Type ("fun", [_, Type ("nat", [])])) $ bin) =
   935       Type ("fun", [_, Type ("nat", [])])) $ bin) =
   936         SOME (Codegen.invoke_codegen thy defs s thyname b (gr,
   936         SOME (Codegen.invoke_codegen thy defs s thyname b (gr,
   937           Const ("IntDef.nat", HOLogic.intT --> HOLogic.natT) $
   937           Const ("IntDef.nat", HOLogic.intT --> HOLogic.natT) $
   938             (Const ("Numeral.number_of", HOLogic.binT --> HOLogic.intT) $ bin)))
   938             (Const ("Numeral.number_of", HOLogic.intT --> HOLogic.intT) $ bin)))
   939   | number_of_codegen _ _ _ _ _ _ _ = NONE;
   939   | number_of_codegen _ _ _ _ _ _ _ = NONE;
   940 *}
   940 *}
   941 
   941 
   942 setup {*
   942 setup {*
   943   Codegen.add_codegen "number_of_codegen" number_of_codegen
   943   Codegen.add_codegen "number_of_codegen" number_of_codegen