src/HOL/Tools/Predicate_Compile/predicate_compile_core.ML
changeset 38072 7b8c295af291
parent 37678 0040bafffdef
child 38549 d0385f2764d8
--- a/src/HOL/Tools/Predicate_Compile/predicate_compile_core.ML	Thu Jul 29 15:07:52 2010 +0200
+++ b/src/HOL/Tools/Predicate_Compile/predicate_compile_core.ML	Thu Jul 29 17:27:51 2010 +0200
@@ -27,6 +27,7 @@
   val all_modes_of : compilation -> Proof.context -> (string * mode list) list
   val all_random_modes_of : Proof.context -> (string * mode list) list
   val intros_of : Proof.context -> string -> thm list
+  val intros_graph_of : Proof.context -> thm list Graph.T
   val add_intro : thm -> theory -> theory
   val set_elim : thm -> theory -> theory
   val register_alternative_function : string -> mode -> string -> theory -> theory
@@ -295,6 +296,9 @@
 
 val predfun_neg_intro_of = #neg_intro ooo the_predfun_data
 
+val intros_graph_of =
+  Graph.map_nodes (#intros o rep_pred_data) o PredData.get o ProofContext.theory_of
+
 (* diagnostic display functions *)
 
 fun print_modes options modes =