aboutsummaryrefslogtreecommitdiffstats
path: root/src/SMT_terms.v
diff options
context:
space:
mode:
authorChantal Keller <Chantal.Keller@lri.fr>2016-04-26 23:07:38 +0200
committerChantal Keller <Chantal.Keller@lri.fr>2016-04-26 23:07:38 +0200
commita5bd782f300c3767936fc3f45df6a09cda185370 (patch)
treebb3c0753a54e035fec56f78edbae84485a50b878 /src/SMT_terms.v
parent048f0170612ee39f6bc736246fca82d960e79a18 (diff)
downloadsmtcoq-a5bd782f300c3767936fc3f45df6a09cda185370.tar.gz
smtcoq-a5bd782f300c3767936fc3f45df6a09cda185370.zip
Both native-coq and Coq 8.5 are fully supported
Diffstat (limited to 'src/SMT_terms.v')
-rw-r--r--src/SMT_terms.v16
1 files changed, 16 insertions, 0 deletions
diff --git a/src/SMT_terms.v b/src/SMT_terms.v
index 2d16d3e..6c5ba27 100644
--- a/src/SMT_terms.v
+++ b/src/SMT_terms.v
@@ -234,6 +234,22 @@ Record typ_eqb : Type := Typ_eqb {
te_reflect : forall x y, reflect (x = y) (te_eqb x y)
}.
+Section Typ_eqb_param.
+
+ Variable A : Type.
+
+ Record typ_eqb_param : Type := Typ_eqb_param {
+ te_eqb_param : A -> A -> bool;
+ te_reflect_param : forall x y, reflect (x = y) (te_eqb_param x y)
+ }.
+
+ Variable r : typ_eqb_param.
+
+ Definition typ_eqb_of_typ_eqb_param :=
+ Typ_eqb A (te_eqb_param r) (te_reflect_param r).
+
+End Typ_eqb_param.
+
(* Common used types into which we interpret *)
(* Unit *)