src/Pure/context_position.ML
changeset 56294 85911b8a6868
parent 55923 4bdae9403baf
child 56333 38f1422ef473
--- a/src/Pure/context_position.ML	Wed Mar 26 14:15:34 2014 +0100
+++ b/src/Pure/context_position.ML	Wed Mar 26 14:41:52 2014 +0100
@@ -9,8 +9,6 @@
   val is_visible_generic: Context.generic -> bool
   val is_visible: Proof.context -> bool
   val is_visible_global: theory -> bool
-  val if_visible: Proof.context -> ('a -> unit) -> 'a -> unit
-  val if_visible_global: theory -> ('a -> unit) -> 'a -> unit
   val set_visible: bool -> Proof.context -> Proof.context
   val set_visible_global: bool -> theory -> theory
   val restore_visible: Proof.context -> Proof.context -> Proof.context
@@ -40,9 +38,6 @@
 val is_visible = is_visible_generic o Context.Proof;
 val is_visible_global = is_visible_generic o Context.Theory;
 
-fun if_visible ctxt f x = if is_visible ctxt then f x else ();
-fun if_visible_global thy f x = if is_visible_global thy then f x else ();
-
 val set_visible = Context.proof_map o Data.put o SOME;
 val set_visible_global = Context.theory_map o Data.put o SOME;