src/HOL/HOL.thy
changeset 78799 807b249f1061
parent 78794 c74fd21af246
child 78800 0b3700d31758
--- a/src/HOL/HOL.thy	Thu Oct 19 11:30:16 2023 +0200
+++ b/src/HOL/HOL.thy	Thu Oct 19 16:31:17 2023 +0200
@@ -1542,15 +1542,14 @@
 
 ML_file \<open>~~/src/Tools/induction.ML\<close>
 
-simproc_setup swap_induct_false ("induct_false \<Longrightarrow> PROP P \<Longrightarrow> PROP Q") =
+simproc_setup passive swap_induct_false ("induct_false \<Longrightarrow> PROP P \<Longrightarrow> PROP Q") =
   \<open>fn _ => fn _ => fn ct =>
     (case Thm.term_of ct of
       _ $ (P as _ $ \<^Const_>\<open>induct_false\<close>) $ (_ $ Q $ _) =>
         if P <> Q then SOME Drule.swap_prems_eq else NONE
     | _ => NONE)\<close>
- (passive)
-
-simproc_setup induct_equal_conj_curry ("induct_conj P Q \<Longrightarrow> PROP R") =
+
+simproc_setup passive induct_equal_conj_curry ("induct_conj P Q \<Longrightarrow> PROP R") =
   \<open>fn _ => fn _ => fn ct =>
     (case Thm.term_of ct of
       _ $ (_ $ P) $ _ =>
@@ -1562,7 +1561,6 @@
             | is_conj _ = false
         in if is_conj P then SOME @{thm induct_conj_curry} else NONE end
       | _ => NONE)\<close>
- (passive)
 
 declaration \<open>
   K (Induct.map_simpset (fn ss => ss
@@ -1934,12 +1932,11 @@
 declare eq_equal [symmetric, code_post]
 declare eq_equal [code]
 
-simproc_setup equal (HOL.eq) =
+simproc_setup passive equal (HOL.eq) =
   \<open>fn _ => fn _ => fn ct =>
     (case Thm.term_of ct of
       Const (_, Type (\<^type_name>\<open>fun\<close>, [Type _, _])) => SOME @{thm eq_equal}
     | _ => NONE)\<close>
-  (passive)
 
 setup \<open>Code_Preproc.map_pre (fn ctxt => ctxt addsimprocs [\<^simproc>\<open>equal\<close>])\<close>