src/HOL/Code_Numeral.thy
changeset 35687 564a49e8be44
parent 35028 108662d50512
child 36049 0ce5b7a5c2fd
     1.1 --- a/src/HOL/Code_Numeral.thy	Wed Mar 10 08:04:50 2010 +0100
     1.2 +++ b/src/HOL/Code_Numeral.thy	Wed Mar 10 15:29:21 2010 +0100
     1.3 @@ -247,7 +247,7 @@
     1.4    "nat_of i = nat_of_aux i 0"
     1.5    by (simp add: nat_of_aux_def)
     1.6  
     1.7 -definition div_mod_code_numeral ::  "code_numeral \<Rightarrow> code_numeral \<Rightarrow> code_numeral \<times> code_numeral" where
     1.8 +definition div_mod_code_numeral :: "code_numeral \<Rightarrow> code_numeral \<Rightarrow> code_numeral \<times> code_numeral" where
     1.9    [code del]: "div_mod_code_numeral n m = (n div m, n mod m)"
    1.10  
    1.11  lemma [code]: