Quot/QuotMain.thy
changeset 1077 44461d5615eb
parent 1068 62e54830590f
child 1113 9f6c606d5b59
equal deleted inserted replaced
1076:9a3d2a4f8956 1077:44461d5615eb
   179 method_setup cleaning =
   179 method_setup cleaning =
   180   {* Scan.succeed (mk_method2 Quotient_Tacs.clean_tac) *}
   180   {* Scan.succeed (mk_method2 Quotient_Tacs.clean_tac) *}
   181   {* Proves automatically the cleaning goals from the lifting procedure. *}
   181   {* Proves automatically the cleaning goals from the lifting procedure. *}
   182 
   182 
   183 attribute_setup quot_lifted =
   183 attribute_setup quot_lifted =
   184   {* Scan.succeed Quotient_Tacs.lifted_attr *}
   184   {* Scan.succeed Quotient_Tacs.lifted_attrib *}
   185   {* Lifting of theorems to quotient types. *}
   185   {* Lifting of theorems to quotient types. *}
   186 
   186 
   187 end
   187 end
   188 
   188