aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories
diff options
context:
space:
mode:
authorGravatar Maxime Dénès <mail@maximedenes.fr>2017-06-23 17:10:41 +0200
committerGravatar Maxime Dénès <mail@maximedenes.fr>2017-06-23 17:10:41 +0200
commit42dc32440b4b30d05e3f83d24031bc7b207149d6 (patch)
tree15871fee3601513f84e4d3849bcccce7f6f64af1 /theories
parentf5a746eca3866b4652ead49548d08b2fe460960c (diff)
parentdb601b06b0880f573b6d1fa83de471679ce87ee7 (diff)
Merge PR#794: Cleanup of ltac cmxs
Diffstat (limited to 'theories')
-rw-r--r--theories/Init/Notations.v6
-rw-r--r--theories/Init/Tauto.v2
2 files changed, 1 insertions, 7 deletions
diff --git a/theories/Init/Notations.v b/theories/Init/Notations.v
index edcd53005..2b0fe1362 100644
--- a/theories/Init/Notations.v
+++ b/theories/Init/Notations.v
@@ -89,11 +89,5 @@ Open Scope type_scope.
(** ML Tactic Notations *)
Declare ML Module "ltac_plugin".
-Declare ML Module "coretactics".
-Declare ML Module "extratactics".
-Declare ML Module "g_auto".
-Declare ML Module "g_class".
-Declare ML Module "g_eqdecide".
-Declare ML Module "g_rewrite".
Global Set Default Proof Mode "Classic".
diff --git a/theories/Init/Tauto.v b/theories/Init/Tauto.v
index 1e409607a..886533586 100644
--- a/theories/Init/Tauto.v
+++ b/theories/Init/Tauto.v
@@ -2,7 +2,7 @@ Require Import Notations.
Require Import Datatypes.
Require Import Logic.
-Local Declare ML Module "tauto".
+Declare ML Module "tauto_plugin".
Local Ltac not_dep_intros :=
repeat match goal with