# HG changeset patch # User wenzelm # Date 1747830837 -7200 # Node ID ccc21bb6004da787963069ebd2d6c5ac30f86d7c # Parent c994245a696588a479607c5890a03acd313a9790 tuned: more antiquotations; diff -r c994245a6965 -r ccc21bb6004d src/HOL/HOLCF/Cpo.thy --- a/src/HOL/HOLCF/Cpo.thy Wed May 21 13:50:40 2025 +0200 +++ b/src/HOL/HOLCF/Cpo.thy Wed May 21 14:33:57 2025 +0200 @@ -1105,8 +1105,8 @@ using cont_id by (rule cont2cont_fun) simproc_setup apply_cont (\cont (\f. E f)\) = \ - fn _ => fn ctxt => fn ct => - (case Thm.term_of ct of + fn _ => fn ctxt => fn lhs => + (case Thm.term_of lhs of \<^Const_>\cont _ _ for \Abs (_, _, expr)\\ => if Term.head_of expr = Bound 0 (* since \\f. E f\ is too permissive, we ensure that the term is of the @@ -1114,9 +1114,10 @@ then let val tac = Metis_Tactic.metis_tac ["no_types"] "combs" ctxt @{thms cont2cont_fun cont_id} - val rwrt_ct = HOLogic.mk_judgment (Thm.apply \<^cterm>\\lhs. lhs = True\ ct) - val rwrt_thm = Goal.prove_internal ctxt [] rwrt_ct (fn _ => tac 1) - in SOME (mk_meta_eq rwrt_thm) end + val thm = + Goal.prove_internal ctxt [] \<^instantiate>\lhs in cprop \lhs = True\\ + (fn _ => tac 1) + in SOME (mk_meta_eq thm) end else NONE | _ => NONE) \