aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/Abstr.v
diff options
context:
space:
mode:
authorYann Herklotz <git@yannherklotz.com>2021-11-14 15:58:08 +0000
committerYann Herklotz <git@yannherklotz.com>2021-11-14 15:58:08 +0000
commit9afc00b337eb4eb704bf95d642073135f3345dca (patch)
treec71b2a0a4522db14be9f8375ec192468227d7ca1 /src/hls/Abstr.v
parentdc9ad1382ee548019e6ff546a24954057cdd8ff0 (diff)
downloadvericert-9afc00b337eb4eb704bf95d642073135f3345dca.tar.gz
vericert-9afc00b337eb4eb704bf95d642073135f3345dca.zip
Add the tseytin transformation instead
Diffstat (limited to 'src/hls/Abstr.v')
-rw-r--r--src/hls/Abstr.v9
1 files changed, 0 insertions, 9 deletions
diff --git a/src/hls/Abstr.v b/src/hls/Abstr.v
index abc4181..2ab79cf 100644
--- a/src/hls/Abstr.v
+++ b/src/hls/Abstr.v
@@ -630,15 +630,6 @@ Definition encode_expression max pe h :=
(Pand (Por (Pnot p) (Pvar p')) p'', h'')
end.*)
-Fixpoint max_predicate (p: pred_op) : positive :=
- match p with
- | Plit (b, p) => p
- | Ptrue => 1
- | Pfalse => 1
- | Pand a b => Pos.max (max_predicate a) (max_predicate b)
- | Por a b => Pos.max (max_predicate a) (max_predicate b)
- end.
-
Fixpoint max_pred_expr (pe: pred_expr) : positive :=
match pe with
| NE.singleton (p, e) => max_predicate p