src/HOL/Library/Complete_Partial_Order2.thy
changeset 75582 6fb4a0829cc4
parent 74334 ead56ad40e15
child 75650 6d4fb57eb66c
--- a/src/HOL/Library/Complete_Partial_Order2.thy	Mon Jun 20 11:06:33 2022 +0200
+++ b/src/HOL/Library/Complete_Partial_Order2.thy	Tue Jun 21 13:39:06 2022 +0200
@@ -373,9 +373,9 @@
       | NONE => NONE
   in
     case Thm.term_of ct of
-      t as Const (\<^const_name>\<open>ccpo.admissible\<close>, _) $ _ $ _ $ _ => mk_thm t
-    | t as Const (\<^const_name>\<open>mcont\<close>, _) $ _ $ _ $ _ $ _ $ _ => mk_thm t
-    | t as Const (\<^const_name>\<open>monotone\<close>, _) $ _ $ _ $ _ => mk_thm t
+      t as \<^Const_>\<open>ccpo.admissible _ for _ _ _\<close> => mk_thm t
+    | t as \<^Const_>\<open>mcont _ _ for _ _ _ _ _\<close> => mk_thm t
+    | t as \<^Const_>\<open>monotone_on _ _ for \<^Const_>\<open>Orderings.top _\<close> _ _ _\<close> => mk_thm t
     | _ => NONE
   end
   handle THM _ => NONE