src/HOL/Set.thy
changeset 80662 ad9647592a81
parent 79566 f783490c6c99
child 80760 be8c0e039a5e
--- a/src/HOL/Set.thy	Wed Aug 07 14:44:51 2024 +0200
+++ b/src/HOL/Set.thy	Wed Aug 07 15:11:54 2024 +0200
@@ -251,7 +251,7 @@
       else raise Match;
 
     fun tr' q = (q, fn _ =>
-      (fn [Const (\<^syntax_const>\<open>_bound\<close>, _) $ Free (v, Type (\<^type_name>\<open>set\<close>, _)),
+      (fn [Const (\<^syntax_const>\<open>_bound\<close>, _) $ Free (v, \<^Type>\<open>set _\<close>),
           Const (c, _) $
             (Const (d, _) $ (Const (\<^syntax_const>\<open>_bound\<close>, _) $ Free (v', T)) $ n) $ P] =>
           (case AList.lookup (=) trans (q, c, d) of