src/HOL/List.thy
changeset 18622 4524643feecc
parent 18490 434e34392c40
child 18702 7dc7dcd63224
--- a/src/HOL/List.thy	Mon Jan 09 00:05:10 2006 +0100
+++ b/src/HOL/List.thy	Mon Jan 09 13:27:44 2006 +0100
@@ -1728,9 +1728,13 @@
 lemma nth_Cons': "(x # xs)!n = (if n = 0 then x else xs!(n - 1))"
 by (cases n) simp_all
 
-lemmas [simp] = take_Cons'[of "number_of v",standard]
-                drop_Cons'[of "number_of v",standard]
-                nth_Cons'[of _ _ "number_of v",standard]
+lemmas take_Cons_number_of = take_Cons'[of "number_of v",standard]
+lemmas drop_Cons_number_of = drop_Cons'[of "number_of v",standard]
+lemmas nth_Cons_number_of = nth_Cons'[of _ _ "number_of v",standard]
+
+declare take_Cons_number_of [simp] 
+        drop_Cons_number_of [simp] 
+        nth_Cons_number_of [simp] 
 
 
 subsubsection {* @{text "distinct"} and @{text remdups} *}