src/HOL/Code_Numeral.thy
changeset 35028 108662d50512
parent 34944 970e1466028d
child 35687 564a49e8be44
equal deleted inserted replaced
35027:ed7d12bcf8f8 35028:108662d50512
   142 code_datatype "number_of \<Colon> int \<Rightarrow> code_numeral"
   142 code_datatype "number_of \<Colon> int \<Rightarrow> code_numeral"
   143 
   143 
   144 
   144 
   145 subsection {* Basic arithmetic *}
   145 subsection {* Basic arithmetic *}
   146 
   146 
   147 instantiation code_numeral :: "{minus, ordered_semidom, semiring_div, linorder}"
   147 instantiation code_numeral :: "{minus, linordered_semidom, semiring_div, linorder}"
   148 begin
   148 begin
   149 
   149 
   150 definition [simp, code del]:
   150 definition [simp, code del]:
   151   "(1\<Colon>code_numeral) = of_nat 1"
   151   "(1\<Colon>code_numeral) = of_nat 1"
   152 
   152