src/HOL/Library/List_Cset.thy
changeset 43979 9f27d2bf4087
parent 43971 892030194015
child 44556 c0fd385a41f4
--- a/src/HOL/Library/List_Cset.thy	Tue Jul 26 12:44:36 2011 +0200
+++ b/src/HOL/Library/List_Cset.thy	Tue Jul 26 14:05:28 2011 +0200
@@ -133,7 +133,7 @@
 
 end
 
-declare single_code [code del]
+declare Cset.single_code [code del]
 lemma single_set [code]:
   "Cset.single a = Cset.set [a]"
 by(simp add: Cset.single_code)