From db601b06b0880f573b6d1fa83de471679ce87ee7 Mon Sep 17 00:00:00 2001 From: Pierre Letouzey Date: Wed, 14 Jun 2017 18:18:37 +0200 Subject: plugins/ltac : avoid spurious .cmxs files In the previous setting, all plugins/ltac/*.cmxs except ltac_plugin.cmxs (for instance coretactics.cmxs, g_auto.cmxs, ...) were utterly bogus : - wrong -for-pack used for their inner .cmx - dependency over modules not provided (for instance Tacenv, that ends up being a submodule of the pack ltac_plugin). But we were lucky, those files were actually never loaded, thanks to the several DECLARE PLUGIN inside coretactics and co, that end up in ltac_plugin, and hence tell Coq that these modules are already known, preventing any attempt to load them. Anyway, this commit cleans up this mess (thanks PMP for the help) --- theories/Init/Notations.v | 6 ------ theories/Init/Tauto.v | 2 +- 2 files changed, 1 insertion(+), 7 deletions(-) (limited to 'theories') 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 -- cgit v1.2.3