simplified use of tacticals;
authorwenzelm
Tue, 14 Feb 2012 20:09:35 +0100
changeset 46468 4db76d47b51a
parent 46467 39e412f9ffdf
child 46469 0632b8e56e46
simplified use of tacticals;
src/HOL/Quotient.thy
src/HOL/Tools/Quotient/quotient_tacs.ML
--- a/src/HOL/Quotient.thy	Tue Feb 14 20:08:59 2012 +0100
+++ b/src/HOL/Quotient.thy	Tue Feb 14 20:09:35 2012 +0100
@@ -738,41 +738,41 @@
 
 method_setup lifting =
   {* Attrib.thms >> (fn thms => fn ctxt => 
-       SIMPLE_METHOD (HEADGOAL (Quotient_Tacs.lift_tac ctxt [] thms))) *}
+       SIMPLE_METHOD' (Quotient_Tacs.lift_tac ctxt [] thms)) *}
   {* lift theorems to quotient types *}
 
 method_setup lifting_setup =
   {* Attrib.thm >> (fn thm => fn ctxt => 
-       SIMPLE_METHOD (HEADGOAL (Quotient_Tacs.lift_procedure_tac ctxt [] thm))) *}
+       SIMPLE_METHOD' (Quotient_Tacs.lift_procedure_tac ctxt [] thm)) *}
   {* set up the three goals for the quotient lifting procedure *}
 
 method_setup descending =
-  {* Scan.succeed (fn ctxt => SIMPLE_METHOD (HEADGOAL (Quotient_Tacs.descend_tac ctxt []))) *}
+  {* Scan.succeed (fn ctxt => SIMPLE_METHOD' (Quotient_Tacs.descend_tac ctxt [])) *}
   {* decend theorems to the raw level *}
 
 method_setup descending_setup =
-  {* Scan.succeed (fn ctxt => SIMPLE_METHOD (HEADGOAL (Quotient_Tacs.descend_procedure_tac ctxt []))) *}
+  {* Scan.succeed (fn ctxt => SIMPLE_METHOD' (Quotient_Tacs.descend_procedure_tac ctxt [])) *}
   {* set up the three goals for the decending theorems *}
 
 method_setup partiality_descending =
-  {* Scan.succeed (fn ctxt => SIMPLE_METHOD (HEADGOAL (Quotient_Tacs.partiality_descend_tac ctxt []))) *}
+  {* Scan.succeed (fn ctxt => SIMPLE_METHOD' (Quotient_Tacs.partiality_descend_tac ctxt [])) *}
   {* decend theorems to the raw level *}
 
 method_setup partiality_descending_setup =
   {* Scan.succeed (fn ctxt => 
-       SIMPLE_METHOD (HEADGOAL (Quotient_Tacs.partiality_descend_procedure_tac ctxt []))) *}
+       SIMPLE_METHOD' (Quotient_Tacs.partiality_descend_procedure_tac ctxt [])) *}
   {* set up the three goals for the decending theorems *}
 
 method_setup regularize =
-  {* Scan.succeed (fn ctxt => SIMPLE_METHOD (HEADGOAL (Quotient_Tacs.regularize_tac ctxt))) *}
+  {* Scan.succeed (fn ctxt => SIMPLE_METHOD' (Quotient_Tacs.regularize_tac ctxt)) *}
   {* prove the regularization goals from the quotient lifting procedure *}
 
 method_setup injection =
-  {* Scan.succeed (fn ctxt => SIMPLE_METHOD (HEADGOAL (Quotient_Tacs.all_injection_tac ctxt))) *}
+  {* Scan.succeed (fn ctxt => SIMPLE_METHOD' (Quotient_Tacs.all_injection_tac ctxt)) *}
   {* prove the rep/abs injection goals from the quotient lifting procedure *}
 
 method_setup cleaning =
-  {* Scan.succeed (fn ctxt => SIMPLE_METHOD (HEADGOAL (Quotient_Tacs.clean_tac ctxt))) *}
+  {* Scan.succeed (fn ctxt => SIMPLE_METHOD' (Quotient_Tacs.clean_tac ctxt)) *}
   {* prove the cleaning goals from the quotient lifting procedure *}
 
 attribute_setup quot_lifted =
--- a/src/HOL/Tools/Quotient/quotient_tacs.ML	Tue Feb 14 20:08:59 2012 +0100
+++ b/src/HOL/Tools/Quotient/quotient_tacs.ML	Tue Feb 14 20:09:35 2012 +0100
@@ -364,7 +364,7 @@
   | (_ $
       (Const(@{const_name Babs},_) $ (Const (@{const_name Respects}, _) $ _) $ _) $
       (Const(@{const_name Babs},_) $ (Const (@{const_name Respects}, _) $ _) $ _))
-        => rtac @{thm babs_rsp} THEN' RANGE [quotient_tac ctxt]
+        => rtac @{thm babs_rsp} THEN' quotient_tac ctxt
 
   | Const (@{const_name HOL.eq},_) $ (R $ _ $ _) $ (_ $ _ $ _) =>
      (rtac @{thm refl} ORELSE'