src/Pure/Isar/isar_thy.ML
changeset 14598 7009f59711e3
parent 14564 3667b4616e9a
child 14649 8ad41d25c152
--- a/src/Pure/Isar/isar_thy.ML	Fri Apr 16 18:44:39 2004 +0200
+++ b/src/Pure/Isar/isar_thy.ML	Fri Apr 16 18:45:56 2004 +0200
@@ -565,7 +565,7 @@
     \val thms = PureThy.get_thms_closure (Context.the_context ());\n\
     \val method: bstring * (Args.src -> Proof.context -> Proof.method) * string"
     "PureIsar.Method.add_method method"
-    ("(" ^ quote name ^ ", " ^ txt ^ ", " ^ quote cmt ^ ")");
+    ("(" ^ Library.quote name ^ ", " ^ txt ^ ", " ^ Library.quote cmt ^ ")");
 
 
 (* add_oracle *)
@@ -574,7 +574,7 @@
   Context.use_let
     "val oracle: bstring * (Sign.sg * Object.T -> term)"
     "Theory.add_oracle oracle"
-    ("(" ^ quote name ^ ", " ^ txt ^ ")");
+    ("(" ^ Library.quote name ^ ", " ^ txt ^ ")");
 
 
 (* add_locale *)