src/HOL/Library/Code_Index.thy
changeset 26264 89e25cc8da7a
parent 26140 e45375135052
child 26304 02fbd0e7954a
--- a/src/HOL/Library/Code_Index.thy	Wed Mar 12 17:29:09 2008 +0100
+++ b/src/HOL/Library/Code_Index.thy	Wed Mar 12 19:38:13 2008 +0100
@@ -139,6 +139,10 @@
 
 end
 
+lemma nat_of_index_number [simp]:
+  "nat_of_index (number_of k) = number_of k"
+  by (simp add: number_of_index_def nat_number_of_def number_of_is_id)
+
 code_datatype "number_of \<Colon> int \<Rightarrow> index"