diff -r 8d0294d877bd -r 107941e8fa01 src/HOL/HOL.thy --- a/src/HOL/HOL.thy Tue Sep 28 22:14:02 2021 +0200 +++ b/src/HOL/HOL.thy Tue Sep 28 22:14:44 2021 +0200 @@ -888,7 +888,7 @@ structure Blast = Blast ( structure Classical = Classical - val Trueprop_const = dest_Const \<^const>\Trueprop\ + val Trueprop_const = dest_Const \<^Const>\Trueprop\ val equality_name = \<^const_name>\HOL.eq\ val not_name = \<^const_name>\Not\ val notE = @{thm notE} @@ -1549,7 +1549,7 @@ {lhss = [\<^term>\induct_false \ PROP P \ PROP Q\], proc = fn _ => fn _ => fn ct => (case Thm.term_of ct of - _ $ (P as _ $ \<^const>\induct_false\) $ (_ $ Q $ _) => + _ $ (P as _ $ \<^Const_>\induct_false\) $ (_ $ Q $ _) => if P <> Q then SOME Drule.swap_prems_eq else NONE | _ => NONE)}, Simplifier.make_simproc \<^context> "induct_equal_conj_curry" @@ -1558,11 +1558,11 @@ (case Thm.term_of ct of _ $ (_ $ P) $ _ => let - fun is_conj (\<^const>\induct_conj\ $ P $ Q) = + fun is_conj \<^Const_>\induct_conj for P Q\ = is_conj P andalso is_conj Q - | is_conj (Const (\<^const_name>\induct_equal\, _) $ _ $ _) = true - | is_conj \<^const>\induct_true\ = true - | is_conj \<^const>\induct_false\ = true + | is_conj \<^Const_>\induct_equal _ for _ _\ = true + | is_conj \<^Const_>\induct_true\ = true + | is_conj \<^Const_>\induct_false\ = true | is_conj _ = false in if is_conj P then SOME @{thm induct_conj_curry} else NONE end | _ => NONE)}]