src/HOL/ex/Cartouche_Examples.thy
changeset 69187 d8849cfad60f
parent 68823 5e7b1ae10eb8
child 69216 1a52baa70aed
--- a/src/HOL/ex/Cartouche_Examples.thy	Thu Oct 25 17:08:04 2018 +0200
+++ b/src/HOL/ex/Cartouche_Examples.thy	Thu Oct 25 21:29:08 2018 +0200
@@ -176,7 +176,7 @@
   fun ml_tactic source ctxt =
     let
       val ctxt' = ctxt |> Context.proof_map
-        (ML_Context.expression (Input.range_of source) "tactic" "Proof.context -> tactic"
+        (ML_Context.expression ("tactic", Position.thread_data ()) "Proof.context -> tactic"
           "Context.map_proof (ML_Tactic.set tactic)"
           (ML_Lex.read "fn ctxt: Proof.context =>" @ ML_Lex.read_source source));
     in Data.get ctxt' ctxt end;