aboutsummaryrefslogtreecommitdiffstats
path: root/src/hls/Predicate.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/hls/Predicate.v')
-rw-r--r--src/hls/Predicate.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/src/hls/Predicate.v b/src/hls/Predicate.v
index c6fe853..087b119 100644
--- a/src/hls/Predicate.v
+++ b/src/hls/Predicate.v
@@ -566,8 +566,8 @@ Defined.
#[local] Open Scope positive.
-Compute tseytin_simple (Por (negate (Pand (Por (Plit (true, 1)) (Plit (true, 2))) (Plit (true, 3)))) (Plit (false, 4))).
-Compute sat_pred_simple (Por Pfalse (Pand (Plit (true, 1)) (Plit (false, 1)))).
+(* Compute tseytin_simple (Por (negate (Pand (Por (Plit (true, 1)) (Plit (true, 2))) (Plit (true, 3)))) (Plit (false, 4))). *)
+(* Compute sat_pred_simple (Por Pfalse (Pand (Plit (true, 1)) (Plit (false, 1)))). *)
Lemma sat_dec a: {sat a} + {unsat a}.
Proof.
@@ -584,7 +584,7 @@ Definition equiv_check p1 p2 :=
| _ => false
end.
-Compute equiv_check Pfalse (Pand (Plit (true, 1%positive)) (Plit (false, 1%positive))).
+(* Compute equiv_check Pfalse (Pand (Plit (true, 1%positive)) (Plit (false, 1%positive))). *)
Lemma equiv_check_correct :
forall p1 p2, equiv_check p1 p2 = true -> p1 == p2.