diff options
| author | Jason Gross | 2020-04-19 16:18:22 -0400 |
|---|---|---|
| committer | Jason Gross | 2020-04-24 17:28:54 -0400 |
| commit | 087804f288e82a5e4538b7b2387bdc324bebe7b6 (patch) | |
| tree | e6dcf4b05879f92528b5dc65193699ccb5fb4fe3 /theories/nsatz | |
| parent | 1b258168882c17f2afed9e25d51732013bafa184 (diff) | |
Make the nsatz test-suite pass
Diffstat (limited to 'theories/nsatz')
| -rw-r--r-- | theories/nsatz/Nsatz.v | 2 | ||||
| -rw-r--r-- | theories/nsatz/NsatzTactic.v | 8 |
2 files changed, 8 insertions, 2 deletions
diff --git a/theories/nsatz/Nsatz.v b/theories/nsatz/Nsatz.v index aa0ac144c5..70180f47c7 100644 --- a/theories/nsatz/Nsatz.v +++ b/theories/nsatz/Nsatz.v @@ -34,6 +34,8 @@ Require Import ZArith. Require Import Lia. Require Export NsatzTactic. +(** Make use of [discrR] in [nsatz] *) +Ltac nsatz_internal_discrR ::= discrR. (* Real numbers *) Require Import Reals. diff --git a/theories/nsatz/NsatzTactic.v b/theories/nsatz/NsatzTactic.v index 79253009f4..db7dab2c46 100644 --- a/theories/nsatz/NsatzTactic.v +++ b/theories/nsatz/NsatzTactic.v @@ -29,7 +29,6 @@ Require Export Ncring. Require Export Ncring_initial. Require Export Ncring_tac. Require Export Integral_domain. -Require Import DiscrR. Require Import ZArith. Require Import Lia. @@ -347,6 +346,11 @@ Ltac get_lpol g := let l := get_lpol g in constr:(p::l) end. +(** We only make use of [discrR] if [nsatz] support for reals is + loaded. To do this, we redefine this tactic in Nsatz.v to make + use of real discrimination. *) +Ltac nsatz_internal_discrR := idtac. + Ltac nsatz_generic radicalmax info lparam lvar := let nparam := eval compute in (Z.of_nat (List.length lparam)) in match goal with @@ -414,7 +418,7 @@ Ltac nsatz_generic radicalmax info lparam lvar := try exact integral_domain_minus_one_zero || (solve [simpl; unfold R2, equality, eq_notation, addition, add_notation, one, one_notation, multiplication, mul_notation, zero, zero_notation; - discrR || lia ]) + nsatz_internal_discrR || lia ]) || ((*simpl*) idtac) || idtac "could not prove discrimination result" ] ] |
