--- a/src/CCL/CCL.thy Sun May 15 17:06:35 2011 +0200
+++ b/src/CCL/CCL.thy Sun May 15 17:45:53 2011 +0200
@@ -205,7 +205,7 @@
method_setup inj_rl = {*
Attrib.thms >> (fn rews => fn ctxt => SIMPLE_METHOD' (inj_rl_tac ctxt rews))
-*} ""
+*}
lemma ccl_injs:
"<a,b> = <a',b'> <-> (a=a' & b=b')"