src/Pure/context_position.ML
changeset 52699 abed4121c17e
parent 48767 7f0c469cc796
child 52700 d63f80f93025
--- a/src/Pure/context_position.ML	Thu Jul 18 21:06:21 2013 +0200
+++ b/src/Pure/context_position.ML	Thu Jul 18 21:20:09 2013 +0200
@@ -10,8 +10,6 @@
   val set_visible: bool -> Proof.context -> Proof.context
   val restore_visible: Proof.context -> Proof.context -> Proof.context
   val if_visible: Proof.context -> ('a -> unit) -> 'a -> unit
-  val is_visible_proof: Context.generic -> bool
-  val if_visible_proof: Context.generic -> ('a -> unit) -> 'a -> unit
   val report_generic: Context.generic -> Position.T -> Markup.T -> unit
   val reported_text: Proof.context -> Position.T -> Markup.T -> string -> string
   val report_text: Proof.context -> Position.T -> Markup.T -> string -> unit
@@ -38,11 +36,6 @@
 
 fun if_visible ctxt f x = if is_visible ctxt then f x else ();
 
-fun is_visible_proof (Context.Proof ctxt) = is_visible ctxt
-  | is_visible_proof _ = false;
-
-fun if_visible_proof context f x = if is_visible_proof context then f x else ();
-
 fun report_generic context pos markup =
   if is_visible_generic context then
     Output.report (Position.reported_text pos markup "")