type signature for bin_sign
authorhuffman
Tue, 13 Dec 2011 12:10:43 +0100
changeset 45846 518a245a1ab6
parent 45845 4158f35a5c6f
child 45847 b4254b2e2b4a
type signature for bin_sign
src/HOL/Word/Bit_Representation.thy
--- a/src/HOL/Word/Bit_Representation.thy	Tue Dec 13 12:05:47 2011 +0100
+++ b/src/HOL/Word/Bit_Representation.thy	Tue Dec 13 12:10:43 2011 +0100
@@ -296,7 +296,7 @@
 
 subsection {* Truncating binary integers *}
 
-definition
+definition bin_sign :: "int \<Rightarrow> int" where
   bin_sign_def: "bin_sign k = (if k \<ge> 0 then 0 else - 1)"
 
 lemma bin_sign_simps [simp]: