changeset 80322 | b10f7c981df6 |
parent 79597 | 76a1c0ea6777 |
--- 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 \<equiv> (x, y) \<in> R" -lemma wf_in_rel: "wf R \<Longrightarrow> wfP (in_rel R)" - by (simp add: wfP_def) +lemma wf_in_rel: "wf R \<Longrightarrow> wfp (in_rel R)" + by (simp add: wfp_def) ML_file \<open>Tools/Function/function_core.ML\<close> ML_file \<open>Tools/Function/mutual.ML\<close>