proper lemma [source] antiquotation
authorhaftmann
Mon, 26 May 2008 17:55:37 +0200
changeset 26996 090a619e7d87
parent 26995 2511a72dd73c
child 26997 40552bbac005
proper lemma [source] antiquotation
src/Pure/Thy/thy_output.ML
--- a/src/Pure/Thy/thy_output.ML	Mon May 26 17:55:36 2008 +0200
+++ b/src/Pure/Thy/thy_output.ML	Mon May 26 17:55:37 2008 +0200
@@ -468,6 +468,8 @@
       |> Proof.global_terminal_proof (method_text, NONE);
   in pretty_term ctxt prop end;
 
+val hd_src = Args.src o (apfst o apsnd) (single o hd) o Args.dest_src;
+
 fun pretty_thm ctxt = pretty_term ctxt o Thm.full_prop_of;
 
 fun pretty_term_style ctxt (name, t) =
@@ -529,7 +531,7 @@
  [("thm", args Attrib.thms (output_list pretty_thm)),
   ("thm_style", args (Scan.lift Args.liberal_name -- Attrib.thm) (output pretty_thm_style)),
   ("prop", args Args.prop (output pretty_term)),
-  ("lemma", args (Args.prop -- Scan.lift Method.simple_text) (output pretty_fact)),
+  ("lemma", args (Args.prop -- Scan.lift Method.simple_text) (output pretty_fact o hd_src)),
   ("term", args Args.term (output pretty_term)),
   ("term_style", args (Scan.lift Args.liberal_name -- Args.term) (output pretty_term_style)),
   ("term_type", args Args.term (output pretty_term_typ)),