src/CCL/CCL.thy
changeset 39159 0dec18004e75
parent 36452 d37c6eed8117
child 40844 5895c525739d
--- a/src/CCL/CCL.thy	Mon Sep 06 19:11:01 2010 +0200
+++ b/src/CCL/CCL.thy	Mon Sep 06 19:13:10 2010 +0200
@@ -238,9 +238,9 @@
 
   fun mk_thm_str thy a b = "~ " ^ (saturate thy a "a") ^ " = " ^ (saturate thy b "b")
 
-  val lemma = thm "lem";
-  val eq_lemma = thm "eq_lemma";
-  val distinctness = thm "distinctness";
+  val lemma = @{thm lem};
+  val eq_lemma = @{thm eq_lemma};
+  val distinctness = @{thm distinctness};
   fun mk_lemma (ra,rb) = [lemma] RL [ra RS (rb RS eq_lemma)] RL
                            [distinctness RS notE, @{thm sym} RS (distinctness RS notE)]
 in