src/HOL/Library/Efficient_Nat.thy
changeset 28694 4e9edaef64dc
parent 28683 59c01ec6cb8d
child 28969 4ed63cdda799
--- a/src/HOL/Library/Efficient_Nat.thy	Mon Oct 27 16:15:48 2008 +0100
+++ b/src/HOL/Library/Efficient_Nat.thy	Mon Oct 27 16:15:49 2008 +0100
@@ -6,7 +6,7 @@
 header {* Implementation of natural numbers by target-language integers *}
 
 theory Efficient_Nat
-imports Plain Code_Index Code_Integer
+imports Code_Index Code_Integer
 begin
 
 text {*
@@ -56,9 +56,7 @@
 text {* Specialized @{term "op div \<Colon> nat \<Rightarrow> nat \<Rightarrow> nat"} 
   and @{term "op mod \<Colon> nat \<Rightarrow> nat \<Rightarrow> nat"} operations. *}
 
-definition
-  divmod_aux ::  "nat \<Rightarrow> nat \<Rightarrow> nat \<times> nat"
-where
+definition divmod_aux ::  "nat \<Rightarrow> nat \<Rightarrow> nat \<times> nat" where
   [code del]: "divmod_aux = divmod"
 
 lemma [code]: