undone the previous change: show_hyps not supported anymore
authorwebertj
Tue, 20 Sep 2005 17:01:43 +0200
changeset 17523 73571cefff44
parent 17522 8d25bb07d8ed
child 17524 42d56a6dec6e
undone the previous change: show_hyps not supported anymore
src/Pure/proof_general.ML
--- a/src/Pure/proof_general.ML	Tue Sep 20 16:19:51 2005 +0200
+++ b/src/Pure/proof_general.ML	Tue Sep 20 17:01:43 2005 +0200
@@ -565,9 +565,6 @@
      ("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))]),