equal
deleted
inserted
replaced
24 |
24 |
25 fun print_term ctxt t = |
25 fun print_term ctxt t = |
26 t |
26 t |
27 |> singleton (Syntax.uncheck_terms ctxt) |
27 |> singleton (Syntax.uncheck_terms ctxt) |
28 |> Sledgehammer_Isar_Annotate.annotate_types_in_term ctxt |
28 |> Sledgehammer_Isar_Annotate.annotate_types_in_term ctxt |
29 |> Print_Mode.setmp [] (Syntax.unparse_term ctxt #> Pretty.string_of) |
29 |> Syntax.unparse_term ctxt |
|
30 |> Pretty.pure_string_of |
30 |> Sledgehammer_Util.simplify_spaces |
31 |> Sledgehammer_Util.simplify_spaces |
31 |> ATP_Util.maybe_quote ctxt; |
32 |> ATP_Util.maybe_quote ctxt; |
32 |
33 |
33 fun eigen_context_for_statement (params, assms, concl) ctxt = |
34 fun eigen_context_for_statement (params, assms, concl) ctxt = |
34 let |
35 let |