aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/setoid_ring/Field_tac.v
diff options
context:
space:
mode:
authorGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-04-16 17:27:00 +0000
committerGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-04-16 17:27:00 +0000
commit665761c4e82504a579d335b529b2e61f0414665c (patch)
treef24a021023e53a0b092a42e89c4cc65cefaf800f /plugins/setoid_ring/Field_tac.v
parentb596e8303c0d22c5df1aed3c7a56b6af863a1b9e (diff)
nouvelle version de la tactique groebner proposee par Loic:
- algo de Janet (finalement pas utilise) - le hash-cons des certificats de Benjamin et Laurent pas encore integre - traitement des puissances jusqu'a 6 (methode totalement naive) git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12088 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'plugins/setoid_ring/Field_tac.v')
-rw-r--r--plugins/setoid_ring/Field_tac.v4
1 files changed, 4 insertions, 0 deletions
diff --git a/plugins/setoid_ring/Field_tac.v b/plugins/setoid_ring/Field_tac.v
index b31ebda55..0082eb9af 100644
--- a/plugins/setoid_ring/Field_tac.v
+++ b/plugins/setoid_ring/Field_tac.v
@@ -488,6 +488,10 @@ Ltac reduce_field_expr ope kont FLD fv expr :=
(* Hack to let a Ltac return a term in the context of a primitive tactic *)
Ltac return_term x := generalize (refl_equal x).
+Ltac get_term :=
+ match goal with
+ | |- ?x = _ -> _ => x
+ end.
(* Turn an operation on field expressions (FExpr) into a reduction
on terms (in the field carrier). Because of field_lookup,