src/Pure/Isar/context_rules.ML
changeset 20289 ba7a7c56bed5
parent 19482 9f11af8f7ef9
child 21506 b2a673894ce5
--- a/src/Pure/Isar/context_rules.ML	Wed Aug 02 22:26:40 2006 +0200
+++ b/src/Pure/Isar/context_rules.ML	Wed Aug 02 22:26:41 2006 +0200
@@ -10,16 +10,16 @@
 sig
   type netpair
   type T
-  val netpair_bang: ProofContext.context -> netpair
-  val netpair: ProofContext.context -> netpair
+  val netpair_bang: Proof.context -> netpair
+  val netpair: Proof.context -> netpair
   val orderlist: ((int * int) * 'a) list -> 'a list
   val find_rules_netpair: bool -> thm list -> term -> netpair -> thm list
-  val find_rules: bool -> thm list -> term -> ProofContext.context -> thm list list
+  val find_rules: bool -> thm list -> term -> Proof.context -> thm list list
   val print_rules: Context.generic -> unit
   val addSWrapper: ((int -> tactic) -> int -> tactic) -> theory -> theory
   val addWrapper: ((int -> tactic) -> int -> tactic) -> theory -> theory
-  val Swrap: ProofContext.context -> (int -> tactic) -> int -> tactic
-  val wrap: ProofContext.context -> (int -> tactic) -> int -> tactic
+  val Swrap: Proof.context -> (int -> tactic) -> int -> tactic
+  val wrap: Proof.context -> (int -> tactic) -> int -> tactic
   val intro_bang: int option -> attribute
   val elim_bang: int option -> attribute
   val dest_bang: int option -> attribute