aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init/Prelude.v
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-02-21 17:13:26 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-02-22 22:28:17 +0100
commit33fe6e61ff2f1f8184373ed8fccc403591c4605a (patch)
tree4c1e0602138994d92be25ba71d80da4e6f0dece0 /theories/Init/Prelude.v
parentf358d7b4c962f5288ad9ce2dc35802666c882422 (diff)
Moving the Tauto tactic to proper Ltac.
This gets rid of brittle code written in ML files through Ltac quotations, and reduces the dependance of Coq to such a feature. This also fixes the particular instance of bug #2800, although the underlying issue is still there.
Diffstat (limited to 'theories/Init/Prelude.v')
-rw-r--r--theories/Init/Prelude.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/theories/Init/Prelude.v b/theories/Init/Prelude.v
index 04a263ad9..03f2328de 100644
--- a/theories/Init/Prelude.v
+++ b/theories/Init/Prelude.v
@@ -15,6 +15,7 @@ Require Coq.Init.Nat.
Require Export Peano.
Require Export Coq.Init.Wf.
Require Export Coq.Init.Tactics.
+Require Export Coq.Init.Tauto.
(* Initially available plugins
(+ nat_syntax_plugin loaded in Datatypes) *)
Declare ML Module "extraction_plugin".