tuned whitespace
authorhaftmann
Wed, 10 Mar 2010 15:29:21 +0100
changeset 35687 564a49e8be44
parent 35686 abf91fba0a70
child 35688 cfe0accda6e3
tuned whitespace
src/HOL/Code_Numeral.thy
--- a/src/HOL/Code_Numeral.thy	Wed Mar 10 08:04:50 2010 +0100
+++ b/src/HOL/Code_Numeral.thy	Wed Mar 10 15:29:21 2010 +0100
@@ -247,7 +247,7 @@
   "nat_of i = nat_of_aux i 0"
   by (simp add: nat_of_aux_def)
 
-definition div_mod_code_numeral ::  "code_numeral \<Rightarrow> code_numeral \<Rightarrow> code_numeral \<times> code_numeral" where
+definition div_mod_code_numeral :: "code_numeral \<Rightarrow> code_numeral \<Rightarrow> code_numeral \<times> code_numeral" where
   [code del]: "div_mod_code_numeral n m = (n div m, n mod m)"
 
 lemma [code]: