src/Pure/Isar/method.ML
changeset 68823 5e7b1ae10eb8
parent 67504 310114bec0d7
child 69187 d8849cfad60f
--- a/src/Pure/Isar/method.ML	Mon Aug 27 19:29:07 2018 +0200
+++ b/src/Pure/Isar/method.ML	Mon Aug 27 20:43:01 2018 +0200
@@ -373,7 +373,7 @@
             "tactic" "Morphism.morphism -> thm list -> tactic"
             "Method.set_tactic tactic"
             (ML_Lex.read "fn morphism: Morphism.morphism => fn facts: thm list =>" @
-             ML_Lex.read_source false source);
+             ML_Lex.read_source source);
         val tac = the_tactic context';
       in
         fn phi => set_tactic (fn _ => Context.setmp_generic_context (SOME context) (tac phi))
@@ -476,7 +476,7 @@
 fun local_setup binding scan comment = define binding (method_syntax scan) comment #> snd;
 
 fun method_setup name source comment =
-  ML_Lex.read_source false source
+  ML_Lex.read_source source
   |> ML_Context.expression (Input.range_of source) "parser"
     "(Proof.context -> Proof.method) context_parser"
     ("Context.map_proof (Method.local_setup " ^ ML_Syntax.atomic (ML_Syntax.make_binding name) ^