aboutsummaryrefslogtreecommitdiff
path: root/theories/micromega
diff options
context:
space:
mode:
authorJasper Hugunin2020-08-26 07:38:53 -0700
committerJasper Hugunin2020-08-26 07:38:53 -0700
commit179a23ad345c6d0753bbb1771fc01f402dc1cb33 (patch)
tree8dcb1469b398c7c92d6c4ab2b78947c69b5b82e5 /theories/micromega
parent4e6b029805a74ea16166da2c5f59f9669fd34eb8 (diff)
Modify lia to work with -mangle-names
We used to be refreshing the names for intros but not using the refreshed names. The same pattern of `intro_using` (which is what `intros ?name` effectively is) messing things up as in coq/coq#12881.
Diffstat (limited to 'theories/micromega')
-rw-r--r--theories/micromega/Lia.v5
1 files changed, 4 insertions, 1 deletions
diff --git a/theories/micromega/Lia.v b/theories/micromega/Lia.v
index b2c5884ed7..ef2f139133 100644
--- a/theories/micromega/Lia.v
+++ b/theories/micromega/Lia.v
@@ -20,7 +20,10 @@ Require Coq.micromega.Tauto.
Declare ML Module "micromega_plugin".
Ltac zchecker :=
- intros ?__wit ?__varmap ?__ff ;
+ let __wit := fresh "__wit" in
+ let __varmap := fresh "__varmap" in
+ let __ff := fresh "__ff" in
+ intros __wit __varmap __ff ;
exact (ZTautoChecker_sound __ff __wit
(@eq_refl bool true <: @eq bool (ZTautoChecker __ff __wit) true)
(@find Z Z0 __varmap)).