src/HOL/Quotient.thy
changeset 45782 f82020ca3248
parent 45680 a61510361b89
child 45802 b16f976db515
equal deleted inserted replaced
45776:714100f5fda4 45782:f82020ca3248
   745 
   745 
   746 method_setup descending_setup =
   746 method_setup descending_setup =
   747   {* Scan.succeed (fn ctxt => SIMPLE_METHOD (HEADGOAL (Quotient_Tacs.descend_procedure_tac ctxt []))) *}
   747   {* Scan.succeed (fn ctxt => SIMPLE_METHOD (HEADGOAL (Quotient_Tacs.descend_procedure_tac ctxt []))) *}
   748   {* set up the three goals for the decending theorems *}
   748   {* set up the three goals for the decending theorems *}
   749 
   749 
       
   750 method_setup partiality_descending =
       
   751   {* Scan.succeed (fn ctxt => SIMPLE_METHOD (HEADGOAL (Quotient_Tacs.partiality_descend_tac ctxt []))) *}
       
   752   {* decend theorems to the raw level *}
       
   753 
       
   754 method_setup partiality_descending_setup =
       
   755   {* Scan.succeed (fn ctxt => 
       
   756        SIMPLE_METHOD (HEADGOAL (Quotient_Tacs.partiality_descend_procedure_tac ctxt []))) *}
       
   757   {* set up the three goals for the decending theorems *}
       
   758 
   750 method_setup regularize =
   759 method_setup regularize =
   751   {* Scan.succeed (fn ctxt => SIMPLE_METHOD (HEADGOAL (Quotient_Tacs.regularize_tac ctxt))) *}
   760   {* Scan.succeed (fn ctxt => SIMPLE_METHOD (HEADGOAL (Quotient_Tacs.regularize_tac ctxt))) *}
   752   {* prove the regularization goals from the quotient lifting procedure *}
   761   {* prove the regularization goals from the quotient lifting procedure *}
   753 
   762 
   754 method_setup injection =
   763 method_setup injection =