src/HOL/Quotient.thy
changeset 45782 f82020ca3248
parent 45680 a61510361b89
child 45802 b16f976db515
--- a/src/HOL/Quotient.thy	Mon Dec 05 15:10:15 2011 +0100
+++ b/src/HOL/Quotient.thy	Wed Dec 07 14:00:02 2011 +0000
@@ -747,6 +747,15 @@
   {* Scan.succeed (fn ctxt => SIMPLE_METHOD (HEADGOAL (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 []))) *}
+  {* 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 []))) *}
+  {* set up the three goals for the decending theorems *}
+
 method_setup regularize =
   {* Scan.succeed (fn ctxt => SIMPLE_METHOD (HEADGOAL (Quotient_Tacs.regularize_tac ctxt))) *}
   {* prove the regularization goals from the quotient lifting procedure *}