new menu item show-sort-hypotheses to toggle show_hyps
authorwebertj
Tue, 20 Sep 2005 15:12:40 +0200
changeset 17520 8581c151adea
parent 17519 9c10585a238c
child 17521 0f1c48de39f5
new menu item show-sort-hypotheses to toggle show_hyps
src/Pure/proof_general.ML
--- a/src/Pure/proof_general.ML	Tue Sep 20 14:20:58 2005 +0200
+++ b/src/Pure/proof_general.ML	Tue Sep 20 15:12:40 2005 +0200
@@ -565,6 +565,9 @@
      ("show-main-goal",
       ("Show main goal in proof state display",
        bool_option Proof.show_main_goal)),
+     ("show-sort-hypotheses",
+      ("Include sort hypotheses in display of Isabelle theorems",
+       bool_option show_hyps)),
      ("eta-contract",
       ("Print terms eta-contracted",
        bool_option Syntax.eta_contract))]),