aboutsummaryrefslogtreecommitdiff
path: root/coq/coq-showdiff.el
diff options
context:
space:
mode:
authorErik Martin-Dorel2020-05-15 15:50:48 +0200
committerAnaclet2020-05-29 11:05:58 +0200
commitaba3f2bfe2bffde6d2df21b098740100459a84be (patch)
treebe6f6bef28652affcfed4425f8aacc9baf1ecd79 /coq/coq-showdiff.el
parentecb47478c9f9959ea25ce509076f6e3959d2c620 (diff)
Fix name clash & rephrase some strings
Diffstat (limited to 'coq/coq-showdiff.el')
-rw-r--r--coq/coq-showdiff.el4
1 files changed, 2 insertions, 2 deletions
diff --git a/coq/coq-showdiff.el b/coq/coq-showdiff.el
index f42431af..0daf98f8 100644
--- a/coq/coq-showdiff.el
+++ b/coq/coq-showdiff.el
@@ -2,11 +2,11 @@
(defun coq-show-proof-fun ()
(interactive)
;; TODO: Check if we are in a proof
- (when coq-show-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.")))
- ) \ No newline at end of file
+ )