| author | bulwahn | 
| Wed, 08 Dec 2010 14:25:08 +0100 | |
| changeset 41078 | 051251fde456 | 
| parent 39508 | dfacdb01e1ec | 
| child 41470 | 890b25753bf7 | 
| permissions | -rw-r--r-- | 
| 28405 | 1 | (* Title: Pure/context_position.ML | 
| 2 | Author: Makarius | |
| 3 | ||
| 28409 | 4 | Context position visibility flag. | 
| 28405 | 5 | *) | 
| 6 | ||
| 7 | signature CONTEXT_POSITION = | |
| 8 | sig | |
| 9 | val is_visible: Proof.context -> bool | |
| 10 | val set_visible: bool -> Proof.context -> Proof.context | |
| 11 | val restore_visible: Proof.context -> Proof.context -> Proof.context | |
| 38831 
4933a3dfd745
more careful treatment of context visibility flag wrt. spurious warnings;
 wenzelm parents: 
38481diff
changeset | 12 |   val if_visible: Proof.context -> ('a -> unit) -> 'a -> unit
 | 
| 39507 
839873937ddd
tuned signature of (Context_)Position.report variants;
 wenzelm parents: 
39440diff
changeset | 13 | val reported_text: Proof.context -> Position.T -> Markup.T -> string -> string | 
| 
839873937ddd
tuned signature of (Context_)Position.report variants;
 wenzelm parents: 
39440diff
changeset | 14 | val report_text: Proof.context -> Position.T -> Markup.T -> string -> unit | 
| 
839873937ddd
tuned signature of (Context_)Position.report variants;
 wenzelm parents: 
39440diff
changeset | 15 | val report: Proof.context -> Position.T -> Markup.T -> unit | 
| 28405 | 16 | end; | 
| 17 | ||
| 33383 | 18 | structure Context_Position: CONTEXT_POSITION = | 
| 28405 | 19 | struct | 
| 20 | ||
| 39508 
dfacdb01e1ec
simplified some internal flags using Config.T instead of full-blown Proof_Data;
 wenzelm parents: 
39507diff
changeset | 21 | val visible = Config.bool (Config.declare "Context_Position.visible" (K (Config.Bool true))); | 
| 
dfacdb01e1ec
simplified some internal flags using Config.T instead of full-blown Proof_Data;
 wenzelm parents: 
39507diff
changeset | 22 | fun is_visible ctxt = Config.get ctxt visible; | 
| 
dfacdb01e1ec
simplified some internal flags using Config.T instead of full-blown Proof_Data;
 wenzelm parents: 
39507diff
changeset | 23 | val set_visible = Config.put visible; | 
| 28405 | 24 | val restore_visible = set_visible o is_visible; | 
| 25 | ||
| 38831 
4933a3dfd745
more careful treatment of context visibility flag wrt. spurious warnings;
 wenzelm parents: 
38481diff
changeset | 26 | fun if_visible ctxt f x = if is_visible ctxt then f x else (); | 
| 
4933a3dfd745
more careful treatment of context visibility flag wrt. spurious warnings;
 wenzelm parents: 
38481diff
changeset | 27 | |
| 39507 
839873937ddd
tuned signature of (Context_)Position.report variants;
 wenzelm parents: 
39440diff
changeset | 28 | fun reported_text ctxt pos markup txt = | 
| 
839873937ddd
tuned signature of (Context_)Position.report variants;
 wenzelm parents: 
39440diff
changeset | 29 | if is_visible ctxt then Position.reported_text pos markup txt else ""; | 
| 38481 
81ec258c4cd3
Output_Position.report_text -- markup with potential "arguments";
 wenzelm parents: 
38237diff
changeset | 30 | |
| 39507 
839873937ddd
tuned signature of (Context_)Position.report variants;
 wenzelm parents: 
39440diff
changeset | 31 | fun report_text ctxt pos markup txt = Output.report (reported_text ctxt pos markup txt); | 
| 
839873937ddd
tuned signature of (Context_)Position.report variants;
 wenzelm parents: 
39440diff
changeset | 32 | fun report ctxt pos markup = report_text ctxt pos markup ""; | 
| 28405 | 33 | |
| 34 | end; |