aboutsummaryrefslogtreecommitdiffstats
path: root/src/euf/Euf.v
diff options
context:
space:
mode:
authorChantal Keller <Chantal.Keller@inria.fr>2015-02-10 18:41:46 +0100
committerChantal Keller <Chantal.Keller@inria.fr>2015-02-10 18:41:46 +0100
commitff9b5494cb1943339543eeac41683a8ec2dda437 (patch)
tree21af4c0fff64fbd03c6c2006da1e305e849ebbff /src/euf/Euf.v
parent5311b1fa064949089b8d17e34eb31a62426f71fd (diff)
downloadsmtcoq-ff9b5494cb1943339543eeac41683a8ec2dda437.tar.gz
smtcoq-ff9b5494cb1943339543eeac41683a8ec2dda437.zip
More on the support for standard Coq (not working yet)
Diffstat (limited to 'src/euf/Euf.v')
-rw-r--r--src/euf/Euf.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/src/euf/Euf.v b/src/euf/Euf.v
index 9b86bf3..e3d73f6 100644
--- a/src/euf/Euf.v
+++ b/src/euf/Euf.v
@@ -36,7 +36,7 @@ Section certif.
end
| _ => C._true
end.
- Register get_eq as PrimInline.
+ (* Register get_eq as PrimInline. *)
Fixpoint check_trans_aux (t1 t2:int)
(eqs:list _lit) (res:_lit) (clause:C.t) : C.t :=