aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics
diff options
context:
space:
mode:
authorGravatar Théo Zimmermann <theo.zimmermann@univ-paris-diderot.fr>2016-10-19 18:30:44 +0200
committerGravatar Théo Zimmermann <theo.zimmermann@univ-paris-diderot.fr>2016-10-25 16:06:13 +0200
commitd2e713c3913c995ba3796863f778556e00cc5051 (patch)
tree110d408563b1b65438599f33ba1926e53bf88053 /tactics
parent67b49d4d5afdd67bb0a81e3fdf6876387d28a36e (diff)
Remove warning now that info_auto is fixed.
Removes a warning dating from 8.5 signaling that info_auto and info_trivial are broken and advising to use Info 1 auto instead. Now, these tactics are fixed and thus they can be used again. They do not do exactly the same thing as Info 1 auto and may be more useful for the learner.
Diffstat (limited to 'tactics')
-rw-r--r--tactics/tacinterp.ml13
1 files changed, 1 insertions, 12 deletions
diff --git a/tactics/tacinterp.ml b/tactics/tacinterp.ml
index c3f7fa143..23d188aa7 100644
--- a/tactics/tacinterp.ml
+++ b/tactics/tacinterp.ml
@@ -2023,12 +2023,6 @@ and interp_atomic ist tac : unit Proofview.tactic =
(* Automation tactics *)
| TacTrivial (debug,lems,l) ->
- begin if debug == Tacexpr.Info then
- msg_warning
- (strbrk"The \"info_trivial\" tactic" ++ spc ()
- ++strbrk"does not print traces anymore." ++ spc()
- ++strbrk"Use \"Info 1 trivial\", instead.")
- end;
Proofview.Goal.enter begin fun gl ->
let env = Proofview.Goal.env gl in
let sigma = Proofview.Goal.sigma gl in
@@ -2039,13 +2033,8 @@ and interp_atomic ist tac : unit Proofview.tactic =
lems
(Option.map (List.map (interp_hint_base ist)) l))
end
+
| TacAuto (debug,n,lems,l) ->
- begin if debug == Tacexpr.Info then
- msg_warning
- (strbrk"The \"info_auto\" tactic" ++ spc ()
- ++strbrk"does not print traces anymore." ++ spc()
- ++strbrk"Use \"Info 1 auto\", instead.")
- end;
Proofview.Goal.enter begin fun gl ->
let env = Proofview.Goal.env gl in
let sigma = Proofview.Goal.sigma gl in