src/HOL/Library/Word.thy
changeset 81609 3458f17e7cba
parent 81142 6ad2c917dd2e
child 81763 2cf8f8e4c1fd
--- a/src/HOL/Library/Word.thy	Mon Dec 16 19:22:54 2024 +0100
+++ b/src/HOL/Library/Word.thy	Mon Dec 16 21:08:43 2024 +0100
@@ -415,6 +415,18 @@
   \<open>nat (uint w) = unat w\<close>
   by transfer simp
 
+lemma nat_of_natural_unsigned_eq [simp]:
+  \<open>nat_of_natural (unsigned w) = unat w\<close>
+  by transfer simp
+
+lemma int_of_integer_unsigned_eq [simp]:
+  \<open>int_of_integer (unsigned w) = uint w\<close>
+  by transfer simp
+
+lemma int_of_integer_signed_eq [simp]:
+  \<open>int_of_integer (signed w) = sint w\<close>
+  by transfer simp
+
 lemma sgn_uint_eq [simp]:
   \<open>sgn (uint w) = of_bool (w \<noteq> 0)\<close>
   by transfer (simp add: less_le)