changeset 76588 | 82a36e3d1b55 |
parent 76559 | 4352d0ff165a |
child 76682 | e260dabc88e6 |
--- a/src/HOL/Wellfounded.thy Tue Dec 06 20:08:51 2022 +0100 +++ b/src/HOL/Wellfounded.thy Tue Dec 06 18:56:28 2022 +0100 @@ -75,7 +75,7 @@ using wf_irrefl [OF assms] by (auto simp add: irrefl_def) lemma wfP_imp_irreflp: "wfP r \<Longrightarrow> irreflp r" - by (rule wf_imp_irrefl[to_pred, folded top_set_def]) + by (rule wf_imp_irrefl[to_pred]) lemma wf_wellorderI: assumes wf: "wf {(x::'a::ord, y). x < y}"