src/HOL/Library/Pure_term.thy
changeset 22845 5f9138bcb3d7
parent 22804 d3c23b90c6c6
child 23063 b4ee6ec4f9c6
--- a/src/HOL/Library/Pure_term.thy	Sun May 06 21:49:44 2007 +0200
+++ b/src/HOL/Library/Pure_term.thy	Sun May 06 21:50:17 2007 +0200
@@ -92,8 +92,8 @@
 
 code_datatype Const App Fix Absp Bound
 lemmas [code func] = Bnd_Bound Abs_Absp
-lemmas [code nofunc] = term.recs term.cases term.size
-lemma [code func, code nofunc]: "(t1\<Colon>term) = t2 \<longleftrightarrow> t1 = t2" ..
+lemmas [code func del] = term.recs term.cases term.size
+lemma [code func, code func del]: "(t1\<Colon>term) = t2 \<longleftrightarrow> t1 = t2" ..
 
 code_type "typ" and "term"
   (SML "Term.typ" and "Term.term")