src/HOL/Nominal/nominal_thmdecls.ML
changeset 22715 381e6c45f13b
parent 22562 80b814fe284b
child 22846 fb79144af9a3
--- a/src/HOL/Nominal/nominal_thmdecls.ML	Mon Apr 16 06:45:22 2007 +0200
+++ b/src/HOL/Nominal/nominal_thmdecls.ML	Mon Apr 16 07:32:23 2007 +0200
@@ -15,6 +15,8 @@
   val print_data: Proof.context -> unit
   val eqvt_add: attribute
   val eqvt_del: attribute
+  val eqvt_force_add: attribute
+  val eqvt_force_del: attribute
   val setup: theory -> theory
   val get_eqvt_thms: theory -> thm list
   val get_fresh_thms: theory -> thm list
@@ -205,19 +207,22 @@
 
 val eqvt_add  = Thm.declaration_attribute (eqvt_add_del_aux (eqvt_map Drule.add_rule)); 
 val eqvt_del  = Thm.declaration_attribute (eqvt_add_del_aux (eqvt_map Drule.del_rule)); 
+val eqvt_force_add  = Thm.declaration_attribute (eqvt_force_add_del_aux (eqvt_map Drule.add_rule)); 
+val eqvt_force_del  = Thm.declaration_attribute (eqvt_force_add_del_aux (eqvt_map Drule.del_rule)); 
+
 val bij_add   = Thm.declaration_attribute (bij_add_del_aux (bij_map Drule.add_rule)); 
 val bij_del   = Thm.declaration_attribute (bij_add_del_aux (bij_map Drule.del_rule));
 val fresh_add = Thm.declaration_attribute (fresh_add_del_aux (fresh_map Drule.add_rule)); 
 val fresh_del = Thm.declaration_attribute (fresh_add_del_aux (fresh_map Drule.del_rule));
 
-val eqvt_force_add  = Thm.declaration_attribute (eqvt_force_add_del_aux (eqvt_map Drule.add_rule)); 
-val eqvt_force_del  = Thm.declaration_attribute (eqvt_force_add_del_aux (eqvt_map Drule.del_rule)); 
+
 
 val setup =
   Data.init #>
   Attrib.add_attributes 
      [("eqvt",  Attrib.add_del_args eqvt_add eqvt_del,   "equivariance theorem declaration"),
-      ("eqvt_force",  Attrib.add_del_args eqvt_force_add eqvt_force_del,"equivariance theorem declaration (without checking the form of the lemma)"),
+      ("eqvt_force", Attrib.add_del_args eqvt_force_add eqvt_force_del,
+                             "equivariance theorem declaration (without checking the form of the lemma)"),
       ("fresh", Attrib.add_del_args fresh_add fresh_del, "freshness theorem declaration"),
       ("bij",   Attrib.add_del_args bij_add bij_del,     "bijection theorem declaration")];