src/HOL/Library/RType.thy
changeset 28562 4e74209f113e
parent 28394 b9c8e3a12a98
--- a/src/HOL/Library/RType.thy	Fri Oct 10 06:45:50 2008 +0200
+++ b/src/HOL/Library/RType.thy	Fri Oct 10 06:45:53 2008 +0200
@@ -89,7 +89,7 @@
   #> TypedefPackage.interpretation Typerep.perhaps_add_def
 *}
 
-lemma [code func]:
+lemma [code]:
   "eq_class.eq (Typerep tyco1 tys1) (Typerep tyco2 tys2) \<longleftrightarrow> eq_class.eq tyco1 tyco2
      \<and> list_all2 eq_class.eq tys1 tys2"
   by (auto simp add: equals_eq [symmetric] list_all2_eq [symmetric])