renamed SIMPLE_METHOD' to SIMPLE_METHOD'';
authorwenzelm
Wed, 29 Nov 2006 15:44:59 +0100
changeset 21592 8831206d7f41
parent 21591 5e0f2340caa7
child 21593 282c40fb001a
renamed SIMPLE_METHOD' to SIMPLE_METHOD''; added simple version of SIMPLE_METHOD';
src/Pure/Isar/method.ML
--- a/src/Pure/Isar/method.ML	Wed Nov 29 15:44:58 2006 +0100
+++ b/src/Pure/Isar/method.ML	Wed Nov 29 15:44:59 2006 +0100
@@ -29,7 +29,8 @@
   val insert: thm list -> method
   val insert_facts: method
   val SIMPLE_METHOD: tactic -> method
-  val SIMPLE_METHOD': ((int -> tactic) -> tactic) -> (int -> tactic) -> method
+  val SIMPLE_METHOD': (int -> tactic) -> method
+  val SIMPLE_METHOD'': ((int -> tactic) -> tactic) -> (int -> tactic) -> method
   val defer: int option -> method
   val prefer: int -> method
   val cheating: bool -> Proof.context -> method
@@ -163,7 +164,8 @@
 fun insert thms = METHOD (fn _ => ALLGOALS (insert_tac thms));
 
 fun SIMPLE_METHOD tac = METHOD (fn facts => ALLGOALS (insert_tac facts) THEN tac);
-fun SIMPLE_METHOD' quant tac = METHOD (fn facts => quant (insert_tac facts THEN' tac));
+fun SIMPLE_METHOD'' quant tac = METHOD (fn facts => quant (insert_tac facts THEN' tac));
+val SIMPLE_METHOD' = SIMPLE_METHOD'' HEADGOAL;
 
 end;
 
@@ -182,8 +184,8 @@
 
 (* unfold intro/elim rules *)
 
-fun intro ths = SIMPLE_METHOD' HEADGOAL (CHANGED_PROP o REPEAT_ALL_NEW (Tactic.match_tac ths));
-fun elim ths = SIMPLE_METHOD' HEADGOAL (CHANGED_PROP o REPEAT_ALL_NEW (Tactic.ematch_tac ths));
+fun intro ths = SIMPLE_METHOD' (CHANGED_PROP o REPEAT_ALL_NEW (Tactic.match_tac ths));
+fun elim ths = SIMPLE_METHOD' (CHANGED_PROP o REPEAT_ALL_NEW (Tactic.ematch_tac ths));
 
 
 (* unfold/fold definitions *)
@@ -194,7 +196,7 @@
 
 (* atomize rule statements *)
 
-fun atomize false = SIMPLE_METHOD' HEADGOAL (CHANGED_PROP o ObjectLogic.atomize_tac)
+fun atomize false = SIMPLE_METHOD' (CHANGED_PROP o ObjectLogic.atomize_tac)
   | atomize true = RAW_METHOD (K (HEADGOAL (CHANGED_PROP o ObjectLogic.full_atomize_tac)));
 
 
@@ -205,8 +207,8 @@
 
 (* fact -- composition by facts from context *)
 
-fun fact [] ctxt = SIMPLE_METHOD' HEADGOAL (ProofContext.some_fact_tac ctxt)
-  | fact rules _ = SIMPLE_METHOD' HEADGOAL (ProofContext.fact_tac rules);
+fun fact [] ctxt = SIMPLE_METHOD' (ProofContext.some_fact_tac ctxt)
+  | fact rules _ = SIMPLE_METHOD' (ProofContext.fact_tac rules);
 
 
 (* assumption *)
@@ -538,13 +540,13 @@
   (#2 oo syntax (Scan.lift (Scan.optional (Args.parens Args.nat) 0) -- Attrib.thms));
 
 fun goal_args' args tac src ctxt = #2 (syntax (Args.goal_spec HEADGOAL -- args >>
-  (fn (quant, s) => SIMPLE_METHOD' quant (tac s))) src ctxt);
+  (fn (quant, s) => SIMPLE_METHOD'' quant (tac s))) src ctxt);
 
 fun goal_args args tac = goal_args' (Scan.lift args) tac;
 
 fun goal_args_ctxt' args tac src ctxt =
   #2 (syntax (Args.goal_spec HEADGOAL -- args >>
-  (fn (quant, s) => SIMPLE_METHOD' quant (tac ctxt s))) src ctxt);
+  (fn (quant, s) => SIMPLE_METHOD'' quant (tac ctxt s))) src ctxt);
 
 fun goal_args_ctxt args tac = goal_args_ctxt' (Scan.lift args) tac;