aboutsummaryrefslogtreecommitdiff
path: root/coq/coq-showdiff.el
blob: 0daf98f8d705c1ec212b67b09ccea798f5e7587e (plain)
1
2
3
4
5
6
7
8
9
10
11
12
;; Temporary file, just for test
(defun coq-show-proof-fun ()
  (interactive)
  ;; TODO: Check if we are in a proof
  (when coq-show-proof-stepwise
    (when (eq coq-diffs 'off)
      (proof-shell-invisible-command "Show Proof." ))
    (when (eq coq-diffs 'on)
      (proof-shell-invisible-command "Show Proof Diffs."))
    (when (eq coq-diffs 'removed)
      (proof-shell-invisible-command "Show Proof Diffs removed.")))
 )