src/HOL/Inductive.thy
changeset 81506 f76a5849b570
parent 81505 01f2936ec85e
--- a/src/HOL/Inductive.thy	Fri Nov 29 00:25:03 2024 +0100
+++ b/src/HOL/Inductive.thy	Fri Nov 29 11:26:17 2024 +0100
@@ -532,7 +532,7 @@
   let
     fun fun_tr ctxt [cs] =
       let
-        val x = Syntax.free (fst (Name.variant "x" (Term.declare_free_names cs Name.context)));
+        val x = Syntax.free (#1 (Name.variant "x" (Name.build_context (Term.declare_free_names cs))));
         val ft = Case_Translation.case_tr true ctxt [x, cs];
       in lambda x ft end
   in [(\<^syntax_const>\<open>_lam_pats_syntax\<close>, fun_tr)] end