src/HOL/List.thy
changeset 25563 cab4f808f791
parent 25559 f14305fb698c
child 25571 c9e39eafc7a0
--- a/src/HOL/List.thy	Thu Dec 06 16:56:00 2007 +0100
+++ b/src/HOL/List.thy	Thu Dec 06 17:05:44 2007 +0100
@@ -109,6 +109,7 @@
 where
   append_Nil:"[] @ ys = ys"
   | append_Cons: "(x#xs) @ ys = x # xs @ ys"
+declare append.simps [code]
 
 primrec
   "rev([]) = []"
@@ -3177,6 +3178,7 @@
 where 
   "x mem [] \<longleftrightarrow> False"
   | "x mem (y#ys) \<longleftrightarrow> (if y = x then True else x mem ys)"
+declare member.simps [code]
 
 primrec
   "null [] = True"