src/Pure/Isar/method.ML
changeset 58978 e42da880c61e
parent 58963 26bf09b95dda
child 58979 162a4c2e97bc
--- a/src/Pure/Isar/method.ML	Tue Nov 11 15:55:31 2014 +0100
+++ b/src/Pure/Isar/method.ML	Tue Nov 11 18:16:25 2014 +0100
@@ -282,7 +282,7 @@
     Scan.lift (Args.text_declaration (fn source =>
       let
         val context' = context |>
-          ML_Context.expression (#pos source)
+          ML_Context.expression (#range source)
             "fun tactic (morphism: Morphism.morphism) (facts: thm list) : tactic"
             "Method.set_tactic tactic" (ML_Lex.read_source false source);
         val tac = the_tactic context';
@@ -381,7 +381,7 @@
   (ML_Lex.read Position.none ("(" ^ ML_Syntax.make_binding name ^ ", ") @
     ML_Lex.read_source false source @
     ML_Lex.read Position.none (", " ^ ML_Syntax.print_string cmt ^ ")"))
-  |> ML_Context.expression (#pos source)
+  |> ML_Context.expression (#range source)
     "val (name, scan, comment): binding * (Proof.context -> Proof.method) context_parser * string"
     "Context.map_proof (Method.local_setup name scan comment)"
   |> Context.proof_map;