equal
deleted
inserted
replaced
893 (T, NONE) => NONE |
893 (T, NONE) => NONE |
894 | (T, SOME rhs) => |
894 | (T, SOME rhs) => |
895 SOME (Goal.prove ctxt [] [] (Logic.mk_equals (t, rhs)) |
895 SOME (Goal.prove ctxt [] [] (Logic.mk_equals (t, rhs)) |
896 (fn _ => |
896 (fn _ => |
897 rtac eq_reflection 1 THEN |
897 rtac eq_reflection 1 THEN |
898 rtac ext 1 THEN |
898 rtac @{thm ext} 1 THEN |
899 simp_tac (put_simpset ss ctxt) 1)) |
899 simp_tac (put_simpset ss ctxt) 1)) |
900 end |
900 end |
901 in proc end |
901 in proc end |
902 *} |
902 *} |
903 |
903 |