changeset 78799 | 807b249f1061 |
parent 78798 | 200daaab2578 |
child 78805 | 62616d8422c5 |
--- a/src/Pure/ex/Def.thy Thu Oct 19 11:30:16 2023 +0200 +++ b/src/Pure/ex/Def.thy Thu Oct 19 16:31:17 2023 +0200 @@ -67,7 +67,7 @@ val _ = Simplifier.simproc_setup - {name = \<^binding>\<open>expand_def\<close>, lhss = ["x::'a"], passive = false, proc = K get_def}; + {passive = false, name = \<^binding>\<open>expand_def\<close>, lhss = ["x::'a"], proc = K get_def}; (* Isar command *)