src/HOL/ex/Cartouche_Examples.thy
changeset 58991 92b6f4e68c5a
parent 58978 e42da880c61e
child 58999 ed09ae4ea2d8
--- a/src/HOL/ex/Cartouche_Examples.thy	Tue Nov 11 21:14:19 2014 +0100
+++ b/src/HOL/ex/Cartouche_Examples.thy	Wed Nov 12 10:30:59 2014 +0100
@@ -214,9 +214,10 @@
   fun ml_tactic source ctxt =
     let
       val ctxt' = ctxt |> Context.proof_map
-        (ML_Context.expression (#range source)
-          "fun tactic (ctxt : Proof.context) : tactic"
-          "Context.map_proof (ML_Tactic.set tactic)" (ML_Lex.read_source false source));
+        (ML_Context.expression (#range source) "tactic" "Proof.context -> tactic"
+          "Context.map_proof (ML_Tactic.set tactic)"
+          (ML_Lex.read Position.none "fn ctxt: Proof.context =>" @
+           ML_Lex.read_source false source));
     in Data.get ctxt' ctxt end;
 end;
 *}