equal
deleted
inserted
replaced
8 (if fastype_of t = Sign.certify_typ (ProofContext.theory_of ctxt) T then () |
8 (if fastype_of t = Sign.certify_typ (ProofContext.theory_of ctxt) T then () |
9 else error "term_type_only: type mismatch"; |
9 else error "term_type_only: type mismatch"; |
10 Syntax.pretty_typ ctxt T) |
10 Syntax.pretty_typ ctxt T) |
11 |
11 |
12 val _ = Thy_Output.antiquotation "term_type_only" (Args.term -- Args.typ_abbrev) |
12 val _ = Thy_Output.antiquotation "term_type_only" (Args.term -- Args.typ_abbrev) |
13 (fn {source, context, ...} => fn arg => |
13 (fn {source, context = ctxt, ...} => fn arg => |
14 Thy_Output.output |
14 Thy_Output.output ctxt |
15 (Thy_Output.maybe_pretty_source (pretty_term_type_only context) source [arg])); |
15 (Thy_Output.maybe_pretty_source pretty_term_type_only ctxt source [arg])); |
16 *} |
16 *} |
17 (*>*) |
17 (*>*) |
18 text{* |
18 text{* |
19 |
19 |
20 \begin{abstract} |
20 \begin{abstract} |