tuned signature for print_nested_cases;
authorwenzelm
Mon, 27 Jul 2015 16:35:12 +0200
changeset 60799 57dd0b45fc21
parent 60798 9a9694087cda
child 60800 7d04351c795a
child 60801 7664e0916eec
tuned signature for print_nested_cases;
src/Pure/Isar/proof_context.ML
--- a/src/Pure/Isar/proof_context.ML	Mon Jul 27 15:13:05 2015 +0200
+++ b/src/Pure/Isar/proof_context.ML	Mon Jul 27 16:35:12 2015 +0200
@@ -139,6 +139,7 @@
   val add_assms_cmd: Assumption.export ->
     (Thm.binding * (string * string list) list) list ->
     Proof.context -> (string * thm list) list * Proof.context
+  val dest_cases: Proof.context -> (string * (Rule_Cases.T * {legacy: bool})) list
   val update_cases: (string * Rule_Cases.T option) list -> Proof.context -> Proof.context
   val update_cases_legacy: (string * Rule_Cases.T option) list -> Proof.context -> Proof.context
   val apply_case: Rule_Cases.T -> Proof.context -> (string * term list) list * Proof.context