--- a/NEWS Wed Feb 28 16:35:00 2007 +0100
+++ b/NEWS Wed Feb 28 22:05:41 2007 +0100
@@ -769,6 +769,8 @@
ML {* @{cprop "x == y"} *}
ML {* @{thm asm_rl} *}
ML {* @{thms asm_rl} *}
+ML {* @{const_name c} *}
+ML {* @{const_syntax c} *}
ML {* @{context} *}
ML {* @{theory} *}
ML {* @{theory Pure} *}
--- a/src/Pure/Thy/ml_context.ML Wed Feb 28 16:35:00 2007 +0100
+++ b/src/Pure/Thy/ml_context.ML Wed Feb 28 22:05:41 2007 +0100
@@ -206,6 +206,15 @@
"Thm.cterm_of (ML_Context.the_context ()) " ^ ML_Syntax.atomic (ML_Syntax.print_term t))));
+fun const syn = (Scan.state >> Context.proof_of) -- Scan.lift Args.name >> (fn (ctxt, c) =>
+ #1 (Term.dest_Const (Consts.read_const (ProofContext.consts_of ctxt) c))
+ |> syn ? ProofContext.const_syntax_name ctxt
+ |> ML_Syntax.print_string);
+
+val _ = inline_antiq "const_name" (const false);
+val _ = inline_antiq "const_syntax" (const true);
+
+
(** fact references **)