temporary code generator work arounds
authorhaftmann
Thu, 06 Dec 2007 17:05:44 +0100
changeset 25563 cab4f808f791
parent 25562 f0fc8531c909
child 25564 4ca31a3706a4
temporary code generator work arounds
src/HOL/List.thy
src/HOL/Nat.thy
--- 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"
--- a/src/HOL/Nat.thy	Thu Dec 06 16:56:00 2007 +0100
+++ b/src/HOL/Nat.thy	Thu Dec 06 17:05:44 2007 +0100
@@ -1162,6 +1162,7 @@
 where
   of_nat_0:     "of_nat 0 = 0"
   | of_nat_Suc: "of_nat (Suc m) = 1 + of_nat m"
+declare of_nat.simps [code]
 
 lemma of_nat_1 [simp]: "of_nat 1 = 1"
   by simp