changeset 74342 | 5d411d85da8c |
parent 73015 | 2d7060a3ea11 |
child 80754 | 701912f5645a |
--- a/src/FOL/IFOL.thy Tue Sep 21 13:12:14 2021 +0200 +++ b/src/FOL/IFOL.thy Tue Sep 21 13:14:18 2021 +0200 @@ -527,7 +527,7 @@ structure Hypsubst = Hypsubst ( val dest_eq = FOLogic.dest_eq - val dest_Trueprop = FOLogic.dest_Trueprop + val dest_Trueprop = \<^dest_judgment> val dest_imp = FOLogic.dest_imp val eq_reflection = @{thm eq_reflection} val rev_eq_reflection = @{thm meta_eq_to_obj_eq}