src/Pure/Isar/method.ML
changeset 58004 1b064162ec57
parent 58003 250ecd2502ad
child 58005 c28e6bc6635d
--- a/src/Pure/Isar/method.ML	Tue Aug 19 14:51:25 2014 +0200
+++ b/src/Pure/Isar/method.ML	Tue Aug 19 15:10:37 2014 +0200
@@ -69,7 +69,7 @@
     local_theory -> local_theory
   val method_setup: bstring * Position.T -> Symbol_Pos.source -> string ->
     local_theory -> local_theory
-  val evaluate: Proof.context -> text -> Proof.context -> method
+  val evaluate: text -> Proof.context -> Proof.context -> method
   type modifier = (Proof.context -> Proof.context) * attribute
   val section: modifier parser list -> thm list context_parser
   val sections: modifier parser list -> thm list list context_parser
@@ -413,7 +413,7 @@
 
 in
 
-fun evaluate static_ctxt text =
+fun evaluate text static_ctxt =
   let
     fun eval (Basic meth) = APPEND_CASES oo meth
       | eval (Source src) = APPEND_CASES oo method_cmd static_ctxt src