misc tuning: more concise operations on prems (without change of exceptions);
discontinue odd clone Drule.cprems_of (see also 991a3feaf270);
(* Title: HOL/Library/Code_Target_Numeral.thy
Author: Florian Haftmann, TU Muenchen
*)
section \<open>Implementation of natural and integer numbers by target-language integers\<close>
theory Code_Target_Numeral
imports Code_Target_Nat Code_Target_Int Code_Target_Bit_Shifts
begin
end