diff -r 31b9dfbe534c -r b10f7c981df6 src/HOL/Fun_Def.thy --- a/src/HOL/Fun_Def.thy Mon Jun 10 13:44:46 2024 +0200 +++ b/src/HOL/Fun_Def.thy Mon Jun 10 14:09:55 2024 +0200 @@ -68,8 +68,8 @@ definition in_rel_def[simp]: "in_rel R x y \ (x, y) \ R" -lemma wf_in_rel: "wf R \ wfP (in_rel R)" - by (simp add: wfP_def) +lemma wf_in_rel: "wf R \ wfp (in_rel R)" + by (simp add: wfp_def) ML_file \Tools/Function/function_core.ML\ ML_file \Tools/Function/mutual.ML\