merge
authorblanchet
Tue, 03 Jun 2014 16:27:31 +0200
changeset 57171 3fc8bbf089a2
parent 57170 3afada8f820d (diff)
parent 57166 5cfcc616d485 (current diff)
child 57172 bcc6dc6c1d1c
merge
--- a/Admin/components/components.sha1	Tue Jun 03 16:22:01 2014 +0200
+++ b/Admin/components/components.sha1	Tue Jun 03 16:27:31 2014 +0200
@@ -95,3 +95,4 @@
 d94a716502c8503d63952bcb4d4176fac8b28704  z3-4.0.tar.gz
 86e721296c400ada440e4a9ce11b9e845eec9e25  z3-4.3.0.tar.gz
 06b30757ff23aefbc30479785c212685ffd39f4d  z3-4.3.2pre.tar.gz
+a8917c31b31c182edeec0aaa48870844960c8a61  z3-4.3.2pre-1.tar.gz
--- a/Admin/components/main	Tue Jun 03 16:22:01 2014 +0200
+++ b/Admin/components/main	Tue Jun 03 16:27:31 2014 +0200
@@ -12,6 +12,6 @@
 scala-2.11.1
 spass-3.8ds
 z3-3.2-1
-z3-4.3.2pre
+z3-4.3.2pre-1
 xz-java-1.2-1
 ProofGeneral-4.2-1
--- a/src/HOL/SMT2.thy	Tue Jun 03 16:22:01 2014 +0200
+++ b/src/HOL/SMT2.thy	Tue Jun 03 16:27:31 2014 +0200
@@ -298,20 +298,20 @@
   if_True if_False not_not
 
 lemma [z3_new_rule]:
-  "(P \<and> Q) = (\<not>(\<not>P \<or> \<not>Q))"
-  "(P \<and> Q) = (\<not>(\<not>Q \<or> \<not>P))"
-  "(\<not>P \<and> Q) = (\<not>(P \<or> \<not>Q))"
-  "(\<not>P \<and> Q) = (\<not>(\<not>Q \<or> P))"
-  "(P \<and> \<not>Q) = (\<not>(\<not>P \<or> Q))"
-  "(P \<and> \<not>Q) = (\<not>(Q \<or> \<not>P))"
-  "(\<not>P \<and> \<not>Q) = (\<not>(P \<or> Q))"
-  "(\<not>P \<and> \<not>Q) = (\<not>(Q \<or> P))"
+  "(P \<and> Q) = (\<not> (\<not> P \<or> \<not> Q))"
+  "(P \<and> Q) = (\<not> (\<not> Q \<or> \<not> P))"
+  "(\<not> P \<and> Q) = (\<not> (P \<or> \<not> Q))"
+  "(\<not> P \<and> Q) = (\<not> (\<not> Q \<or> P))"
+  "(P \<and> \<not> Q) = (\<not> (\<not> P \<or> Q))"
+  "(P \<and> \<not> Q) = (\<not> (Q \<or> \<not> P))"
+  "(\<not> P \<and> \<not> Q) = (\<not> (P \<or> Q))"
+  "(\<not> P \<and> \<not> Q) = (\<not> (Q \<or> P))"
   by auto
 
 lemma [z3_new_rule]:
-  "(P \<longrightarrow> Q) = (Q \<or> \<not>P)"
-  "(\<not>P \<longrightarrow> Q) = (P \<or> Q)"
-  "(\<not>P \<longrightarrow> Q) = (Q \<or> P)"
+  "(P \<longrightarrow> Q) = (Q \<or> \<not> P)"
+  "(\<not> P \<longrightarrow> Q) = (P \<or> Q)"
+  "(\<not> P \<longrightarrow> Q) = (Q \<or> P)"
   "(True \<longrightarrow> P) = P"
   "(P \<longrightarrow> True) = True"
   "(False \<longrightarrow> P) = True"
@@ -319,41 +319,41 @@
   by auto
 
 lemma [z3_new_rule]:
-  "((P = Q) \<longrightarrow> R) = (R | (Q = (\<not>P)))"
+  "((P = Q) \<longrightarrow> R) = (R | (Q = (\<not> P)))"
   by auto
 
 lemma [z3_new_rule]:
-  "(\<not>True) = False"
-  "(\<not>False) = True"
+  "(\<not> True) = False"
+  "(\<not> False) = True"
   "(x = x) = True"
   "(P = True) = P"
   "(True = P) = P"
-  "(P = False) = (\<not>P)"
-  "(False = P) = (\<not>P)"
-  "((\<not>P) = P) = False"
-  "(P = (\<not>P)) = False"
-  "((\<not>P) = (\<not>Q)) = (P = Q)"
-  "\<not>(P = (\<not>Q)) = (P = Q)"
-  "\<not>((\<not>P) = Q) = (P = Q)"
-  "(P \<noteq> Q) = (Q = (\<not>P))"
-  "(P = Q) = ((\<not>P \<or> Q) \<and> (P \<or> \<not>Q))"
-  "(P \<noteq> Q) = ((\<not>P \<or> \<not>Q) \<and> (P \<or> Q))"
+  "(P = False) = (\<not> P)"
+  "(False = P) = (\<not> P)"
+  "((\<not> P) = P) = False"
+  "(P = (\<not> P)) = False"
+  "((\<not> P) = (\<not> Q)) = (P = Q)"
+  "\<not> (P = (\<not> Q)) = (P = Q)"
+  "\<not> ((\<not> P) = Q) = (P = Q)"
+  "(P \<noteq> Q) = (Q = (\<not> P))"
+  "(P = Q) = ((\<not> P \<or> Q) \<and> (P \<or> \<not> Q))"
+  "(P \<noteq> Q) = ((\<not> P \<or> \<not> Q) \<and> (P \<or> Q))"
   by auto
 
 lemma [z3_new_rule]:
-  "(if P then P else \<not>P) = True"
-  "(if \<not>P then \<not>P else P) = True"
+  "(if P then P else \<not> P) = True"
+  "(if \<not> P then \<not> P else P) = True"
   "(if P then True else False) = P"
-  "(if P then False else True) = (\<not>P)"
-  "(if P then Q else True) = ((\<not>P) \<or> Q)"
-  "(if P then Q else True) = (Q \<or> (\<not>P))"
-  "(if P then Q else \<not>Q) = (P = Q)"
-  "(if P then Q else \<not>Q) = (Q = P)"
-  "(if P then \<not>Q else Q) = (P = (\<not>Q))"
-  "(if P then \<not>Q else Q) = ((\<not>Q) = P)"
-  "(if \<not>P then x else y) = (if P then y else x)"
-  "(if P then (if Q then x else y) else x) = (if P \<and> (\<not>Q) then y else x)"
-  "(if P then (if Q then x else y) else x) = (if (\<not>Q) \<and> P then y else x)"
+  "(if P then False else True) = (\<not> P)"
+  "(if P then Q else True) = ((\<not> P) \<or> Q)"
+  "(if P then Q else True) = (Q \<or> (\<not> P))"
+  "(if P then Q else \<not> Q) = (P = Q)"
+  "(if P then Q else \<not> Q) = (Q = P)"
+  "(if P then \<not> Q else Q) = (P = (\<not> Q))"
+  "(if P then \<not> Q else Q) = ((\<not> Q) = P)"
+  "(if \<not> P then x else y) = (if P then y else x)"
+  "(if P then (if Q then x else y) else x) = (if P \<and> (\<not> Q) then y else x)"
+  "(if P then (if Q then x else y) else x) = (if (\<not> Q) \<and> P then y else x)"
   "(if P then (if Q then x else y) else y) = (if P \<and> Q then x else y)"
   "(if P then (if Q then x else y) else y) = (if Q \<and> P then x else y)"
   "(if P then x else if P then y else z) = (if P then x else z)"
@@ -375,31 +375,31 @@
 
 lemma [z3_new_rule]:  (* for def-axiom *)
   "P = Q \<or> P \<or> Q"
-  "P = Q \<or> \<not>P \<or> \<not>Q"
-  "(\<not>P) = Q \<or> \<not>P \<or> Q"
-  "(\<not>P) = Q \<or> P \<or> \<not>Q"
-  "P = (\<not>Q) \<or> \<not>P \<or> Q"
-  "P = (\<not>Q) \<or> P \<or> \<not>Q"
-  "P \<noteq> Q \<or> P \<or> \<not>Q"
-  "P \<noteq> Q \<or> \<not>P \<or> Q"
-  "P \<noteq> (\<not>Q) \<or> P \<or> Q"
-  "(\<not>P) \<noteq> Q \<or> P \<or> Q"
-  "P \<or> Q \<or> P \<noteq> (\<not>Q)"
-  "P \<or> Q \<or> (\<not>P) \<noteq> Q"
-  "P \<or> \<not>Q \<or> P \<noteq> Q"
-  "\<not>P \<or> Q \<or> P \<noteq> Q"
+  "P = Q \<or> \<not> P \<or> \<not> Q"
+  "(\<not> P) = Q \<or> \<not> P \<or> Q"
+  "(\<not> P) = Q \<or> P \<or> \<not> Q"
+  "P = (\<not> Q) \<or> \<not> P \<or> Q"
+  "P = (\<not> Q) \<or> P \<or> \<not> Q"
+  "P \<noteq> Q \<or> P \<or> \<not> Q"
+  "P \<noteq> Q \<or> \<not> P \<or> Q"
+  "P \<noteq> (\<not> Q) \<or> P \<or> Q"
+  "(\<not> P) \<noteq> Q \<or> P \<or> Q"
+  "P \<or> Q \<or> P \<noteq> (\<not> Q)"
+  "P \<or> Q \<or> (\<not> P) \<noteq> Q"
+  "P \<or> \<not> Q \<or> P \<noteq> Q"
+  "\<not> P \<or> Q \<or> P \<noteq> Q"
   "P \<or> y = (if P then x else y)"
   "P \<or> (if P then x else y) = y"
-  "\<not>P \<or> x = (if P then x else y)"
-  "\<not>P \<or> (if P then x else y) = x"
-  "P \<or> R \<or> \<not>(if P then Q else R)"
-  "\<not>P \<or> Q \<or> \<not>(if P then Q else R)"
-  "\<not>(if P then Q else R) \<or> \<not>P \<or> Q"
-  "\<not>(if P then Q else R) \<or> P \<or> R"
-  "(if P then Q else R) \<or> \<not>P \<or> \<not>Q"
-  "(if P then Q else R) \<or> P \<or> \<not>R"
-  "(if P then \<not>Q else R) \<or> \<not>P \<or> Q"
-  "(if P then Q else \<not>R) \<or> P \<or> R"
+  "\<not> P \<or> x = (if P then x else y)"
+  "\<not> P \<or> (if P then x else y) = x"
+  "P \<or> R \<or> \<not> (if P then Q else R)"
+  "\<not> P \<or> Q \<or> \<not> (if P then Q else R)"
+  "\<not> (if P then Q else R) \<or> \<not> P \<or> Q"
+  "\<not> (if P then Q else R) \<or> P \<or> R"
+  "(if P then Q else R) \<or> \<not> P \<or> \<not> Q"
+  "(if P then Q else R) \<or> P \<or> \<not> R"
+  "(if P then \<not> Q else R) \<or> \<not> P \<or> Q"
+  "(if P then Q else \<not> R) \<or> P \<or> R"
   by auto
 
 hide_type (open) pattern
--- a/src/HOL/SMT_Examples/Boogie_Dijkstra.certs2	Tue Jun 03 16:22:01 2014 +0200
+++ b/src/HOL/SMT_Examples/Boogie_Dijkstra.certs2	Tue Jun 03 16:27:31 2014 +0200
@@ -1,3139 +1,3045 @@
-4130cc2c7db4aedd246ade86526a1512dc2d3ec1 3138 0
-unsat
-((set-logic AUFLIA)
-(declare-fun ?v0!19 () B_Vertex$)
-(declare-fun ?v1!18 () B_Vertex$)
-(declare-fun ?v0!20 () B_Vertex$)
-(declare-fun ?v0!17 () B_Vertex$)
-(declare-fun ?v1!16 () B_Vertex$)
-(declare-fun ?v0!15 () B_Vertex$)
-(declare-fun ?v0!14 () B_Vertex$)
-(declare-fun ?v0!13 () B_Vertex$)
-(declare-fun ?v0!12 () B_Vertex$)
-(declare-fun ?v0!11 () B_Vertex$)
-(declare-fun ?v1!10 () B_Vertex$)
-(declare-fun ?v1!9 (B_Vertex$) B_Vertex$)
-(declare-fun ?v0!8 () B_Vertex$)
-(declare-fun ?v1!7 (B_Vertex$) B_Vertex$)
-(declare-fun ?v1!6 (B_Vertex$) B_Vertex$)
-(declare-fun ?v0!5 () B_Vertex$)
-(declare-fun ?v0!4 () B_Vertex$)
-(declare-fun ?v1!3 () B_Vertex$)
-(declare-fun ?v0!2 () B_Vertex$)
-(declare-fun ?v1!1 () B_Vertex$)
-(declare-fun ?v0!0 () B_Vertex$)
-(proof
-(let ((?x2200 (* (- 1) (v_b_SP_G_2$ ?v0!19))))
-(let ((?x2198 (v_b_SP_G_2$ ?v1!18)))
-(let ((?x2191 (b_G$ (pair$ ?v1!18 ?v0!19))))
-(let (($x2202 (>= (+ ?x2191 ?x2198 ?x2200) 0)))
-(let (($x2194 (<= (+ b_Infinity$ (* (- 1) ?x2191)) 0)))
-(let (($x2189 (fun_app$ v_b_Visited_G_2$ ?v1!18)))
-(let (($x3065 (not $x2189)))
-(let (($x3080 (or $x3065 $x2194 $x2202)))
-(let (($x3085 (not $x3080)))
-(let (($x3977 (forall ((?v1 B_Vertex$) )(!(let ((?x2217 (v_b_SP_G_2$ ?v0!20)))
-(let ((?x2218 (* (- 1) ?x2217)))
-(let ((?x220 (v_b_SP_G_2$ ?v1)))
-(let (($x2528 (= (+ ?x220 ?x2218 (b_G$ (pair$ ?v1 ?v0!20))) 0)))
-(let (($x238 (fun_app$ v_b_Visited_G_2$ ?v1)))
-(let (($x247 (not $x238)))
-(or (>= (+ ?x220 ?x2218) 0) $x247 (not $x2528)))))))) :pattern ( (v_b_SP_G_2$ ?v1) ) :pattern ( (fun_app$ v_b_Visited_G_2$ ?v1) ) :pattern ( (pair$ ?v1 ?v0!20) )))
-))
-(let (($x3982 (not $x3977)))
-(let (($x2220 (<= (+ b_Infinity$ (* (- 1) (v_b_SP_G_2$ ?v0!20))) 0)))
-(let (($x2215 (= ?v0!20 b_Source$)))
-(let (($x3968 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(!(let ((?x220 (v_b_SP_G_2$ ?v1)))
-(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let (($x1621 (>= (+ ?x102 ?x220 (* (- 1) (v_b_SP_G_2$ ?v0))) 0)))
-(let (($x1303 (<= (+ b_Infinity$ (* (- 1) ?x102)) 0)))
-(let (($x238 (fun_app$ v_b_Visited_G_2$ ?v1)))
-(let (($x247 (not $x238)))
-(or $x247 $x1303 $x1621))))))) :pattern ( (pair$ ?v1 ?v0) )))
-))
-(let (($x3973 (not $x3968)))
-(let (($x3985 (or $x3973 $x2215 $x2220 $x3982)))
-(let (($x3988 (not $x3985)))
-(let (($x3991 (or $x3085 $x3988)))
-(let (($x3994 (not $x3991)))
-(let (($x3960 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(!(let (($x1601 (>= (+ (v_b_SP_G_2$ ?v1) (* (- 1) (v_b_SP_G_2$ ?v0))) 0)))
-(let (($x238 (fun_app$ v_b_Visited_G_2$ ?v1)))
-(or $x238 (not (fun_app$ v_b_Visited_G_2$ ?v0)) $x1601))) :pattern ( (v_b_SP_G_2$ ?v1) (v_b_SP_G_2$ ?v0) )))
-))
-(let (($x3997 (or (not $x3960) $x3994)))
-(let (($x4000 (not $x3997)))
-(let (($x2175 (>= (+ (v_b_SP_G_2$ ?v1!16) (* (- 1) (v_b_SP_G_2$ ?v0!17))) 0)))
-(let (($x2168 (fun_app$ v_b_Visited_G_2$ ?v0!17)))
-(let (($x3019 (not $x2168)))
-(let (($x2166 (fun_app$ v_b_Visited_G_2$ ?v1!16)))
-(let (($x3034 (or $x2166 $x3019 $x2175)))
-(let (($x3943 (forall ((?v0 B_Vertex$) )(!(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v0)))
-(let ((?x220 (v_b_SP_G_2$ ?v0)))
-(let (($x225 (= ?x220 ?x121)))
-(let (($x238 (fun_app$ v_b_Visited_G_2$ ?v0)))
-(let (($x247 (not $x238)))
-(or $x247 $x225)))))) :pattern ( (fun_app$ v_b_Visited_G_2$ ?v0) ) :pattern ( (v_b_SP_G_2$ ?v0) ) :pattern ( (fun_app$c v_b_SP_G_1$ ?v0) )))
-))
-(let (($x3039 (not $x3034)))
-(let (($x4003 (or $x3039 $x4000)))
-(let (($x4006 (not $x4003)))
-(let (($x3951 (forall ((?v0 B_Vertex$) )(!(let ((?x220 (v_b_SP_G_2$ ?v0)))
-(>= ?x220 0)) :pattern ( (v_b_SP_G_2$ ?v0) )))
-))
-(let (($x4009 (or (not $x3951) $x4006)))
-(let (($x4012 (not $x4009)))
-(let ((?x2152 (v_b_SP_G_2$ ?v0!15)))
-(let (($x2153 (>= ?x2152 0)))
-(let (($x2154 (not $x2153)))
-(let ((?x243 (v_b_SP_G_2$ b_Source$)))
-(let (($x244 (= ?x243 0)))
-(let (($x913 (not $x244)))
-(let (($x4015 (or $x913 $x2154 $x4012)))
-(let (($x4018 (not $x4015)))
-(let (($x3948 (not $x3943)))
-(let (($x4021 (or $x3948 $x4018)))
-(let (($x4024 (not $x4021)))
-(let ((?x2136 (fun_app$c v_b_SP_G_1$ ?v0!14)))
-(let ((?x2135 (v_b_SP_G_2$ ?v0!14)))
-(let (($x2137 (= ?x2135 ?x2136)))
-(let (($x2133 (fun_app$ v_b_Visited_G_2$ ?v0!14)))
-(let (($x2134 (not $x2133)))
-(let (($x2138 (or $x2134 $x2137)))
-(let ((@x8891 (unit-resolution (def-axiom (or $x2138 $x2133)) (hypothesis (not $x2138)) $x2133)))
-(let (($x3646 (not $x2137)))
-(let ((@x8820 (unit-resolution (def-axiom (or $x2138 $x3646)) (hypothesis (not $x2138)) $x3646)))
-(let ((?x212 (fun_app$a (fun_app$b (fun_upd$ v_b_Visited_G_1$) v_b_v_G_1$) true)))
-(let (($x213 (= v_b_Visited_G_2$ ?x212)))
-(let (($x2139 (not $x2138)))
-(let (($x4027 (or $x2139 $x4024)))
-(let (($x4030 (not $x4027)))
-(let (($x3934 (forall ((?v0 B_Vertex$) )(!(>= (+ (fun_app$c v_b_SP_G_1$ ?v0) (* (- 1) (v_b_SP_G_2$ ?v0))) 0) :pattern ( (fun_app$c v_b_SP_G_1$ ?v0) ) :pattern ( (v_b_SP_G_2$ ?v0) )))
-))
-(let (($x3939 (not $x3934)))
-(let (($x4033 (or $x3939 $x4030)))
-(let (($x4036 (not $x4033)))
-(let (($x2121 (>= (+ (fun_app$c v_b_SP_G_1$ ?v0!13) (* (- 1) (v_b_SP_G_2$ ?v0!13))) 0)))
-(let (($x2122 (not $x2121)))
-(let (($x4039 (or $x2122 $x4036)))
-(let (($x4042 (not $x4039)))
-(let (($x3926 (forall ((?v0 B_Vertex$) )(!(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v0)))
-(let ((?x220 (v_b_SP_G_2$ ?v0)))
-(let (($x225 (= ?x220 ?x121)))
-(let ((?x204 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
-(let ((?x1520 (* (- 1) ?x204)))
-(let (($x1547 (<= (+ ?x121 ?x1520 (* (- 1) (b_G$ (pair$ v_b_v_G_1$ ?v0)))) 0)))
-(let (($x1540 (<= (+ b_Infinity$ (* (- 1) (b_G$ (pair$ v_b_v_G_1$ ?v0)))) 0)))
-(let (($x2991 (or $x1540 $x1547)))
-(let (($x2992 (not $x2991)))
-(or $x2992 $x225)))))))))) :pattern ( (pair$ v_b_v_G_1$ ?v0) ) :pattern ( (fun_app$c v_b_SP_G_1$ ?v0) ) :pattern ( (v_b_SP_G_2$ ?v0) )))
-))
-(let (($x3931 (not $x3926)))
-(let (($x3918 (forall ((?v0 B_Vertex$) )(!(let ((?x220 (v_b_SP_G_2$ ?v0)))
-(let ((?x1560 (* (- 1) ?x220)))
-(let ((?x215 (b_G$ (pair$ v_b_v_G_1$ ?v0))))
-(let ((?x204 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
-(let (($x1559 (= (+ ?x204 ?x215 ?x1560) 0)))
-(let (($x1547 (<= (+ (fun_app$c v_b_SP_G_1$ ?v0) (* (- 1) ?x204) (* (- 1) ?x215)) 0)))
-(let (($x1540 (<= (+ b_Infinity$ (* (- 1) ?x215)) 0)))
-(or $x1540 $x1547 $x1559)))))))) :pattern ( (pair$ v_b_v_G_1$ ?v0) ) :pattern ( (fun_app$c v_b_SP_G_1$ ?v0) ) :pattern ( (v_b_SP_G_2$ ?v0) )))
-))
-(let (($x3923 (not $x3918)))
-(let (($x3196 (not $x213)))
-(let (($x3908 (forall ((?v0 B_Vertex$) )(!(let ((?x204 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
-(let ((?x1520 (* (- 1) ?x204)))
-(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v0)))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v0)))
-(or $x125 (>= (+ ?x121 ?x1520) 0)))))) :pattern ( (fun_app$ v_b_Visited_G_1$ ?v0) ) :pattern ( (fun_app$c v_b_SP_G_1$ ?v0) )))
-))
-(let (($x3913 (not $x3908)))
-(let (($x1522 (<= (+ b_Infinity$ (* (- 1) (fun_app$c v_b_SP_G_1$ v_b_v_G_1$))) 0)))
-(let (($x202 (fun_app$ v_b_Visited_G_1$ v_b_v_G_1$)))
-(let (($x2087 (<= (+ b_Infinity$ (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0!12))) 0)))
-(let (($x2082 (fun_app$ v_b_Visited_G_1$ ?v0!12)))
-(let (($x4045 (or $x2082 $x2087 $x202 $x1522 $x3913 $x3196 $x3923 $x3931 $x4042)))
-(let (($x4048 (not $x4045)))
-(let (($x193 (= (fun_app$c v_b_SP_G_3$ b_Source$) 0)))
-(let (($x3870 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(!(let ((?x177 (fun_app$c v_b_SP_G_3$ ?v1)))
-(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let (($x1493 (>= (+ ?x102 ?x177 (* (- 1) (fun_app$c v_b_SP_G_3$ ?v0))) 0)))
-(let (($x1303 (<= (+ b_Infinity$ (* (- 1) ?x102)) 0)))
-(let (($x1448 (<= (+ b_Infinity$ (* (- 1) ?x177)) 0)))
-(or $x1448 $x1303 $x1493)))))) :pattern ( (pair$ ?v1 ?v0) )))
-))
-(let (($x3878 (or (not $x3870) $x193)))
-(let (($x3881 (not $x3878)))
-(let ((?x2036 (b_G$ (pair$ ?v1!10 ?v0!11))))
-(let ((?x2030 (fun_app$c v_b_SP_G_3$ ?v1!10)))
-(let (($x2497 (>= (+ ?x2030 ?x2036 (* (- 1) (fun_app$c v_b_SP_G_3$ ?v0!11))) 0)))
-(let (($x2039 (<= (+ b_Infinity$ (* (- 1) ?x2036)) 0)))
-(let (($x2033 (<= (+ b_Infinity$ (* (- 1) ?x2030)) 0)))
-(let (($x2919 (or $x2033 $x2039 $x2497)))
-(let (($x2924 (not $x2919)))
-(let (($x3884 (or $x2924 $x3881)))
-(let (($x3887 (not $x3884)))
-(let (($x3862 (forall ((?v0 B_Vertex$) )(!(let ((?x177 (fun_app$c v_b_SP_G_3$ ?v0)))
-(let ((?x2479 (+ ?x177 (* (- 1) (fun_app$c v_b_SP_G_3$ (?v1!9 ?v0))) (* (- 1) (b_G$ (pair$ (?v1!9 ?v0) ?v0))))))
-(let (($x2480 (= ?x2479 0)))
-(let (($x2464 (<= (+ ?x177 (* (- 1) (fun_app$c v_b_SP_G_3$ (?v1!9 ?v0)))) 0)))
-(let (($x2891 (not (or $x2464 (not $x2480)))))
-(let (($x1448 (<= (+ b_Infinity$ (* (- 1) ?x177)) 0)))
-(let (($x74 (= ?v0 b_Source$)))
-(or $x74 $x1448 $x2891)))))))) :pattern ( (fun_app$c v_b_SP_G_3$ ?v0) )))
-))
-(let (($x3890 (or (not $x3862) $x3887)))
-(let (($x3893 (not $x3890)))
-(let (($x3848 (forall ((?v1 B_Vertex$) )(!(let ((?x1970 (fun_app$c v_b_SP_G_3$ ?v0!8)))
-(let ((?x1971 (* (- 1) ?x1970)))
-(let ((?x177 (fun_app$c v_b_SP_G_3$ ?v1)))
-(let (($x2436 (= (+ ?x177 ?x1971 (b_G$ (pair$ ?v1 ?v0!8))) 0)))
-(or (>= (+ ?x177 ?x1971) 0) (not $x2436)))))) :pattern ( (fun_app$c v_b_SP_G_3$ ?v1) ) :pattern ( (pair$ ?v1 ?v0!8) )))
-))
-(let (($x3853 (not $x3848)))
-(let (($x1973 (<= (+ b_Infinity$ (* (- 1) (fun_app$c v_b_SP_G_3$ ?v0!8))) 0)))
-(let (($x1968 (= ?v0!8 b_Source$)))
-(let (($x3856 (or $x1968 $x1973 $x3853)))
-(let (($x3859 (not $x3856)))
-(let (($x3896 (or $x3859 $x3893)))
-(let (($x3899 (not $x3896)))
-(let (($x164 (= v_b_SP_G_3$ v_b_SP_G_1$)))
-(let (($x2982 (not $x164)))
-(let (($x3838 (forall ((?v0 B_Vertex$) )(!(let (($x1395 (<= (+ b_Infinity$ (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0))) 0)))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v0)))
-(or $x125 $x1395))) :pattern ( (fun_app$ v_b_Visited_G_1$ ?v0) ) :pattern ( (fun_app$c v_b_SP_G_1$ ?v0) )))
-))
-(let (($x3843 (not $x3838)))
-(let (($x3902 (or $x3843 (not (= v_b_Visited_G_3$ v_b_Visited_G_1$)) (not (= v_b_v_G_2$ v_b_v_G_0$)) $x2982 (not (= v_b_oldSP_G_1$ v_b_oldSP_G_0$)) $x3899)))
-(let (($x5759 (>= (+ ?x2030 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v1!10))) 0)))
-(let ((?x4698 (fun_app$c v_b_SP_G_1$ ?v1!10)))
-(let (($x6220 (= ?x2030 ?x4698)))
-(let (($x3905 (not $x3902)))
-(let ((@x5698 (hypothesis $x3905)))
-(let ((@x5699 (unit-resolution (def-axiom (or $x3902 $x164)) @x5698 $x164)))
-(let ((@x7384 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x6220) $x5759)) (monotonicity @x5699 $x6220) $x5759)))
-(let (($x3668 (not $x2497)))
-(let (($x4677 (>= (+ ?x2036 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0!11)) ?x4698) 0)))
-(let (($x4697 (fun_app$ v_b_Visited_G_1$ ?v1!10)))
-(let (($x4492 (<= (+ b_Infinity$ (* (- 1) ?x4698)) 0)))
-(let (($x5659 (not $x4492)))
-(let (($x2034 (not $x2033)))
-(let ((?x119 (fun_app$c v_b_SP_G_1$ b_Source$)))
-(let (($x120 (= ?x119 0)))
-(let (($x4051 (or $x3905 $x4048)))
-(let (($x4054 (not $x4051)))
-(let (($x3829 (forall ((?v0 B_Vertex$) )(!(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v0)))
-(let ((?x2416 (+ ?x121 (* (- 1) (fun_app$c v_b_SP_G_1$ (?v1!7 ?v0))) (* (- 1) (b_G$ (pair$ (?v1!7 ?v0) ?v0))))))
-(let (($x2417 (= ?x2416 0)))
-(let (($x2401 (<= (+ ?x121 (* (- 1) (fun_app$c v_b_SP_G_1$ (?v1!7 ?v0)))) 0)))
-(let (($x2825 (not (or $x2401 (not (fun_app$ v_b_Visited_G_1$ (?v1!7 ?v0))) (not $x2417)))))
-(let (($x1395 (<= (+ b_Infinity$ (* (- 1) ?x121)) 0)))
-(let (($x74 (= ?v0 b_Source$)))
-(or $x74 $x1395 $x2825)))))))) :pattern ( (fun_app$c v_b_SP_G_1$ ?v0) )))
-))
-(let (($x3834 (not $x3829)))
-(let (($x3821 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(!(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v1)))
-(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let (($x1384 (>= (+ ?x102 ?x121 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0))) 0)))
-(let (($x1303 (<= (+ b_Infinity$ (* (- 1) ?x102)) 0)))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v1)))
-(let (($x126 (not $x125)))
-(or $x126 $x1303 $x1384))))))) :pattern ( (pair$ ?v1 ?v0) )))
-))
-(let (($x3826 (not $x3821)))
-(let (($x3813 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(!(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v1)))
-(let (($x1367 (>= (+ ?x121 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0))) 0)))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v1)))
-(or $x125 (not (fun_app$ v_b_Visited_G_1$ ?v0)) $x1367)))) :pattern ( (fun_app$ v_b_Visited_G_1$ ?v1) (fun_app$ v_b_Visited_G_1$ ?v0) )))
-))
-(let (($x3818 (not $x3813)))
-(let (($x3804 (forall ((?v0 B_Vertex$) )(!(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v0)))
-(>= ?x121 0)) :pattern ( (fun_app$c v_b_SP_G_1$ ?v0) )))
-))
-(let (($x3809 (not $x3804)))
-(let (($x3213 (not $x120)))
-(let (($x3795 (forall ((?v0 B_Vertex$) )(!(let ((?x75 (v_b_SP_G_0$ ?v0)))
-(let ((?x2378 (+ ?x75 (* (- 1) (v_b_SP_G_0$ (?v1!6 ?v0))) (* (- 1) (b_G$ (pair$ (?v1!6 ?v0) ?v0))))))
-(let (($x2379 (= ?x2378 0)))
-(let (($x2363 (<= (+ ?x75 (* (- 1) (v_b_SP_G_0$ (?v1!6 ?v0)))) 0)))
-(let (($x2752 (not (or $x2363 (not (v_b_Visited_G_0$ (?v1!6 ?v0))) (not $x2379)))))
-(let (($x1330 (<= (+ b_Infinity$ (* (- 1) ?x75)) 0)))
-(let (($x74 (= ?v0 b_Source$)))
-(or $x74 $x1330 $x2752)))))))) :pattern ( (v_b_SP_G_0$ ?v0) )))
-))
-(let (($x4057 (or (not $x3795) $x3213 $x3809 $x3818 $x3826 $x3834 $x4054)))
-(let (($x4060 (not $x4057)))
-(let (($x3781 (forall ((?v1 B_Vertex$) )(!(let ((?x1849 (v_b_SP_G_0$ ?v0!5)))
-(let ((?x1850 (* (- 1) ?x1849)))
-(let ((?x75 (v_b_SP_G_0$ ?v1)))
-(let (($x83 (v_b_Visited_G_0$ ?v1)))
-(let (($x84 (not $x83)))
-(or (>= (+ ?x75 ?x1850) 0) $x84 (not (= (+ ?x75 ?x1850 (b_G$ (pair$ ?v1 ?v0!5))) 0)))))))) :pattern ( (v_b_SP_G_0$ ?v1) ) :pattern ( (v_b_Visited_G_0$ ?v1) ) :pattern ( (pair$ ?v1 ?v0!5) )))
-))
-(let (($x1852 (<= (+ b_Infinity$ (* (- 1) (v_b_SP_G_0$ ?v0!5))) 0)))
-(let (($x1847 (= ?v0!5 b_Source$)))
-(let (($x3789 (or $x1847 $x1852 (not $x3781))))
-(let (($x3792 (not $x3789)))
-(let (($x4063 (or $x3792 $x4060)))
-(let (($x4066 (not $x4063)))
-(let (($x3772 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(!(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let ((?x75 (v_b_SP_G_0$ ?v1)))
-(let (($x1316 (>= (+ ?x75 (* (- 1) (v_b_SP_G_0$ ?v0)) ?x102) 0)))
-(let (($x1303 (<= (+ b_Infinity$ (* (- 1) ?x102)) 0)))
-(let (($x83 (v_b_Visited_G_0$ ?v1)))
-(let (($x84 (not $x83)))
-(or $x84 $x1303 $x1316))))))) :pattern ( (pair$ ?v1 ?v0) )))
-))
-(let (($x4069 (or (not $x3772) $x4066)))
-(let (($x4072 (not $x4069)))
-(let ((?x1823 (b_G$ (pair$ ?v1!3 ?v0!4))))
-(let (($x2336 (>= (+ ?x1823 (v_b_SP_G_0$ ?v1!3) (* (- 1) (v_b_SP_G_0$ ?v0!4))) 0)))
-(let (($x1826 (<= (+ b_Infinity$ (* (- 1) ?x1823)) 0)))
-(let (($x1821 (v_b_Visited_G_0$ ?v1!3)))
-(let (($x2668 (not $x1821)))
-(let (($x2683 (or $x2668 $x1826 $x2336)))
-(let (($x3748 (forall ((?v0 B_Vertex$) )(!(let (($x83 (v_b_Visited_G_0$ ?v0)))
-(not $x83)) :pattern ( (v_b_Visited_G_0$ ?v0) )))
-))
-(let (($x85 (forall ((?v0 B_Vertex$) )(let (($x83 (v_b_Visited_G_0$ ?v0)))
-(not $x83)))
-))
-(let ((@x3752 (quant-intro (refl (= (not (v_b_Visited_G_0$ ?0)) (not (v_b_Visited_G_0$ ?0)))) (= $x85 $x3748))))
-(let ((@x1779 (nnf-pos (refl (~ (not (v_b_Visited_G_0$ ?0)) (not (v_b_Visited_G_0$ ?0)))) (~ $x85 $x85))))
-(let (($x343 (forall ((?v0 B_Vertex$) )(let (($x74 (= ?v0 b_Source$)))
-(or $x74 (= (v_b_SP_G_0$ ?v0) b_Infinity$))))
-))
-(let (($x337 (forall ((?v0 B_Vertex$) )(let (($x74 (= ?v0 b_Source$)))
-(let (($x79 (not $x74)))
-(or $x79 (= (v_b_SP_G_0$ ?v0) 0)))))
-))
-(let (($x354 (and $x337 $x343 $x85)))
-(let (($x850 (forall ((?v0 B_Vertex$) )(let (($x838 (exists ((?v1 B_Vertex$) )(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let ((?x220 (v_b_SP_G_2$ ?v1)))
-(let ((?x255 (+ ?x220 ?x102)))
-(let ((?x250 (v_b_SP_G_2$ ?v0)))
-(let (($x262 (= ?x250 ?x255)))
-(let (($x238 (fun_app$ v_b_Visited_G_2$ ?v1)))
-(let (($x251 (<= ?x250 ?x220)))
-(let (($x827 (not $x251)))
-(and $x827 $x238 $x262))))))))))
-))
-(let (($x821 (not (<= b_Infinity$ (v_b_SP_G_2$ ?v0)))))
-(let (($x74 (= ?v0 b_Source$)))
-(let (($x79 (not $x74)))
-(let (($x824 (and $x79 $x821)))
-(let (($x844 (not $x824)))
-(or $x844 $x838))))))))
-))
-(let (($x817 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let ((?x220 (v_b_SP_G_2$ ?v1)))
-(let ((?x255 (+ ?x220 ?x102)))
-(let ((?x250 (v_b_SP_G_2$ ?v0)))
-(let (($x256 (<= ?x250 ?x255)))
-(let (($x378 (not (<= b_Infinity$ ?x102))))
-(let (($x238 (fun_app$ v_b_Visited_G_2$ ?v1)))
-(let (($x805 (and $x238 $x378)))
-(let (($x811 (not $x805)))
-(or $x811 $x256)))))))))))
-))
-(let (($x878 (or (not $x817) $x850)))
-(let (($x883 (and $x817 $x878)))
-(let (($x802 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x220 (v_b_SP_G_2$ ?v1)))
-(let ((?x250 (v_b_SP_G_2$ ?v0)))
-(let (($x251 (<= ?x250 ?x220)))
-(let (($x238 (fun_app$ v_b_Visited_G_2$ ?v1)))
-(let (($x247 (not $x238)))
-(let (($x249 (and $x247 (fun_app$ v_b_Visited_G_2$ ?v0))))
-(let (($x798 (not $x249)))
-(or $x798 $x251)))))))))
-))
-(let (($x889 (not $x802)))
-(let (($x890 (or $x889 $x883)))
-(let (($x895 (and $x802 $x890)))
-(let (($x246 (forall ((?v0 B_Vertex$) )(let ((?x220 (v_b_SP_G_2$ ?v0)))
-(<= 0 ?x220)))
-))
-(let (($x901 (not $x246)))
-(let (($x902 (or $x901 $x895)))
-(let (($x907 (and $x246 $x902)))
-(let (($x914 (or $x913 $x907)))
-(let (($x919 (and $x244 $x914)))
-(let (($x786 (forall ((?v0 B_Vertex$) )(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v0)))
-(let ((?x220 (v_b_SP_G_2$ ?v0)))
-(let (($x225 (= ?x220 ?x121)))
-(let (($x238 (fun_app$ v_b_Visited_G_2$ ?v0)))
-(let (($x247 (not $x238)))
-(or $x247 $x225)))))))
-))
-(let (($x925 (not $x786)))
-(let (($x926 (or $x925 $x919)))
-(let (($x931 (and $x786 $x926)))
-(let (($x237 (forall ((?v0 B_Vertex$) )(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v0)))
-(let ((?x220 (v_b_SP_G_2$ ?v0)))
-(<= ?x220 ?x121))))
-))
-(let (($x937 (not $x237)))
-(let (($x938 (or $x937 $x931)))
-(let (($x943 (and $x237 $x938)))
-(let (($x726 (forall ((?v0 B_Vertex$) )(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v0)))
-(let ((?x220 (v_b_SP_G_2$ ?v0)))
-(let (($x225 (= ?x220 ?x121)))
-(let ((?x215 (b_G$ (pair$ v_b_v_G_1$ ?v0))))
-(let ((?x204 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
-(let ((?x217 (+ ?x204 ?x215)))
-(let (($x698 (not (<= ?x121 ?x217))))
-(let (($x694 (not (<= b_Infinity$ ?x215))))
-(let (($x701 (and $x694 $x698)))
-(or $x701 $x225)))))))))))
-))
-(let (($x713 (forall ((?v0 B_Vertex$) )(let ((?x215 (b_G$ (pair$ v_b_v_G_1$ ?v0))))
-(let ((?x204 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
-(let ((?x217 (+ ?x204 ?x215)))
-(let ((?x220 (v_b_SP_G_2$ ?v0)))
-(let (($x221 (= ?x220 ?x217)))
-(let (($x698 (not (<= (fun_app$c v_b_SP_G_1$ ?v0) ?x217))))
-(let (($x694 (not (<= b_Infinity$ ?x215))))
-(let (($x701 (and $x694 $x698)))
-(let (($x707 (not $x701)))
-(or $x707 $x221)))))))))))
-))
-(let (($x690 (forall ((?v0 B_Vertex$) )(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v0)))
-(let ((?x204 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
-(let (($x206 (<= ?x204 ?x121)))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v0)))
-(or $x125 $x206))))))
-))
-(let (($x684 (not (<= b_Infinity$ (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))))
-(let (($x203 (not $x202)))
-(let (($x540 (exists ((?v0 B_Vertex$) )(let (($x452 (not (<= b_Infinity$ (fun_app$c v_b_SP_G_1$ ?v0)))))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v0)))
-(let (($x126 (not $x125)))
-(and $x126 $x452)))))
-))
-(let (($x767 (and $x540 $x203 $x684 $x690 $x213 $x713 $x726)))
-(let (($x949 (not $x767)))
-(let (($x950 (or $x949 $x943)))
-(let (($x638 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let ((?x177 (fun_app$c v_b_SP_G_3$ ?v1)))
-(let ((?x182 (+ ?x177 ?x102)))
-(let ((?x180 (fun_app$c v_b_SP_G_3$ ?v0)))
-(let (($x189 (<= ?x180 ?x182)))
-(let (($x378 (not (<= b_Infinity$ ?x102))))
-(let (($x598 (not (<= b_Infinity$ ?x177))))
-(let (($x626 (and $x598 $x378)))
-(let (($x632 (not $x626)))
-(or $x632 $x189)))))))))))
-))
-(let (($x654 (or (not $x638) $x193)))
-(let (($x659 (and $x638 $x654)))
-(let (($x623 (forall ((?v0 B_Vertex$) )(let (($x611 (exists ((?v1 B_Vertex$) )(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let ((?x177 (fun_app$c v_b_SP_G_3$ ?v1)))
-(let ((?x182 (+ ?x177 ?x102)))
-(let ((?x180 (fun_app$c v_b_SP_G_3$ ?v0)))
-(let (($x183 (= ?x180 ?x182)))
-(let (($x605 (not (<= ?x180 ?x177))))
-(and $x605 $x183))))))))
-))
-(let (($x598 (not (<= b_Infinity$ (fun_app$c v_b_SP_G_3$ ?v0)))))
-(let (($x74 (= ?v0 b_Source$)))
-(let (($x79 (not $x74)))
-(let (($x601 (and $x79 $x598)))
-(let (($x617 (not $x601)))
-(or $x617 $x611))))))))
-))
-(let (($x666 (or (not $x623) $x659)))
-(let (($x671 (and $x623 $x666)))
-(let (($x167 (= v_b_oldSP_G_1$ v_b_oldSP_G_0$)))
-(let (($x162 (= v_b_v_G_2$ v_b_v_G_0$)))
-(let (($x159 (= v_b_Visited_G_3$ v_b_Visited_G_1$)))
-(let (($x543 (not $x540)))
-(let (($x581 (and $x543 $x159 $x162 $x164 $x167)))
-(let (($x677 (not $x581)))
-(let (($x678 (or $x677 $x671)))
-(let (($x955 (and $x678 $x950)))
-(let (($x481 (forall ((?v0 B_Vertex$) )(let (($x469 (exists ((?v1 B_Vertex$) )(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v1)))
-(let ((?x134 (+ ?x121 ?x102)))
-(let ((?x129 (fun_app$c v_b_SP_G_1$ ?v0)))
-(let (($x141 (= ?x129 ?x134)))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v1)))
-(let (($x130 (<= ?x129 ?x121)))
-(let (($x458 (not $x130)))
-(and $x458 $x125 $x141))))))))))
-))
-(let (($x452 (not (<= b_Infinity$ (fun_app$c v_b_SP_G_1$ ?v0)))))
-(let (($x74 (= ?v0 b_Source$)))
-(let (($x79 (not $x74)))
-(let (($x455 (and $x79 $x452)))
-(let (($x475 (not $x455)))
-(or $x475 $x469))))))))
-))
-(let (($x448 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v1)))
-(let ((?x134 (+ ?x121 ?x102)))
-(let ((?x129 (fun_app$c v_b_SP_G_1$ ?v0)))
-(let (($x135 (<= ?x129 ?x134)))
-(let (($x378 (not (<= b_Infinity$ ?x102))))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v1)))
-(let (($x436 (and $x125 $x378)))
-(let (($x442 (not $x436)))
-(or $x442 $x135)))))))))))
-))
-(let (($x433 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v1)))
-(let ((?x129 (fun_app$c v_b_SP_G_1$ ?v0)))
-(let (($x130 (<= ?x129 ?x121)))
-(let (($x127 (fun_app$ v_b_Visited_G_1$ ?v0)))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v1)))
-(let (($x126 (not $x125)))
-(let (($x128 (and $x126 $x127)))
-(let (($x429 (not $x128)))
-(or $x429 $x130))))))))))
-))
-(let (($x123 (forall ((?v0 B_Vertex$) )(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v0)))
-(<= 0 ?x121)))
-))
-(let (($x426 (forall ((?v0 B_Vertex$) )(let (($x414 (exists ((?v1 B_Vertex$) )(let ((?x97 (v_b_SP_G_0$ ?v0)))
-(let (($x112 (= ?x97 (+ (v_b_SP_G_0$ ?v1) (b_G$ (pair$ ?v1 ?v0))))))
-(let (($x83 (v_b_Visited_G_0$ ?v1)))
-(let ((?x75 (v_b_SP_G_0$ ?v1)))
-(let (($x98 (<= ?x97 ?x75)))
-(let (($x403 (not $x98)))
-(and $x403 $x83 $x112))))))))
-))
-(let (($x397 (not (<= b_Infinity$ (v_b_SP_G_0$ ?v0)))))
-(let (($x74 (= ?v0 b_Source$)))
-(let (($x79 (not $x74)))
-(let (($x400 (and $x79 $x397)))
-(or (not $x400) $x414)))))))
-))
-(let (($x532 (and $x426 $x120 $x123 $x433 $x448 $x481)))
-(let (($x961 (not $x532)))
-(let (($x962 (or $x961 $x955)))
-(let (($x967 (and $x426 $x962)))
-(let (($x393 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x97 (v_b_SP_G_0$ ?v0)))
-(let (($x106 (<= ?x97 (+ (v_b_SP_G_0$ ?v1) (b_G$ (pair$ ?v1 ?v0))))))
-(let (($x378 (not (<= b_Infinity$ (b_G$ (pair$ ?v1 ?v0))))))
-(let (($x83 (v_b_Visited_G_0$ ?v1)))
-(let (($x381 (and $x83 $x378)))
-(or (not $x381) $x106)))))))
-))
-(let (($x973 (not $x393)))
-(let (($x974 (or $x973 $x967)))
-(let (($x979 (and $x393 $x974)))
-(let (($x374 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x75 (v_b_SP_G_0$ ?v1)))
-(let ((?x97 (v_b_SP_G_0$ ?v0)))
-(let (($x98 (<= ?x97 ?x75)))
-(let (($x95 (v_b_Visited_G_0$ ?v0)))
-(let (($x83 (v_b_Visited_G_0$ ?v1)))
-(let (($x84 (not $x83)))
-(let (($x96 (and $x84 $x95)))
-(let (($x370 (not $x96)))
-(or $x370 $x98))))))))))
-))
-(let (($x985 (not $x374)))
-(let (($x986 (or $x985 $x979)))
-(let (($x991 (and $x374 $x986)))
-(let (($x94 (forall ((?v0 B_Vertex$) )(let ((?x75 (v_b_SP_G_0$ ?v0)))
-(<= 0 ?x75)))
-))
-(let (($x997 (not $x94)))
-(let (($x998 (or $x997 $x991)))
-(let (($x1003 (and $x94 $x998)))
-(let (($x92 (= (v_b_SP_G_0$ b_Source$) 0)))
-(let (($x1009 (not $x92)))
-(let (($x1010 (or $x1009 $x1003)))
-(let (($x1015 (and $x92 $x1010)))
-(let (($x1022 (or (not $x354) $x1015)))
-(let (($x267 (forall ((?v0 B_Vertex$) )(let (($x265 (exists ((?v1 B_Vertex$) )(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let ((?x220 (v_b_SP_G_2$ ?v1)))
-(let ((?x255 (+ ?x220 ?x102)))
-(let ((?x250 (v_b_SP_G_2$ ?v0)))
-(let (($x262 (= ?x250 ?x255)))
-(let (($x238 (fun_app$ v_b_Visited_G_2$ ?v1)))
-(and (< ?x220 ?x250) (and $x238 $x262)))))))))
-))
-(=> (and (not (= ?v0 b_Source$)) (< (v_b_SP_G_2$ ?v0) b_Infinity$)) $x265)))
-))
-(let (($x268 (and $x267 false)))
-(let (($x269 (=> $x268 true)))
-(let (($x270 (and $x267 $x269)))
-(let (($x258 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let ((?x220 (v_b_SP_G_2$ ?v1)))
-(let ((?x255 (+ ?x220 ?x102)))
-(let ((?x250 (v_b_SP_G_2$ ?v0)))
-(let (($x256 (<= ?x250 ?x255)))
-(=> (and (fun_app$ v_b_Visited_G_2$ ?v1) (< ?x102 b_Infinity$)) $x256)))))))
-))
-(let (($x271 (=> $x258 $x270)))
-(let (($x253 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x220 (v_b_SP_G_2$ ?v1)))
-(let ((?x250 (v_b_SP_G_2$ ?v0)))
-(let (($x251 (<= ?x250 ?x220)))
-(let (($x238 (fun_app$ v_b_Visited_G_2$ ?v1)))
-(let (($x247 (not $x238)))
-(let (($x249 (and $x247 (fun_app$ v_b_Visited_G_2$ ?v0))))
-(=> $x249 $x251))))))))
-))
-(let (($x273 (=> $x253 (and $x258 $x271))))
-(let (($x275 (=> $x246 (and $x253 $x273))))
-(let (($x277 (=> $x244 (and $x246 $x275))))
-(let (($x240 (forall ((?v0 B_Vertex$) )(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v0)))
-(let ((?x220 (v_b_SP_G_2$ ?v0)))
-(let (($x225 (= ?x220 ?x121)))
-(let (($x238 (fun_app$ v_b_Visited_G_2$ ?v0)))
-(=> $x238 $x225))))))
-))
-(let (($x242 (and $x240 (and true true))))
-(let (($x279 (=> $x242 (and $x244 $x277))))
-(let (($x281 (=> $x237 (and $x240 $x279))))
-(let (($x227 (forall ((?v0 B_Vertex$) )(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v0)))
-(let ((?x220 (v_b_SP_G_2$ ?v0)))
-(let (($x225 (= ?x220 ?x121)))
-(let ((?x215 (b_G$ (pair$ v_b_v_G_1$ ?v0))))
-(let ((?x204 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
-(let ((?x217 (+ ?x204 ?x215)))
-(let (($x219 (and (< ?x215 b_Infinity$) (< ?x217 ?x121))))
-(=> (not $x219) $x225)))))))))
-))
-(let (($x223 (forall ((?v0 B_Vertex$) )(let ((?x215 (b_G$ (pair$ v_b_v_G_1$ ?v0))))
-(let ((?x204 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
-(let ((?x217 (+ ?x204 ?x215)))
-(let ((?x220 (v_b_SP_G_2$ ?v0)))
-(let (($x221 (= ?x220 ?x217)))
-(let (($x219 (and (< ?x215 b_Infinity$) (< ?x217 (fun_app$c v_b_SP_G_1$ ?v0)))))
-(=> $x219 $x221))))))))
-))
-(let (($x229 (and $x213 (and $x223 $x227))))
-(let (($x208 (forall ((?v0 B_Vertex$) )(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v0)))
-(let ((?x204 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
-(let (($x206 (<= ?x204 ?x121)))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v0)))
-(let (($x126 (not $x125)))
-(=> $x126 $x206)))))))
-))
-(let (($x230 (and $x208 $x229)))
-(let (($x231 (and (< (fun_app$c v_b_SP_G_1$ v_b_v_G_1$) b_Infinity$) $x230)))
-(let (($x232 (and $x203 $x231)))
-(let (($x156 (exists ((?v0 B_Vertex$) )(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v0)))
-(let (($x138 (< ?x121 b_Infinity$)))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v0)))
-(let (($x126 (not $x125)))
-(and $x126 $x138))))))
-))
-(let (($x233 (and $x156 $x232)))
-(let (($x234 (and true $x233)))
-(let (($x235 (and true $x234)))
-(let (($x283 (=> $x235 (and $x237 $x281))))
-(let (($x195 (and $x193 (=> $x193 true))))
-(let (($x191 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let ((?x177 (fun_app$c v_b_SP_G_3$ ?v1)))
-(let ((?x182 (+ ?x177 ?x102)))
-(let ((?x180 (fun_app$c v_b_SP_G_3$ ?v0)))
-(let (($x189 (<= ?x180 ?x182)))
-(=> (and (< ?x177 b_Infinity$) (< ?x102 b_Infinity$)) $x189)))))))
-))
-(let (($x196 (=> $x191 $x195)))
-(let (($x187 (forall ((?v0 B_Vertex$) )(let (($x185 (exists ((?v1 B_Vertex$) )(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let ((?x177 (fun_app$c v_b_SP_G_3$ ?v1)))
-(let ((?x182 (+ ?x177 ?x102)))
-(let ((?x180 (fun_app$c v_b_SP_G_3$ ?v0)))
-(let (($x183 (= ?x180 ?x182)))
-(and (< ?x177 ?x180) $x183)))))))
-))
-(let ((?x177 (fun_app$c v_b_SP_G_3$ ?v0)))
-(let (($x178 (< ?x177 b_Infinity$)))
-(let (($x74 (= ?v0 b_Source$)))
-(let (($x79 (not $x74)))
-(=> (and $x79 $x178) $x185)))))))
-))
-(let (($x198 (=> $x187 (and $x191 $x196))))
-(let (($x170 (and $x162 (and $x164 (and $x167 true)))))
-(let (($x171 (and $x159 $x170)))
-(let (($x172 (and true $x171)))
-(let (($x173 (and true $x172)))
-(let (($x174 (and (not $x156) $x173)))
-(let (($x175 (and true $x174)))
-(let (($x176 (and true $x175)))
-(let (($x200 (=> $x176 (and $x187 $x198))))
-(let (($x146 (forall ((?v0 B_Vertex$) )(let (($x144 (exists ((?v1 B_Vertex$) )(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v1)))
-(let ((?x134 (+ ?x121 ?x102)))
-(let ((?x129 (fun_app$c v_b_SP_G_1$ ?v0)))
-(let (($x141 (= ?x129 ?x134)))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v1)))
-(and (< ?x121 ?x129) (and $x125 $x141)))))))))
-))
-(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v0)))
-(let (($x138 (< ?x121 b_Infinity$)))
-(let (($x74 (= ?v0 b_Source$)))
-(let (($x79 (not $x74)))
-(=> (and $x79 $x138) $x144)))))))
-))
-(let (($x147 (and $x146 true)))
-(let (($x137 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v1)))
-(let ((?x134 (+ ?x121 ?x102)))
-(let ((?x129 (fun_app$c v_b_SP_G_1$ ?v0)))
-(let (($x135 (<= ?x129 ?x134)))
-(=> (and (fun_app$ v_b_Visited_G_1$ ?v1) (< ?x102 b_Infinity$)) $x135)))))))
-))
-(let (($x132 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v1)))
-(let ((?x129 (fun_app$c v_b_SP_G_1$ ?v0)))
-(let (($x130 (<= ?x129 ?x121)))
-(let (($x127 (fun_app$ v_b_Visited_G_1$ ?v0)))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v1)))
-(let (($x126 (not $x125)))
-(let (($x128 (and $x126 $x127)))
-(=> $x128 $x130)))))))))
-))
-(let (($x149 (and $x132 (and $x137 $x147))))
-(let (($x150 (and $x123 $x149)))
-(let (($x151 (and $x120 $x150)))
-(let (($x152 (and true $x151)))
-(let (($x153 (and true $x152)))
-(let (($x117 (forall ((?v0 B_Vertex$) )(let (($x115 (exists ((?v1 B_Vertex$) )(let ((?x97 (v_b_SP_G_0$ ?v0)))
-(let (($x112 (= ?x97 (+ (v_b_SP_G_0$ ?v1) (b_G$ (pair$ ?v1 ?v0))))))
-(let (($x83 (v_b_Visited_G_0$ ?v1)))
-(and (< (v_b_SP_G_0$ ?v1) ?x97) (and $x83 $x112))))))
-))
-(=> (and (not (= ?v0 b_Source$)) (< (v_b_SP_G_0$ ?v0) b_Infinity$)) $x115)))
-))
-(let (($x154 (and $x117 $x153)))
-(let (($x285 (=> $x154 (and $x200 $x283))))
-(let (($x108 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x97 (v_b_SP_G_0$ ?v0)))
-(let (($x106 (<= ?x97 (+ (v_b_SP_G_0$ ?v1) (b_G$ (pair$ ?v1 ?v0))))))
-(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let (($x103 (< ?x102 b_Infinity$)))
-(let (($x83 (v_b_Visited_G_0$ ?v1)))
-(=> (and $x83 $x103) $x106)))))))
-))
-(let (($x287 (=> $x108 (and $x117 $x285))))
-(let (($x100 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x75 (v_b_SP_G_0$ ?v1)))
-(let ((?x97 (v_b_SP_G_0$ ?v0)))
-(let (($x98 (<= ?x97 ?x75)))
-(let (($x95 (v_b_Visited_G_0$ ?v0)))
-(let (($x83 (v_b_Visited_G_0$ ?v1)))
-(let (($x84 (not $x83)))
-(let (($x96 (and $x84 $x95)))
-(=> $x96 $x98)))))))))
-))
-(let (($x289 (=> $x100 (and $x108 $x287))))
-(let (($x291 (=> $x94 (and $x100 $x289))))
-(let (($x293 (=> $x92 (and $x94 $x291))))
-(let (($x82 (forall ((?v0 B_Vertex$) )(let (($x74 (= ?v0 b_Source$)))
-(let (($x79 (not $x74)))
-(=> $x79 (= (v_b_SP_G_0$ ?v0) b_Infinity$)))))
-))
-(let (($x78 (forall ((?v0 B_Vertex$) )(let (($x74 (= ?v0 b_Source$)))
-(=> $x74 (= (v_b_SP_G_0$ ?v0) 0))))
-))
-(let (($x88 (and $x78 (and $x82 (and $x85 true)))))
-(let (($x89 (and true $x88)))
-(let (($x90 (and true $x89)))
-(let (($x295 (=> $x90 (and $x92 $x293))))
-(let (($x296 (not $x295)))
-(let (($x838 (exists ((?v1 B_Vertex$) )(let ((?x102 (b_G$ (pair$ ?v1 ?0))))
-(let ((?x220 (v_b_SP_G_2$ ?v1)))
-(let ((?x255 (+ ?x220 ?x102)))
-(let ((?x250 (v_b_SP_G_2$ ?0)))
-(let (($x262 (= ?x250 ?x255)))
-(let (($x238 (fun_app$ v_b_Visited_G_2$ ?v1)))
-(let (($x251 (<= ?x250 ?x220)))
-(let (($x827 (not $x251)))
-(and $x827 $x238 $x262))))))))))
-))
-(let (($x821 (not (<= b_Infinity$ (v_b_SP_G_2$ ?0)))))
-(let (($x74 (= ?0 b_Source$)))
-(let (($x79 (not $x74)))
-(let (($x824 (and $x79 $x821)))
-(let (($x844 (not $x824)))
-(let (($x845 (or $x844 $x838)))
-(let (($x265 (exists ((?v1 B_Vertex$) )(let ((?x102 (b_G$ (pair$ ?v1 ?0))))
-(let ((?x220 (v_b_SP_G_2$ ?v1)))
-(let ((?x255 (+ ?x220 ?x102)))
-(let ((?x250 (v_b_SP_G_2$ ?0)))
-(let (($x262 (= ?x250 ?x255)))
-(let (($x238 (fun_app$ v_b_Visited_G_2$ ?v1)))
-(and (< ?x220 ?x250) (and $x238 $x262)))))))))
-))
-(let (($x266 (=> (and $x79 (< (v_b_SP_G_2$ ?0) b_Infinity$)) $x265)))
-(let ((?x102 (b_G$ (pair$ ?0 ?1))))
-(let ((?x220 (v_b_SP_G_2$ ?0)))
-(let ((?x255 (+ ?x220 ?x102)))
-(let ((?x250 (v_b_SP_G_2$ ?1)))
-(let (($x262 (= ?x250 ?x255)))
-(let (($x238 (fun_app$ v_b_Visited_G_2$ ?0)))
-(let (($x251 (<= ?x250 ?x220)))
-(let (($x827 (not $x251)))
-(let (($x833 (and $x827 $x238 $x262)))
-(let (($x264 (and (< ?x220 ?x250) (and $x238 $x262))))
-(let ((@x832 (monotonicity (rewrite (= (< ?x220 ?x250) $x827)) (= $x264 (and $x827 (and $x238 $x262))))))
-(let ((@x837 (trans @x832 (rewrite (= (and $x827 (and $x238 $x262)) $x833)) (= $x264 $x833))))
-(let ((@x826 (monotonicity (rewrite (= (< ?x220 b_Infinity$) $x821)) (= (and $x79 (< ?x220 b_Infinity$)) $x824))))
-(let ((@x843 (monotonicity @x826 (quant-intro @x837 (= $x265 $x838)) (= $x266 (=> $x824 $x838)))))
-(let ((@x852 (quant-intro (trans @x843 (rewrite (= (=> $x824 $x838) $x845)) (= $x266 $x845)) (= $x267 $x850))))
-(let ((@x859 (trans (monotonicity @x852 (= $x268 (and $x850 false))) (rewrite (= (and $x850 false) false)) (= $x268 false))))
-(let ((@x866 (trans (monotonicity @x859 (= $x269 (=> false true))) (rewrite (= (=> false true) true)) (= $x269 true))))
-(let ((@x873 (trans (monotonicity @x852 @x866 (= $x270 (and $x850 true))) (rewrite (= (and $x850 true) $x850)) (= $x270 $x850))))
-(let (($x256 (<= ?x250 ?x255)))
-(let (($x378 (not (<= b_Infinity$ ?x102))))
-(let (($x805 (and $x238 $x378)))
-(let (($x811 (not $x805)))
-(let (($x812 (or $x811 $x256)))
-(let (($x257 (=> (and $x238 (< ?x102 b_Infinity$)) $x256)))
-(let ((@x380 (rewrite (= (< ?x102 b_Infinity$) $x378))))
-(let ((@x810 (monotonicity (monotonicity @x380 (= (and $x238 (< ?x102 b_Infinity$)) $x805)) (= $x257 (=> $x805 $x256)))))
-(let ((@x819 (quant-intro (trans @x810 (rewrite (= (=> $x805 $x256) $x812)) (= $x257 $x812)) (= $x258 $x817))))
-(let ((@x882 (trans (monotonicity @x819 @x873 (= $x271 (=> $x817 $x850))) (rewrite (= (=> $x817 $x850) $x878)) (= $x271 $x878))))
-(let (($x247 (not $x238)))
-(let (($x249 (and $x247 (fun_app$ v_b_Visited_G_2$ ?1))))
-(let (($x798 (not $x249)))
-(let (($x799 (or $x798 $x251)))
-(let ((@x888 (monotonicity (quant-intro (rewrite (= (=> $x249 $x251) $x799)) (= $x253 $x802)) (monotonicity @x819 @x882 (= (and $x258 $x271) $x883)) (= $x273 (=> $x802 $x883)))))
-(let ((@x897 (monotonicity (quant-intro (rewrite (= (=> $x249 $x251) $x799)) (= $x253 $x802)) (trans @x888 (rewrite (= (=> $x802 $x883) $x890)) (= $x273 $x890)) (= (and $x253 $x273) $x895))))
-(let ((@x906 (trans (monotonicity @x897 (= $x275 (=> $x246 $x895))) (rewrite (= (=> $x246 $x895) $x902)) (= $x275 $x902))))
-(let ((@x912 (monotonicity (monotonicity @x906 (= (and $x246 $x275) $x907)) (= $x277 (=> $x244 $x907)))))
-(let ((@x921 (monotonicity (trans @x912 (rewrite (= (=> $x244 $x907) $x914)) (= $x277 $x914)) (= (and $x244 $x277) $x919))))
-(let ((?x121 (fun_app$c v_b_SP_G_1$ ?0)))
-(let (($x225 (= ?x220 ?x121)))
-(let (($x783 (or $x247 $x225)))
-(let ((@x793 (monotonicity (quant-intro (rewrite (= (=> $x238 $x225) $x783)) (= $x240 $x786)) (rewrite (= (and true true) true)) (= $x242 (and $x786 true)))))
-(let ((@x924 (monotonicity (trans @x793 (rewrite (= (and $x786 true) $x786)) (= $x242 $x786)) @x921 (= $x279 (=> $x786 $x919)))))
-(let ((@x933 (monotonicity (quant-intro (rewrite (= (=> $x238 $x225) $x783)) (= $x240 $x786)) (trans @x924 (rewrite (= (=> $x786 $x919) $x926)) (= $x279 $x926)) (= (and $x240 $x279) $x931))))
-(let ((@x942 (trans (monotonicity @x933 (= $x281 (=> $x237 $x931))) (rewrite (= (=> $x237 $x931) $x938)) (= $x281 $x938))))
-(let (($x759 (and $x203 $x684 $x690 $x213 $x713 $x726)))
-(let (($x751 (and $x684 $x690 $x213 $x713 $x726)))
-(let ((@x745 (rewrite (= (and $x690 (and $x213 $x713 $x726)) (and $x690 $x213 $x713 $x726)))))
-(let ((?x215 (b_G$ (pair$ v_b_v_G_1$ ?0))))
-(let ((?x204 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
-(let ((?x217 (+ ?x204 ?x215)))
-(let (($x698 (not (<= ?x121 ?x217))))
-(let (($x694 (not (<= b_Infinity$ ?x215))))
-(let (($x701 (and $x694 $x698)))
-(let (($x721 (or $x701 $x225)))
-(let (($x226 (=> (not (and (< ?x215 b_Infinity$) (< ?x217 ?x121))) $x225)))
-(let ((@x703 (monotonicity (rewrite (= (< ?x215 b_Infinity$) $x694)) (rewrite (= (< ?x217 ?x121) $x698)) (= (and (< ?x215 b_Infinity$) (< ?x217 ?x121)) $x701))))
-(let ((@x717 (monotonicity @x703 (= (not (and (< ?x215 b_Infinity$) (< ?x217 ?x121))) (not $x701)))))
-(let ((@x725 (trans (monotonicity @x717 (= $x226 (=> (not $x701) $x225))) (rewrite (= (=> (not $x701) $x225) $x721)) (= $x226 $x721))))
-(let (($x221 (= ?x220 ?x217)))
-(let (($x707 (not $x701)))
-(let (($x708 (or $x707 $x221)))
-(let (($x219 (and (< ?x215 b_Infinity$) (< ?x217 ?x121))))
-(let (($x222 (=> $x219 $x221)))
-(let ((@x712 (trans (monotonicity @x703 (= $x222 (=> $x701 $x221))) (rewrite (= (=> $x701 $x221) $x708)) (= $x222 $x708))))
-(let ((@x731 (monotonicity (quant-intro @x712 (= $x223 $x713)) (quant-intro @x725 (= $x227 $x726)) (= (and $x223 $x227) (and $x713 $x726)))))
-(let ((@x739 (trans (monotonicity @x731 (= $x229 (and $x213 (and $x713 $x726)))) (rewrite (= (and $x213 (and $x713 $x726)) (and $x213 $x713 $x726))) (= $x229 (and $x213 $x713 $x726)))))
-(let (($x206 (<= ?x204 ?x121)))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?0)))
-(let (($x687 (or $x125 $x206)))
-(let ((@x692 (quant-intro (rewrite (= (=> (not $x125) $x206) $x687)) (= $x208 $x690))))
-(let ((@x747 (trans (monotonicity @x692 @x739 (= $x230 (and $x690 (and $x213 $x713 $x726)))) @x745 (= $x230 (and $x690 $x213 $x713 $x726)))))
-(let ((@x750 (monotonicity (rewrite (= (< ?x204 b_Infinity$) $x684)) @x747 (= $x231 (and $x684 (and $x690 $x213 $x713 $x726))))))
-(let ((@x755 (trans @x750 (rewrite (= (and $x684 (and $x690 $x213 $x713 $x726)) $x751)) (= $x231 $x751))))
-(let ((@x763 (trans (monotonicity @x755 (= $x232 (and $x203 $x751))) (rewrite (= (and $x203 $x751) $x759)) (= $x232 $x759))))
-(let (($x452 (not (<= b_Infinity$ ?x121))))
-(let (($x126 (not $x125)))
-(let (($x537 (and $x126 $x452)))
-(let ((@x539 (monotonicity (rewrite (= (< ?x121 b_Infinity$) $x452)) (= (and $x126 (< ?x121 b_Infinity$)) $x537))))
-(let ((@x766 (monotonicity (quant-intro @x539 (= $x156 $x540)) @x763 (= $x233 (and $x540 $x759)))))
-(let ((@x774 (monotonicity (trans @x766 (rewrite (= (and $x540 $x759) $x767)) (= $x233 $x767)) (= $x234 (and true $x767)))))
-(let ((@x780 (monotonicity (trans @x774 (rewrite (= (and true $x767) $x767)) (= $x234 $x767)) (= $x235 (and true $x767)))))
-(let ((@x948 (monotonicity (trans @x780 (rewrite (= (and true $x767) $x767)) (= $x235 $x767)) (monotonicity @x942 (= (and $x237 $x281) $x943)) (= $x283 (=> $x767 $x943)))))
-(let ((@x645 (monotonicity (rewrite (= (=> $x193 true) true)) (= $x195 (and $x193 true)))))
-(let ((?x177 (fun_app$c v_b_SP_G_3$ ?0)))
-(let ((?x182 (+ ?x177 ?x102)))
-(let ((?x180 (fun_app$c v_b_SP_G_3$ ?1)))
-(let (($x189 (<= ?x180 ?x182)))
-(let (($x598 (not (<= b_Infinity$ ?x177))))
-(let (($x626 (and $x598 $x378)))
-(let (($x632 (not $x626)))
-(let (($x633 (or $x632 $x189)))
-(let (($x190 (=> (and (< ?x177 b_Infinity$) (< ?x102 b_Infinity$)) $x189)))
-(let ((@x628 (monotonicity (rewrite (= (< ?x177 b_Infinity$) $x598)) @x380 (= (and (< ?x177 b_Infinity$) (< ?x102 b_Infinity$)) $x626))))
-(let ((@x637 (trans (monotonicity @x628 (= $x190 (=> $x626 $x189))) (rewrite (= (=> $x626 $x189) $x633)) (= $x190 $x633))))
-(let ((@x652 (monotonicity (quant-intro @x637 (= $x191 $x638)) (trans @x645 (rewrite (= (and $x193 true) $x193)) (= $x195 $x193)) (= $x196 (=> $x638 $x193)))))
-(let ((@x661 (monotonicity (quant-intro @x637 (= $x191 $x638)) (trans @x652 (rewrite (= (=> $x638 $x193) $x654)) (= $x196 $x654)) (= (and $x191 $x196) $x659))))
-(let (($x611 (exists ((?v1 B_Vertex$) )(let ((?x102 (b_G$ (pair$ ?v1 ?0))))
-(let ((?x177 (fun_app$c v_b_SP_G_3$ ?v1)))
-(let ((?x182 (+ ?x177 ?x102)))
-(let ((?x180 (fun_app$c v_b_SP_G_3$ ?0)))
-(let (($x183 (= ?x180 ?x182)))
-(let (($x605 (not (<= ?x180 ?x177))))
-(and $x605 $x183))))))))
-))
-(let (($x601 (and $x79 $x598)))
-(let (($x617 (not $x601)))
-(let (($x618 (or $x617 $x611)))
-(let (($x185 (exists ((?v1 B_Vertex$) )(let ((?x102 (b_G$ (pair$ ?v1 ?0))))
-(let ((?x177 (fun_app$c v_b_SP_G_3$ ?v1)))
-(let ((?x182 (+ ?x177 ?x102)))
-(let ((?x180 (fun_app$c v_b_SP_G_3$ ?0)))
-(let (($x183 (= ?x180 ?x182)))
-(and (< ?x177 ?x180) $x183)))))))
-))
-(let (($x186 (=> (and $x79 (< ?x177 b_Infinity$)) $x185)))
-(let (($x183 (= ?x180 ?x182)))
-(let (($x605 (not (<= ?x180 ?x177))))
-(let (($x608 (and $x605 $x183)))
-(let ((@x610 (monotonicity (rewrite (= (< ?x177 ?x180) $x605)) (= (and (< ?x177 ?x180) $x183) $x608))))
-(let ((@x603 (monotonicity (rewrite (= (< ?x177 b_Infinity$) $x598)) (= (and $x79 (< ?x177 b_Infinity$)) $x601))))
-(let ((@x616 (monotonicity @x603 (quant-intro @x610 (= $x185 $x611)) (= $x186 (=> $x601 $x611)))))
-(let ((@x625 (quant-intro (trans @x616 (rewrite (= (=> $x601 $x611) $x618)) (= $x186 $x618)) (= $x187 $x623))))
-(let ((@x670 (trans (monotonicity @x625 @x661 (= $x198 (=> $x623 $x659))) (rewrite (= (=> $x623 $x659) $x666)) (= $x198 $x666))))
-(let (($x562 (and $x159 $x162 $x164 $x167)))
-(let (($x567 (and true $x562)))
-(let ((@x550 (monotonicity (rewrite (= (and $x167 true) $x167)) (= (and $x164 (and $x167 true)) (and $x164 $x167)))))
-(let ((@x558 (trans (monotonicity @x550 (= $x170 (and $x162 (and $x164 $x167)))) (rewrite (= (and $x162 (and $x164 $x167)) (and $x162 $x164 $x167))) (= $x170 (and $x162 $x164 $x167)))))
-(let ((@x566 (trans (monotonicity @x558 (= $x171 (and $x159 (and $x162 $x164 $x167)))) (rewrite (= (and $x159 (and $x162 $x164 $x167)) $x562)) (= $x171 $x562))))
-(let ((@x573 (trans (monotonicity @x566 (= $x172 $x567)) (rewrite (= $x567 $x562)) (= $x172 $x562))))
-(let ((@x577 (trans (monotonicity @x573 (= $x173 $x567)) (rewrite (= $x567 $x562)) (= $x173 $x562))))
-(let ((@x545 (monotonicity (quant-intro @x539 (= $x156 $x540)) (= (not $x156) $x543))))
-(let ((@x585 (trans (monotonicity @x545 @x577 (= $x174 (and $x543 $x562))) (rewrite (= (and $x543 $x562) $x581)) (= $x174 $x581))))
-(let ((@x592 (trans (monotonicity @x585 (= $x175 (and true $x581))) (rewrite (= (and true $x581) $x581)) (= $x175 $x581))))
-(let ((@x596 (trans (monotonicity @x592 (= $x176 (and true $x581))) (rewrite (= (and true $x581) $x581)) (= $x176 $x581))))
-(let ((@x676 (monotonicity @x596 (monotonicity @x625 @x670 (= (and $x187 $x198) $x671)) (= $x200 (=> $x581 $x671)))))
-(let ((@x957 (monotonicity (trans @x676 (rewrite (= (=> $x581 $x671) $x678)) (= $x200 $x678)) (trans @x948 (rewrite (= (=> $x767 $x943) $x950)) (= $x283 $x950)) (= (and $x200 $x283) $x955))))
-(let (($x513 (and $x120 $x123 $x433 $x448 $x481)))
-(let (($x518 (and true $x513)))
-(let ((@x507 (rewrite (= (and $x123 (and $x433 $x448 $x481)) (and $x123 $x433 $x448 $x481)))))
-(let (($x469 (exists ((?v1 B_Vertex$) )(let ((?x102 (b_G$ (pair$ ?v1 ?0))))
-(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v1)))
-(let ((?x134 (+ ?x121 ?x102)))
-(let ((?x129 (fun_app$c v_b_SP_G_1$ ?0)))
-(let (($x141 (= ?x129 ?x134)))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v1)))
-(let (($x130 (<= ?x129 ?x121)))
-(let (($x458 (not $x130)))
-(and $x458 $x125 $x141))))))))))
-))
-(let (($x455 (and $x79 $x452)))
-(let (($x475 (not $x455)))
-(let (($x476 (or $x475 $x469)))
-(let (($x144 (exists ((?v1 B_Vertex$) )(let ((?x102 (b_G$ (pair$ ?v1 ?0))))
-(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v1)))
-(let ((?x134 (+ ?x121 ?x102)))
-(let ((?x129 (fun_app$c v_b_SP_G_1$ ?0)))
-(let (($x141 (= ?x129 ?x134)))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v1)))
-(and (< ?x121 ?x129) (and $x125 $x141)))))))))
-))
-(let (($x145 (=> (and $x79 (< ?x121 b_Infinity$)) $x144)))
-(let ((?x134 (+ ?x121 ?x102)))
-(let ((?x129 (fun_app$c v_b_SP_G_1$ ?1)))
-(let (($x141 (= ?x129 ?x134)))
-(let (($x130 (<= ?x129 ?x121)))
-(let (($x458 (not $x130)))
-(let (($x464 (and $x458 $x125 $x141)))
-(let (($x143 (and (< ?x121 ?x129) (and $x125 $x141))))
-(let ((@x463 (monotonicity (rewrite (= (< ?x121 ?x129) $x458)) (= $x143 (and $x458 (and $x125 $x141))))))
-(let ((@x468 (trans @x463 (rewrite (= (and $x458 (and $x125 $x141)) $x464)) (= $x143 $x464))))
-(let ((@x457 (monotonicity (rewrite (= (< ?x121 b_Infinity$) $x452)) (= (and $x79 (< ?x121 b_Infinity$)) $x455))))
-(let ((@x474 (monotonicity @x457 (quant-intro @x468 (= $x144 $x469)) (= $x145 (=> $x455 $x469)))))
-(let ((@x483 (quant-intro (trans @x474 (rewrite (= (=> $x455 $x469) $x476)) (= $x145 $x476)) (= $x146 $x481))))
-(let ((@x490 (trans (monotonicity @x483 (= $x147 (and $x481 true))) (rewrite (= (and $x481 true) $x481)) (= $x147 $x481))))
-(let (($x135 (<= ?x129 ?x134)))
-(let (($x436 (and $x125 $x378)))
-(let (($x442 (not $x436)))
-(let (($x443 (or $x442 $x135)))
-(let (($x136 (=> (and $x125 (< ?x102 b_Infinity$)) $x135)))
-(let ((@x441 (monotonicity (monotonicity @x380 (= (and $x125 (< ?x102 b_Infinity$)) $x436)) (= $x136 (=> $x436 $x135)))))
-(let ((@x450 (quant-intro (trans @x441 (rewrite (= (=> $x436 $x135) $x443)) (= $x136 $x443)) (= $x137 $x448))))
-(let (($x127 (fun_app$ v_b_Visited_G_1$ ?1)))
-(let (($x128 (and $x126 $x127)))
-(let (($x429 (not $x128)))
-(let (($x430 (or $x429 $x130)))
-(let ((@x496 (monotonicity (quant-intro (rewrite (= (=> $x128 $x130) $x430)) (= $x132 $x433)) (monotonicity @x450 @x490 (= (and $x137 $x147) (and $x448 $x481))) (= $x149 (and $x433 (and $x448 $x481))))))
-(let ((@x501 (trans @x496 (rewrite (= (and $x433 (and $x448 $x481)) (and $x433 $x448 $x481))) (= $x149 (and $x433 $x448 $x481)))))
-(let ((@x509 (trans (monotonicity @x501 (= $x150 (and $x123 (and $x433 $x448 $x481)))) @x507 (= $x150 (and $x123 $x433 $x448 $x481)))))
-(let ((@x517 (trans (monotonicity @x509 (= $x151 (and $x120 (and $x123 $x433 $x448 $x481)))) (rewrite (= (and $x120 (and $x123 $x433 $x448 $x481)) $x513)) (= $x151 $x513))))
-(let ((@x524 (trans (monotonicity @x517 (= $x152 $x518)) (rewrite (= $x518 $x513)) (= $x152 $x513))))
-(let ((@x528 (trans (monotonicity @x524 (= $x153 $x518)) (rewrite (= $x518 $x513)) (= $x153 $x513))))
-(let (($x414 (exists ((?v1 B_Vertex$) )(let ((?x97 (v_b_SP_G_0$ ?0)))
-(let (($x112 (= ?x97 (+ (v_b_SP_G_0$ ?v1) (b_G$ (pair$ ?v1 ?0))))))
-(let (($x83 (v_b_Visited_G_0$ ?v1)))
-(let ((?x75 (v_b_SP_G_0$ ?v1)))
-(let (($x98 (<= ?x97 ?x75)))
-(let (($x403 (not $x98)))
-(and $x403 $x83 $x112))))))))
-))
-(let (($x421 (or (not (and $x79 (not (<= b_Infinity$ (v_b_SP_G_0$ ?0))))) $x414)))
-(let (($x115 (exists ((?v1 B_Vertex$) )(let ((?x97 (v_b_SP_G_0$ ?0)))
-(let (($x112 (= ?x97 (+ (v_b_SP_G_0$ ?v1) (b_G$ (pair$ ?v1 ?0))))))
-(let (($x83 (v_b_Visited_G_0$ ?v1)))
-(and (< (v_b_SP_G_0$ ?v1) ?x97) (and $x83 $x112))))))
-))
-(let (($x116 (=> (and $x79 (< (v_b_SP_G_0$ ?0) b_Infinity$)) $x115)))
-(let (($x422 (= (=> (and $x79 (not (<= b_Infinity$ (v_b_SP_G_0$ ?0)))) $x414) $x421)))
-(let (($x418 (= $x116 (=> (and $x79 (not (<= b_Infinity$ (v_b_SP_G_0$ ?0)))) $x414))))
-(let ((?x97 (v_b_SP_G_0$ ?1)))
-(let (($x112 (= ?x97 (+ (v_b_SP_G_0$ ?0) ?x102))))
-(let (($x83 (v_b_Visited_G_0$ ?0)))
-(let ((?x75 (v_b_SP_G_0$ ?0)))
-(let (($x98 (<= ?x97 ?x75)))
-(let (($x403 (not $x98)))
-(let (($x409 (and $x403 $x83 $x112)))
-(let (($x114 (and (< ?x75 ?x97) (and $x83 $x112))))
-(let ((@x408 (monotonicity (rewrite (= (< ?x75 ?x97) $x403)) (= $x114 (and $x403 (and $x83 $x112))))))
-(let ((@x413 (trans @x408 (rewrite (= (and $x403 (and $x83 $x112)) $x409)) (= $x114 $x409))))
-(let (($x397 (not (<= b_Infinity$ ?x75))))
-(let (($x400 (and $x79 $x397)))
-(let ((@x402 (monotonicity (rewrite (= (< ?x75 b_Infinity$) $x397)) (= (and $x79 (< ?x75 b_Infinity$)) $x400))))
-(let ((@x425 (trans (monotonicity @x402 (quant-intro @x413 (= $x115 $x414)) $x418) (rewrite $x422) (= $x116 $x421))))
-(let ((@x531 (monotonicity (quant-intro @x425 (= $x117 $x426)) @x528 (= $x154 (and $x426 $x513)))))
-(let ((@x960 (monotonicity (trans @x531 (rewrite (= (and $x426 $x513) $x532)) (= $x154 $x532)) @x957 (= $x285 (=> $x532 $x955)))))
-(let ((@x969 (monotonicity (quant-intro @x425 (= $x117 $x426)) (trans @x960 (rewrite (= (=> $x532 $x955) $x962)) (= $x285 $x962)) (= (and $x117 $x285) $x967))))
-(let (($x106 (<= ?x97 (+ ?x75 ?x102))))
-(let (($x388 (or (not (and $x83 $x378)) $x106)))
-(let (($x107 (=> (and $x83 (< ?x102 b_Infinity$)) $x106)))
-(let ((@x383 (monotonicity @x380 (= (and $x83 (< ?x102 b_Infinity$)) (and $x83 $x378)))))
-(let ((@x392 (trans (monotonicity @x383 (= $x107 (=> (and $x83 $x378) $x106))) (rewrite (= (=> (and $x83 $x378) $x106) $x388)) (= $x107 $x388))))
-(let ((@x972 (monotonicity (quant-intro @x392 (= $x108 $x393)) @x969 (= $x287 (=> $x393 $x967)))))
-(let ((@x981 (monotonicity (quant-intro @x392 (= $x108 $x393)) (trans @x972 (rewrite (= (=> $x393 $x967) $x974)) (= $x287 $x974)) (= (and $x108 $x287) $x979))))
-(let (($x95 (v_b_Visited_G_0$ ?1)))
-(let (($x84 (not $x83)))
-(let (($x96 (and $x84 $x95)))
-(let (($x370 (not $x96)))
-(let (($x371 (or $x370 $x98)))
-(let ((@x984 (monotonicity (quant-intro (rewrite (= (=> $x96 $x98) $x371)) (= $x100 $x374)) @x981 (= $x289 (=> $x374 $x979)))))
-(let ((@x993 (monotonicity (quant-intro (rewrite (= (=> $x96 $x98) $x371)) (= $x100 $x374)) (trans @x984 (rewrite (= (=> $x374 $x979) $x986)) (= $x289 $x986)) (= (and $x100 $x289) $x991))))
-(let ((@x1002 (trans (monotonicity @x993 (= $x291 (=> $x94 $x991))) (rewrite (= (=> $x94 $x991) $x998)) (= $x291 $x998))))
-(let ((@x1008 (monotonicity (monotonicity @x1002 (= (and $x94 $x291) $x1003)) (= $x293 (=> $x92 $x1003)))))
-(let ((@x1017 (monotonicity (trans @x1008 (rewrite (= (=> $x92 $x1003) $x1010)) (= $x293 $x1010)) (= (and $x92 $x293) $x1015))))
-(let (($x340 (or $x74 (= ?x75 b_Infinity$))))
-(let ((@x345 (quant-intro (rewrite (= (=> $x79 (= ?x75 b_Infinity$)) $x340)) (= $x82 $x343))))
-(let ((@x350 (monotonicity @x345 (rewrite (= (and $x85 true) $x85)) (= (and $x82 (and $x85 true)) (and $x343 $x85)))))
-(let ((@x339 (quant-intro (rewrite (= (=> $x74 (= ?x75 0)) (or $x79 (= ?x75 0)))) (= $x78 $x337))))
-(let ((@x358 (trans (monotonicity @x339 @x350 (= $x88 (and $x337 (and $x343 $x85)))) (rewrite (= (and $x337 (and $x343 $x85)) $x354)) (= $x88 $x354))))
-(let ((@x365 (trans (monotonicity @x358 (= $x89 (and true $x354))) (rewrite (= (and true $x354) $x354)) (= $x89 $x354))))
-(let ((@x369 (trans (monotonicity @x365 (= $x90 (and true $x354))) (rewrite (= (and true $x354) $x354)) (= $x90 $x354))))
-(let ((@x1026 (trans (monotonicity @x369 @x1017 (= $x295 (=> $x354 $x1015))) (rewrite (= (=> $x354 $x1015) $x1022)) (= $x295 $x1022))))
-(let ((@x1030 (mp (asserted $x296) (monotonicity @x1026 (= $x296 (not $x1022))) (not $x1022))))
-(let ((@x1031 (not-or-elim @x1030 $x354)))
-(let ((@x1780 (mp~ (mp (and-elim @x1031 $x85) (rewrite* (= $x85 $x85)) $x85) @x1779 $x85)))
-(let ((@x4210 (unit-resolution ((_ quant-inst ?v1!3) (or (not $x3748) $x2668)) (mp @x1780 @x3752 $x3748) (hypothesis $x1821) false)))
-(let (($x2688 (not $x2683)))
-(let (($x4075 (or $x2688 $x4072)))
-(let (($x4078 (not $x4075)))
-(let (($x3763 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(!(let (($x1288 (>= (+ (v_b_SP_G_0$ ?v1) (* (- 1) (v_b_SP_G_0$ ?v0))) 0)))
-(let (($x83 (v_b_Visited_G_0$ ?v1)))
-(or $x83 (not (v_b_Visited_G_0$ ?v0)) $x1288))) :pattern ( (v_b_Visited_G_0$ ?v1) (v_b_Visited_G_0$ ?v0) )))
-))
-(let (($x4081 (or (not $x3763) $x4078)))
-(let (($x4084 (not $x4081)))
-(let (($x1807 (>= (+ (v_b_SP_G_0$ ?v1!1) (* (- 1) (v_b_SP_G_0$ ?v0!2))) 0)))
-(let (($x1800 (v_b_Visited_G_0$ ?v0!2)))
-(let (($x2622 (not $x1800)))
-(let (($x1798 (v_b_Visited_G_0$ ?v1!1)))
-(let (($x2637 (or $x1798 $x2622 $x1807)))
-(let (($x2642 (not $x2637)))
-(let (($x4087 (or $x2642 $x4084)))
-(let (($x4090 (not $x4087)))
-(let (($x3754 (forall ((?v0 B_Vertex$) )(!(let ((?x75 (v_b_SP_G_0$ ?v0)))
-(>= ?x75 0)) :pattern ( (v_b_SP_G_0$ ?v0) )))
-))
-(let (($x4093 (or (not $x3754) $x4090)))
-(let (($x4096 (not $x4093)))
-(let ((?x1784 (v_b_SP_G_0$ ?v0!0)))
-(let (($x1785 (>= ?x1784 0)))
-(let (($x307 (not (<= b_Infinity$ 0))))
-(let ((@x310 (mp (asserted (< 0 b_Infinity$)) (rewrite (= (< 0 b_Infinity$) $x307)) $x307)))
-(let (($x3424 (= b_Infinity$ ?x1784)))
-(let ((@x3416 (symm (commutativity (= $x3424 (= ?x1784 b_Infinity$))) (= (= ?x1784 b_Infinity$) $x3424))))
-(let (($x3481 (= ?x1784 b_Infinity$)))
-(let (($x5544 (= ?v0!0 b_Source$)))
-(let (($x5542 (not $x5544)))
-(let ((@x3411 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x1784 0)) $x1785)) (hypothesis (not $x1785)) (not (= ?x1784 0)))))
-(let (($x3735 (forall ((?v0 B_Vertex$) )(!(let (($x74 (= ?v0 b_Source$)))
-(let (($x79 (not $x74)))
-(or $x79 (= (v_b_SP_G_0$ ?v0) 0)))) :pattern ( (v_b_SP_G_0$ ?v0) )))
-))
-(let ((@x3739 (quant-intro (refl (= (or $x79 (= ?x75 0)) (or $x79 (= ?x75 0)))) (= $x337 $x3735))))
-(let ((@x1769 (nnf-pos (refl (~ (or $x79 (= ?x75 0)) (or $x79 (= ?x75 0)))) (~ $x337 $x337))))
-(let ((@x1770 (mp~ (mp (and-elim @x1031 $x337) (rewrite* (= $x337 $x337)) $x337) @x1769 $x337)))
-(let (($x3446 (= (or (not $x3735) (or $x5542 (= ?x1784 0))) (or (not $x3735) $x5542 (= ?x1784 0)))))
-(let ((@x3448 (mp ((_ quant-inst ?v0!0) (or (not $x3735) (or $x5542 (= ?x1784 0)))) (rewrite $x3446) (or (not $x3735) $x5542 (= ?x1784 0)))))
-(let (($x3741 (forall ((?v0 B_Vertex$) )(!(let (($x74 (= ?v0 b_Source$)))
-(or $x74 (= (v_b_SP_G_0$ ?v0) b_Infinity$))) :pattern ( (v_b_SP_G_0$ ?v0) )))
-))
-(let ((@x1775 (mp~ (mp (and-elim @x1031 $x343) (rewrite* (= $x343 $x343)) $x343) (nnf-pos (refl (~ $x340 $x340)) (~ $x343 $x343)) $x343)))
-(let ((@x3440 (rewrite (= (or (not $x3741) (or $x5544 $x3481)) (or (not $x3741) $x5544 $x3481)))))
-(let ((@x3430 (mp ((_ quant-inst ?v0!0) (or (not $x3741) (or $x5544 $x3481))) @x3440 (or (not $x3741) $x5544 $x3481))))
-(let ((@x3417 (unit-resolution @x3430 (mp @x1775 (quant-intro (refl (= $x340 $x340)) (= $x343 $x3741)) $x3741) (unit-resolution @x3448 (mp @x1770 @x3739 $x3735) @x3411 $x5542) $x3481)))
-(let ((@x3399 ((_ th-lemma arith triangle-eq) (or (not $x3424) (<= (+ b_Infinity$ (* (- 1) ?x1784)) 0)))))
-(let ((@x3400 (unit-resolution @x3399 (mp @x3417 @x3416 $x3424) (<= (+ b_Infinity$ (* (- 1) ?x1784)) 0))))
-(let ((@x3331 (unit-resolution ((_ th-lemma arith farkas 1 1) (or (<= ?x1784 0) $x1785)) (hypothesis (not $x1785)) (<= ?x1784 0))))
-(let ((@x3301 ((_ th-lemma arith farkas 1 -1 1) @x3331 @x3400 (mp @x310 (rewrite* (= $x307 $x307)) $x307) false)))
-(let (($x3437 (not $x3735)))
-(let (($x3312 (or $x3437 $x92)))
-(let ((@x3294 (monotonicity (rewrite (= (= b_Source$ b_Source$) true)) (= (not (= b_Source$ b_Source$)) (not true)))))
-(let ((@x3309 (trans @x3294 (rewrite (= (not true) false)) (= (not (= b_Source$ b_Source$)) false))))
-(let ((@x3315 (monotonicity @x3309 (= (or (not (= b_Source$ b_Source$)) $x92) (or false $x92)))))
-(let ((@x3319 (trans @x3315 (rewrite (= (or false $x92) $x92)) (= (or (not (= b_Source$ b_Source$)) $x92) $x92))))
-(let ((@x3291 (monotonicity @x3319 (= (or $x3437 (or (not (= b_Source$ b_Source$)) $x92)) $x3312))))
-(let ((@x3299 (trans @x3291 (rewrite (= $x3312 $x3312)) (= (or $x3437 (or (not (= b_Source$ b_Source$)) $x92)) $x3312))))
-(let ((@x3300 (mp ((_ quant-inst b_Source$) (or $x3437 (or (not (= b_Source$ b_Source$)) $x92))) @x3299 $x3312)))
-(let ((@x4116 (lemma (unit-resolution @x3300 (mp @x1770 @x3739 $x3735) (hypothesis $x1009) false) $x92)))
-(let (($x3122 (forall ((?v1 B_Vertex$) )(let ((?x2217 (v_b_SP_G_2$ ?v0!20)))
-(let ((?x2218 (* (- 1) ?x2217)))
-(let ((?x220 (v_b_SP_G_2$ ?v1)))
-(let (($x2528 (= (+ ?x220 ?x2218 (b_G$ (pair$ ?v1 ?v0!20))) 0)))
-(let (($x238 (fun_app$ v_b_Visited_G_2$ ?v1)))
-(let (($x247 (not $x238)))
-(or (>= (+ ?x220 ?x2218) 0) $x247 (not $x2528)))))))))
-))
-(let (($x3107 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x220 (v_b_SP_G_2$ ?v1)))
-(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let (($x1621 (>= (+ ?x102 ?x220 (* (- 1) (v_b_SP_G_2$ ?v0))) 0)))
-(let (($x1303 (<= (+ b_Infinity$ (* (- 1) ?x102)) 0)))
-(let (($x238 (fun_app$ v_b_Visited_G_2$ ?v1)))
-(let (($x247 (not $x238)))
-(or $x247 $x1303 $x1621))))))))
-))
-(let (($x3131 (not (or (not $x3107) $x2215 $x2220 (not $x3122)))))
-(let (($x3136 (or $x3085 $x3131)))
-(let (($x3062 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let (($x1601 (>= (+ (v_b_SP_G_2$ ?v1) (* (- 1) (v_b_SP_G_2$ ?v0))) 0)))
-(let (($x238 (fun_app$ v_b_Visited_G_2$ ?v1)))
-(or $x238 (not (fun_app$ v_b_Visited_G_2$ ?v0)) $x1601))))
-))
-(let (($x3145 (not (or (not $x3062) (not $x3136)))))
-(let (($x3150 (or $x3039 $x3145)))
-(let (($x1595 (forall ((?v0 B_Vertex$) )(let ((?x220 (v_b_SP_G_2$ ?v0)))
-(>= ?x220 0)))
-))
-(let (($x1598 (not $x1595)))
-(let (($x3158 (not (or $x1598 (not $x3150)))))
-(let (($x3163 (or $x913 $x2154 $x3158)))
-(let (($x3171 (not (or $x925 (not $x3163)))))
-(let (($x3176 (or $x2139 $x3171)))
-(let (($x1586 (forall ((?v0 B_Vertex$) )(>= (+ (fun_app$c v_b_SP_G_1$ ?v0) (* (- 1) (v_b_SP_G_2$ ?v0))) 0))
-))
-(let (($x1589 (not $x1586)))
-(let (($x3184 (not (or $x1589 (not $x3176)))))
-(let (($x3189 (or $x2122 $x3184)))
-(let (($x3016 (forall ((?v0 B_Vertex$) )(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v0)))
-(let ((?x220 (v_b_SP_G_2$ ?v0)))
-(let (($x225 (= ?x220 ?x121)))
-(let ((?x204 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
-(let ((?x1520 (* (- 1) ?x204)))
-(let (($x1547 (<= (+ ?x121 ?x1520 (* (- 1) (b_G$ (pair$ v_b_v_G_1$ ?v0)))) 0)))
-(let (($x1540 (<= (+ b_Infinity$ (* (- 1) (b_G$ (pair$ v_b_v_G_1$ ?v0)))) 0)))
-(let (($x2991 (or $x1540 $x1547)))
-(let (($x2992 (not $x2991)))
-(or $x2992 $x225)))))))))))
-))
-(let (($x3010 (forall ((?v0 B_Vertex$) )(let ((?x220 (v_b_SP_G_2$ ?v0)))
-(let ((?x1560 (* (- 1) ?x220)))
-(let ((?x215 (b_G$ (pair$ v_b_v_G_1$ ?v0))))
-(let ((?x204 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
-(let (($x1559 (= (+ ?x204 ?x215 ?x1560) 0)))
-(let (($x1547 (<= (+ (fun_app$c v_b_SP_G_1$ ?v0) (* (- 1) ?x204) (* (- 1) ?x215)) 0)))
-(let (($x1540 (<= (+ b_Infinity$ (* (- 1) ?x215)) 0)))
-(or $x1540 $x1547 $x1559)))))))))
-))
-(let (($x1535 (forall ((?v0 B_Vertex$) )(let ((?x204 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
-(let ((?x1520 (* (- 1) ?x204)))
-(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v0)))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v0)))
-(or $x125 (>= (+ ?x121 ?x1520) 0)))))))
-))
-(let (($x3200 (or $x2082 $x2087 $x202 $x1522 (not $x1535) $x3196 (not $x3010) (not $x3016) (not $x3189))))
-(let (($x3201 (not $x3200)))
-(let (($x2946 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x177 (fun_app$c v_b_SP_G_3$ ?v1)))
-(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let (($x1493 (>= (+ ?x102 ?x177 (* (- 1) (fun_app$c v_b_SP_G_3$ ?v0))) 0)))
-(let (($x1303 (<= (+ b_Infinity$ (* (- 1) ?x102)) 0)))
-(let (($x1448 (<= (+ b_Infinity$ (* (- 1) ?x177)) 0)))
-(or $x1448 $x1303 $x1493)))))))
-))
-(let (($x2954 (not (or (not $x2946) $x193))))
-(let (($x2959 (or $x2924 $x2954)))
-(let (($x2902 (forall ((?v0 B_Vertex$) )(let ((?x177 (fun_app$c v_b_SP_G_3$ ?v0)))
-(let ((?x2479 (+ ?x177 (* (- 1) (fun_app$c v_b_SP_G_3$ (?v1!9 ?v0))) (* (- 1) (b_G$ (pair$ (?v1!9 ?v0) ?v0))))))
-(let (($x2480 (= ?x2479 0)))
-(let (($x2464 (<= (+ ?x177 (* (- 1) (fun_app$c v_b_SP_G_3$ (?v1!9 ?v0)))) 0)))
-(let (($x2891 (not (or $x2464 (not $x2480)))))
-(let (($x1448 (<= (+ b_Infinity$ (* (- 1) ?x177)) 0)))
-(let (($x74 (= ?v0 b_Source$)))
-(or $x74 $x1448 $x2891)))))))))
-))
-(let (($x2968 (not (or (not $x2902) (not $x2959)))))
-(let (($x2865 (forall ((?v1 B_Vertex$) )(let ((?x1970 (fun_app$c v_b_SP_G_3$ ?v0!8)))
-(let ((?x1971 (* (- 1) ?x1970)))
-(let ((?x177 (fun_app$c v_b_SP_G_3$ ?v1)))
-(let (($x2436 (= (+ ?x177 ?x1971 (b_G$ (pair$ ?v1 ?v0!8))) 0)))
-(or (>= (+ ?x177 ?x1971) 0) (not $x2436)))))))
-))
-(let (($x2873 (not (or $x1968 $x1973 (not $x2865)))))
-(let (($x2973 (or $x2873 $x2968)))
-(let (($x2850 (forall ((?v0 B_Vertex$) )(let (($x1395 (<= (+ b_Infinity$ (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0))) 0)))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v0)))
-(or $x125 $x1395))))
-))
-(let (($x2986 (not (or (not $x2850) (not $x159) (not $x162) $x2982 (not $x167) (not $x2973)))))
-(let (($x3206 (or $x2986 $x3201)))
-(let (($x2836 (forall ((?v0 B_Vertex$) )(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v0)))
-(let ((?x2416 (+ ?x121 (* (- 1) (fun_app$c v_b_SP_G_1$ (?v1!7 ?v0))) (* (- 1) (b_G$ (pair$ (?v1!7 ?v0) ?v0))))))
-(let (($x2417 (= ?x2416 0)))
-(let (($x2401 (<= (+ ?x121 (* (- 1) (fun_app$c v_b_SP_G_1$ (?v1!7 ?v0)))) 0)))
-(let (($x2825 (not (or $x2401 (not (fun_app$ v_b_Visited_G_1$ (?v1!7 ?v0))) (not $x2417)))))
-(let (($x1395 (<= (+ b_Infinity$ (* (- 1) ?x121)) 0)))
-(let (($x74 (= ?v0 b_Source$)))
-(or $x74 $x1395 $x2825)))))))))
-))
-(let (($x2808 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v1)))
-(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let (($x1384 (>= (+ ?x102 ?x121 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0))) 0)))
-(let (($x1303 (<= (+ b_Infinity$ (* (- 1) ?x102)) 0)))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v1)))
-(let (($x126 (not $x125)))
-(or $x126 $x1303 $x1384))))))))
-))
-(let (($x2786 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v1)))
-(let (($x1367 (>= (+ ?x121 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0))) 0)))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v1)))
-(or $x125 (not (fun_app$ v_b_Visited_G_1$ ?v0)) $x1367)))))
-))
-(let (($x1363 (forall ((?v0 B_Vertex$) )(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v0)))
-(>= ?x121 0)))
-))
-(let (($x2763 (forall ((?v0 B_Vertex$) )(let ((?x75 (v_b_SP_G_0$ ?v0)))
-(let ((?x2378 (+ ?x75 (* (- 1) (v_b_SP_G_0$ (?v1!6 ?v0))) (* (- 1) (b_G$ (pair$ (?v1!6 ?v0) ?v0))))))
-(let (($x2379 (= ?x2378 0)))
-(let (($x2363 (<= (+ ?x75 (* (- 1) (v_b_SP_G_0$ (?v1!6 ?v0)))) 0)))
-(let (($x2752 (not (or $x2363 (not (v_b_Visited_G_0$ (?v1!6 ?v0))) (not $x2379)))))
-(let (($x1330 (<= (+ b_Infinity$ (* (- 1) ?x75)) 0)))
-(let (($x74 (= ?v0 b_Source$)))
-(or $x74 $x1330 $x2752)))))))))
-))
-(let (($x3219 (or (not $x2763) $x3213 (not $x1363) (not $x2786) (not $x2808) (not $x2836) (not $x3206))))
-(let (($x3220 (not $x3219)))
-(let (($x2725 (forall ((?v1 B_Vertex$) )(let ((?x1849 (v_b_SP_G_0$ ?v0!5)))
-(let ((?x1850 (* (- 1) ?x1849)))
-(let ((?x75 (v_b_SP_G_0$ ?v1)))
-(let (($x83 (v_b_Visited_G_0$ ?v1)))
-(let (($x84 (not $x83)))
-(or (>= (+ ?x75 ?x1850) 0) $x84 (not (= (+ ?x75 ?x1850 (b_G$ (pair$ ?v1 ?v0!5))) 0)))))))))
-))
-(let (($x2733 (not (or $x1847 $x1852 (not $x2725)))))
-(let (($x3225 (or $x2733 $x3220)))
-(let (($x2710 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let ((?x75 (v_b_SP_G_0$ ?v1)))
-(let (($x1316 (>= (+ ?x75 (* (- 1) (v_b_SP_G_0$ ?v0)) ?x102) 0)))
-(let (($x1303 (<= (+ b_Infinity$ (* (- 1) ?x102)) 0)))
-(let (($x83 (v_b_Visited_G_0$ ?v1)))
-(let (($x84 (not $x83)))
-(or $x84 $x1303 $x1316))))))))
-))
-(let (($x3234 (not (or (not $x2710) (not $x3225)))))
-(let (($x3239 (or $x2688 $x3234)))
-(let (($x2665 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let (($x1288 (>= (+ (v_b_SP_G_0$ ?v1) (* (- 1) (v_b_SP_G_0$ ?v0))) 0)))
-(let (($x83 (v_b_Visited_G_0$ ?v1)))
-(or $x83 (not (v_b_Visited_G_0$ ?v0)) $x1288))))
-))
-(let (($x3248 (not (or (not $x2665) (not $x3239)))))
-(let (($x3253 (or $x2642 $x3248)))
-(let (($x1280 (forall ((?v0 B_Vertex$) )(let ((?x75 (v_b_SP_G_0$ ?v0)))
-(>= ?x75 0)))
-))
-(let (($x1283 (not $x1280)))
-(let (($x3261 (not (or $x1283 (not $x3253)))))
-(let (($x1786 (not $x1785)))
-(let (($x3266 (or $x1009 $x1786 $x3261)))
-(let (($x2528 (= (+ ?x220 (* (- 1) (v_b_SP_G_2$ ?v0!20)) (b_G$ (pair$ ?0 ?v0!20))) 0)))
-(let (($x3111 (or (>= (+ ?x220 (* (- 1) (v_b_SP_G_2$ ?v0!20))) 0) $x247 (not $x2528))))
-(let ((@x3984 (monotonicity (quant-intro (refl (= $x3111 $x3111)) (= $x3122 $x3977)) (= (not $x3122) $x3982))))
-(let (($x1621 (>= (+ ?x102 ?x220 (* (- 1) ?x250)) 0)))
-(let (($x1303 (<= (+ b_Infinity$ (* (- 1) ?x102)) 0)))
-(let (($x3102 (or $x247 $x1303 $x1621)))
-(let ((@x3975 (monotonicity (quant-intro (refl (= $x3102 $x3102)) (= $x3107 $x3968)) (= (not $x3107) $x3973))))
-(let ((@x3987 (monotonicity @x3975 @x3984 (= (or (not $x3107) $x2215 $x2220 (not $x3122)) $x3985))))
-(let ((@x3996 (monotonicity (monotonicity (monotonicity @x3987 (= $x3131 $x3988)) (= $x3136 $x3991)) (= (not $x3136) $x3994))))
-(let (($x1601 (>= (+ ?x220 (* (- 1) ?x250)) 0)))
-(let (($x3057 (or $x238 (not (fun_app$ v_b_Visited_G_2$ ?1)) $x1601)))
-(let ((@x3967 (monotonicity (quant-intro (refl (= $x3057 $x3057)) (= $x3062 $x3960)) (= (not $x3062) (not $x3960)))))
-(let ((@x4002 (monotonicity (monotonicity @x3967 @x3996 (= (or (not $x3062) (not $x3136)) $x3997)) (= $x3145 $x4000))))
-(let ((@x4008 (monotonicity (monotonicity @x4002 (= $x3150 $x4003)) (= (not $x3150) $x4006))))
-(let ((@x3955 (quant-intro (refl (= (>= ?x220 0) (>= ?x220 0))) (= $x1595 $x3951))))
-(let ((@x4011 (monotonicity (monotonicity @x3955 (= $x1598 (not $x3951))) @x4008 (= (or $x1598 (not $x3150)) $x4009))))
-(let ((@x4020 (monotonicity (monotonicity (monotonicity @x4011 (= $x3158 $x4012)) (= $x3163 $x4015)) (= (not $x3163) $x4018))))
-(let ((@x3950 (monotonicity (quant-intro (refl (= $x783 $x783)) (= $x786 $x3943)) (= $x925 $x3948))))
-(let ((@x4026 (monotonicity (monotonicity @x3950 @x4020 (= (or $x925 (not $x3163)) $x4021)) (= $x3171 $x4024))))
-(let ((@x4032 (monotonicity (monotonicity @x4026 (= $x3176 $x4027)) (= (not $x3176) $x4030))))
-(let (($x1582 (>= (+ ?x121 (* (- 1) ?x220)) 0)))
-(let ((@x3941 (monotonicity (quant-intro (refl (= $x1582 $x1582)) (= $x1586 $x3934)) (= $x1589 $x3939))))
-(let ((@x4038 (monotonicity (monotonicity @x3941 @x4032 (= (or $x1589 (not $x3176)) $x4033)) (= $x3184 $x4036))))
-(let ((@x4044 (monotonicity (monotonicity @x4038 (= $x3189 $x4039)) (= (not $x3189) $x4042))))
-(let (($x1547 (<= (+ ?x121 (* (- 1) ?x204) (* (- 1) ?x215)) 0)))
-(let (($x1540 (<= (+ b_Infinity$ (* (- 1) ?x215)) 0)))
-(let (($x2991 (or $x1540 $x1547)))
-(let (($x2992 (not $x2991)))
-(let (($x3013 (or $x2992 $x225)))
-(let ((@x3933 (monotonicity (quant-intro (refl (= $x3013 $x3013)) (= $x3016 $x3926)) (= (not $x3016) $x3931))))
-(let (($x1559 (= (+ ?x204 ?x215 (* (- 1) ?x220)) 0)))
-(let (($x3005 (or $x1540 $x1547 $x1559)))
-(let ((@x3925 (monotonicity (quant-intro (refl (= $x3005 $x3005)) (= $x3010 $x3918)) (= (not $x3010) $x3923))))
-(let (($x1532 (or $x125 (>= (+ ?x121 (* (- 1) ?x204)) 0))))
-(let ((@x3915 (monotonicity (quant-intro (refl (= $x1532 $x1532)) (= $x1535 $x3908)) (= (not $x1535) $x3913))))
-(let ((@x4050 (monotonicity (monotonicity @x3915 @x3925 @x3933 @x4044 (= $x3200 $x4045)) (= $x3201 $x4048))))
-(let (($x3903 (= (or (not $x2850) (not $x159) (not $x162) $x2982 (not $x167) (not $x2973)) $x3902)))
-(let (($x1493 (>= (+ ?x102 ?x177 (* (- 1) ?x180)) 0)))
-(let (($x1448 (<= (+ b_Infinity$ (* (- 1) ?x177)) 0)))
-(let (($x2941 (or $x1448 $x1303 $x1493)))
-(let ((@x3877 (monotonicity (quant-intro (refl (= $x2941 $x2941)) (= $x2946 $x3870)) (= (not $x2946) (not $x3870)))))
-(let ((@x3883 (monotonicity (monotonicity @x3877 (= (or (not $x2946) $x193) $x3878)) (= $x2954 $x3881))))
-(let ((@x3889 (monotonicity (monotonicity @x3883 (= $x2959 $x3884)) (= (not $x2959) $x3887))))
-(let ((?x2479 (+ ?x177 (* (- 1) (fun_app$c v_b_SP_G_3$ (?v1!9 ?0))) (* (- 1) (b_G$ (pair$ (?v1!9 ?0) ?0))))))
-(let (($x2480 (= ?x2479 0)))
-(let (($x2464 (<= (+ ?x177 (* (- 1) (fun_app$c v_b_SP_G_3$ (?v1!9 ?0)))) 0)))
-(let (($x2891 (not (or $x2464 (not $x2480)))))
-(let (($x2897 (or $x74 $x1448 $x2891)))
-(let ((@x3869 (monotonicity (quant-intro (refl (= $x2897 $x2897)) (= $x2902 $x3862)) (= (not $x2902) (not $x3862)))))
-(let ((@x3895 (monotonicity (monotonicity @x3869 @x3889 (= (or (not $x2902) (not $x2959)) $x3890)) (= $x2968 $x3893))))
-(let ((?x1970 (fun_app$c v_b_SP_G_3$ ?v0!8)))
-(let ((?x1971 (* (- 1) ?x1970)))
-(let (($x2436 (= (+ ?x177 ?x1971 (b_G$ (pair$ ?0 ?v0!8))) 0)))
-(let (($x2854 (or (>= (+ ?x177 ?x1971) 0) (not $x2436))))
-(let ((@x3855 (monotonicity (quant-intro (refl (= $x2854 $x2854)) (= $x2865 $x3848)) (= (not $x2865) $x3853))))
-(let ((@x3861 (monotonicity (monotonicity @x3855 (= (or $x1968 $x1973 (not $x2865)) $x3856)) (= $x2873 $x3859))))
-(let ((@x3901 (monotonicity (monotonicity @x3861 @x3895 (= $x2973 $x3896)) (= (not $x2973) $x3899))))
-(let (($x1395 (<= (+ b_Infinity$ (* (- 1) ?x121)) 0)))
-(let (($x2839 (or $x125 $x1395)))
-(let ((@x3845 (monotonicity (quant-intro (refl (= $x2839 $x2839)) (= $x2850 $x3838)) (= (not $x2850) $x3843))))
-(let ((@x4053 (monotonicity (monotonicity (monotonicity @x3845 @x3901 $x3903) (= $x2986 $x3905)) @x4050 (= $x3206 $x4051))))
-(let ((?x2416 (+ ?x121 (* (- 1) (fun_app$c v_b_SP_G_1$ (?v1!7 ?0))) (* (- 1) (b_G$ (pair$ (?v1!7 ?0) ?0))))))
-(let (($x2417 (= ?x2416 0)))
-(let (($x2401 (<= (+ ?x121 (* (- 1) (fun_app$c v_b_SP_G_1$ (?v1!7 ?0)))) 0)))
-(let (($x2825 (not (or $x2401 (not (fun_app$ v_b_Visited_G_1$ (?v1!7 ?0))) (not $x2417)))))
-(let (($x2831 (or $x74 $x1395 $x2825)))
-(let ((@x3836 (monotonicity (quant-intro (refl (= $x2831 $x2831)) (= $x2836 $x3829)) (= (not $x2836) $x3834))))
-(let (($x1384 (>= (+ ?x102 ?x121 (* (- 1) ?x129)) 0)))
-(let (($x2803 (or $x126 $x1303 $x1384)))
-(let ((@x3828 (monotonicity (quant-intro (refl (= $x2803 $x2803)) (= $x2808 $x3821)) (= (not $x2808) $x3826))))
-(let (($x1367 (>= (+ ?x121 (* (- 1) ?x129)) 0)))
-(let (($x2781 (or $x125 (not $x127) $x1367)))
-(let ((@x3820 (monotonicity (quant-intro (refl (= $x2781 $x2781)) (= $x2786 $x3813)) (= (not $x2786) $x3818))))
-(let ((@x3808 (quant-intro (refl (= (>= ?x121 0) (>= ?x121 0))) (= $x1363 $x3804))))
-(let ((?x2378 (+ ?x75 (* (- 1) (v_b_SP_G_0$ (?v1!6 ?0))) (* (- 1) (b_G$ (pair$ (?v1!6 ?0) ?0))))))
-(let (($x2379 (= ?x2378 0)))
-(let (($x2363 (<= (+ ?x75 (* (- 1) (v_b_SP_G_0$ (?v1!6 ?0)))) 0)))
-(let (($x2752 (not (or $x2363 (not (v_b_Visited_G_0$ (?v1!6 ?0))) (not $x2379)))))
-(let (($x1330 (<= (+ b_Infinity$ (* (- 1) ?x75)) 0)))
-(let (($x2758 (or $x74 $x1330 $x2752)))
-(let ((@x3802 (monotonicity (quant-intro (refl (= $x2758 $x2758)) (= $x2763 $x3795)) (= (not $x2763) (not $x3795)))))
-(let ((@x4059 (monotonicity @x3802 (monotonicity @x3808 (= (not $x1363) $x3809)) @x3820 @x3828 @x3836 (monotonicity @x4053 (= (not $x3206) $x4054)) (= $x3219 $x4057))))
-(let (($x1862 (= (+ ?x75 (* (- 1) (v_b_SP_G_0$ ?v0!5)) (b_G$ (pair$ ?0 ?v0!5))) 0)))
-(let (($x2714 (or (>= (+ ?x75 (* (- 1) (v_b_SP_G_0$ ?v0!5))) 0) $x84 (not $x1862))))
-(let ((@x3788 (monotonicity (quant-intro (refl (= $x2714 $x2714)) (= $x2725 $x3781)) (= (not $x2725) (not $x3781)))))
-(let ((@x3794 (monotonicity (monotonicity @x3788 (= (or $x1847 $x1852 (not $x2725)) $x3789)) (= $x2733 $x3792))))
-(let ((@x4065 (monotonicity @x3794 (monotonicity @x4059 (= $x3220 $x4060)) (= $x3225 $x4063))))
-(let (($x1316 (>= (+ ?x75 (* (- 1) ?x97) ?x102) 0)))
-(let (($x2705 (or $x84 $x1303 $x1316)))
-(let ((@x3779 (monotonicity (quant-intro (refl (= $x2705 $x2705)) (= $x2710 $x3772)) (= (not $x2710) (not $x3772)))))
-(let ((@x4071 (monotonicity @x3779 (monotonicity @x4065 (= (not $x3225) $x4066)) (= (or (not $x2710) (not $x3225)) $x4069))))
-(let ((@x4080 (monotonicity (monotonicity (monotonicity @x4071 (= $x3234 $x4072)) (= $x3239 $x4075)) (= (not $x3239) $x4078))))
-(let (($x1288 (>= (+ ?x75 (* (- 1) ?x97)) 0)))
-(let (($x2660 (or $x83 (not $x95) $x1288)))
-(let ((@x3770 (monotonicity (quant-intro (refl (= $x2660 $x2660)) (= $x2665 $x3763)) (= (not $x2665) (not $x3763)))))
-(let ((@x4086 (monotonicity (monotonicity @x3770 @x4080 (= (or (not $x2665) (not $x3239)) $x4081)) (= $x3248 $x4084))))
-(let ((@x4092 (monotonicity (monotonicity @x4086 (= $x3253 $x4087)) (= (not $x3253) $x4090))))
-(let ((@x3758 (quant-intro (refl (= (>= ?x75 0) (>= ?x75 0))) (= $x1280 $x3754))))
-(let ((@x4095 (monotonicity (monotonicity @x3758 (= $x1283 (not $x3754))) @x4092 (= (or $x1283 (not $x3253)) $x4093))))
-(let ((@x4101 (monotonicity (monotonicity @x4095 (= $x3261 $x4096)) (= $x3266 (or $x1009 $x1786 $x4096)))))
-(let (($x2537 (forall ((?v1 B_Vertex$) )(let ((?x2217 (v_b_SP_G_2$ ?v0!20)))
-(let ((?x2218 (* (- 1) ?x2217)))
-(let ((?x220 (v_b_SP_G_2$ ?v1)))
-(let (($x2528 (= (+ ?x220 ?x2218 (b_G$ (pair$ ?v1 ?v0!20))) 0)))
-(let (($x238 (fun_app$ v_b_Visited_G_2$ ?v1)))
-(let (($x2531 (and (not (>= (+ ?x220 ?x2218) 0)) $x238 $x2528)))
-(not $x2531))))))))
-))
-(let (($x2221 (not $x2220)))
-(let (($x2216 (not $x2215)))
-(let (($x1628 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x220 (v_b_SP_G_2$ ?v1)))
-(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let (($x1621 (>= (+ ?x102 ?x220 (* (- 1) (v_b_SP_G_2$ ?v0))) 0)))
-(let (($x1303 (<= (+ b_Infinity$ (* (- 1) ?x102)) 0)))
-(let (($x1306 (not $x1303)))
-(let (($x238 (fun_app$ v_b_Visited_G_2$ ?v1)))
-(let (($x1615 (and $x238 $x1306)))
-(let (($x1618 (not $x1615)))
-(or $x1618 $x1621))))))))))
-))
-(let (($x2546 (and $x1628 $x2216 $x2221 $x2537)))
-(let (($x2197 (not (and $x2189 (not $x2194)))))
-(let (($x2203 (or $x2197 $x2202)))
-(let (($x2204 (not $x2203)))
-(let (($x2551 (or $x2204 $x2546)))
-(let (($x1609 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let (($x1601 (>= (+ (v_b_SP_G_2$ ?v1) (* (- 1) (v_b_SP_G_2$ ?v0))) 0)))
-(let (($x238 (fun_app$ v_b_Visited_G_2$ ?v1)))
-(let (($x247 (not $x238)))
-(let (($x249 (and $x247 (fun_app$ v_b_Visited_G_2$ ?v0))))
-(let (($x798 (not $x249)))
-(or $x798 $x1601)))))))
-))
-(let (($x2554 (and $x1609 $x2551)))
-(let (($x2170 (not (and (not $x2166) $x2168))))
-(let (($x2176 (or $x2170 $x2175)))
-(let (($x2177 (not $x2176)))
-(let (($x2557 (or $x2177 $x2554)))
-(let (($x2560 (and $x1595 $x2557)))
-(let (($x2563 (or $x913 $x2154 $x2560)))
-(let (($x2566 (and $x786 $x2563)))
-(let (($x2569 (or $x2139 $x2566)))
-(let (($x2572 (and $x1586 $x2569)))
-(let (($x2575 (or $x2122 $x2572)))
-(let (($x1573 (forall ((?v0 B_Vertex$) )(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v0)))
-(let ((?x220 (v_b_SP_G_2$ ?v0)))
-(let (($x225 (= ?x220 ?x121)))
-(let ((?x204 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
-(let ((?x1520 (* (- 1) ?x204)))
-(let (($x1547 (<= (+ ?x121 ?x1520 (* (- 1) (b_G$ (pair$ v_b_v_G_1$ ?v0)))) 0)))
-(let (($x1540 (<= (+ b_Infinity$ (* (- 1) (b_G$ (pair$ v_b_v_G_1$ ?v0)))) 0)))
-(let (($x1553 (and (not $x1540) (not $x1547))))
-(or $x1553 $x225))))))))))
-))
-(let (($x1567 (forall ((?v0 B_Vertex$) )(let ((?x220 (v_b_SP_G_2$ ?v0)))
-(let ((?x1560 (* (- 1) ?x220)))
-(let ((?x215 (b_G$ (pair$ v_b_v_G_1$ ?v0))))
-(let ((?x204 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
-(let (($x1559 (= (+ ?x204 ?x215 ?x1560) 0)))
-(let (($x1547 (<= (+ (fun_app$c v_b_SP_G_1$ ?v0) (* (- 1) ?x204) (* (- 1) ?x215)) 0)))
-(let (($x1553 (and (not (<= (+ b_Infinity$ (* (- 1) ?x215)) 0)) (not $x1547))))
-(let (($x1556 (not $x1553)))
-(or $x1556 $x1559))))))))))
-))
-(let (($x1525 (not $x1522)))
-(let (($x2088 (not $x2087)))
-(let (($x2083 (not $x2082)))
-(let (($x2581 (and $x2083 $x2088 $x203 $x1525 $x1535 $x213 $x1567 $x1573 $x2575)))
-(let (($x2058 (not $x193)))
-(let (($x1499 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x177 (fun_app$c v_b_SP_G_3$ ?v1)))
-(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let (($x1493 (>= (+ ?x102 ?x177 (* (- 1) (fun_app$c v_b_SP_G_3$ ?v0))) 0)))
-(let (($x1303 (<= (+ b_Infinity$ (* (- 1) ?x102)) 0)))
-(let (($x1306 (not $x1303)))
-(let (($x1448 (<= (+ b_Infinity$ (* (- 1) ?x177)) 0)))
-(let (($x1451 (not $x1448)))
-(let (($x1487 (and $x1451 $x1306)))
-(let (($x1490 (not $x1487)))
-(or $x1490 $x1493)))))))))))
-))
-(let (($x2061 (and $x1499 $x2058)))
-(let (($x2042 (not (and $x2034 (not $x2039)))))
-(let (($x2500 (or $x2042 $x2497)))
-(let (($x2503 (not $x2500)))
-(let (($x2506 (or $x2503 $x2061)))
-(let (($x2491 (forall ((?v0 B_Vertex$) )(let ((?x177 (fun_app$c v_b_SP_G_3$ ?v0)))
-(let ((?x2479 (+ ?x177 (* (- 1) (fun_app$c v_b_SP_G_3$ (?v1!9 ?v0))) (* (- 1) (b_G$ (pair$ (?v1!9 ?v0) ?v0))))))
-(let (($x2480 (= ?x2479 0)))
-(let (($x2464 (<= (+ ?x177 (* (- 1) (fun_app$c v_b_SP_G_3$ (?v1!9 ?v0)))) 0)))
-(let (($x2485 (and (not $x2464) $x2480)))
-(let (($x1448 (<= (+ b_Infinity$ (* (- 1) ?x177)) 0)))
-(let (($x1451 (not $x1448)))
-(let (($x74 (= ?v0 b_Source$)))
-(let (($x79 (not $x74)))
-(let (($x1454 (and $x79 $x1451)))
-(let (($x1457 (not $x1454)))
-(or $x1457 $x2485)))))))))))))
-))
-(let (($x2509 (and $x2491 $x2506)))
-(let (($x2445 (forall ((?v1 B_Vertex$) )(let ((?x1970 (fun_app$c v_b_SP_G_3$ ?v0!8)))
-(let ((?x1971 (* (- 1) ?x1970)))
-(let ((?x177 (fun_app$c v_b_SP_G_3$ ?v1)))
-(let (($x2436 (= (+ ?x177 ?x1971 (b_G$ (pair$ ?v1 ?v0!8))) 0)))
-(let (($x2439 (and (not (>= (+ ?x177 ?x1971) 0)) $x2436)))
-(not $x2439)))))))
-))
-(let (($x1974 (not $x1973)))
-(let (($x1969 (not $x1968)))
-(let (($x2451 (and $x1969 $x1974 $x2445)))
-(let (($x2512 (or $x2451 $x2509)))
-(let (($x1950 (forall ((?v0 B_Vertex$) )(let (($x1395 (<= (+ b_Infinity$ (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0))) 0)))
-(let (($x1398 (not $x1395)))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v0)))
-(let (($x126 (not $x125)))
-(let (($x1431 (and $x126 $x1398)))
-(not $x1431)))))))
-))
-(let (($x2518 (and $x1950 $x159 $x162 $x164 $x167 $x2512)))
-(let (($x2586 (or $x2518 $x2581)))
-(let (($x2428 (forall ((?v0 B_Vertex$) )(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v0)))
-(let ((?x2416 (+ ?x121 (* (- 1) (fun_app$c v_b_SP_G_1$ (?v1!7 ?v0))) (* (- 1) (b_G$ (pair$ (?v1!7 ?v0) ?v0))))))
-(let (($x2417 (= ?x2416 0)))
-(let ((?x1922 (?v1!7 ?v0)))
-(let (($x1927 (fun_app$ v_b_Visited_G_1$ ?x1922)))
-(let (($x2422 (and (not (<= (+ ?x121 (* (- 1) (fun_app$c v_b_SP_G_1$ ?x1922))) 0)) $x1927 $x2417)))
-(let (($x1395 (<= (+ b_Infinity$ (* (- 1) ?x121)) 0)))
-(let (($x1398 (not $x1395)))
-(let (($x74 (= ?v0 b_Source$)))
-(let (($x79 (not $x74)))
-(let (($x1401 (and $x79 $x1398)))
-(let (($x1404 (not $x1401)))
-(or $x1404 $x2422))))))))))))))
-))
-(let (($x1390 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v1)))
-(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let (($x1384 (>= (+ ?x102 ?x121 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0))) 0)))
-(let (($x1303 (<= (+ b_Infinity$ (* (- 1) ?x102)) 0)))
-(let (($x1306 (not $x1303)))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v1)))
-(let (($x1377 (and $x125 $x1306)))
-(let (($x1380 (not $x1377)))
-(or $x1380 $x1384))))))))))
-))
-(let (($x1374 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v1)))
-(let (($x1367 (>= (+ ?x121 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0))) 0)))
-(let (($x127 (fun_app$ v_b_Visited_G_1$ ?v0)))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v1)))
-(let (($x126 (not $x125)))
-(let (($x128 (and $x126 $x127)))
-(let (($x429 (not $x128)))
-(or $x429 $x1367)))))))))
-))
-(let (($x2390 (forall ((?v0 B_Vertex$) )(let ((?x75 (v_b_SP_G_0$ ?v0)))
-(let ((?x2378 (+ ?x75 (* (- 1) (v_b_SP_G_0$ (?v1!6 ?v0))) (* (- 1) (b_G$ (pair$ (?v1!6 ?v0) ?v0))))))
-(let (($x2379 (= ?x2378 0)))
-(let ((?x1887 (?v1!6 ?v0)))
-(let (($x1892 (v_b_Visited_G_0$ ?x1887)))
-(let (($x2384 (and (not (<= (+ ?x75 (* (- 1) (v_b_SP_G_0$ ?x1887))) 0)) $x1892 $x2379)))
-(let (($x74 (= ?v0 b_Source$)))
-(let (($x79 (not $x74)))
-(let (($x1336 (and $x79 (not (<= (+ b_Infinity$ (* (- 1) ?x75)) 0)))))
-(let (($x1339 (not $x1336)))
-(or $x1339 $x2384))))))))))))
-))
-(let (($x2595 (and $x2390 $x120 $x1363 $x1374 $x1390 $x2428 $x2586)))
-(let (($x1876 (forall ((?v1 B_Vertex$) )(let ((?x1849 (v_b_SP_G_0$ ?v0!5)))
-(let ((?x1850 (* (- 1) ?x1849)))
-(let ((?x75 (v_b_SP_G_0$ ?v1)))
-(let (($x83 (v_b_Visited_G_0$ ?v1)))
-(let (($x1863 (and (not (>= (+ ?x75 ?x1850) 0)) $x83 (= (+ ?x75 ?x1850 (b_G$ (pair$ ?v1 ?v0!5))) 0))))
-(not $x1863)))))))
-))
-(let (($x1853 (not $x1852)))
-(let (($x1848 (not $x1847)))
-(let (($x2350 (and $x1848 $x1853 $x1876)))
-(let (($x2600 (or $x2350 $x2595)))
-(let (($x1322 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let ((?x75 (v_b_SP_G_0$ ?v1)))
-(let (($x1316 (>= (+ ?x75 (* (- 1) (v_b_SP_G_0$ ?v0)) ?x102) 0)))
-(let (($x1303 (<= (+ b_Infinity$ (* (- 1) ?x102)) 0)))
-(let (($x1306 (not $x1303)))
-(let (($x83 (v_b_Visited_G_0$ ?v1)))
-(let (($x1309 (and $x83 $x1306)))
-(let (($x1312 (not $x1309)))
-(or $x1312 $x1316))))))))))
-))
-(let (($x2603 (and $x1322 $x2600)))
-(let (($x1829 (not (and $x1821 (not $x1826)))))
-(let (($x2339 (or $x1829 $x2336)))
-(let (($x2342 (not $x2339)))
-(let (($x2606 (or $x2342 $x2603)))
-(let (($x1295 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let (($x1288 (>= (+ (v_b_SP_G_0$ ?v1) (* (- 1) (v_b_SP_G_0$ ?v0))) 0)))
-(let (($x95 (v_b_Visited_G_0$ ?v0)))
-(let (($x83 (v_b_Visited_G_0$ ?v1)))
-(let (($x84 (not $x83)))
-(let (($x96 (and $x84 $x95)))
-(let (($x370 (not $x96)))
-(or $x370 $x1288))))))))
-))
-(let (($x2609 (and $x1295 $x2606)))
-(let (($x1802 (not (and (not $x1798) $x1800))))
-(let (($x1808 (or $x1802 $x1807)))
-(let (($x1809 (not $x1808)))
-(let (($x2612 (or $x1809 $x2609)))
-(let (($x2615 (and $x1280 $x2612)))
-(let (($x2618 (or $x1009 $x1786 $x2615)))
-(let ((@x3203 (rewrite (= (and $x2083 $x2088 $x203 $x1525 $x1535 $x213 $x3010 $x3016 $x3189) $x3201))))
-(let (($x2531 (and (not (>= (+ ?x220 (* (- 1) (v_b_SP_G_2$ ?v0!20))) 0)) $x238 $x2528)))
-(let (($x2534 (not $x2531)))
-(let ((@x3117 (monotonicity (rewrite (= $x2531 (not $x3111))) (= $x2534 (not (not $x3111))))))
-(let ((@x3124 (quant-intro (trans @x3117 (rewrite (= (not (not $x3111)) $x3111)) (= $x2534 $x3111)) (= $x2537 $x3122))))
-(let (($x1306 (not $x1303)))
-(let (($x1615 (and $x238 $x1306)))
-(let (($x1618 (not $x1615)))
-(let (($x1625 (or $x1618 $x1621)))
-(let ((@x3094 (monotonicity (rewrite (= $x1615 (not (or $x247 $x1303)))) (= $x1618 (not (not (or $x247 $x1303)))))))
-(let ((@x3098 (trans @x3094 (rewrite (= (not (not (or $x247 $x1303))) (or $x247 $x1303))) (= $x1618 (or $x247 $x1303)))))
-(let ((@x3106 (trans (monotonicity @x3098 (= $x1625 (or (or $x247 $x1303) $x1621))) (rewrite (= (or (or $x247 $x1303) $x1621) $x3102)) (= $x1625 $x3102))))
-(let ((@x3127 (monotonicity (quant-intro @x3106 (= $x1628 $x3107)) @x3124 (= $x2546 (and $x3107 $x2216 $x2221 $x3122)))))
-(let ((@x3135 (trans @x3127 (rewrite (= (and $x3107 $x2216 $x2221 $x3122) $x3131)) (= $x2546 $x3131))))
-(let ((@x3072 (monotonicity (rewrite (= (and $x2189 (not $x2194)) (not (or $x3065 $x2194)))) (= $x2197 (not (not (or $x3065 $x2194)))))))
-(let ((@x3076 (trans @x3072 (rewrite (= (not (not (or $x3065 $x2194))) (or $x3065 $x2194))) (= $x2197 (or $x3065 $x2194)))))
-(let ((@x3084 (trans (monotonicity @x3076 (= $x2203 (or (or $x3065 $x2194) $x2202))) (rewrite (= (or (or $x3065 $x2194) $x2202) $x3080)) (= $x2203 $x3080))))
-(let ((@x3138 (monotonicity (monotonicity @x3084 (= $x2204 $x3085)) @x3135 (= $x2551 $x3136))))
-(let (($x3058 (= (or (or $x238 (not (fun_app$ v_b_Visited_G_2$ ?1))) $x1601) $x3057)))
-(let (($x1606 (or $x798 $x1601)))
-(let (($x3055 (= $x1606 (or (or $x238 (not (fun_app$ v_b_Visited_G_2$ ?1))) $x1601))))
-(let (($x3043 (or $x238 (not (fun_app$ v_b_Visited_G_2$ ?1)))))
-(let ((@x3049 (monotonicity (rewrite (= $x249 (not $x3043))) (= $x798 (not (not $x3043))))))
-(let ((@x3056 (monotonicity (trans @x3049 (rewrite (= (not (not $x3043)) $x3043)) (= $x798 $x3043)) $x3055)))
-(let ((@x3064 (quant-intro (trans @x3056 (rewrite $x3058) (= $x1606 $x3057)) (= $x1609 $x3062))))
-(let ((@x3149 (trans (monotonicity @x3064 @x3138 (= $x2554 (and $x3062 $x3136))) (rewrite (= (and $x3062 $x3136) $x3145)) (= $x2554 $x3145))))
-(let ((@x3026 (monotonicity (rewrite (= (and (not $x2166) $x2168) (not (or $x2166 $x3019)))) (= $x2170 (not (not (or $x2166 $x3019)))))))
-(let ((@x3030 (trans @x3026 (rewrite (= (not (not (or $x2166 $x3019))) (or $x2166 $x3019))) (= $x2170 (or $x2166 $x3019)))))
-(let ((@x3038 (trans (monotonicity @x3030 (= $x2176 (or (or $x2166 $x3019) $x2175))) (rewrite (= (or (or $x2166 $x3019) $x2175) $x3034)) (= $x2176 $x3034))))
-(let ((@x3152 (monotonicity (monotonicity @x3038 (= $x2177 $x3039)) @x3149 (= $x2557 $x3150))))
-(let ((@x3162 (trans (monotonicity @x3152 (= $x2560 (and $x1595 $x3150))) (rewrite (= (and $x1595 $x3150) $x3158)) (= $x2560 $x3158))))
-(let ((@x3168 (monotonicity (monotonicity @x3162 (= $x2563 $x3163)) (= $x2566 (and $x786 $x3163)))))
-(let ((@x3178 (monotonicity (trans @x3168 (rewrite (= (and $x786 $x3163) $x3171)) (= $x2566 $x3171)) (= $x2569 $x3176))))
-(let ((@x3188 (trans (monotonicity @x3178 (= $x2572 (and $x1586 $x3176))) (rewrite (= (and $x1586 $x3176) $x3184)) (= $x2572 $x3184))))
-(let ((@x3015 (monotonicity (rewrite (= (and (not $x1540) (not $x1547)) $x2992)) (= (or (and (not $x1540) (not $x1547)) $x225) $x3013))))
-(let ((@x2997 (monotonicity (rewrite (= (and (not $x1540) (not $x1547)) $x2992)) (= (not (and (not $x1540) (not $x1547))) (not $x2992)))))
-(let ((@x3001 (trans @x2997 (rewrite (= (not $x2992) $x2991)) (= (not (and (not $x1540) (not $x1547))) $x2991))))
-(let ((@x3004 (monotonicity @x3001 (= (or (not (and (not $x1540) (not $x1547))) $x1559) (or $x2991 $x1559)))))
-(let ((@x3009 (trans @x3004 (rewrite (= (or $x2991 $x1559) $x3005)) (= (or (not (and (not $x1540) (not $x1547))) $x1559) $x3005))))
-(let ((@x3194 (monotonicity (quant-intro @x3009 (= $x1567 $x3010)) (quant-intro @x3015 (= $x1573 $x3016)) (monotonicity @x3188 (= $x2575 $x3189)) (= $x2581 (and $x2083 $x2088 $x203 $x1525 $x1535 $x213 $x3010 $x3016 $x3189)))))
-(let (($x1451 (not $x1448)))
-(let (($x1487 (and $x1451 $x1306)))
-(let (($x1490 (not $x1487)))
-(let (($x1496 (or $x1490 $x1493)))
-(let ((@x2933 (monotonicity (rewrite (= $x1487 (not (or $x1448 $x1303)))) (= $x1490 (not (not (or $x1448 $x1303)))))))
-(let ((@x2937 (trans @x2933 (rewrite (= (not (not (or $x1448 $x1303))) (or $x1448 $x1303))) (= $x1490 (or $x1448 $x1303)))))
-(let ((@x2945 (trans (monotonicity @x2937 (= $x1496 (or (or $x1448 $x1303) $x1493))) (rewrite (= (or (or $x1448 $x1303) $x1493) $x2941)) (= $x1496 $x2941))))
-(let ((@x2951 (monotonicity (quant-intro @x2945 (= $x1499 $x2946)) (= $x2061 (and $x2946 $x2058)))))
-(let ((@x2911 (monotonicity (rewrite (= (and $x2034 (not $x2039)) (not (or $x2033 $x2039)))) (= $x2042 (not (not (or $x2033 $x2039)))))))
-(let ((@x2915 (trans @x2911 (rewrite (= (not (not (or $x2033 $x2039))) (or $x2033 $x2039))) (= $x2042 (or $x2033 $x2039)))))
-(let ((@x2923 (trans (monotonicity @x2915 (= $x2500 (or (or $x2033 $x2039) $x2497))) (rewrite (= (or (or $x2033 $x2039) $x2497) $x2919)) (= $x2500 $x2919))))
-(let ((@x2961 (monotonicity (monotonicity @x2923 (= $x2503 $x2924)) (trans @x2951 (rewrite (= (and $x2946 $x2058) $x2954)) (= $x2061 $x2954)) (= $x2506 $x2959))))
-(let (($x2485 (and (not $x2464) $x2480)))
-(let (($x1454 (and $x79 $x1451)))
-(let (($x1457 (not $x1454)))
-(let (($x2488 (or $x1457 $x2485)))
-(let ((@x2884 (monotonicity (rewrite (= $x1454 (not (or $x74 $x1448)))) (= $x1457 (not (not (or $x74 $x1448)))))))
-(let ((@x2888 (trans @x2884 (rewrite (= (not (not (or $x74 $x1448))) (or $x74 $x1448))) (= $x1457 (or $x74 $x1448)))))
-(let ((@x2896 (monotonicity @x2888 (rewrite (= $x2485 $x2891)) (= $x2488 (or (or $x74 $x1448) $x2891)))))
-(let ((@x2901 (trans @x2896 (rewrite (= (or (or $x74 $x1448) $x2891) $x2897)) (= $x2488 $x2897))))
-(let ((@x2964 (monotonicity (quant-intro @x2901 (= $x2491 $x2902)) @x2961 (= $x2509 (and $x2902 $x2959)))))
-(let (($x2439 (and (not (>= (+ ?x177 ?x1971) 0)) $x2436)))
-(let (($x2442 (not $x2439)))
-(let ((@x2860 (monotonicity (rewrite (= $x2439 (not $x2854))) (= $x2442 (not (not $x2854))))))
-(let ((@x2867 (quant-intro (trans @x2860 (rewrite (= (not (not $x2854)) $x2854)) (= $x2442 $x2854)) (= $x2445 $x2865))))
-(let ((@x2877 (trans (monotonicity @x2867 (= $x2451 (and $x1969 $x1974 $x2865))) (rewrite (= (and $x1969 $x1974 $x2865) $x2873)) (= $x2451 $x2873))))
-(let ((@x2975 (monotonicity @x2877 (trans @x2964 (rewrite (= (and $x2902 $x2959) $x2968)) (= $x2509 $x2968)) (= $x2512 $x2973))))
-(let ((@x2845 (monotonicity (rewrite (= (and $x126 (not $x1395)) (not $x2839))) (= (not (and $x126 (not $x1395))) (not (not $x2839))))))
-(let ((@x2849 (trans @x2845 (rewrite (= (not (not $x2839)) $x2839)) (= (not (and $x126 (not $x1395))) $x2839))))
-(let ((@x2978 (monotonicity (quant-intro @x2849 (= $x1950 $x2850)) @x2975 (= $x2518 (and $x2850 $x159 $x162 $x164 $x167 $x2973)))))
-(let ((@x2990 (trans @x2978 (rewrite (= (and $x2850 $x159 $x162 $x164 $x167 $x2973) $x2986)) (= $x2518 $x2986))))
-(let ((?x1922 (?v1!7 ?0)))
-(let (($x1927 (fun_app$ v_b_Visited_G_1$ ?x1922)))
-(let (($x2422 (and (not $x2401) $x1927 $x2417)))
-(let (($x1398 (not $x1395)))
-(let (($x1401 (and $x79 $x1398)))
-(let (($x1404 (not $x1401)))
-(let (($x2425 (or $x1404 $x2422)))
-(let ((@x2817 (monotonicity (rewrite (= $x1401 (not (or $x74 $x1395)))) (= $x1404 (not (not (or $x74 $x1395)))))))
-(let ((@x2821 (trans @x2817 (rewrite (= (not (not (or $x74 $x1395))) (or $x74 $x1395))) (= $x1404 (or $x74 $x1395)))))
-(let ((@x2830 (monotonicity @x2821 (rewrite (= $x2422 $x2825)) (= $x2425 (or (or $x74 $x1395) $x2825)))))
-(let ((@x2835 (trans @x2830 (rewrite (= (or (or $x74 $x1395) $x2825) $x2831)) (= $x2425 $x2831))))
-(let ((@x2795 (monotonicity (rewrite (= (and $x125 $x1306) (not (or $x126 $x1303)))) (= (not (and $x125 $x1306)) (not (not (or $x126 $x1303)))))))
-(let ((@x2799 (trans @x2795 (rewrite (= (not (not (or $x126 $x1303))) (or $x126 $x1303))) (= (not (and $x125 $x1306)) (or $x126 $x1303)))))
-(let ((@x2802 (monotonicity @x2799 (= (or (not (and $x125 $x1306)) $x1384) (or (or $x126 $x1303) $x1384)))))
-(let ((@x2807 (trans @x2802 (rewrite (= (or (or $x126 $x1303) $x1384) $x2803)) (= (or (not (and $x125 $x1306)) $x1384) $x2803))))
-(let ((@x2775 (rewrite (= (not (not (or $x125 (not $x127)))) (or $x125 (not $x127))))))
-(let ((@x2773 (monotonicity (rewrite (= $x128 (not (or $x125 (not $x127))))) (= $x429 (not (not (or $x125 (not $x127))))))))
-(let ((@x2780 (monotonicity (trans @x2773 @x2775 (= $x429 (or $x125 (not $x127)))) (= (or $x429 $x1367) (or (or $x125 (not $x127)) $x1367)))))
-(let ((@x2785 (trans @x2780 (rewrite (= (or (or $x125 (not $x127)) $x1367) $x2781)) (= (or $x429 $x1367) $x2781))))
-(let ((?x1887 (?v1!6 ?0)))
-(let (($x1892 (v_b_Visited_G_0$ ?x1887)))
-(let (($x2384 (and (not $x2363) $x1892 $x2379)))
-(let (($x1336 (and $x79 (not $x1330))))
-(let (($x1339 (not $x1336)))
-(let (($x2387 (or $x1339 $x2384)))
-(let ((@x2744 (monotonicity (rewrite (= $x1336 (not (or $x74 $x1330)))) (= $x1339 (not (not (or $x74 $x1330)))))))
-(let ((@x2748 (trans @x2744 (rewrite (= (not (not (or $x74 $x1330))) (or $x74 $x1330))) (= $x1339 (or $x74 $x1330)))))
-(let ((@x2757 (monotonicity @x2748 (rewrite (= $x2384 $x2752)) (= $x2387 (or (or $x74 $x1330) $x2752)))))
-(let ((@x2762 (trans @x2757 (rewrite (= (or (or $x74 $x1330) $x2752) $x2758)) (= $x2387 $x2758))))
-(let ((@x3211 (monotonicity (quant-intro @x2762 (= $x2390 $x2763)) (quant-intro @x2785 (= $x1374 $x2786)) (quant-intro @x2807 (= $x1390 $x2808)) (quant-intro @x2835 (= $x2428 $x2836)) (monotonicity @x2990 (trans @x3194 @x3203 (= $x2581 $x3201)) (= $x2586 $x3206)) (= $x2595 (and $x2763 $x120 $x1363 $x2786 $x2808 $x2836 $x3206)))))
-(let ((@x3224 (trans @x3211 (rewrite (= (and $x2763 $x120 $x1363 $x2786 $x2808 $x2836 $x3206) $x3220)) (= $x2595 $x3220))))
-(let (($x1863 (and (not (>= (+ ?x75 (* (- 1) (v_b_SP_G_0$ ?v0!5))) 0)) $x83 $x1862)))
-(let (($x1873 (not $x1863)))
-(let ((@x2720 (monotonicity (rewrite (= $x1863 (not $x2714))) (= $x1873 (not (not $x2714))))))
-(let ((@x2727 (quant-intro (trans @x2720 (rewrite (= (not (not $x2714)) $x2714)) (= $x1873 $x2714)) (= $x1876 $x2725))))
-(let ((@x2737 (trans (monotonicity @x2727 (= $x2350 (and $x1848 $x1853 $x2725))) (rewrite (= (and $x1848 $x1853 $x2725) $x2733)) (= $x2350 $x2733))))
-(let ((@x2697 (monotonicity (rewrite (= (and $x83 $x1306) (not (or $x84 $x1303)))) (= (not (and $x83 $x1306)) (not (not (or $x84 $x1303)))))))
-(let ((@x2701 (trans @x2697 (rewrite (= (not (not (or $x84 $x1303))) (or $x84 $x1303))) (= (not (and $x83 $x1306)) (or $x84 $x1303)))))
-(let ((@x2704 (monotonicity @x2701 (= (or (not (and $x83 $x1306)) $x1316) (or (or $x84 $x1303) $x1316)))))
-(let ((@x2709 (trans @x2704 (rewrite (= (or (or $x84 $x1303) $x1316) $x2705)) (= (or (not (and $x83 $x1306)) $x1316) $x2705))))
-(let ((@x3230 (monotonicity (quant-intro @x2709 (= $x1322 $x2710)) (monotonicity @x2737 @x3224 (= $x2600 $x3225)) (= $x2603 (and $x2710 $x3225)))))
-(let ((@x2675 (monotonicity (rewrite (= (and $x1821 (not $x1826)) (not (or $x2668 $x1826)))) (= $x1829 (not (not (or $x2668 $x1826)))))))
-(let ((@x2679 (trans @x2675 (rewrite (= (not (not (or $x2668 $x1826))) (or $x2668 $x1826))) (= $x1829 (or $x2668 $x1826)))))
-(let ((@x2687 (trans (monotonicity @x2679 (= $x2339 (or (or $x2668 $x1826) $x2336))) (rewrite (= (or (or $x2668 $x1826) $x2336) $x2683)) (= $x2339 $x2683))))
-(let ((@x3241 (monotonicity (monotonicity @x2687 (= $x2342 $x2688)) (trans @x3230 (rewrite (= (and $x2710 $x3225) $x3234)) (= $x2603 $x3234)) (= $x2606 $x3239))))
-(let ((@x2654 (rewrite (= (not (not (or $x83 (not $x95)))) (or $x83 (not $x95))))))
-(let ((@x2652 (monotonicity (rewrite (= $x96 (not (or $x83 (not $x95))))) (= $x370 (not (not (or $x83 (not $x95))))))))
-(let ((@x2659 (monotonicity (trans @x2652 @x2654 (= $x370 (or $x83 (not $x95)))) (= (or $x370 $x1288) (or (or $x83 (not $x95)) $x1288)))))
-(let ((@x2664 (trans @x2659 (rewrite (= (or (or $x83 (not $x95)) $x1288) $x2660)) (= (or $x370 $x1288) $x2660))))
-(let ((@x3244 (monotonicity (quant-intro @x2664 (= $x1295 $x2665)) @x3241 (= $x2609 (and $x2665 $x3239)))))
-(let ((@x2629 (monotonicity (rewrite (= (and (not $x1798) $x1800) (not (or $x1798 $x2622)))) (= $x1802 (not (not (or $x1798 $x2622)))))))
-(let ((@x2633 (trans @x2629 (rewrite (= (not (not (or $x1798 $x2622))) (or $x1798 $x2622))) (= $x1802 (or $x1798 $x2622)))))
-(let ((@x2641 (trans (monotonicity @x2633 (= $x1808 (or (or $x1798 $x2622) $x1807))) (rewrite (= (or (or $x1798 $x2622) $x1807) $x2637)) (= $x1808 $x2637))))
-(let ((@x3255 (monotonicity (monotonicity @x2641 (= $x1809 $x2642)) (trans @x3244 (rewrite (= (and $x2665 $x3239) $x3248)) (= $x2609 $x3248)) (= $x2612 $x3253))))
-(let ((@x3265 (trans (monotonicity @x3255 (= $x2615 (and $x1280 $x3253))) (rewrite (= (and $x1280 $x3253) $x3261)) (= $x2615 $x3261))))
-(let (($x2244 (forall ((?v1 B_Vertex$) )(let ((?x2217 (v_b_SP_G_2$ ?v0!20)))
-(let ((?x2218 (* (- 1) ?x2217)))
-(let ((?x220 (v_b_SP_G_2$ ?v1)))
-(let (($x238 (fun_app$ v_b_Visited_G_2$ ?v1)))
-(let (($x2231 (and (not (>= (+ ?x220 ?x2218) 0)) $x238 (= (+ (b_G$ (pair$ ?v1 ?v0!20)) ?x220 ?x2218) 0))))
-(not $x2231)))))))
-))
-(let (($x2238 (not (not (and $x2216 $x2221)))))
-(let (($x2248 (and $x2238 $x2244)))
-(let (($x2253 (and $x1628 $x2248)))
-(let (($x2257 (or $x2204 $x2253)))
-(let (($x2261 (and $x1609 $x2257)))
-(let (($x2265 (or $x2177 $x2261)))
-(let (($x2269 (and $x1595 $x2265)))
-(let (($x2273 (or $x913 $x2154 $x2269)))
-(let (($x2277 (and $x786 $x2273)))
-(let (($x2281 (or $x2139 $x2277)))
-(let (($x2285 (and $x1586 $x2281)))
-(let (($x2289 (or $x2122 $x2285)))
-(let (($x2110 (and (and $x2083 $x2088) $x203 $x1525 $x1535 $x213 $x1567 $x1573)))
-(let (($x2293 (and $x2110 $x2289)))
-(let (($x2047 (or $x2042 (>= (+ ?x2036 ?x2030 (* (- 1) (fun_app$c v_b_SP_G_3$ ?v0!11))) 0))))
-(let (($x2048 (not $x2047)))
-(let (($x2065 (or $x2048 $x2061)))
-(let (($x2022 (forall ((?v0 B_Vertex$) )(let ((?x177 (fun_app$c v_b_SP_G_3$ ?v0)))
-(let ((?x1446 (* (- 1) ?x177)))
-(let ((?x2008 (fun_app$c v_b_SP_G_3$ (?v1!9 ?v0))))
-(let ((?x2013 (b_G$ (pair$ (?v1!9 ?v0) ?v0))))
-(let (($x2015 (= (+ ?x2013 ?x2008 ?x1446) 0)))
-(let (($x2016 (and (not (>= (+ ?x2008 ?x1446) 0)) $x2015)))
-(let (($x1448 (<= (+ b_Infinity$ ?x1446) 0)))
-(let (($x1451 (not $x1448)))
-(let (($x74 (= ?v0 b_Source$)))
-(let (($x79 (not $x74)))
-(let (($x1454 (and $x79 $x1451)))
-(let (($x1457 (not $x1454)))
-(or $x1457 $x2016))))))))))))))
-))
-(let (($x2069 (and $x2022 $x2065)))
-(let (($x1996 (forall ((?v1 B_Vertex$) )(let ((?x1970 (fun_app$c v_b_SP_G_3$ ?v0!8)))
-(let ((?x1971 (* (- 1) ?x1970)))
-(let ((?x177 (fun_app$c v_b_SP_G_3$ ?v1)))
-(let (($x1984 (and (not (>= (+ ?x177 ?x1971) 0)) (= (+ (b_G$ (pair$ ?v1 ?v0!8)) ?x177 ?x1971) 0))))
-(not $x1984))))))
-))
-(let (($x1990 (not (not (and $x1969 $x1974)))))
-(let (($x2000 (and $x1990 $x1996)))
-(let (($x2073 (or $x2000 $x2069)))
-(let (($x1961 (and $x1950 $x159 $x162 $x164 $x167)))
-(let (($x2077 (and $x1961 $x2073)))
-(let (($x2297 (or $x2077 $x2293)))
-(let (($x1938 (forall ((?v0 B_Vertex$) )(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v0)))
-(let ((?x1393 (* (- 1) ?x121)))
-(let ((?x1922 (?v1!7 ?v0)))
-(let ((?x1923 (fun_app$c v_b_SP_G_1$ ?x1922)))
-(let ((?x1929 (b_G$ (pair$ ?x1922 ?v0))))
-(let (($x1931 (= (+ ?x1929 ?x1923 ?x1393) 0)))
-(let (($x1927 (fun_app$ v_b_Visited_G_1$ ?x1922)))
-(let (($x1932 (and (not (>= (+ ?x1923 ?x1393) 0)) $x1927 $x1931)))
-(let (($x1395 (<= (+ b_Infinity$ ?x1393) 0)))
-(let (($x1398 (not $x1395)))
-(let (($x74 (= ?v0 b_Source$)))
-(let (($x79 (not $x74)))
-(let (($x1401 (and $x79 $x1398)))
-(let (($x1404 (not $x1401)))
-(or $x1404 $x1932))))))))))))))))
-))
-(let (($x1903 (forall ((?v0 B_Vertex$) )(let ((?x1894 (b_G$ (pair$ (?v1!6 ?v0) ?v0))))
-(let ((?x75 (v_b_SP_G_0$ ?v0)))
-(let ((?x1328 (* (- 1) ?x75)))
-(let ((?x1887 (?v1!6 ?v0)))
-(let ((?x1888 (v_b_SP_G_0$ ?x1887)))
-(let (($x1896 (= (+ ?x1888 ?x1328 ?x1894) 0)))
-(let (($x1892 (v_b_Visited_G_0$ ?x1887)))
-(let (($x1897 (and (not (>= (+ ?x1888 ?x1328) 0)) $x1892 $x1896)))
-(let (($x74 (= ?v0 b_Source$)))
-(let (($x79 (not $x74)))
-(let (($x1336 (and $x79 (not (<= (+ b_Infinity$ ?x1328) 0)))))
-(let (($x1339 (not $x1336)))
-(or $x1339 $x1897))))))))))))))
-))
-(let (($x1941 (and $x1903 $x120 $x1363 $x1374 $x1390 $x1938)))
-(let (($x2301 (and $x1941 $x2297)))
-(let (($x1870 (not (not (and $x1848 $x1853)))))
-(let (($x1880 (and $x1870 $x1876)))
-(let (($x2305 (or $x1880 $x2301)))
-(let (($x2309 (and $x1322 $x2305)))
-(let (($x1834 (>= (+ (v_b_SP_G_0$ ?v1!3) (* (- 1) (v_b_SP_G_0$ ?v0!4)) ?x1823) 0)))
-(let (($x1836 (not (or $x1829 $x1834))))
-(let (($x2313 (or $x1836 $x2309)))
-(let (($x2317 (and $x1295 $x2313)))
-(let (($x2321 (or $x1809 $x2317)))
-(let (($x2325 (and $x1280 $x2321)))
-(let (($x2329 (or $x1009 $x1786 $x2325)))
-(let (($x2230 (= (+ (b_G$ (pair$ ?0 ?v0!20)) ?x220 (* (- 1) (v_b_SP_G_2$ ?v0!20))) 0)))
-(let (($x2231 (and (not (>= (+ ?x220 (* (- 1) (v_b_SP_G_2$ ?v0!20))) 0)) $x238 $x2230)))
-(let (($x2241 (not $x2231)))
-(let (($x2526 (= (+ (b_G$ (pair$ ?0 ?v0!20)) ?x220 (* (- 1) (v_b_SP_G_2$ ?v0!20))) (+ ?x220 (* (- 1) (v_b_SP_G_2$ ?v0!20)) (b_G$ (pair$ ?0 ?v0!20))))))
-(let ((@x2533 (monotonicity (monotonicity (rewrite $x2526) (= $x2230 $x2528)) (= $x2231 $x2531))))
-(let ((@x2542 (monotonicity (rewrite (= $x2238 (and $x2216 $x2221))) (quant-intro (monotonicity @x2533 (= $x2241 $x2534)) (= $x2244 $x2537)) (= $x2248 (and (and $x2216 $x2221) $x2537)))))
-(let ((@x2550 (trans (monotonicity @x2542 (= $x2253 (and $x1628 (and (and $x2216 $x2221) $x2537)))) (rewrite (= (and $x1628 (and (and $x2216 $x2221) $x2537)) $x2546)) (= $x2253 $x2546))))
-(let ((@x2559 (monotonicity (monotonicity (monotonicity @x2550 (= $x2257 $x2551)) (= $x2261 $x2554)) (= $x2265 $x2557))))
-(let ((@x2568 (monotonicity (monotonicity (monotonicity @x2559 (= $x2269 $x2560)) (= $x2273 $x2563)) (= $x2277 $x2566))))
-(let ((@x2577 (monotonicity (monotonicity (monotonicity @x2568 (= $x2281 $x2569)) (= $x2285 $x2572)) (= $x2289 $x2575))))
-(let ((@x2585 (trans (monotonicity @x2577 (= $x2293 (and $x2110 $x2575))) (rewrite (= (and $x2110 $x2575) $x2581)) (= $x2293 $x2581))))
-(let (($x2498 (= (>= (+ ?x2036 ?x2030 (* (- 1) (fun_app$c v_b_SP_G_3$ ?v0!11))) 0) $x2497)))
-(let (($x2495 (= (+ ?x2036 ?x2030 (* (- 1) (fun_app$c v_b_SP_G_3$ ?v0!11))) (+ ?x2030 ?x2036 (* (- 1) (fun_app$c v_b_SP_G_3$ ?v0!11))))))
-(let ((@x2505 (monotonicity (monotonicity (monotonicity (rewrite $x2495) $x2498) (= $x2047 $x2500)) (= $x2048 $x2503))))
-(let ((?x1446 (* (- 1) ?x177)))
-(let ((?x2008 (fun_app$c v_b_SP_G_3$ (?v1!9 ?0))))
-(let ((?x2013 (b_G$ (pair$ (?v1!9 ?0) ?0))))
-(let (($x2015 (= (+ ?x2013 ?x2008 ?x1446) 0)))
-(let (($x2016 (and (not (>= (+ ?x2008 ?x1446) 0)) $x2015)))
-(let (($x2019 (or $x1457 $x2016)))
-(let ((@x2477 (monotonicity (rewrite (= (+ ?x2013 ?x2008 ?x1446) (+ ?x1446 ?x2008 ?x2013))) (= $x2015 (= (+ ?x1446 ?x2008 ?x2013) 0)))))
-(let ((@x2484 (trans @x2477 (rewrite (= (= (+ ?x1446 ?x2008 ?x2013) 0) $x2480)) (= $x2015 $x2480))))
-(let ((@x2461 (monotonicity (rewrite (= (+ ?x2008 ?x1446) (+ ?x1446 ?x2008))) (= (>= (+ ?x2008 ?x1446) 0) (>= (+ ?x1446 ?x2008) 0)))))
-(let ((@x2468 (trans @x2461 (rewrite (= (>= (+ ?x1446 ?x2008) 0) $x2464)) (= (>= (+ ?x2008 ?x1446) 0) $x2464))))
-(let ((@x2487 (monotonicity (monotonicity @x2468 (= (not (>= (+ ?x2008 ?x1446) 0)) (not $x2464))) @x2484 (= $x2016 $x2485))))
-(let ((@x2511 (monotonicity (quant-intro (monotonicity @x2487 (= $x2019 $x2488)) (= $x2022 $x2491)) (monotonicity @x2505 (= $x2065 $x2506)) (= $x2069 $x2509))))
-(let (($x1984 (and (not (>= (+ ?x177 ?x1971) 0)) (= (+ (b_G$ (pair$ ?0 ?v0!8)) ?x177 ?x1971) 0))))
-(let (($x1993 (not $x1984)))
-(let (($x2434 (= (+ (b_G$ (pair$ ?0 ?v0!8)) ?x177 ?x1971) (+ ?x177 ?x1971 (b_G$ (pair$ ?0 ?v0!8))))))
-(let ((@x2438 (monotonicity (rewrite $x2434) (= (= (+ (b_G$ (pair$ ?0 ?v0!8)) ?x177 ?x1971) 0) $x2436))))
-(let ((@x2447 (quant-intro (monotonicity (monotonicity @x2438 (= $x1984 $x2439)) (= $x1993 $x2442)) (= $x1996 $x2445))))
-(let ((@x2450 (monotonicity (rewrite (= $x1990 (and $x1969 $x1974))) @x2447 (= $x2000 (and (and $x1969 $x1974) $x2445)))))
-(let ((@x2455 (trans @x2450 (rewrite (= (and (and $x1969 $x1974) $x2445) $x2451)) (= $x2000 $x2451))))
-(let ((@x2517 (monotonicity (monotonicity @x2455 @x2511 (= $x2073 $x2512)) (= $x2077 (and $x1961 $x2512)))))
-(let ((@x2588 (monotonicity (trans @x2517 (rewrite (= (and $x1961 $x2512) $x2518)) (= $x2077 $x2518)) @x2585 (= $x2297 $x2586))))
-(let ((?x1393 (* (- 1) ?x121)))
-(let ((?x1923 (fun_app$c v_b_SP_G_1$ ?x1922)))
-(let ((?x1929 (b_G$ (pair$ ?x1922 ?0))))
-(let (($x1931 (= (+ ?x1929 ?x1923 ?x1393) 0)))
-(let (($x1932 (and (not (>= (+ ?x1923 ?x1393) 0)) $x1927 $x1931)))
-(let (($x1935 (or $x1404 $x1932)))
-(let ((@x2414 (monotonicity (rewrite (= (+ ?x1929 ?x1923 ?x1393) (+ ?x1393 ?x1923 ?x1929))) (= $x1931 (= (+ ?x1393 ?x1923 ?x1929) 0)))))
-(let ((@x2421 (trans @x2414 (rewrite (= (= (+ ?x1393 ?x1923 ?x1929) 0) $x2417)) (= $x1931 $x2417))))
-(let ((@x2398 (monotonicity (rewrite (= (+ ?x1923 ?x1393) (+ ?x1393 ?x1923))) (= (>= (+ ?x1923 ?x1393) 0) (>= (+ ?x1393 ?x1923) 0)))))
-(let ((@x2405 (trans @x2398 (rewrite (= (>= (+ ?x1393 ?x1923) 0) $x2401)) (= (>= (+ ?x1923 ?x1393) 0) $x2401))))
-(let ((@x2424 (monotonicity (monotonicity @x2405 (= (not (>= (+ ?x1923 ?x1393) 0)) (not $x2401))) @x2421 (= $x1932 $x2422))))
-(let (($x1896 (= (+ (v_b_SP_G_0$ ?x1887) (* (- 1) ?x75) (b_G$ (pair$ ?x1887 ?0))) 0)))
-(let (($x1897 (and (not (>= (+ (v_b_SP_G_0$ ?x1887) (* (- 1) ?x75)) 0)) $x1892 $x1896)))
-(let (($x1900 (or $x1339 $x1897)))
-(let (($x2374 (= (+ (* (- 1) ?x75) (v_b_SP_G_0$ ?x1887) (b_G$ (pair$ ?x1887 ?0))) 0)))
-(let (($x2372 (= (+ (v_b_SP_G_0$ ?x1887) (* (- 1) ?x75) (b_G$ (pair$ ?x1887 ?0))) (+ (* (- 1) ?x75) (v_b_SP_G_0$ ?x1887) (b_G$ (pair$ ?x1887 ?0))))))
-(let ((@x2383 (trans (monotonicity (rewrite $x2372) (= $x1896 $x2374)) (rewrite (= $x2374 $x2379)) (= $x1896 $x2379))))
-(let (($x2369 (= (not (>= (+ (v_b_SP_G_0$ ?x1887) (* (- 1) ?x75)) 0)) (not $x2363))))
-(let (($x1890 (>= (+ (v_b_SP_G_0$ ?x1887) (* (- 1) ?x75)) 0)))
-(let (($x2356 (= (+ (v_b_SP_G_0$ ?x1887) (* (- 1) ?x75)) (+ (* (- 1) ?x75) (v_b_SP_G_0$ ?x1887)))))
-(let ((@x2360 (monotonicity (rewrite $x2356) (= $x1890 (>= (+ (* (- 1) ?x75) (v_b_SP_G_0$ ?x1887)) 0)))))
-(let ((@x2367 (trans @x2360 (rewrite (= (>= (+ (* (- 1) ?x75) (v_b_SP_G_0$ ?x1887)) 0) $x2363)) (= $x1890 $x2363))))
-(let ((@x2389 (monotonicity (monotonicity (monotonicity @x2367 $x2369) @x2383 (= $x1897 $x2384)) (= $x1900 $x2387))))
-(let ((@x2591 (monotonicity (quant-intro @x2389 (= $x1903 $x2390)) (quant-intro (monotonicity @x2424 (= $x1935 $x2425)) (= $x1938 $x2428)) (= $x1941 (and $x2390 $x120 $x1363 $x1374 $x1390 $x2428)))))
-(let ((@x2594 (monotonicity @x2591 @x2588 (= $x2301 (and (and $x2390 $x120 $x1363 $x1374 $x1390 $x2428) $x2586)))))
-(let ((@x2599 (trans @x2594 (rewrite (= (and (and $x2390 $x120 $x1363 $x1374 $x1390 $x2428) $x2586) $x2595)) (= $x2301 $x2595))))
-(let ((@x2349 (monotonicity (rewrite (= $x1870 (and $x1848 $x1853))) (= $x1880 (and (and $x1848 $x1853) $x1876)))))
-(let ((@x2354 (trans @x2349 (rewrite (= (and (and $x1848 $x1853) $x1876) $x2350)) (= $x1880 $x2350))))
-(let ((@x2605 (monotonicity (monotonicity @x2354 @x2599 (= $x2305 $x2600)) (= $x2309 $x2603))))
-(let (($x2334 (= (+ (v_b_SP_G_0$ ?v1!3) (* (- 1) (v_b_SP_G_0$ ?v0!4)) ?x1823) (+ ?x1823 (v_b_SP_G_0$ ?v1!3) (* (- 1) (v_b_SP_G_0$ ?v0!4))))))
-(let ((@x2341 (monotonicity (monotonicity (rewrite $x2334) (= $x1834 $x2336)) (= (or $x1829 $x1834) $x2339))))
-(let ((@x2608 (monotonicity (monotonicity @x2341 (= $x1836 $x2342)) @x2605 (= $x2313 $x2606))))
-(let ((@x2617 (monotonicity (monotonicity (monotonicity @x2608 (= $x2317 $x2609)) (= $x2321 $x2612)) (= $x2325 $x2615))))
-(let (($x1662 (forall ((?v0 B_Vertex$) )(let (($x1656 (exists ((?v1 B_Vertex$) )(let ((?x220 (v_b_SP_G_2$ ?v1)))
-(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let (($x238 (fun_app$ v_b_Visited_G_2$ ?v1)))
-(and (not (>= (+ ?x220 (* (- 1) (v_b_SP_G_2$ ?v0))) 0)) $x238 (= (+ ?x102 ?x220 (* (- 1) (v_b_SP_G_2$ ?v0))) 0))))))
-))
-(let (($x74 (= ?v0 b_Source$)))
-(let (($x79 (not $x74)))
-(let (($x1641 (and $x79 (not (<= (+ b_Infinity$ (* (- 1) (v_b_SP_G_2$ ?v0))) 0)))))
-(or (not $x1641) $x1656))))))
-))
-(let (($x1631 (not $x1628)))
-(let (($x1665 (or $x1631 $x1662)))
-(let (($x1668 (and $x1628 $x1665)))
-(let (($x1612 (not $x1609)))
-(let (($x1671 (or $x1612 $x1668)))
-(let (($x1674 (and $x1609 $x1671)))
-(let (($x1677 (or $x1598 $x1674)))
-(let (($x1680 (and $x244 $x1595 $x1677)))
-(let (($x1683 (or $x925 $x1680)))
-(let (($x1686 (and $x786 $x1683)))
-(let (($x1689 (or $x1589 $x1686)))
-(let (($x1692 (and $x1586 $x1689)))
-(let (($x1434 (exists ((?v0 B_Vertex$) )(let (($x1395 (<= (+ b_Infinity$ (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0))) 0)))
-(let (($x1398 (not $x1395)))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v0)))
-(let (($x126 (not $x125)))
-(and $x126 $x1398))))))
-))
-(let (($x1576 (and $x1434 $x203 $x1525 $x1535 $x213 $x1567 $x1573)))
-(let (($x1579 (not $x1576)))
-(let (($x1695 (or $x1579 $x1692)))
-(let (($x1502 (not $x1499)))
-(let (($x1505 (or $x1502 $x193)))
-(let (($x1508 (and $x1499 $x1505)))
-(let (($x1481 (forall ((?v0 B_Vertex$) )(let (($x1475 (exists ((?v1 B_Vertex$) )(let ((?x177 (fun_app$c v_b_SP_G_3$ ?v1)))
-(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(and (not (>= (+ ?x177 (* (- 1) (fun_app$c v_b_SP_G_3$ ?v0))) 0)) (= (+ ?x102 ?x177 (* (- 1) (fun_app$c v_b_SP_G_3$ ?v0))) 0)))))
-))
-(let (($x1448 (<= (+ b_Infinity$ (* (- 1) (fun_app$c v_b_SP_G_3$ ?v0))) 0)))
-(let (($x1451 (not $x1448)))
-(let (($x74 (= ?v0 b_Source$)))
-(let (($x79 (not $x74)))
-(let (($x1454 (and $x79 $x1451)))
-(let (($x1457 (not $x1454)))
-(or $x1457 $x1475)))))))))
-))
-(let (($x1484 (not $x1481)))
-(let (($x1511 (or $x1484 $x1508)))
-(let (($x1514 (and $x1481 $x1511)))
-(let (($x1437 (not $x1434)))
-(let (($x1440 (and $x1437 $x159 $x162 $x164 $x167)))
-(let (($x1443 (not $x1440)))
-(let (($x1517 (or $x1443 $x1514)))
-(let (($x1698 (and $x1517 $x1695)))
-(let (($x1422 (forall ((?v0 B_Vertex$) )(let (($x1416 (exists ((?v1 B_Vertex$) )(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v1)))
-(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v1)))
-(and (not (>= (+ ?x121 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0))) 0)) $x125 (= (+ ?x102 ?x121 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0))) 0))))))
-))
-(let (($x1395 (<= (+ b_Infinity$ (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0))) 0)))
-(let (($x1398 (not $x1395)))
-(let (($x74 (= ?v0 b_Source$)))
-(let (($x79 (not $x74)))
-(let (($x1401 (and $x79 $x1398)))
-(let (($x1404 (not $x1401)))
-(or $x1404 $x1416)))))))))
-))
-(let (($x1357 (forall ((?v0 B_Vertex$) )(let (($x1351 (exists ((?v1 B_Vertex$) )(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let ((?x75 (v_b_SP_G_0$ ?v1)))
-(let (($x83 (v_b_Visited_G_0$ ?v1)))
-(and (not (>= (+ ?x75 (* (- 1) (v_b_SP_G_0$ ?v0))) 0)) $x83 (= (+ ?x75 (* (- 1) (v_b_SP_G_0$ ?v0)) ?x102) 0))))))
-))
-(let (($x74 (= ?v0 b_Source$)))
-(let (($x79 (not $x74)))
-(let (($x1336 (and $x79 (not (<= (+ b_Infinity$ (* (- 1) (v_b_SP_G_0$ ?v0))) 0)))))
-(let (($x1339 (not $x1336)))
-(or $x1339 $x1351)))))))
-))
-(let (($x1425 (and $x1357 $x120 $x1363 $x1374 $x1390 $x1422)))
-(let (($x1428 (not $x1425)))
-(let (($x1701 (or $x1428 $x1698)))
-(let (($x1704 (and $x1357 $x1701)))
-(let (($x1325 (not $x1322)))
-(let (($x1707 (or $x1325 $x1704)))
-(let (($x1710 (and $x1322 $x1707)))
-(let (($x1298 (not $x1295)))
-(let (($x1713 (or $x1298 $x1710)))
-(let (($x1716 (and $x1295 $x1713)))
-(let (($x1719 (or $x1283 $x1716)))
-(let (($x1725 (not (and $x92 $x1280 $x1719))))
-(let (($x2232 (exists ((?v1 B_Vertex$) )(let ((?x2217 (v_b_SP_G_2$ ?v0!20)))
-(let ((?x2218 (* (- 1) ?x2217)))
-(let ((?x220 (v_b_SP_G_2$ ?v1)))
-(let (($x238 (fun_app$ v_b_Visited_G_2$ ?v1)))
-(and (not (>= (+ ?x220 ?x2218) 0)) $x238 (= (+ (b_G$ (pair$ ?v1 ?v0!20)) ?x220 ?x2218) 0)))))))
-))
-(let ((@x2250 (nnf-neg (refl (~ $x2238 $x2238)) (nnf-neg (refl (~ $x2241 $x2241)) (~ (not $x2232) $x2244)) (~ (not (or (not (and $x2216 $x2221)) $x2232)) $x2248))))
-(let ((@x2252 (trans (sk (~ (not $x1662) (not (or (not (and $x2216 $x2221)) $x2232)))) @x2250 (~ (not $x1662) $x2248))))
-(let ((@x2213 (nnf-neg (nnf-pos (refl (~ $x1625 $x1625)) (~ $x1628 $x1628)) (~ (not $x1631) $x1628))))
-(let ((@x2260 (nnf-neg (sk (~ $x1631 $x2204)) (nnf-neg @x2213 @x2252 (~ (not $x1665) $x2253)) (~ (not $x1668) $x2257))))
-(let ((@x2186 (nnf-neg (nnf-pos (refl (~ $x1606 $x1606)) (~ $x1609 $x1609)) (~ (not $x1612) $x1609))))
-(let ((@x2268 (nnf-neg (sk (~ $x1612 $x2177)) (nnf-neg @x2186 @x2260 (~ (not $x1671) $x2261)) (~ (not $x1674) $x2265))))
-(let ((@x2163 (nnf-neg (nnf-pos (refl (~ (>= ?x220 0) (>= ?x220 0))) (~ $x1595 $x1595)) (~ (not $x1598) $x1595))))
-(let ((@x2276 (nnf-neg (refl (~ $x913 $x913)) (sk (~ $x1598 $x2154)) (nnf-neg @x2163 @x2268 (~ (not $x1677) $x2269)) (~ (not $x1680) $x2273))))
-(let ((@x2148 (nnf-neg (nnf-pos (refl (~ $x783 $x783)) (~ $x786 $x786)) (~ (not $x925) $x786))))
-(let ((@x2284 (nnf-neg (sk (~ $x925 $x2139)) (nnf-neg @x2148 @x2276 (~ (not $x1683) $x2277)) (~ (not $x1686) $x2281))))
-(let ((@x2131 (nnf-neg (nnf-pos (refl (~ $x1582 $x1582)) (~ $x1586 $x1586)) (~ (not $x1589) $x1586))))
-(let ((@x2292 (nnf-neg (sk (~ $x1589 $x2122)) (nnf-neg @x2131 @x2284 (~ (not $x1689) $x2285)) (~ (not $x1692) $x2289))))
-(let (($x1553 (and (not $x1540) (not $x1547))))
-(let (($x1570 (or $x1553 $x225)))
-(let ((@x2105 (nnf-pos (refl (~ (or (not $x1553) $x1559) (or (not $x1553) $x1559))) (~ $x1567 $x1567))))
-(let ((@x2112 (monotonicity (sk (~ $x1434 (and $x2083 $x2088))) (refl (~ $x203 $x203)) (refl (~ $x1525 $x1525)) (nnf-pos (refl (~ $x1532 $x1532)) (~ $x1535 $x1535)) (refl (~ $x213 $x213)) @x2105 (nnf-pos (refl (~ $x1570 $x1570)) (~ $x1573 $x1573)) (~ $x1576 $x2110))))
-(let ((@x2296 (nnf-neg (nnf-neg @x2112 (~ (not $x1579) $x2110)) @x2292 (~ (not $x1695) $x2293))))
-(let ((@x2057 (nnf-neg (nnf-pos (refl (~ $x1496 $x1496)) (~ $x1499 $x1499)) (~ (not $x1502) $x1499))))
-(let ((@x2068 (nnf-neg (sk (~ $x1502 $x2048)) (nnf-neg @x2057 (refl (~ $x2058 $x2058)) (~ (not $x1505) $x2061)) (~ (not $x1508) $x2065))))
-(let (($x1475 (exists ((?v1 B_Vertex$) )(let ((?x177 (fun_app$c v_b_SP_G_3$ ?v1)))
-(let ((?x102 (b_G$ (pair$ ?v1 ?0))))
-(and (not (>= (+ ?x177 (* (- 1) (fun_app$c v_b_SP_G_3$ ?0))) 0)) (= (+ ?x102 ?x177 (* (- 1) (fun_app$c v_b_SP_G_3$ ?0))) 0)))))
-))
-(let (($x1478 (or $x1457 $x1475)))
-(let ((@x2024 (nnf-pos (monotonicity (refl (~ $x1457 $x1457)) (sk (~ $x1475 $x2016)) (~ $x1478 $x2019)) (~ $x1481 $x2022))))
-(let ((@x2072 (nnf-neg (nnf-neg @x2024 (~ (not $x1484) $x2022)) @x2068 (~ (not $x1511) $x2069))))
-(let (($x1985 (exists ((?v1 B_Vertex$) )(let ((?x1970 (fun_app$c v_b_SP_G_3$ ?v0!8)))
-(let ((?x1971 (* (- 1) ?x1970)))
-(let ((?x177 (fun_app$c v_b_SP_G_3$ ?v1)))
-(and (not (>= (+ ?x177 ?x1971) 0)) (= (+ (b_G$ (pair$ ?v1 ?v0!8)) ?x177 ?x1971) 0))))))
-))
-(let ((@x2002 (nnf-neg (refl (~ $x1990 $x1990)) (nnf-neg (refl (~ $x1993 $x1993)) (~ (not $x1985) $x1996)) (~ (not (or (not (and $x1969 $x1974)) $x1985)) $x2000))))
-(let ((@x2004 (trans (sk (~ $x1484 (not (or (not (and $x1969 $x1974)) $x1985)))) @x2002 (~ $x1484 $x2000))))
-(let ((@x1952 (nnf-neg (refl (~ (not (and $x126 $x1398)) (not (and $x126 $x1398)))) (~ $x1437 $x1950))))
-(let ((@x1963 (monotonicity @x1952 (refl (~ $x159 $x159)) (refl (~ $x162 $x162)) (refl (~ $x164 $x164)) (refl (~ $x167 $x167)) (~ $x1440 $x1961))))
-(let ((@x2080 (nnf-neg (nnf-neg @x1963 (~ (not $x1443) $x1961)) (nnf-neg @x2004 @x2072 (~ (not $x1514) $x2073)) (~ (not $x1517) $x2077))))
-(let (($x1416 (exists ((?v1 B_Vertex$) )(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v1)))
-(let ((?x102 (b_G$ (pair$ ?v1 ?0))))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v1)))
-(and (not (>= (+ ?x121 (* (- 1) (fun_app$c v_b_SP_G_1$ ?0))) 0)) $x125 (= (+ ?x102 ?x121 (* (- 1) (fun_app$c v_b_SP_G_1$ ?0))) 0))))))
-))
-(let (($x1419 (or $x1404 $x1416)))
-(let ((@x1940 (nnf-pos (monotonicity (refl (~ $x1404 $x1404)) (sk (~ $x1416 $x1932)) (~ $x1419 $x1935)) (~ $x1422 $x1938))))
-(let ((@x1917 (refl (~ (or (not (and $x125 $x1306)) $x1384) (or (not (and $x125 $x1306)) $x1384)))))
-(let (($x1351 (exists ((?v1 B_Vertex$) )(let ((?x102 (b_G$ (pair$ ?v1 ?0))))
-(let ((?x75 (v_b_SP_G_0$ ?v1)))
-(let (($x83 (v_b_Visited_G_0$ ?v1)))
-(and (not (>= (+ ?x75 (* (- 1) (v_b_SP_G_0$ ?0))) 0)) $x83 (= (+ ?x75 (* (- 1) (v_b_SP_G_0$ ?0)) ?x102) 0))))))
-))
-(let (($x1354 (or $x1339 $x1351)))
-(let ((@x1905 (nnf-pos (monotonicity (refl (~ $x1339 $x1339)) (sk (~ $x1351 $x1897)) (~ $x1354 $x1900)) (~ $x1357 $x1903))))
-(let ((@x1943 (monotonicity @x1905 (refl (~ $x120 $x120)) (nnf-pos (refl (~ (>= ?x121 0) (>= ?x121 0))) (~ $x1363 $x1363)) (nnf-pos (refl (~ (or $x429 $x1367) (or $x429 $x1367))) (~ $x1374 $x1374)) (nnf-pos @x1917 (~ $x1390 $x1390)) @x1940 (~ $x1425 $x1941))))
-(let ((@x2304 (nnf-neg (nnf-neg @x1943 (~ (not $x1428) $x1941)) (nnf-neg @x2080 @x2296 (~ (not $x1698) $x2297)) (~ (not $x1701) $x2301))))
-(let (($x1864 (exists ((?v1 B_Vertex$) )(let ((?x1849 (v_b_SP_G_0$ ?v0!5)))
-(let ((?x1850 (* (- 1) ?x1849)))
-(let ((?x75 (v_b_SP_G_0$ ?v1)))
-(let (($x83 (v_b_Visited_G_0$ ?v1)))
-(and (not (>= (+ ?x75 ?x1850) 0)) $x83 (= (+ ?x75 ?x1850 (b_G$ (pair$ ?v1 ?v0!5))) 0)))))))
-))
-(let ((@x1882 (nnf-neg (refl (~ $x1870 $x1870)) (nnf-neg (refl (~ $x1873 $x1873)) (~ (not $x1864) $x1876)) (~ (not (or (not (and $x1848 $x1853)) $x1864)) $x1880))))
-(let ((@x1884 (trans (sk (~ (not $x1357) (not (or (not (and $x1848 $x1853)) $x1864)))) @x1882 (~ (not $x1357) $x1880))))
-(let ((@x1840 (refl (~ (or (not (and $x83 $x1306)) $x1316) (or (not (and $x83 $x1306)) $x1316)))))
-(let ((@x2312 (nnf-neg (nnf-neg (nnf-pos @x1840 (~ $x1322 $x1322)) (~ (not $x1325) $x1322)) (nnf-neg @x1884 @x2304 (~ (not $x1704) $x2305)) (~ (not $x1707) $x2309))))
-(let ((@x1818 (nnf-neg (nnf-pos (refl (~ (or $x370 $x1288) (or $x370 $x1288))) (~ $x1295 $x1295)) (~ (not $x1298) $x1295))))
-(let ((@x2320 (nnf-neg @x1818 (nnf-neg (sk (~ $x1325 $x1836)) @x2312 (~ (not $x1710) $x2313)) (~ (not $x1713) $x2317))))
-(let ((@x1795 (nnf-neg (nnf-pos (refl (~ (>= ?x75 0) (>= ?x75 0))) (~ $x1280 $x1280)) (~ (not $x1283) $x1280))))
-(let ((@x2328 (nnf-neg @x1795 (nnf-neg (sk (~ $x1298 $x1809)) @x2320 (~ (not $x1716) $x2321)) (~ (not $x1719) $x2325))))
-(let ((@x2331 (nnf-neg (refl (~ $x1009 $x1009)) (sk (~ $x1283 $x1786)) @x2328 (~ $x1725 $x2329))))
-(let (($x1075 (or $x949 (and $x237 (or $x937 (and $x786 (or $x925 (and $x244 $x246 $x902))))))))
-(let (($x1082 (and $x374 (or $x985 (and $x393 (or $x973 (and $x426 (or $x961 (and $x678 $x1075)))))))))
-(let (($x1084 (not (and $x92 $x94 (or $x997 $x1082)))))
-(let (($x1211 (forall ((?v0 B_Vertex$) )(let (($x1205 (exists ((?v1 B_Vertex$) )(let ((?x220 (v_b_SP_G_2$ ?v1)))
-(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let ((?x1184 (+ ?x102 ?x220)))
-(let ((?x250 (v_b_SP_G_2$ ?v0)))
-(let (($x1199 (= ?x250 ?x1184)))
-(let (($x238 (fun_app$ v_b_Visited_G_2$ ?v1)))
-(let (($x251 (<= ?x250 ?x220)))
-(let (($x827 (not $x251)))
-(and $x827 $x238 $x1199))))))))))
-))
-(let (($x821 (not (<= b_Infinity$ (v_b_SP_G_2$ ?v0)))))
-(let (($x74 (= ?v0 b_Source$)))
-(let (($x79 (not $x74)))
-(let (($x824 (and $x79 $x821)))
-(let (($x844 (not $x824)))
-(or $x844 $x1205))))))))
-))
-(let (($x1193 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x220 (v_b_SP_G_2$ ?v1)))
-(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let ((?x1184 (+ ?x102 ?x220)))
-(let ((?x250 (v_b_SP_G_2$ ?v0)))
-(let (($x1187 (<= ?x250 ?x1184)))
-(let (($x378 (not (<= b_Infinity$ ?x102))))
-(let (($x238 (fun_app$ v_b_Visited_G_2$ ?v1)))
-(let (($x805 (and $x238 $x378)))
-(let (($x811 (not $x805)))
-(or $x811 $x1187)))))))))))
-))
-(let (($x1196 (not $x1193)))
-(let (($x1214 (or $x1196 $x1211)))
-(let (($x1217 (and $x1193 $x1214)))
-(let (($x1220 (or $x889 $x1217)))
-(let (($x1223 (and $x802 $x1220)))
-(let (($x1226 (or $x901 $x1223)))
-(let (($x1229 (and $x244 $x246 $x1226)))
-(let (($x1232 (or $x925 $x1229)))
-(let (($x1235 (and $x786 $x1232)))
-(let (($x1238 (or $x937 $x1235)))
-(let (($x1241 (and $x237 $x1238)))
-(let (($x1244 (or $x949 $x1241)))
-(let (($x1163 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x177 (fun_app$c v_b_SP_G_3$ ?v1)))
-(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let ((?x1136 (+ ?x102 ?x177)))
-(let ((?x180 (fun_app$c v_b_SP_G_3$ ?v0)))
-(let (($x1157 (<= ?x180 ?x1136)))
-(let (($x378 (not (<= b_Infinity$ ?x102))))
-(let (($x598 (not (<= b_Infinity$ ?x177))))
-(let (($x626 (and $x598 $x378)))
-(let (($x632 (not $x626)))
-(or $x632 $x1157)))))))))))
-))
-(let (($x1166 (not $x1163)))
-(let (($x1169 (or $x1166 $x193)))
-(let (($x1172 (and $x1163 $x1169)))
-(let (($x1151 (forall ((?v0 B_Vertex$) )(let (($x1145 (exists ((?v1 B_Vertex$) )(let ((?x177 (fun_app$c v_b_SP_G_3$ ?v1)))
-(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let ((?x1136 (+ ?x102 ?x177)))
-(let ((?x180 (fun_app$c v_b_SP_G_3$ ?v0)))
-(let (($x1139 (= ?x180 ?x1136)))
-(let (($x605 (not (<= ?x180 ?x177))))
-(and $x605 $x1139))))))))
-))
-(let (($x598 (not (<= b_Infinity$ (fun_app$c v_b_SP_G_3$ ?v0)))))
-(let (($x74 (= ?v0 b_Source$)))
-(let (($x79 (not $x74)))
-(let (($x601 (and $x79 $x598)))
-(let (($x617 (not $x601)))
-(or $x617 $x1145))))))))
-))
-(let (($x1154 (not $x1151)))
-(let (($x1175 (or $x1154 $x1172)))
-(let (($x1178 (and $x1151 $x1175)))
-(let (($x1181 (or $x677 $x1178)))
-(let (($x1247 (and $x1181 $x1244)))
-(let (($x1127 (forall ((?v0 B_Vertex$) )(let (($x1121 (exists ((?v1 B_Vertex$) )(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v1)))
-(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let ((?x1102 (+ ?x102 ?x121)))
-(let ((?x129 (fun_app$c v_b_SP_G_1$ ?v0)))
-(let (($x1115 (= ?x129 ?x1102)))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v1)))
-(let (($x130 (<= ?x129 ?x121)))
-(let (($x458 (not $x130)))
-(and $x458 $x125 $x1115))))))))))
-))
-(let (($x452 (not (<= b_Infinity$ (fun_app$c v_b_SP_G_1$ ?v0)))))
-(let (($x74 (= ?v0 b_Source$)))
-(let (($x79 (not $x74)))
-(let (($x455 (and $x79 $x452)))
-(let (($x475 (not $x455)))
-(or $x475 $x1121))))))))
-))
-(let (($x1112 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v1)))
-(let ((?x102 (b_G$ (pair$ ?v1 ?v0))))
-(let ((?x1102 (+ ?x102 ?x121)))
-(let ((?x129 (fun_app$c v_b_SP_G_1$ ?v0)))
-(let (($x1106 (<= ?x129 ?x1102)))
-(let (($x378 (not (<= b_Infinity$ ?x102))))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v1)))
-(let (($x436 (and $x125 $x378)))
-(let (($x442 (not $x436)))
-(or $x442 $x1106)))))))))))
-))
-(let (($x1130 (and $x426 $x120 $x123 $x433 $x1112 $x1127)))
-(let (($x1133 (not $x1130)))
-(let (($x1250 (or $x1133 $x1247)))
-(let (($x1253 (and $x426 $x1250)))
-(let (($x1256 (or $x973 $x1253)))
-(let (($x1259 (and $x393 $x1256)))
-(let (($x1262 (or $x985 $x1259)))
-(let (($x1265 (and $x374 $x1262)))
-(let (($x1268 (or $x997 $x1265)))
-(let (($x1271 (and $x92 $x94 $x1268)))
-(let (($x1656 (exists ((?v1 B_Vertex$) )(let ((?x220 (v_b_SP_G_2$ ?v1)))
-(let ((?x102 (b_G$ (pair$ ?v1 ?0))))
-(let (($x238 (fun_app$ v_b_Visited_G_2$ ?v1)))
-(and (not (>= (+ ?x220 (* (- 1) (v_b_SP_G_2$ ?0))) 0)) $x238 (= (+ ?x102 ?x220 (* (- 1) (v_b_SP_G_2$ ?0))) 0))))))
-))
-(let (($x1659 (or (not (and $x79 (not (<= (+ b_Infinity$ (* (- 1) ?x220)) 0)))) $x1656)))
-(let (($x1205 (exists ((?v1 B_Vertex$) )(let ((?x220 (v_b_SP_G_2$ ?v1)))
-(let ((?x102 (b_G$ (pair$ ?v1 ?0))))
-(let ((?x1184 (+ ?x102 ?x220)))
-(let ((?x250 (v_b_SP_G_2$ ?0)))
-(let (($x1199 (= ?x250 ?x1184)))
-(let (($x238 (fun_app$ v_b_Visited_G_2$ ?v1)))
-(let (($x251 (<= ?x250 ?x220)))
-(let (($x827 (not $x251)))
-(and $x827 $x238 $x1199))))))))))
-))
-(let (($x1208 (or $x844 $x1205)))
-(let ((?x1184 (+ ?x102 ?x220)))
-(let (($x1199 (= ?x250 ?x1184)))
-(let (($x1202 (and $x827 $x238 $x1199)))
-(let (($x1654 (= $x1202 (and (not $x1601) $x238 (= (+ ?x102 ?x220 (* (- 1) ?x250)) 0)))))
-(let ((@x1655 (monotonicity (monotonicity (rewrite (= $x251 $x1601)) (= $x827 (not $x1601))) (rewrite (= $x1199 (= (+ ?x102 ?x220 (* (- 1) ?x250)) 0))) $x1654)))
-(let (($x1645 (= $x844 (not (and $x79 (not (<= (+ b_Infinity$ (* (- 1) ?x220)) 0)))))))
-(let (($x1642 (= $x824 (and $x79 (not (<= (+ b_Infinity$ (* (- 1) ?x220)) 0))))))
-(let (($x1636 (= (<= b_Infinity$ ?x220) (<= (+ b_Infinity$ (* (- 1) ?x220)) 0))))
-(let ((@x1640 (monotonicity (rewrite $x1636) (= $x821 (not (<= (+ b_Infinity$ (* (- 1) ?x220)) 0))))))
-(let ((@x1661 (monotonicity (monotonicity (monotonicity @x1640 $x1642) $x1645) (quant-intro @x1655 (= $x1205 $x1656)) (= $x1208 $x1659))))
-(let ((@x1308 (monotonicity (rewrite (= (<= b_Infinity$ ?x102) $x1303)) (= $x378 $x1306))))
-(let ((@x1627 (monotonicity (monotonicity (monotonicity @x1308 (= $x805 $x1615)) (= $x811 $x1618)) (rewrite (= (<= ?x250 ?x1184) $x1621)) (= (or $x811 (<= ?x250 ?x1184)) $x1625))))
-(let ((@x1667 (monotonicity (monotonicity (quant-intro @x1627 (= $x1193 $x1628)) (= $x1196 $x1631)) (quant-intro @x1661 (= $x1211 $x1662)) (= $x1214 $x1665))))
-(let ((@x1611 (quant-intro (monotonicity (rewrite (= $x251 $x1601)) (= $x799 $x1606)) (= $x802 $x1609))))
-(let ((@x1673 (monotonicity (monotonicity @x1611 (= $x889 $x1612)) (monotonicity (quant-intro @x1627 (= $x1193 $x1628)) @x1667 (= $x1217 $x1668)) (= $x1220 $x1671))))
-(let ((@x1597 (quant-intro (rewrite (= (<= 0 ?x220) (>= ?x220 0))) (= $x246 $x1595))))
-(let ((@x1679 (monotonicity (monotonicity @x1597 (= $x901 $x1598)) (monotonicity @x1611 @x1673 (= $x1223 $x1674)) (= $x1226 $x1677))))
-(let ((@x1685 (monotonicity (monotonicity @x1597 @x1679 (= $x1229 $x1680)) (= $x1232 $x1683))))
-(let ((@x1591 (monotonicity (quant-intro (rewrite (= (<= ?x220 ?x121) $x1582)) (= $x237 $x1586)) (= $x937 $x1589))))
-(let ((@x1691 (monotonicity @x1591 (monotonicity @x1685 (= $x1235 $x1686)) (= $x1238 $x1689))))
-(let ((@x1694 (monotonicity (quant-intro (rewrite (= (<= ?x220 ?x121) $x1582)) (= $x237 $x1586)) @x1691 (= $x1241 $x1692))))
-(let ((@x1552 (monotonicity (rewrite (= (<= ?x121 ?x217) $x1547)) (= $x698 (not $x1547)))))
-(let ((@x1545 (monotonicity (rewrite (= (<= b_Infinity$ ?x215) $x1540)) (= $x694 (not $x1540)))))
-(let ((@x1572 (monotonicity (monotonicity @x1545 @x1552 (= $x701 $x1553)) (= $x721 $x1570))))
-(let ((@x1558 (monotonicity (monotonicity @x1545 @x1552 (= $x701 $x1553)) (= $x707 (not $x1553)))))
-(let ((@x1566 (monotonicity @x1558 (rewrite (= $x221 $x1559)) (= $x708 (or (not $x1553) $x1559)))))
-(let ((@x1534 (monotonicity (rewrite (= $x206 (>= (+ ?x121 (* (- 1) ?x204)) 0))) (= $x687 $x1532))))
-(let ((@x1527 (monotonicity (rewrite (= (<= b_Infinity$ ?x204) $x1522)) (= $x684 $x1525))))
-(let ((@x1400 (monotonicity (rewrite (= (<= b_Infinity$ ?x121) $x1395)) (= $x452 $x1398))))
-(let ((@x1436 (quant-intro (monotonicity @x1400 (= $x537 (and $x126 $x1398))) (= $x540 $x1434))))
-(let ((@x1578 (monotonicity @x1436 @x1527 (quant-intro @x1534 (= $x690 $x1535)) (quant-intro @x1566 (= $x713 $x1567)) (quant-intro @x1572 (= $x726 $x1573)) (= $x767 $x1576))))
-(let ((@x1697 (monotonicity (monotonicity @x1578 (= $x949 $x1579)) @x1694 (= $x1244 $x1695))))
-(let ((@x1453 (monotonicity (rewrite (= (<= b_Infinity$ ?x177) $x1448)) (= $x598 $x1451))))
-(let ((@x1492 (monotonicity (monotonicity @x1453 @x1308 (= $x626 $x1487)) (= $x632 $x1490))))
-(let ((@x1498 (monotonicity @x1492 (rewrite (= (<= ?x180 (+ ?x102 ?x177)) $x1493)) (= (or $x632 (<= ?x180 (+ ?x102 ?x177))) $x1496))))
-(let ((@x1507 (monotonicity (monotonicity (quant-intro @x1498 (= $x1163 $x1499)) (= $x1166 $x1502)) (= $x1169 $x1505))))
-(let (($x1145 (exists ((?v1 B_Vertex$) )(let ((?x177 (fun_app$c v_b_SP_G_3$ ?v1)))
-(let ((?x102 (b_G$ (pair$ ?v1 ?0))))
-(let ((?x1136 (+ ?x102 ?x177)))
-(let ((?x180 (fun_app$c v_b_SP_G_3$ ?0)))
-(let (($x1139 (= ?x180 ?x1136)))
-(let (($x605 (not (<= ?x180 ?x177))))
-(and $x605 $x1139))))))))
-))
-(let (($x1148 (or $x617 $x1145)))
-(let (($x1472 (and (not (>= (+ ?x177 (* (- 1) ?x180)) 0)) (= (+ ?x102 ?x177 (* (- 1) ?x180)) 0))))
-(let ((?x1136 (+ ?x102 ?x177)))
-(let (($x1139 (= ?x180 ?x1136)))
-(let (($x1142 (and $x605 $x1139)))
-(let ((@x1467 (monotonicity (rewrite (= (<= ?x180 ?x177) (>= (+ ?x177 (* (- 1) ?x180)) 0))) (= $x605 (not (>= (+ ?x177 (* (- 1) ?x180)) 0))))))
-(let ((@x1474 (monotonicity @x1467 (rewrite (= $x1139 (= (+ ?x102 ?x177 (* (- 1) ?x180)) 0))) (= $x1142 $x1472))))
-(let ((@x1480 (monotonicity (monotonicity (monotonicity @x1453 (= $x601 $x1454)) (= $x617 $x1457)) (quant-intro @x1474 (= $x1145 $x1475)) (= $x1148 $x1478))))
-(let ((@x1513 (monotonicity (monotonicity (quant-intro @x1480 (= $x1151 $x1481)) (= $x1154 $x1484)) (monotonicity (quant-intro @x1498 (= $x1163 $x1499)) @x1507 (= $x1172 $x1508)) (= $x1175 $x1511))))
-(let ((@x1445 (monotonicity (monotonicity (monotonicity @x1436 (= $x543 $x1437)) (= $x581 $x1440)) (= $x677 $x1443))))
-(let ((@x1519 (monotonicity @x1445 (monotonicity (quant-intro @x1480 (= $x1151 $x1481)) @x1513 (= $x1178 $x1514)) (= $x1181 $x1517))))
-(let (($x1121 (exists ((?v1 B_Vertex$) )(let ((?x121 (fun_app$c v_b_SP_G_1$ ?v1)))
-(let ((?x102 (b_G$ (pair$ ?v1 ?0))))
-(let ((?x1102 (+ ?x102 ?x121)))
-(let ((?x129 (fun_app$c v_b_SP_G_1$ ?0)))
-(let (($x1115 (= ?x129 ?x1102)))
-(let (($x125 (fun_app$ v_b_Visited_G_1$ ?v1)))
-(let (($x130 (<= ?x129 ?x121)))
-(let (($x458 (not $x130)))
-(and $x458 $x125 $x1115))))))))))
-))
-(let (($x1124 (or $x475 $x1121)))
-(let ((?x1102 (+ ?x102 ?x121)))
-(let (($x1115 (= ?x129 ?x1102)))
-(let (($x1118 (and $x458 $x125 $x1115)))
-(let (($x1414 (= $x1118 (and (not $x1367) $x125 (= (+ ?x102 ?x121 (* (- 1) ?x129)) 0)))))
-(let ((@x1415 (monotonicity (monotonicity (rewrite (= $x130 $x1367)) (= $x458 (not $x1367))) (rewrite (= $x1115 (= (+ ?x102 ?x121 (* (- 1) ?x129)) 0))) $x1414)))
-(let ((@x1421 (monotonicity (monotonicity (monotonicity @x1400 (= $x455 $x1401)) (= $x475 $x1404)) (quant-intro @x1415 (= $x1121 $x1416)) (= $x1124 $x1419))))
-(let ((@x1382 (monotonicity (monotonicity @x1308 (= $x436 (and $x125 $x1306))) (= $x442 (not (and $x125 $x1306))))))
-(let ((@x1389 (monotonicity @x1382 (rewrite (= (<= ?x129 ?x1102) $x1384)) (= (or $x442 (<= ?x129 ?x1102)) (or (not (and $x125 $x1306)) $x1384)))))
-(let ((@x1376 (quant-intro (monotonicity (rewrite (= $x130 $x1367)) (= $x430 (or $x429 $x1367))) (= $x433 $x1374))))
-(let ((@x1365 (quant-intro (rewrite (= (<= 0 ?x121) (>= ?x121 0))) (= $x123 $x1363))))
-(let (($x1349 (= $x409 (and (not $x1288) $x83 (= (+ ?x75 (* (- 1) ?x97) ?x102) 0)))))
-(let ((@x1350 (monotonicity (monotonicity (rewrite (= $x98 $x1288)) (= $x403 (not $x1288))) (rewrite (= $x112 (= (+ ?x75 (* (- 1) ?x97) ?x102) 0))) $x1349)))
-(let ((@x1335 (monotonicity (rewrite (= (<= b_Infinity$ ?x75) $x1330)) (= $x397 (not $x1330)))))
-(let ((@x1341 (monotonicity (monotonicity @x1335 (= $x400 $x1336)) (= (not $x400) $x1339))))
-(let ((@x1359 (quant-intro (monotonicity @x1341 (quant-intro @x1350 (= $x414 $x1351)) (= $x421 $x1354)) (= $x426 $x1357))))
-(let ((@x1427 (monotonicity @x1359 @x1365 @x1376 (quant-intro @x1389 (= $x1112 $x1390)) (quant-intro @x1421 (= $x1127 $x1422)) (= $x1130 $x1425))))
-(let ((@x1703 (monotonicity (monotonicity @x1427 (= $x1133 $x1428)) (monotonicity @x1519 @x1697 (= $x1247 $x1698)) (= $x1250 $x1701))))
-(let ((@x1314 (monotonicity (monotonicity @x1308 (= (and $x83 $x378) (and $x83 $x1306))) (= (not (and $x83 $x378)) (not (and $x83 $x1306))))))
-(let ((@x1321 (monotonicity @x1314 (rewrite (= $x106 $x1316)) (= $x388 (or (not (and $x83 $x1306)) $x1316)))))
-(let ((@x1709 (monotonicity (monotonicity (quant-intro @x1321 (= $x393 $x1322)) (= $x973 $x1325)) (monotonicity @x1359 @x1703 (= $x1253 $x1704)) (= $x1256 $x1707))))
-(let ((@x1297 (quant-intro (monotonicity (rewrite (= $x98 $x1288)) (= $x371 (or $x370 $x1288))) (= $x374 $x1295))))
-(let ((@x1715 (monotonicity (monotonicity @x1297 (= $x985 $x1298)) (monotonicity (quant-intro @x1321 (= $x393 $x1322)) @x1709 (= $x1259 $x1710)) (= $x1262 $x1713))))
-(let ((@x1282 (quant-intro (rewrite (= (<= 0 ?x75) (>= ?x75 0))) (= $x94 $x1280))))
-(let ((@x1721 (monotonicity (monotonicity @x1282 (= $x997 $x1283)) (monotonicity @x1297 @x1715 (= $x1265 $x1716)) (= $x1268 $x1719))))
-(let ((@x1727 (monotonicity (monotonicity @x1282 @x1721 (= $x1271 (and $x92 $x1280 $x1719))) (= (not $x1271) $x1725))))
-(let (($x1263 (= (or $x985 (and $x393 (or $x973 (and $x426 (or $x961 (and $x678 $x1075)))))) $x1262)))
-(let (($x1260 (= (and $x393 (or $x973 (and $x426 (or $x961 (and $x678 $x1075))))) $x1259)))
-(let (($x1242 (= (and $x237 (or $x937 (and $x786 (or $x925 (and $x244 $x246 $x902))))) $x1241)))
-(let ((@x1204 (monotonicity (monotonicity (rewrite (= ?x255 ?x1184)) (= $x262 $x1199)) (= $x833 $x1202))))
-(let ((@x1213 (quant-intro (monotonicity (quant-intro @x1204 (= $x838 $x1205)) (= $x845 $x1208)) (= $x850 $x1211))))
-(let ((@x1192 (monotonicity (monotonicity (rewrite (= ?x255 ?x1184)) (= $x256 (<= ?x250 ?x1184))) (= $x812 (or $x811 (<= ?x250 ?x1184))))))
-(let ((@x1198 (monotonicity (quant-intro @x1192 (= $x817 $x1193)) (= (not $x817) $x1196))))
-(let ((@x1219 (monotonicity (quant-intro @x1192 (= $x817 $x1193)) (monotonicity @x1198 @x1213 (= $x878 $x1214)) (= $x883 $x1217))))
-(let ((@x1228 (monotonicity (monotonicity (monotonicity @x1219 (= $x890 $x1220)) (= $x895 $x1223)) (= $x902 $x1226))))
-(let ((@x1234 (monotonicity (monotonicity @x1228 (= (and $x244 $x246 $x902) $x1229)) (= (or $x925 (and $x244 $x246 $x902)) $x1232))))
-(let ((@x1237 (monotonicity @x1234 (= (and $x786 (or $x925 (and $x244 $x246 $x902))) $x1235))))
-(let ((@x1240 (monotonicity @x1237 (= (or $x937 (and $x786 (or $x925 (and $x244 $x246 $x902)))) $x1238))))
-(let ((@x1162 (monotonicity (monotonicity (rewrite (= ?x182 ?x1136)) (= $x189 (<= ?x180 ?x1136))) (= $x633 (or $x632 (<= ?x180 ?x1136))))))
-(let ((@x1168 (monotonicity (quant-intro @x1162 (= $x638 $x1163)) (= (not $x638) $x1166))))
-(let ((@x1174 (monotonicity (quant-intro @x1162 (= $x638 $x1163)) (monotonicity @x1168 (= $x654 $x1169)) (= $x659 $x1172))))
-(let ((@x1144 (monotonicity (monotonicity (rewrite (= ?x182 ?x1136)) (= $x183 $x1139)) (= $x608 $x1142))))
-(let ((@x1153 (quant-intro (monotonicity (quant-intro @x1144 (= $x611 $x1145)) (= $x618 $x1148)) (= $x623 $x1151))))
-(let ((@x1177 (monotonicity (monotonicity @x1153 (= (not $x623) $x1154)) @x1174 (= $x666 $x1175))))
-(let ((@x1183 (monotonicity (monotonicity @x1153 @x1177 (= $x671 $x1178)) (= $x678 $x1181))))
-(let ((@x1249 (monotonicity @x1183 (monotonicity (monotonicity @x1240 $x1242) (= $x1075 $x1244)) (= (and $x678 $x1075) $x1247))))
-(let ((@x1120 (monotonicity (monotonicity (rewrite (= ?x134 ?x1102)) (= $x141 $x1115)) (= $x464 $x1118))))
-(let ((@x1129 (quant-intro (monotonicity (quant-intro @x1120 (= $x469 $x1121)) (= $x476 $x1124)) (= $x481 $x1127))))
-(let ((@x1111 (monotonicity (monotonicity (rewrite (= ?x134 ?x1102)) (= $x135 (<= ?x129 ?x1102))) (= $x443 (or $x442 (<= ?x129 ?x1102))))))
-(let ((@x1135 (monotonicity (monotonicity (quant-intro @x1111 (= $x448 $x1112)) @x1129 (= $x532 $x1130)) (= $x961 $x1133))))
-(let ((@x1255 (monotonicity (monotonicity @x1135 @x1249 (= (or $x961 (and $x678 $x1075)) $x1250)) (= (and $x426 (or $x961 (and $x678 $x1075))) $x1253))))
-(let ((@x1258 (monotonicity @x1255 (= (or $x973 (and $x426 (or $x961 (and $x678 $x1075)))) $x1256))))
-(let ((@x1267 (monotonicity (monotonicity (monotonicity @x1258 $x1260) $x1263) (= $x1082 $x1265))))
-(let ((@x1273 (monotonicity (monotonicity @x1267 (= (or $x997 $x1082) $x1268)) (= (and $x92 $x94 (or $x997 $x1082)) $x1271))))
-(let ((@x1729 (trans (monotonicity @x1273 (= $x1084 (not $x1271))) @x1727 (= $x1084 $x1725))))
-(let ((@x1088 (mp (not-or-elim @x1030 (not $x1015)) (rewrite* (= (not $x1015) $x1084)) $x1084)))
-(let ((@x2621 (mp (mp~ (mp @x1088 @x1729 $x1725) @x2331 $x2329) (monotonicity @x2617 (= $x2329 $x2618)) $x2618)))
-(let ((@x4102 (mp (mp @x2621 (monotonicity @x3265 (= $x2618 $x3266)) $x3266) @x4101 (or $x1009 $x1786 $x4096))))
-(let ((@x5459 (unit-resolution (def-axiom (or $x4093 $x4087)) (unit-resolution @x4102 @x4116 (lemma @x3301 $x1785) $x4096) $x4087)))
-(let ((@x4213 (unit-resolution ((_ quant-inst ?v0!2) (or (not $x3748) $x2622)) (mp @x1780 @x3752 $x3748) (hypothesis $x1800) false)))
-(let ((@x5512 (unit-resolution (def-axiom (or $x4090 $x2642 $x4084)) (unit-resolution (def-axiom (or $x2637 $x1800)) (lemma @x4213 $x2622) $x2637) @x5459 $x4084)))
-(let ((@x5451 (unit-resolution (def-axiom (or $x4078 $x2688 $x4072)) (unit-resolution (def-axiom (or $x4081 $x4075)) @x5512 $x4075) (unit-resolution (def-axiom (or $x2683 $x1821)) (lemma @x4210 $x2668) $x2683) $x4072)))
-(let ((?x1849 (v_b_SP_G_0$ ?v0!5)))
-(let (($x4261 (= b_Infinity$ ?x1849)))
-(let ((@x4269 (symm (commutativity (= $x4261 (= ?x1849 b_Infinity$))) (= (= ?x1849 b_Infinity$) $x4261))))
-(let (($x4170 (= ?x1849 b_Infinity$)))
-(let ((@x4259 (rewrite (= (or (not $x3741) (or $x1847 $x4170)) (or (not $x3741) $x1847 $x4170)))))
-(let ((@x4260 (mp ((_ quant-inst ?v0!5) (or (not $x3741) (or $x1847 $x4170))) @x4259 (or (not $x3741) $x1847 $x4170))))
-(let ((@x4263 (unit-resolution @x4260 (mp @x1775 (quant-intro (refl (= $x340 $x340)) (= $x343 $x3741)) $x3741) (unit-resolution (def-axiom (or $x3789 $x1848)) (hypothesis $x3792) $x1848) $x4170)))
-(let ((@x4249 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x4261) $x1852)) (unit-resolution (def-axiom (or $x3789 $x1853)) (hypothesis $x3792) $x1853) (not $x4261))))
-(let ((@x5453 (unit-resolution (def-axiom (or $x4066 $x3792 $x4060)) (lemma (unit-resolution @x4249 (mp @x4263 @x4269 $x4261) false) $x3789) (unit-resolution (def-axiom (or $x4069 $x4063)) @x5451 $x4063) $x4060)))
-(let ((@x5456 (unit-resolution (def-axiom (or $x4057 $x120)) @x5453 $x120)))
-(let ((@x5702 (trans (monotonicity @x5699 (= (fun_app$c v_b_SP_G_3$ b_Source$) ?x119)) @x5456 $x193)))
-(let (($x4338 (<= (+ b_Infinity$ (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0!8))) 0)))
-(let (($x4960 (not $x4338)))
-(let (($x4484 (>= (+ ?x1970 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0!8))) 0)))
-(let ((@x6411 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x1970 (fun_app$c v_b_SP_G_1$ ?v0!8))) $x4484)) (monotonicity @x5699 (= ?x1970 (fun_app$c v_b_SP_G_1$ ?v0!8))) $x4484)))
-(let ((@x4754 (lemma ((_ th-lemma arith farkas 1 -1 1) (hypothesis $x4484) (hypothesis $x4338) (hypothesis $x1974) false) (or $x4960 (not $x4484) $x1973))))
-(let (($x5013 (<= (+ ?x1970 (* (- 1) (fun_app$c v_b_SP_G_3$ (?v1!7 ?v0!8)))) 0)))
-(let ((?x4355 (* (- 1) (fun_app$c v_b_SP_G_1$ (?v1!7 ?v0!8)))))
-(let ((?x4335 (fun_app$c v_b_SP_G_1$ ?v0!8)))
-(let (($x4361 (<= (+ ?x4335 ?x4355) 0)))
-(let (($x4332 (not $x4361)))
-(let ((?x4366 (+ ?x4335 ?x4355 (* (- 1) (b_G$ (pair$ (?v1!7 ?v0!8) ?v0!8))))))
-(let (($x4371 (= ?x4366 0)))
-(let (($x4372 (not $x4371)))
-(let (($x4370 (or $x4361 (not (fun_app$ v_b_Visited_G_1$ (?v1!7 ?v0!8))) $x4372)))
-(let (($x4373 (not $x4370)))
-(let ((@x4406 (unit-resolution (def-axiom (or $x4057 $x3829)) @x5453 $x3829)))
-(let ((@x4343 (rewrite (= (or $x3834 (or $x1968 $x4338 $x4373)) (or $x3834 $x1968 $x4338 $x4373)))))
-(let ((@x4329 (mp ((_ quant-inst ?v0!8) (or $x3834 (or $x1968 $x4338 $x4373))) @x4343 (or $x3834 $x1968 $x4338 $x4373))))
-(let ((@x4408 (unit-resolution @x4329 @x4406 (unit-resolution (def-axiom (or $x3856 $x1969)) (hypothesis $x3859) $x1969) (hypothesis $x4960) $x4373)))
-(let ((@x4463 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x1970 ?x4335)) $x4484)) (monotonicity (hypothesis $x164) (= ?x1970 ?x4335)) $x4484)))
-(let (($x4500 (<= (+ (fun_app$c v_b_SP_G_3$ (?v1!7 ?v0!8)) ?x4355) 0)))
-(let ((?x4341 (?v1!7 ?v0!8)))
-(let ((?x4288 (fun_app$c v_b_SP_G_3$ ?x4341)))
-(let ((@x5080 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x4288 (fun_app$c v_b_SP_G_1$ ?x4341))) $x4500)) (monotonicity (hypothesis $x164) (= ?x4288 (fun_app$c v_b_SP_G_1$ ?x4341))) $x4500)))
-(let ((@x5445 ((_ th-lemma arith farkas 1 -1 -1 1) (hypothesis $x4484) (hypothesis $x5013) (hypothesis $x4500) (hypothesis $x4332) false)))
-(let ((@x4647 (unit-resolution (lemma @x5445 (or (not $x5013) (not $x4484) (not $x4500) $x4361)) @x5080 @x4463 (unit-resolution (def-axiom (or $x4370 $x4332)) @x4408 $x4332) (not $x5013))))
-(let ((?x4700 (+ ?x1970 (* (- 1) ?x4288) (* (- 1) (b_G$ (pair$ ?x4341 ?v0!8))))))
-(let (($x4722 (= ?x4700 0)))
-(let (($x4489 (>= ?x4700 0)))
-(let (($x4331 (>= ?x4366 0)))
-(let ((@x4769 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x4372 $x4331)) (unit-resolution (def-axiom (or $x4370 $x4371)) @x4408 $x4371) $x4331)))
-(let ((@x5050 (unit-resolution ((_ th-lemma arith assign-bounds -1 -1 1) (or $x4489 (not $x4331) (not $x4484) (not $x4500))) @x4769 @x4463 @x5080 $x4489)))
-(let (($x5088 (<= ?x4700 0)))
-(let (($x4912 (>= (+ ?x4288 ?x4355) 0)))
-(let ((@x6226 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x4288 (fun_app$c v_b_SP_G_1$ ?x4341))) $x4912)) (monotonicity (hypothesis $x164) (= ?x4288 (fun_app$c v_b_SP_G_1$ ?x4341))) $x4912)))
-(let (($x4483 (<= (+ ?x1970 (* (- 1) ?x4335)) 0)))
-(let ((@x4788 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x1970 ?x4335)) $x4483)) (monotonicity (hypothesis $x164) (= ?x1970 ?x4335)) $x4483)))
-(let (($x4330 (<= ?x4366 0)))
-(let ((@x4407 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x4372 $x4330)) (unit-resolution (def-axiom (or $x4370 $x4371)) @x4408 $x4371) $x4330)))
-(let ((@x5001 (unit-resolution ((_ th-lemma arith assign-bounds -1 -1 1) (or $x5088 (not $x4330) (not $x4483) (not $x4912))) @x4407 @x4788 @x6226 $x5088)))
-(let ((@x4974 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x4722 (not $x5088) (not $x4489))) @x5001 @x5050 $x4722)))
-(let (($x5094 (not $x4722)))
-(let (($x4624 (or $x5013 $x5094)))
-(let (($x4764 (or $x3853 $x5013 $x5094)))
-(let (($x4299 (>= (+ ?x4288 ?x1971) 0)))
-(let (($x4989 (or $x3853 (or $x4299 (not (= (+ ?x4288 ?x1971 (b_G$ (pair$ ?x4341 ?v0!8))) 0))))))
-(let (($x4626 (= (or $x4299 (not (= (+ ?x4288 ?x1971 (b_G$ (pair$ ?x4341 ?v0!8))) 0))) $x4624)))
-(let ((@x4723 (rewrite (= (= (+ ?x1971 ?x4288 (b_G$ (pair$ ?x4341 ?v0!8))) 0) $x4722))))
-(let (($x4286 (= (+ ?x4288 ?x1971 (b_G$ (pair$ ?x4341 ?v0!8))) 0)))
-(let (($x4839 (= (+ ?x4288 ?x1971 (b_G$ (pair$ ?x4341 ?v0!8))) (+ ?x1971 ?x4288 (b_G$ (pair$ ?x4341 ?v0!8))))))
-(let ((@x4695 (monotonicity (rewrite $x4839) (= $x4286 (= (+ ?x1971 ?x4288 (b_G$ (pair$ ?x4341 ?v0!8))) 0)))))
-(let ((@x4401 (monotonicity (trans @x4695 @x4723 (= $x4286 $x4722)) (= (not $x4286) $x5094))))
-(let ((@x5263 (monotonicity (rewrite (= (+ ?x4288 ?x1971) (+ ?x1971 ?x4288))) (= $x4299 (>= (+ ?x1971 ?x4288) 0)))))
-(let ((@x4841 (trans @x5263 (rewrite (= (>= (+ ?x1971 ?x4288) 0) $x5013)) (= $x4299 $x5013))))
-(let ((@x5186 (trans (monotonicity (monotonicity @x4841 @x4401 $x4626) (= $x4989 (or $x3853 $x4624))) (rewrite (= (or $x3853 $x4624) $x4764)) (= $x4989 $x4764))))
-(let ((@x5499 (unit-resolution (mp ((_ quant-inst (?v1!7 ?v0!8)) $x4989) @x5186 $x4764) (unit-resolution (def-axiom (or $x3856 $x3848)) (hypothesis $x3859) $x3848) $x4624)))
-(let ((@x5708 (unit-resolution (lemma (unit-resolution @x5499 @x4974 @x4647 false) (or $x3856 $x2982 $x4338)) @x5699 (unit-resolution @x4754 @x6411 (hypothesis $x1974) $x4960) $x3856)))
-(let ((@x5837 (unit-resolution (def-axiom (or $x3899 $x3859 $x3893)) @x5708 (unit-resolution (def-axiom (or $x3902 $x3896)) @x5698 $x3896) $x3893)))
-(let ((@x5839 (unit-resolution (def-axiom (or $x3887 $x2924 $x3881)) (unit-resolution (def-axiom (or $x3890 $x3884)) @x5837 $x3884) (unit-resolution (def-axiom (or $x3878 $x2058)) @x5702 $x3878) $x2924)))
-(let ((@x5847 (monotonicity (symm @x5699 (= v_b_SP_G_1$ v_b_SP_G_3$)) (= ?x4698 ?x2030))))
-(let ((@x6414 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x6220) $x5759)) (symm @x5847 $x6220) $x5759)))
-(let ((@x6168 (lemma ((_ th-lemma arith farkas 1 -1 1) (hypothesis $x5759) (hypothesis $x4492) (hypothesis $x2034) false) (or $x5659 (not $x5759) $x2033))))
-(let ((@x5991 (unit-resolution @x6168 @x6414 (unit-resolution (def-axiom (or $x2919 $x2034)) @x5839 $x2034) $x5659)))
-(let ((@x4386 (mp ((_ quant-inst ?v1!10) (or $x3843 (or $x4697 $x4492))) (rewrite (= (or $x3843 (or $x4697 $x4492)) (or $x3843 $x4697 $x4492))) (or $x3843 $x4697 $x4492))))
-(let ((@x5999 (unit-resolution @x4386 (unit-resolution (def-axiom (or $x3902 $x3838)) @x5698 $x3838) (or $x4697 $x4492))))
-(let ((@x6172 (unit-resolution (def-axiom (or $x4057 $x3821)) @x5453 $x3821)))
-(let (($x4384 (not $x4697)))
-(let (($x5846 (or $x3826 $x4384 $x2039 $x4677)))
-(let (($x4673 (or $x4384 $x2039 (>= (+ ?x2036 ?x4698 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0!11))) 0))))
-(let (($x5849 (or $x3826 $x4673)))
-(let (($x4614 (= (>= (+ ?x2036 ?x4698 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0!11))) 0) $x4677)))
-(let (($x4674 (= (+ ?x2036 ?x4698 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0!11))) (+ ?x2036 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0!11)) ?x4698))))
-(let ((@x5516 (monotonicity (monotonicity (rewrite $x4674) $x4614) (= $x4673 (or $x4384 $x2039 $x4677)))))
-(let ((@x5314 (trans (monotonicity @x5516 (= $x5849 (or $x3826 (or $x4384 $x2039 $x4677)))) (rewrite (= (or $x3826 (or $x4384 $x2039 $x4677)) $x5846)) (= $x5849 $x5846))))
-(let ((@x6307 (unit-resolution (mp ((_ quant-inst ?v0!11 ?v1!10) $x5849) @x5314 $x5846) @x6172 (unit-resolution (def-axiom (or $x2919 (not $x2039))) @x5839 (not $x2039)) (or $x4384 $x4677))))
-(let ((?x4518 (fun_app$c v_b_SP_G_1$ ?v0!11)))
-(let ((?x4546 (* (- 1) ?x4518)))
-(let ((?x2043 (fun_app$c v_b_SP_G_3$ ?v0!11)))
-(let ((@x6142 (monotonicity (symm @x5699 (= v_b_SP_G_1$ v_b_SP_G_3$)) (= ?x4518 ?x2043))))
-(let ((@x5800 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x2043 ?x4518)) (<= (+ ?x2043 ?x4546) 0))) (symm @x6142 (= ?x2043 ?x4518)) (<= (+ ?x2043 ?x4546) 0))))
-(let ((@x5815 ((_ th-lemma arith farkas -1 -1 1 1) @x5800 (unit-resolution (def-axiom (or $x2919 $x3668)) @x5839 $x3668) @x6414 (unit-resolution @x6307 (unit-resolution @x5999 @x5991 $x4697) $x4677) false)))
-(let ((@x7385 (unit-resolution (def-axiom (or $x3856 $x1974)) (unit-resolution (lemma @x5815 (or $x3902 $x1973)) @x5698 $x1973) $x3856)))
-(let ((@x7411 (unit-resolution (def-axiom (or $x3899 $x3859 $x3893)) @x7385 (unit-resolution (def-axiom (or $x3902 $x3896)) @x5698 $x3896) $x3893)))
-(let ((@x7356 (unit-resolution (def-axiom (or $x3887 $x2924 $x3881)) (unit-resolution (def-axiom (or $x3878 $x2058)) @x5702 $x3878) (unit-resolution (def-axiom (or $x3890 $x3884)) @x7411 $x3884) $x2924)))
-(let ((@x7398 (unit-resolution @x6168 (unit-resolution (def-axiom (or $x2919 $x2034)) @x7356 $x2034) @x7384 $x5659)))
-(let ((@x7318 (unit-resolution @x4386 (unit-resolution (def-axiom (or $x3902 $x3838)) @x5698 $x3838) @x7398 $x4697)))
-(let ((@x5937 (unit-resolution (mp ((_ quant-inst ?v0!11 ?v1!10) $x5849) @x5314 $x5846) @x6172 (unit-resolution (def-axiom (or $x2919 (not $x2039))) @x7356 (not $x2039)) @x7318 $x4677)))
-(let ((@x6020 ((_ th-lemma arith farkas 1 -1 -1 1) @x5937 @x5800 (unit-resolution (def-axiom (or $x2919 $x3668)) @x7356 $x3668) @x7384 false)))
-(let ((@x8163 (unit-resolution (def-axiom (or $x4054 $x3905 $x4048)) (unit-resolution (def-axiom (or $x4057 $x4051)) @x5453 $x4051) $x4051)))
-(let ((@x8164 (unit-resolution @x8163 (lemma @x6020 $x3902) $x4048)))
-(let ((@x8214 (unit-resolution (def-axiom (or $x4045 $x213)) @x8164 $x213)))
-(let ((@x8302 (unit-resolution (def-axiom (or $x4045 $x3926)) @x8164 $x3926)))
-(let (($x5115 (fun_app$ ?x212 ?v0!14)))
-(let ((@x7409 (monotonicity (symm (hypothesis $x213) (= ?x212 v_b_Visited_G_2$)) (= $x5115 $x2133))))
-(let (($x6262 (fun_app$ v_b_Visited_G_1$ ?v0!14)))
-(let (($x5230 (= ?v0!14 v_b_v_G_1$)))
-(let (($x7438 (or $x5230 $x6262)))
-(let (($x7443 (= $x5115 $x7438)))
-(let (($x3716 (forall ((?v0 B_Vertex_bool_fun$) (?v1 B_Vertex$) (?v2 Bool) (?v3 B_Vertex$) )(!(let (($x56 (fun_app$ (fun_app$a (fun_app$b (fun_upd$ ?v0) ?v1) ?v2) ?v3)))
-(= $x56 (ite (= ?v3 ?v1) ?v2 (fun_app$ ?v0 ?v3)))) :pattern ( (fun_app$ (fun_app$a (fun_app$b (fun_upd$ ?v0) ?v1) ?v2) ?v3) )))
-))
-(let (($x1099 (forall ((?v0 B_Vertex_bool_fun$) (?v1 B_Vertex$) (?v2 Bool) (?v3 B_Vertex$) )(let (($x56 (fun_app$ (fun_app$a (fun_app$b (fun_upd$ ?v0) ?v1) ?v2) ?v3)))
-(= $x56 (ite (= ?v3 ?v1) ?v2 (fun_app$ ?v0 ?v3)))))
-))
-(let (($x56 (fun_app$ (fun_app$a (fun_app$b (fun_upd$ ?3) ?2) ?1) ?0)))
-(let (($x1095 (= $x56 (ite (= ?0 ?2) ?1 (fun_app$ ?3 ?0)))))
-(let (($x61 (forall ((?v0 B_Vertex_bool_fun$) (?v1 B_Vertex$) (?v2 Bool) (?v3 B_Vertex$) )(let (($x56 (fun_app$ (fun_app$a (fun_app$b (fun_upd$ ?v0) ?v1) ?v2) ?v3)))
-(= $x56 (ite (= ?v3 ?v1) ?v2 (fun_app$ ?v0 ?v3)))))
-))
-(let ((@x1098 (rewrite (= (= $x56 (ite (= ?0 ?2) ?1 (fun_app$ ?3 ?0))) $x1095))))
-(let ((@x1104 (mp (mp (asserted $x61) (rewrite* (= $x61 $x61)) $x61) (quant-intro @x1098 (= $x61 $x1099)) $x1099)))
-(let ((@x3721 (mp (mp~ @x1104 (nnf-pos (refl (~ $x1095 $x1095)) (~ $x1099 $x1099)) $x1099) (quant-intro (refl (= $x1095 $x1095)) (= $x1099 $x3716)) $x3716)))
-(let (($x5105 (not $x3716)))
-(let (($x7445 (or $x5105 $x7443)))
-(let ((@x7444 (monotonicity (rewrite (= (ite $x5230 true $x6262) $x7438)) (= (= $x5115 (ite $x5230 true $x6262)) $x7443))))
-(let ((@x7449 (monotonicity @x7444 (= (or $x5105 (= $x5115 (ite $x5230 true $x6262))) $x7445))))
-(let ((@x7452 (trans @x7449 (rewrite (= $x7445 $x7445)) (= (or $x5105 (= $x5115 (ite $x5230 true $x6262))) $x7445))))
-(let ((@x7453 (mp ((_ quant-inst v_b_Visited_G_1$ v_b_v_G_1$ true ?v0!14) (or $x5105 (= $x5115 (ite $x5230 true $x6262)))) @x7452 $x7445)))
-(let (($x7425 (not $x7438)))
-(let (($x6006 (not $x6262)))
-(let (($x7455 (>= (+ ?x204 (* (- 1) ?x2136)) 0)))
-(let (($x7487 (not $x7455)))
-(let (($x5623 (>= (+ ?x204 (* (- 1) ?x2136) (b_G$ (pair$ v_b_v_G_1$ ?v0!14))) 0)))
-(let (($x5890 (not $x5623)))
-(let (($x6101 (<= (+ b_Infinity$ (* (- 1) (b_G$ (pair$ v_b_v_G_1$ ?v0!14)))) 0)))
-(let (($x5590 (or $x6101 $x5623)))
-(let (($x5624 (not $x5590)))
-(let ((@x5806 (hypothesis $x3646)))
-(let ((@x6086 (hypothesis $x3926)))
-(let (($x5930 (or $x3931 $x5624 $x2137)))
-(let ((?x6353 (b_G$ (pair$ v_b_v_G_1$ ?v0!14))))
-(let ((?x6397 (* (- 1) ?x6353)))
-(let ((?x1520 (* (- 1) ?x204)))
-(let (($x6154 (<= (+ ?x2136 ?x1520 ?x6397) 0)))
-(let (($x5925 (or $x3931 (or (not (or $x6101 $x6154)) $x2137))))
-(let ((@x5231 (monotonicity (rewrite (= (+ ?x2136 ?x1520 ?x6397) (+ ?x1520 ?x2136 ?x6397))) (= $x6154 (<= (+ ?x1520 ?x2136 ?x6397) 0)))))
-(let ((@x5207 (trans @x5231 (rewrite (= (<= (+ ?x1520 ?x2136 ?x6397) 0) $x5623)) (= $x6154 $x5623))))
-(let ((@x5636 (monotonicity (monotonicity @x5207 (= (or $x6101 $x6154) $x5590)) (= (not (or $x6101 $x6154)) $x5624))))
-(let ((@x5641 (monotonicity @x5636 (= (or (not (or $x6101 $x6154)) $x2137) (or $x5624 $x2137)))))
-(let ((@x5869 (trans (monotonicity @x5641 (= $x5925 (or $x3931 (or $x5624 $x2137)))) (rewrite (= (or $x3931 (or $x5624 $x2137)) $x5930)) (= $x5925 $x5930))))
-(let ((@x6877 (unit-resolution (def-axiom (or $x5590 $x5890)) (unit-resolution (mp ((_ quant-inst ?v0!14) $x5925) @x5869 $x5930) @x6086 @x5806 $x5624) $x5890)))
-(let (($x5403 (= v_b_v_G_1$ ?v0!14)))
-(let (($x5399 (<= ?x6353 0)))
-(let ((@x6842 (hypothesis $x5890)))
-(let ((@x7496 (unit-resolution ((_ th-lemma arith assign-bounds 1 1) (or $x5399 $x5623 $x7487)) (hypothesis $x7455) @x6842 $x5399)))
-(let (($x3728 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(!(let (($x319 (not (<= (b_G$ (pair$ ?v0 ?v1)) 0))))
-(let (($x64 (= ?v0 ?v1)))
-(or $x64 $x319))) :pattern ( (pair$ ?v0 ?v1) )))
-))
-(let (($x330 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let (($x319 (not (<= (b_G$ (pair$ ?v0 ?v1)) 0))))
-(let (($x64 (= ?v0 ?v1)))
-(or $x64 $x319))))
-))
-(let (($x319 (not (<= (b_G$ (pair$ ?1 ?0)) 0))))
-(let (($x64 (= ?1 ?0)))
-(let (($x325 (or $x64 $x319)))
-(let (($x72 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let (($x64 (= ?v0 ?v1)))
-(let (($x69 (not $x64)))
-(=> $x69 (< 0 (b_G$ (pair$ ?v0 ?v1)))))))
-))
-(let (($x69 (not $x64)))
-(let (($x71 (=> $x69 (< 0 (b_G$ (pair$ ?1 ?0))))))
-(let ((@x324 (monotonicity (rewrite (= (< 0 (b_G$ (pair$ ?1 ?0))) $x319)) (= $x71 (=> $x69 $x319)))))
-(let ((@x332 (quant-intro (trans @x324 (rewrite (= (=> $x69 $x319) $x325)) (= $x71 $x325)) (= $x72 $x330))))
-(let ((@x1765 (mp~ (mp (mp (asserted $x72) @x332 $x330) (rewrite* (= $x330 $x330)) $x330) (nnf-pos (refl (~ $x325 $x325)) (~ $x330 $x330)) $x330)))
-(let ((@x3733 (mp @x1765 (quant-intro (refl (= $x325 $x325)) (= $x330 $x3728)) $x3728)))
-(let (($x7466 (= (or (not $x3728) (or $x5403 (not $x5399))) (or (not $x3728) $x5403 (not $x5399)))))
-(let ((@x7468 (mp ((_ quant-inst v_b_v_G_1$ ?v0!14) (or (not $x3728) (or $x5403 (not $x5399)))) (rewrite $x7466) (or (not $x3728) $x5403 (not $x5399)))))
-(let ((@x7498 (unit-resolution (unit-resolution @x7468 @x3733 (or $x5403 (not $x5399))) @x7496 $x5403)))
-(let ((@x7502 (unit-resolution ((_ th-lemma arith assign-bounds -1 1) (or (not (>= ?x6353 0)) $x5623 $x7487)) (hypothesis $x7455) @x6842 (not (>= ?x6353 0)))))
-(let ((@x7506 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x6353 0)) (>= ?x6353 0))) @x7502 (not (= ?x6353 0)))))
-(let (($x3722 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(!(let (($x64 (= ?v0 ?v1)))
-(let (($x69 (not $x64)))
-(or $x69 (= (b_G$ (pair$ ?v0 ?v1)) 0)))) :pattern ( (pair$ ?v0 ?v1) )))
-))
-(let (($x314 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let (($x64 (= ?v0 ?v1)))
-(let (($x69 (not $x64)))
-(or $x69 (= (b_G$ (pair$ ?v0 ?v1)) 0)))))
-))
-(let (($x311 (or $x69 (= (b_G$ (pair$ ?1 ?0)) 0))))
-(let (($x68 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let (($x64 (= ?v0 ?v1)))
-(=> $x64 (= (b_G$ (pair$ ?v0 ?v1)) 0))))
-))
-(let ((@x316 (quant-intro (rewrite (= (=> $x64 (= (b_G$ (pair$ ?1 ?0)) 0)) $x311)) (= $x68 $x314))))
-(let ((@x1760 (mp~ (mp (mp (asserted $x68) @x316 $x314) (rewrite* (= $x314 $x314)) $x314) (nnf-pos (refl (~ $x311 $x311)) (~ $x314 $x314)) $x314)))
-(let ((@x3727 (mp @x1760 (quant-intro (refl (= $x311 $x311)) (= $x314 $x3722)) $x3722)))
-(let (($x7472 (= (or (not $x3722) (or (not $x5403) (= ?x6353 0))) (or (not $x3722) (not $x5403) (= ?x6353 0)))))
-(let ((@x7474 (mp ((_ quant-inst v_b_v_G_1$ ?v0!14) (or (not $x3722) (or (not $x5403) (= ?x6353 0)))) (rewrite $x7472) (or (not $x3722) (not $x5403) (= ?x6353 0)))))
-(let ((@x7508 (unit-resolution (unit-resolution @x7474 @x3727 (or (not $x5403) (= ?x6353 0))) @x7506 @x7498 false)))
-(let ((@x6970 (unit-resolution (def-axiom (or $x4057 $x3813)) @x5453 $x3813)))
-(let ((@x7100 (rewrite (= (or $x3818 (or $x202 $x6006 $x7455)) (or $x3818 $x202 $x6006 $x7455)))))
-(let ((@x7101 (mp ((_ quant-inst ?v0!14 v_b_v_G_1$) (or $x3818 (or $x202 $x6006 $x7455))) @x7100 (or $x3818 $x202 $x6006 $x7455))))
-(let ((@x5643 (unit-resolution @x7101 @x6970 (hypothesis $x203) (hypothesis $x6262) (hypothesis $x7487) false)))
-(let ((@x7476 (unit-resolution (lemma @x5643 (or $x6006 $x202 $x7455)) (unit-resolution (lemma @x7508 (or $x7487 $x5623)) @x6877 $x7487) (hypothesis $x203) $x6006)))
-(let ((?x3394 (v_b_SP_G_2$ v_b_v_G_1$)))
-(let (($x3329 (= ?x3394 ?x204)))
-(let ((?x3404 (b_G$ (pair$ v_b_v_G_1$ v_b_v_G_1$))))
-(let (($x3390 (>= ?x3404 0)))
-(let (($x4586 (or (<= (+ b_Infinity$ (* (- 1) ?x3404)) 0) $x3390)))
-(let (($x4394 (= ?x3404 0)))
-(let (($x4439 (not $x3722)))
-(let (($x4440 (or $x4439 $x4394)))
-(let ((@x4427 (monotonicity (rewrite (= (= v_b_v_G_1$ v_b_v_G_1$) true)) (= (not (= v_b_v_G_1$ v_b_v_G_1$)) (not true)))))
-(let ((@x4447 (trans @x4427 (rewrite (= (not true) false)) (= (not (= v_b_v_G_1$ v_b_v_G_1$)) false))))
-(let ((@x4434 (monotonicity @x4447 (= (or (not (= v_b_v_G_1$ v_b_v_G_1$)) $x4394) (or false $x4394)))))
-(let ((@x4438 (trans @x4434 (rewrite (= (or false $x4394) $x4394)) (= (or (not (= v_b_v_G_1$ v_b_v_G_1$)) $x4394) $x4394))))
-(let ((@x4450 (monotonicity @x4438 (= (or $x4439 (or (not (= v_b_v_G_1$ v_b_v_G_1$)) $x4394)) $x4440))))
-(let ((@x4451 (trans @x4450 (rewrite (= $x4440 $x4440)) (= (or $x4439 (or (not (= v_b_v_G_1$ v_b_v_G_1$)) $x4394)) $x4440))))
-(let ((@x4452 (mp ((_ quant-inst v_b_v_G_1$ v_b_v_G_1$) (or $x4439 (or (not (= v_b_v_G_1$ v_b_v_G_1$)) $x4394))) @x4451 $x4440)))
-(let ((@x4473 (lemma (unit-resolution @x4452 @x3727 (hypothesis (not $x4394)) false) $x4394)))
-(let ((@x6229 (unit-resolution (def-axiom (or $x4586 (not $x3390))) (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x4394) $x3390)) @x4473 $x3390) $x4586)))
-(let (($x4589 (not $x4586)))
-(let (($x5387 (or $x3931 $x4589 $x3329)))
-(let (($x3393 (<= (+ ?x204 ?x1520 (* (- 1) ?x3404)) 0)))
-(let (($x3330 (or (not (or (<= (+ b_Infinity$ (* (- 1) ?x3404)) 0) $x3393)) $x3329)))
-(let (($x4517 (or $x3931 $x3330)))
-(let (($x4592 (= (not (or (<= (+ b_Infinity$ (* (- 1) ?x3404)) 0) $x3393)) $x4589)))
-(let ((@x3389 (monotonicity (rewrite (= (+ ?x204 ?x1520 (* (- 1) ?x3404)) (* (- 1) ?x3404))) (= $x3393 (<= (* (- 1) ?x3404) 0)))))
-(let ((@x3371 (trans @x3389 (rewrite (= (<= (* (- 1) ?x3404) 0) $x3390)) (= $x3393 $x3390))))
-(let ((@x5175 (monotonicity @x3371 (= (or (<= (+ b_Infinity$ (* (- 1) ?x3404)) 0) $x3393) $x4586))))
-(let ((@x4575 (monotonicity (monotonicity (monotonicity @x5175 $x4592) (= $x3330 (or $x4589 $x3329))) (= $x4517 (or $x3931 (or $x4589 $x3329))))))
-(let ((@x5481 (trans @x4575 (rewrite (= (or $x3931 (or $x4589 $x3329)) $x5387)) (= $x4517 $x5387))))
-(let ((@x6230 (unit-resolution (mp ((_ quant-inst v_b_v_G_1$) $x4517) @x5481 $x5387) @x6086 @x6229 $x3329)))
-(let ((@x7480 (trans (monotonicity (hypothesis $x5230) (= ?x2135 ?x3394)) (hypothesis $x3329) (= ?x2135 ?x204))))
-(let ((@x7483 (trans @x7480 (symm (monotonicity (hypothesis $x5230) (= ?x2136 ?x204)) (= ?x204 ?x2136)) $x2137)))
-(let ((@x7489 (lemma (unit-resolution @x5806 @x7483 false) (or (not $x5230) $x2137 (not $x3329)))))
-(let ((@x7479 (unit-resolution (def-axiom (or $x7425 $x5230 $x6262)) (unit-resolution @x7489 @x5806 @x6230 (not $x5230)) (or $x7425 $x6262))))
-(let ((@x7373 (unit-resolution (def-axiom (or (not $x7443) (not $x5115) $x7438)) (unit-resolution @x7479 @x7476 $x7425) (unit-resolution @x7453 @x3721 $x7443) (not $x5115))))
-(let ((@x7491 (unit-resolution @x7373 (mp (hypothesis $x2133) (symm @x7409 (= $x2133 $x5115)) $x5115) false)))
-(let ((@x5912 (unit-resolution (lemma @x7491 (or $x2134 $x3196 $x202 $x3931 $x2137)) (unit-resolution (def-axiom (or $x4045 $x203)) @x8164 $x203) @x8302 @x8214 $x2138)))
-(let ((@x8165 (unit-resolution (def-axiom (or $x4045 $x3918)) @x8164 $x3918)))
-(let ((?x6546 (b_G$ (pair$ v_b_v_G_1$ ?v0!13))))
-(let ((?x2118 (v_b_SP_G_2$ ?v0!13)))
-(let ((?x2119 (* (- 1) ?x2118)))
-(let ((?x6581 (+ ?x204 ?x2119 ?x6546)))
-(let (($x6584 (= ?x6581 0)))
-(let (($x6576 (>= (+ ?x204 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0!13)) ?x6546) 0)))
-(let (($x6555 (<= (+ b_Infinity$ (* (- 1) ?x6546)) 0)))
-(let (($x6633 (or $x6555 $x6576)))
-(let (($x6635 (not $x6633)))
-(let (($x6716 (not (= (fun_app$c v_b_SP_G_1$ ?v0!13) ?x2118))))
-(let ((?x2117 (fun_app$c v_b_SP_G_1$ ?v0!13)))
-(let (($x6631 (= ?x2118 ?x2117)))
-(let ((@x6726 (monotonicity (commutativity (= (= ?x2117 ?x2118) $x6631)) (= $x6716 (not $x6631)))))
-(let ((@x6727 (mp (unit-resolution ((_ th-lemma arith triangle-eq) (or $x6716 $x2121)) (hypothesis $x2122) $x6716) @x6726 (not $x6631))))
-(let (($x6620 (or $x6635 $x6631)))
-(let (($x6613 (or $x3931 $x6635 $x6631)))
-(let (($x6614 (or $x3931 (or (not (or $x6555 (<= (+ ?x2117 ?x1520 (* (- 1) ?x6546)) 0))) $x6631))))
-(let (($x6610 (= (or (not (or $x6555 (<= (+ ?x2117 ?x1520 (* (- 1) ?x6546)) 0))) $x6631) $x6620)))
-(let (($x6556 (<= (+ ?x2117 ?x1520 (* (- 1) ?x6546)) 0)))
-(let ((@x6595 (rewrite (= (+ ?x2117 ?x1520 (* (- 1) ?x6546)) (+ ?x1520 ?x2117 (* (- 1) ?x6546))))))
-(let ((@x6574 (monotonicity @x6595 (= $x6556 (<= (+ ?x1520 ?x2117 (* (- 1) ?x6546)) 0)))))
-(let ((@x6580 (trans @x6574 (rewrite (= (<= (+ ?x1520 ?x2117 (* (- 1) ?x6546)) 0) $x6576)) (= $x6556 $x6576))))
-(let ((@x6619 (monotonicity (monotonicity @x6580 (= (or $x6555 $x6556) $x6633)) (= (not (or $x6555 $x6556)) $x6635))))
-(let ((@x6624 (trans (monotonicity (monotonicity @x6619 $x6610) (= $x6614 (or $x3931 $x6620))) (rewrite (= (or $x3931 $x6620) $x6613)) (= $x6614 $x6613))))
-(let ((@x6732 (unit-resolution (unit-resolution (mp ((_ quant-inst ?v0!13) $x6614) @x6624 $x6613) @x6086 $x6620) @x6727 $x6635)))
-(let (($x6587 (or $x6555 $x6576 $x6584)))
-(let ((@x4512 (hypothesis $x3918)))
-(let (($x6590 (or $x3923 $x6555 $x6576 $x6584)))
-(let (($x6591 (or $x3923 (or $x6555 $x6556 (= (+ ?x204 ?x6546 ?x2119) 0)))))
-(let ((@x6586 (monotonicity (rewrite (= (+ ?x204 ?x6546 ?x2119) ?x6581)) (= (= (+ ?x204 ?x6546 ?x2119) 0) $x6584))))
-(let ((@x6589 (monotonicity @x6580 @x6586 (= (or $x6555 $x6556 (= (+ ?x204 ?x6546 ?x2119) 0)) $x6587))))
-(let ((@x6601 (trans (monotonicity @x6589 (= $x6591 (or $x3923 $x6587))) (rewrite (= (or $x3923 $x6587) $x6590)) (= $x6591 $x6590))))
-(let ((@x6735 (unit-resolution (unit-resolution (mp ((_ quant-inst ?v0!13) $x6591) @x6601 $x6590) @x4512 $x6587) (unit-resolution (def-axiom (or $x6633 (not $x6576))) @x6732 (not $x6576)) (unit-resolution (def-axiom (or $x6633 (not $x6555))) @x6732 (not $x6555)) $x6584)))
-(let ((@x6746 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x6584) (>= ?x6581 0))) @x6735 (>= ?x6581 0))))
-(let ((@x6748 (unit-resolution ((_ th-lemma arith farkas 1 1) (or (<= (+ ?x2117 ?x2119) 0) $x2121)) (hypothesis $x2122) (<= (+ ?x2117 ?x2119) 0))))
-(let ((@x6749 ((_ th-lemma arith farkas 1 -1 1) @x6748 (unit-resolution (def-axiom (or $x6633 (not $x6576))) @x6732 (not $x6576)) @x6746 false)))
-(let ((@x8304 (unit-resolution (def-axiom (or $x4042 $x2122 $x4036)) (unit-resolution (lemma @x6749 (or $x2121 $x3923 $x3931)) @x8165 @x8302 $x2121) (unit-resolution (def-axiom (or $x4045 $x4039)) @x8164 $x4039) $x4036)))
-(let ((@x8619 (unit-resolution (def-axiom (or $x4030 $x2139 $x4024)) (unit-resolution (def-axiom (or $x4033 $x4027)) @x8304 $x4027) $x4027)))
-(let ((@x10488 (unit-resolution @x8619 (lemma (unit-resolution @x5912 @x8820 @x8891 false) $x2138) $x4024)))
-(let ((@x10489 (unit-resolution (def-axiom (or $x4021 $x3943)) @x10488 $x3943)))
-(let (($x4687 (= ?v0!17 v_b_v_G_1$)))
-(let (($x4718 (fun_app$ v_b_Visited_G_1$ ?v0!17)))
-(let (($x7386 (or $x4687 $x4718)))
-(let (($x4686 (fun_app$ ?x212 ?v0!17)))
-(let (($x7429 (= $x4686 $x7386)))
-(let (($x7431 (or $x5105 $x7429)))
-(let ((@x7423 (monotonicity (rewrite (= (ite $x4687 true $x4718) $x7386)) (= (= $x4686 (ite $x4687 true $x4718)) $x7429))))
-(let ((@x7457 (monotonicity @x7423 (= (or $x5105 (= $x4686 (ite $x4687 true $x4718))) $x7431))))
-(let ((@x7375 (trans @x7457 (rewrite (= $x7431 $x7431)) (= (or $x5105 (= $x4686 (ite $x4687 true $x4718))) $x7431))))
-(let ((@x7402 (mp ((_ quant-inst v_b_Visited_G_1$ v_b_v_G_1$ true ?v0!17) (or $x5105 (= $x4686 (ite $x4687 true $x4718)))) @x7375 $x7431)))
-(let ((@x8181 (symm (monotonicity (symm @x8214 (= ?x212 v_b_Visited_G_2$)) (= $x4686 $x2168)) (= $x2168 $x4686))))
-(let ((@x8115 (mp (unit-resolution (def-axiom (or $x3034 $x2168)) (hypothesis $x3039) $x2168) @x8181 $x4686)))
-(let ((@x8116 (unit-resolution (def-axiom (or (not $x7429) (not $x4686) $x7386)) @x8115 (unit-resolution @x7402 @x3721 $x7429) $x7386)))
-(let (($x7513 (not $x4718)))
-(let (($x8244 (>= (+ ?x204 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0!17))) 0)))
-(let (($x8196 (not $x8244)))
-(let (($x7753 (<= (+ ?x204 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v1!16))) 0)))
-(let (($x4600 (fun_app$ v_b_Visited_G_1$ ?v1!16)))
-(let (($x4599 (= ?v1!16 v_b_v_G_1$)))
-(let (($x7324 (or $x4599 $x4600)))
-(let (($x4598 (fun_app$ ?x212 ?v1!16)))
-(let (($x7351 (= $x4598 $x7324)))
-(let (($x5310 (or $x5105 $x7351)))
-(let ((@x4543 (monotonicity (rewrite (= (ite $x4599 true $x4600) $x7324)) (= (= $x4598 (ite $x4599 true $x4600)) $x7351))))
-(let ((@x7173 (monotonicity @x4543 (= (or $x5105 (= $x4598 (ite $x4599 true $x4600))) $x5310))))
-(let ((@x7233 (trans @x7173 (rewrite (= $x5310 $x5310)) (= (or $x5105 (= $x4598 (ite $x4599 true $x4600))) $x5310))))
-(let ((@x7234 (mp ((_ quant-inst v_b_Visited_G_1$ v_b_v_G_1$ true ?v1!16) (or $x5105 (= $x4598 (ite $x4599 true $x4600)))) @x7233 $x5310)))
-(let ((@x8188 (symm (monotonicity (symm @x8214 (= ?x212 v_b_Visited_G_2$)) (= $x4598 $x2166)) (= $x2166 $x4598))))
-(let (($x2167 (not $x2166)))
-(let ((@x8189 (hypothesis $x3039)))
-(let ((@x7882 (mp (unit-resolution (def-axiom (or $x3034 $x2167)) @x8189 $x2167) (monotonicity @x8188 (= $x2167 (not $x4598))) (not $x4598))))
-(let ((@x7883 (unit-resolution (def-axiom (or (not $x7351) $x4598 (not $x7324))) @x7882 (unit-resolution @x7234 @x3721 $x7351) (not $x7324))))
-(let (($x7758 (or $x4600 $x7753)))
-(let (($x7761 (or $x3913 $x4600 $x7753)))
-(let (($x7762 (or $x3913 (or $x4600 (>= (+ (fun_app$c v_b_SP_G_1$ ?v1!16) ?x1520) 0)))))
-(let (($x7759 (= (or $x4600 (>= (+ (fun_app$c v_b_SP_G_1$ ?v1!16) ?x1520) 0)) $x7758)))
-(let ((@x7755 (rewrite (= (>= (+ ?x1520 (fun_app$c v_b_SP_G_1$ ?v1!16)) 0) $x7753))))
-(let (($x5376 (>= (+ (fun_app$c v_b_SP_G_1$ ?v1!16) ?x1520) 0)))
-(let (($x7728 (= (+ (fun_app$c v_b_SP_G_1$ ?v1!16) ?x1520) (+ ?x1520 (fun_app$c v_b_SP_G_1$ ?v1!16)))))
-(let ((@x7751 (monotonicity (rewrite $x7728) (= $x5376 (>= (+ ?x1520 (fun_app$c v_b_SP_G_1$ ?v1!16)) 0)))))
-(let ((@x7766 (monotonicity (monotonicity (trans @x7751 @x7755 (= $x5376 $x7753)) $x7759) (= $x7762 (or $x3913 $x7758)))))
-(let ((@x7771 (mp ((_ quant-inst ?v1!16) $x7762) (trans @x7766 (rewrite (= (or $x3913 $x7758) $x7761)) (= $x7762 $x7761)) $x7761)))
-(let ((@x7873 (unit-resolution @x7771 (unit-resolution (def-axiom (or $x4045 $x3908)) @x8164 $x3908) $x7758)))
-(let ((@x7874 (unit-resolution @x7873 (unit-resolution (def-axiom (or $x7324 (not $x4600))) @x7883 (not $x4600)) $x7753)))
-(let ((?x4523 (b_G$ (pair$ v_b_v_G_1$ ?v1!16))))
-(let (($x8224 (<= ?x4523 0)))
-(let (($x8225 (not $x8224)))
-(let (($x8223 (= v_b_v_G_1$ ?v1!16)))
-(let (($x8293 (not $x8223)))
-(let ((@x8351 (unit-resolution (hypothesis (not $x4599)) (symm (hypothesis $x8223) $x4599) false)))
-(let ((@x7877 (unit-resolution (lemma @x8351 (or $x8293 $x4599)) (unit-resolution (def-axiom (or $x7324 (not $x4599))) @x7883 (not $x4599)) $x8293)))
-(let ((@x8233 (rewrite (= (or (not $x3728) (or $x8223 $x8225)) (or (not $x3728) $x8223 $x8225)))))
-(let ((@x8234 (mp ((_ quant-inst v_b_v_G_1$ ?v1!16) (or (not $x3728) (or $x8223 $x8225))) @x8233 (or (not $x3728) $x8223 $x8225))))
-(let ((@x6202 (lemma (unit-resolution @x8234 @x3733 (hypothesis $x8224) (hypothesis $x8293) false) (or $x8225 $x8223))))
-(let (($x3634 (not $x2175)))
-(let ((@x8299 (hypothesis $x3634)))
-(let (($x7624 (<= (+ (v_b_SP_G_2$ ?v0!17) (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0!17))) 0)))
-(let ((@x8305 (unit-resolution (def-axiom (or $x4033 $x3934)) @x8304 $x3934)))
-(let (($x7629 (or $x3939 $x7624)))
-(let (($x5070 (>= (+ (fun_app$c v_b_SP_G_1$ ?v0!17) (* (- 1) (v_b_SP_G_2$ ?v0!17))) 0)))
-(let (($x7620 (>= (+ (* (- 1) (v_b_SP_G_2$ ?v0!17)) (fun_app$c v_b_SP_G_1$ ?v0!17)) 0)))
-(let (($x7616 (= (+ (fun_app$c v_b_SP_G_1$ ?v0!17) (* (- 1) (v_b_SP_G_2$ ?v0!17))) (+ (* (- 1) (v_b_SP_G_2$ ?v0!17)) (fun_app$c v_b_SP_G_1$ ?v0!17)))))
-(let ((@x7628 (trans (monotonicity (rewrite $x7616) (= $x5070 $x7620)) (rewrite (= $x7620 $x7624)) (= $x5070 $x7624))))
-(let ((@x7636 (trans (monotonicity @x7628 (= (or $x3939 $x5070) $x7629)) (rewrite (= $x7629 $x7629)) (= (or $x3939 $x5070) $x7629))))
-(let ((@x8222 (hypothesis $x8244)))
-(let (($x7884 (or $x8196 $x2175 (not (<= (+ ?x204 (* (- 1) (v_b_SP_G_2$ ?v1!16)) ?x4523) 0)) $x8224 (not $x7624))))
-(let ((@x8211 (unit-resolution ((_ th-lemma arith assign-bounds 1 1 1 1) $x7884) @x8222 (unit-resolution (mp ((_ quant-inst ?v0!17) (or $x3939 $x5070)) @x7636 $x7629) @x8305 $x7624) (hypothesis $x8225) @x8299 (not (<= (+ ?x204 (* (- 1) (v_b_SP_G_2$ ?v1!16)) ?x4523) 0)))))
-(let (($x8251 (or (not (= (+ ?x204 (* (- 1) (v_b_SP_G_2$ ?v1!16)) ?x4523) 0)) (<= (+ ?x204 (* (- 1) (v_b_SP_G_2$ ?v1!16)) ?x4523) 0))))
-(let ((@x8191 (unit-resolution ((_ th-lemma arith triangle-eq) $x8251) @x8211 (not (= (+ ?x204 (* (- 1) (v_b_SP_G_2$ ?v1!16)) ?x4523) 0)))))
-(let (($x7559 (>= (+ ?x204 ?x4523 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v1!16))) 0)))
-(let (($x4525 (<= (+ b_Infinity$ (* (- 1) ?x4523)) 0)))
-(let (($x7564 (or $x4525 $x7559)))
-(let (($x7567 (not $x7564)))
-(let (($x7592 (>= (+ (v_b_SP_G_2$ ?v1!16) (* (- 1) (fun_app$c v_b_SP_G_1$ ?v1!16))) 0)))
-(let ((@x8198 ((_ th-lemma arith farkas -1 -1 1 1 1) (hypothesis $x7592) @x8222 (unit-resolution (mp ((_ quant-inst ?v0!17) (or $x3939 $x5070)) @x7636 $x7629) @x8305 $x7624) @x8299 (hypothesis $x7753) false)))
-(let ((@x8177 (unit-resolution (lemma @x8198 (or $x8196 (not $x7592) $x2175 (not $x7753))) @x8222 @x8299 (hypothesis $x7753) (not $x7592))))
-(let (($x8284 (or (not (= (v_b_SP_G_2$ ?v1!16) (fun_app$c v_b_SP_G_1$ ?v1!16))) $x7592)))
-(let ((@x8185 (unit-resolution ((_ th-lemma arith triangle-eq) $x8284) @x8177 (not (= (v_b_SP_G_2$ ?v1!16) (fun_app$c v_b_SP_G_1$ ?v1!16))))))
-(let ((?x4855 (fun_app$c v_b_SP_G_1$ ?v1!16)))
-(let ((?x2171 (v_b_SP_G_2$ ?v1!16)))
-(let (($x4497 (= ?x2171 ?x4855)))
-(let (($x7570 (or $x7567 $x4497)))
-(let (($x7573 (or $x3931 $x7567 $x4497)))
-(let (($x7574 (or $x3931 (or (not (or $x4525 (<= (+ ?x4855 ?x1520 (* (- 1) ?x4523)) 0))) $x4497))))
-(let (($x7571 (= (or (not (or $x4525 (<= (+ ?x4855 ?x1520 (* (- 1) ?x4523)) 0))) $x4497) $x7570)))
-(let (($x4527 (<= (+ ?x4855 ?x1520 (* (- 1) ?x4523)) 0)))
-(let ((@x7554 (rewrite (= (+ ?x4855 ?x1520 (* (- 1) ?x4523)) (+ ?x1520 (* (- 1) ?x4523) ?x4855)))))
-(let ((@x7557 (monotonicity @x7554 (= $x4527 (<= (+ ?x1520 (* (- 1) ?x4523) ?x4855) 0)))))
-(let ((@x7563 (trans @x7557 (rewrite (= (<= (+ ?x1520 (* (- 1) ?x4523) ?x4855) 0) $x7559)) (= $x4527 $x7559))))
-(let ((@x7569 (monotonicity (monotonicity @x7563 (= (or $x4525 $x4527) $x7564)) (= (not (or $x4525 $x4527)) $x7567))))
-(let ((@x7582 (trans (monotonicity (monotonicity @x7569 $x7571) (= $x7574 (or $x3931 $x7570))) (rewrite (= (or $x3931 $x7570) $x7573)) (= $x7574 $x7573))))
-(let ((@x7879 (unit-resolution (unit-resolution (mp ((_ quant-inst ?v1!16) $x7574) @x7582 $x7573) @x8302 $x7570) @x8185 $x7567)))
-(let ((?x7593 (+ ?x204 (* (- 1) ?x2171) ?x4523)))
-(let (($x7596 (= ?x7593 0)))
-(let (($x7599 (or $x4525 $x7559 $x7596)))
-(let (($x7602 (or $x3923 $x4525 $x7559 $x7596)))
-(let (($x7603 (or $x3923 (or $x4525 $x4527 (= (+ ?x204 ?x4523 (* (- 1) ?x2171)) 0)))))
-(let ((@x7598 (monotonicity (rewrite (= (+ ?x204 ?x4523 (* (- 1) ?x2171)) ?x7593)) (= (= (+ ?x204 ?x4523 (* (- 1) ?x2171)) 0) $x7596))))
-(let ((@x7601 (monotonicity @x7563 @x7598 (= (or $x4525 $x4527 (= (+ ?x204 ?x4523 (* (- 1) ?x2171)) 0)) $x7599))))
-(let ((@x7611 (trans (monotonicity @x7601 (= $x7603 (or $x3923 $x7599))) (rewrite (= (or $x3923 $x7599) $x7602)) (= $x7603 $x7602))))
-(let ((@x7886 (unit-resolution (unit-resolution (mp ((_ quant-inst ?v1!16) $x7603) @x7611 $x7602) @x8165 $x7599) (unit-resolution (def-axiom (or $x7564 (not $x7559))) @x7879 (not $x7559)) (unit-resolution (def-axiom (or $x7564 (not $x4525))) @x7879 (not $x4525)) @x8191 false)))
-(let ((@x7891 (unit-resolution (lemma @x7886 (or $x8196 $x8224 $x2175 (not $x7753))) (unit-resolution @x6202 @x7877 $x8225) (unit-resolution (def-axiom (or $x3034 $x3634)) @x8189 $x3634) @x7874 $x8196)))
-(let ((@x8258 (rewrite (= (or $x3818 (or $x202 $x7513 $x8244)) (or $x3818 $x202 $x7513 $x8244)))))
-(let ((@x8259 (mp ((_ quant-inst ?v0!17 v_b_v_G_1$) (or $x3818 (or $x202 $x7513 $x8244))) @x8258 (or $x3818 $x202 $x7513 $x8244))))
-(let ((@x8237 (unit-resolution @x8259 @x6970 (unit-resolution (def-axiom (or $x4045 $x203)) @x8164 $x203) (hypothesis $x4718) (hypothesis $x8196) false)))
-(let ((@x7896 (unit-resolution (def-axiom (or (not $x7386) $x4687 $x4718)) (unit-resolution (lemma @x8237 (or $x7513 $x8244)) @x7891 $x7513) @x8116 $x4687)))
-(let ((?x2172 (v_b_SP_G_2$ ?v0!17)))
-(let (($x8143 (= ?x2172 ?x3394)))
-(let (($x8113 (not $x8143)))
-(let (($x3298 (>= (+ ?x204 (* (- 1) ?x3394)) 0)))
-(let ((@x8142 (unit-resolution ((_ quant-inst v_b_v_G_1$) (or $x3939 $x3298)) @x8305 $x3298)))
-(let (($x7700 (>= (+ ?x2172 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0!17))) 0)))
-(let ((?x4678 (fun_app$c v_b_SP_G_1$ ?v0!17)))
-(let (($x4679 (= ?x2172 ?x4678)))
-(let ((@x7441 (mp ((_ quant-inst ?v0!17) (or $x3948 (or $x3019 $x4679))) (rewrite (= (or $x3948 (or $x3019 $x4679)) (or $x3948 $x3019 $x4679))) (or $x3948 $x3019 $x4679))))
-(let ((@x7894 (unit-resolution @x7441 (hypothesis $x3943) (unit-resolution (def-axiom (or $x3034 $x2168)) @x8189 $x2168) $x4679)))
-(let (($x7901 (or $x8244 (not (<= (+ ?x2172 (* (- 1) ?x3394)) 0)) (not $x7700) (not $x3298))))
-(let ((@x5877 (unit-resolution ((_ th-lemma arith assign-bounds 1 -1 -1) $x7901) @x7891 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x4679) $x7700)) @x7894 $x7700) @x8142 (not (<= (+ ?x2172 (* (- 1) ?x3394)) 0)))))
-(let ((@x5587 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x8113 (<= (+ ?x2172 (* (- 1) ?x3394)) 0))) @x5877 $x8113)))
-(let ((@x8137 (unit-resolution (hypothesis $x8113) (monotonicity (hypothesis $x4687) $x8143) false)))
-(let ((@x5143 (lemma (unit-resolution (lemma @x8137 (or (not $x4687) $x8143)) @x5587 @x7896 false) (or $x3034 $x3948))))
-(let ((@x7027 (hypothesis $x2154)))
-(let ((@x5873 (hypothesis $x4048)))
-(let ((@x5974 (unit-resolution (def-axiom (or $x4045 $x3926)) @x5873 $x3926)))
-(let ((@x5247 (unit-resolution (def-axiom (or $x4045 $x3918)) @x5873 $x3918)))
-(let ((?x6040 (b_G$ (pair$ v_b_v_G_1$ ?v0!15))))
-(let ((?x6162 (+ ?x204 (* (- 1) ?x2152) ?x6040)))
-(let (($x5552 (= ?x6162 0)))
-(let (($x7159 (not $x5552)))
-(let (($x6237 (<= ?x6162 0)))
-(let (($x7034 (not $x6237)))
-(let ((?x3280 (?v1!7 v_b_v_G_1$)))
-(let ((?x3281 (fun_app$c v_b_SP_G_1$ ?x3280)))
-(let ((?x3282 (* (- 1) ?x3281)))
-(let (($x4633 (<= (+ b_Infinity$ ?x3282) 0)))
-(let (($x6507 (not $x4633)))
-(let (($x4951 (>= (+ ?x204 ?x3282) 0)))
-(let (($x3284 (<= (+ ?x204 ?x3282) 0)))
-(let (($x4138 (not $x3284)))
-(let (($x4244 (fun_app$ v_b_Visited_G_1$ b_Source$)))
-(let (($x5095 (not $x4244)))
-(let (($x3279 (= v_b_v_G_1$ b_Source$)))
-(let (($x6104 (not (= (+ ?x204 (* (- 1) (b_G$ (pair$ ?x3280 v_b_v_G_1$))) ?x3282) 0))))
-(let (($x5949 (or $x3284 (not (fun_app$ v_b_Visited_G_1$ ?x3280)) $x6104)))
-(let (($x4583 (not $x5949)))
-(let (($x4896 (or $x3834 $x3279 $x1522 $x4583)))
-(let (($x4103 (not (= (+ ?x204 ?x3282 (* (- 1) (b_G$ (pair$ ?x3280 v_b_v_G_1$)))) 0))))
-(let (($x4106 (or $x3279 $x1522 (not (or $x3284 (not (fun_app$ v_b_Visited_G_1$ ?x3280)) $x4103)))))
-(let (($x4926 (or $x3834 $x4106)))
-(let (($x4565 (= (not (or $x3284 (not (fun_app$ v_b_Visited_G_1$ ?x3280)) $x4103)) $x4583)))
-(let (($x5863 (= (= (+ ?x204 ?x3282 (* (- 1) (b_G$ (pair$ ?x3280 v_b_v_G_1$)))) 0) (= (+ ?x204 (* (- 1) (b_G$ (pair$ ?x3280 v_b_v_G_1$))) ?x3282) 0))))
-(let (($x5947 (= (+ ?x204 ?x3282 (* (- 1) (b_G$ (pair$ ?x3280 v_b_v_G_1$)))) (+ ?x204 (* (- 1) (b_G$ (pair$ ?x3280 v_b_v_G_1$))) ?x3282))))
-(let ((@x5489 (monotonicity (monotonicity (monotonicity (rewrite $x5947) $x5863) (= $x4103 $x6104)) (= (or $x3284 (not (fun_app$ v_b_Visited_G_1$ ?x3280)) $x4103) $x5949))))
-(let ((@x4548 (monotonicity (monotonicity (monotonicity @x5489 $x4565) (= $x4106 (or $x3279 $x1522 $x4583))) (= $x4926 (or $x3834 (or $x3279 $x1522 $x4583))))))
-(let ((@x4802 (trans @x4548 (rewrite (= (or $x3834 (or $x3279 $x1522 $x4583)) $x4896)) (= $x4926 $x4896))))
-(let ((@x6065 (unit-resolution (mp ((_ quant-inst v_b_v_G_1$) $x4926) @x4802 $x4896) @x4406 (unit-resolution (def-axiom (or $x4045 $x1525)) @x5873 $x1525) (unit-resolution (def-axiom (or $x5949 $x4138)) (hypothesis $x3284) $x5949) $x3279)))
-(let ((@x5493 (mp (unit-resolution (def-axiom (or $x4045 $x203)) @x5873 $x203) (monotonicity (monotonicity @x6065 (= $x202 $x4244)) (= $x203 $x5095)) $x5095)))
-(let ((@x5435 (unit-resolution (def-axiom (or $x4042 $x2122 $x4036)) (unit-resolution (lemma @x6749 (or $x2121 $x3923 $x3931)) @x5247 @x5974 $x2121) (unit-resolution (def-axiom (or $x4045 $x4039)) @x5873 $x4039) $x4036)))
-(let ((@x7140 (symm (commutativity (= (= b_Source$ ?v0!15) (= ?v0!15 b_Source$))) (= (= ?v0!15 b_Source$) (= b_Source$ ?v0!15)))))
-(let ((@x7142 (monotonicity @x7140 (= (not (= ?v0!15 b_Source$)) (not (= b_Source$ ?v0!15))))))
-(let (($x6380 (= ?v0!15 b_Source$)))
-(let (($x6990 (not $x6380)))
-(let (($x6954 (or $x6380 (fun_app$ v_b_Visited_G_1$ ?v0!15))))
-(let ((?x6005 (fun_app$a (fun_app$b (fun_upd$ v_b_Visited_G_1$) b_Source$) true)))
-(let (($x6887 (fun_app$ ?x6005 ?v0!15)))
-(let (($x6951 (= $x6887 $x6954)))
-(let (($x6959 (or $x5105 $x6951)))
-(let (($x6960 (or $x5105 (= $x6887 (ite $x6380 true (fun_app$ v_b_Visited_G_1$ ?v0!15))))))
-(let (($x6957 (= (= $x6887 (ite $x6380 true (fun_app$ v_b_Visited_G_1$ ?v0!15))) $x6951)))
-(let ((@x6956 (rewrite (= (ite $x6380 true (fun_app$ v_b_Visited_G_1$ ?v0!15)) $x6954))))
-(let ((@x6989 (trans (monotonicity (monotonicity @x6956 $x6957) (= $x6960 $x6959)) (rewrite (= $x6959 $x6959)) (= $x6960 $x6959))))
-(let (($x6793 (= (fun_app$b (fun_upd$ v_b_Visited_G_1$) b_Source$) (fun_app$b (fun_upd$ v_b_Visited_G_1$) v_b_v_G_1$))))
-(let ((@x5780 (hypothesis $x3279)))
-(let ((@x5781 (symm @x5780 (= b_Source$ v_b_v_G_1$))))
-(let ((@x6803 (trans (monotonicity (monotonicity @x5781 $x6793) (= ?x6005 ?x212)) (symm (hypothesis $x213) (= ?x212 v_b_Visited_G_2$)) (= ?x6005 v_b_Visited_G_2$))))
-(let ((@x7131 (symm (monotonicity @x6803 (= $x6887 (fun_app$ v_b_Visited_G_2$ ?v0!15))) (= (fun_app$ v_b_Visited_G_2$ ?v0!15) $x6887))))
-(let ((@x7133 (monotonicity @x7131 (= (not (fun_app$ v_b_Visited_G_2$ ?v0!15)) (not $x6887)))))
-(let (($x5938 (fun_app$ v_b_Visited_G_2$ ?v0!15)))
-(let (($x5943 (not $x5938)))
-(let ((?x5971 (fun_app$c v_b_SP_G_1$ ?v0!15)))
-(let (($x6392 (>= ?x5971 0)))
-(let ((@x5502 (unit-resolution (def-axiom (or $x4057 $x3804)) @x5453 $x3804)))
-(let ((@x7119 ((_ th-lemma arith assign-bounds -1 1) (or (not (>= (+ ?x2152 (* (- 1) ?x5971)) 0)) $x2153 (not $x6392)))))
-(let ((@x7120 (unit-resolution @x7119 (unit-resolution ((_ quant-inst ?v0!15) (or $x3809 $x6392)) @x5502 $x6392) @x7027 (not (>= (+ ?x2152 (* (- 1) ?x5971)) 0)))))
-(let ((@x7123 ((_ th-lemma arith triangle-eq) (or (not (= ?x2152 ?x5971)) (>= (+ ?x2152 (* (- 1) ?x5971)) 0)))))
-(let (($x5994 (= (or $x3948 (or $x5943 (= ?x2152 ?x5971))) (or $x3948 $x5943 (= ?x2152 ?x5971)))))
-(let ((@x6100 (mp ((_ quant-inst ?v0!15) (or $x3948 (or $x5943 (= ?x2152 ?x5971)))) (rewrite $x5994) (or $x3948 $x5943 (= ?x2152 ?x5971)))))
-(let ((@x7127 (unit-resolution (unit-resolution @x6100 (hypothesis $x3943) (or $x5943 (= ?x2152 ?x5971))) (unit-resolution @x7123 @x7120 (not (= ?x2152 ?x5971))) $x5943)))
-(let ((@x7135 (unit-resolution (def-axiom (or (not $x6951) $x6887 (not $x6954))) (mp @x7127 @x7133 (not $x6887)) (unit-resolution (mp ((_ quant-inst v_b_Visited_G_1$ b_Source$ true ?v0!15) $x6960) @x6989 $x6959) @x3721 $x6951) (not $x6954))))
-(let ((@x7143 (mp (unit-resolution (def-axiom (or $x6954 $x6990)) @x7135 $x6990) @x7142 (not (= b_Source$ ?v0!15)))))
-(let ((?x7024 (b_G$ (pair$ b_Source$ ?v0!15))))
-(let (($x7048 (<= ?x7024 0)))
-(let (($x7084 (>= (+ ?x6040 (* (- 1) ?x7024)) 0)))
-(let ((@x7145 (monotonicity @x5781 (= (pair$ b_Source$ ?v0!15) (pair$ v_b_v_G_1$ ?v0!15)))))
-(let ((@x7152 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x6040 ?x7024)) $x7084)) (symm (monotonicity @x7145 (= ?x7024 ?x6040)) (= ?x6040 ?x7024)) $x7084)))
-(let (($x6014 (<= (+ ?x119 ?x1520) 0)))
-(let ((@x5742 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x119 ?x204)) $x6014)) (symm (monotonicity @x5780 (= ?x204 ?x119)) (= ?x119 ?x204)) $x6014)))
-(let (($x3478 (>= ?x119 0)))
-(let ((@x6523 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x3213 $x3478)) @x5456 $x3478)))
-(let (($x5984 (>= (+ ?x204 (* (- 1) ?x5971) ?x6040) 0)))
-(let (($x6042 (<= (+ b_Infinity$ (* (- 1) ?x6040)) 0)))
-(let (($x5545 (or $x6042 $x5984)))
-(let (($x5577 (not $x5545)))
-(let (($x5972 (= ?x2152 ?x5971)))
-(let (($x6132 (or $x5577 $x5972)))
-(let (($x6394 (or $x3931 $x5577 $x5972)))
-(let (($x6213 (or $x3931 (or (not (or $x6042 (<= (+ ?x5971 ?x1520 (* (- 1) ?x6040)) 0))) $x5972))))
-(let (($x6240 (= (or (not (or $x6042 (<= (+ ?x5971 ?x1520 (* (- 1) ?x6040)) 0))) $x5972) $x6132)))
-(let (($x6044 (<= (+ ?x5971 ?x1520 (* (- 1) ?x6040)) 0)))
-(let ((@x6156 (rewrite (= (+ ?x5971 ?x1520 (* (- 1) ?x6040)) (+ ?x1520 ?x5971 (* (- 1) ?x6040))))))
-(let ((@x5992 (monotonicity @x6156 (= $x6044 (<= (+ ?x1520 ?x5971 (* (- 1) ?x6040)) 0)))))
-(let ((@x5651 (trans @x5992 (rewrite (= (<= (+ ?x1520 ?x5971 (* (- 1) ?x6040)) 0) $x5984)) (= $x6044 $x5984))))
-(let ((@x5893 (monotonicity (monotonicity @x5651 (= (or $x6042 $x6044) $x5545)) (= (not (or $x6042 $x6044)) $x5577))))
-(let ((@x5887 (trans (monotonicity (monotonicity @x5893 $x6240) (= $x6213 (or $x3931 $x6132))) (rewrite (= (or $x3931 $x6132) $x6394)) (= $x6213 $x6394))))
-(let ((@x7154 (unit-resolution (unit-resolution (mp ((_ quant-inst ?v0!15) $x6213) @x5887 $x6394) @x6086 $x6132) (unit-resolution @x7123 @x7120 (not $x5972)) $x5577)))
-(let (($x5495 (or $x6042 $x5984 $x5552)))
-(let (($x5652 (or $x3923 $x6042 $x5984 $x5552)))
-(let (($x5496 (or $x3923 (or $x6042 $x6044 (= (+ ?x204 ?x6040 (* (- 1) ?x2152)) 0)))))
-(let ((@x5529 (monotonicity (rewrite (= (+ ?x204 ?x6040 (* (- 1) ?x2152)) ?x6162)) (= (= (+ ?x204 ?x6040 (* (- 1) ?x2152)) 0) $x5552))))
-(let ((@x5649 (monotonicity @x5651 @x5529 (= (or $x6042 $x6044 (= (+ ?x204 ?x6040 (* (- 1) ?x2152)) 0)) $x5495))))
-(let ((@x5906 (trans (monotonicity @x5649 (= $x5496 (or $x3923 $x5495))) (rewrite (= (or $x3923 $x5495) $x5652)) (= $x5496 $x5652))))
-(let ((@x7158 (unit-resolution (unit-resolution (mp ((_ quant-inst ?v0!15) $x5496) @x5906 $x5652) @x4512 $x5495) (unit-resolution (def-axiom (or $x5545 (not $x5984))) @x7154 (not $x5984)) (unit-resolution (def-axiom (or $x5545 (not $x6042))) @x7154 (not $x6042)) $x5552)))
-(let ((@x7166 (unit-resolution ((_ th-lemma arith assign-bounds 1 1 1 1 1) (or $x7048 (not $x7084) $x2153 $x7034 (not $x6014) (not $x3478))) (unit-resolution ((_ th-lemma arith triangle-eq) (or $x7159 $x6237)) @x7158 $x6237) @x6523 @x5742 @x7027 @x7152 $x7048)))
-(let (($x7062 (= (or (not $x3728) (or (= b_Source$ ?v0!15) (not $x7048))) (or (not $x3728) (= b_Source$ ?v0!15) (not $x7048)))))
-(let ((@x7064 (mp ((_ quant-inst b_Source$ ?v0!15) (or (not $x3728) (or (= b_Source$ ?v0!15) (not $x7048)))) (rewrite $x7062) (or (not $x3728) (= b_Source$ ?v0!15) (not $x7048)))))
-(let ((@x7168 (unit-resolution (unit-resolution @x7064 @x3733 (or (= b_Source$ ?v0!15) (not $x7048))) @x7166 @x7143 false)))
-(let ((@x6972 (unit-resolution (lemma @x7168 (or $x3948 $x2153 (not $x3279) $x3196 $x3923 $x3931)) @x6065 @x7027 (unit-resolution (def-axiom (or $x4045 $x213)) @x5873 $x213) @x5247 @x5974 $x3948)))
-(let ((@x6196 (unit-resolution (def-axiom (or $x4030 $x2139 $x4024)) (unit-resolution (def-axiom (or $x4021 $x3943)) @x6972 $x4021) (unit-resolution (def-axiom (or $x4033 $x4027)) @x5435 $x4027) $x2139)))
-(let (($x6189 (>= (+ ?x6353 (* (- 1) (b_G$ (pair$ b_Source$ ?v0!14)))) 0)))
-(let ((@x5870 (monotonicity @x5780 (= (pair$ v_b_v_G_1$ ?v0!14) (pair$ b_Source$ ?v0!14)))))
-(let ((@x6892 ((_ th-lemma arith triangle-eq) (or (not (= ?x6353 (b_G$ (pair$ b_Source$ ?v0!14)))) $x6189))))
-(let ((@x6893 (unit-resolution @x6892 (monotonicity @x5870 (= ?x6353 (b_G$ (pair$ b_Source$ ?v0!14)))) $x6189)))
-(let ((?x6449 (b_G$ (pair$ b_Source$ ?v0!14))))
-(let (($x6497 (<= ?x6449 0)))
-(let (($x6702 (not $x6497)))
-(let (($x6238 (= b_Source$ ?v0!14)))
-(let (($x6704 (not $x6238)))
-(let ((@x5923 (monotonicity (symm (hypothesis $x6238) (= ?v0!14 b_Source$)) (= ?x2136 ?x119))))
-(let ((@x5826 (monotonicity (symm (hypothesis $x6238) (= ?v0!14 b_Source$)) (= ?x2135 ?x243))))
-(let ((@x5929 (trans (trans @x5826 (monotonicity @x5781 (= ?x243 ?x3394)) (= ?x2135 ?x3394)) (hypothesis $x3329) (= ?x2135 ?x204))))
-(let ((@x6701 (trans (trans @x5929 (monotonicity @x5780 (= ?x204 ?x119)) (= ?x2135 ?x119)) (symm @x5923 (= ?x119 ?x2136)) $x2137)))
-(let ((@x6754 (lemma (unit-resolution @x5806 @x6701 false) (or $x6704 $x2137 (not $x3329) (not $x3279)))))
-(let ((@x6858 (rewrite (= (or (not $x3728) (or $x6238 $x6702)) (or (not $x3728) $x6238 $x6702)))))
-(let ((@x6859 (mp ((_ quant-inst b_Source$ ?v0!14) (or (not $x3728) (or $x6238 $x6702))) @x6858 (or (not $x3728) $x6238 $x6702))))
-(let ((@x6879 (unit-resolution @x6859 @x3733 (unit-resolution @x6754 @x5806 @x6230 @x5780 $x6704) $x6702)))
-(let (($x5364 (= ?v0!14 b_Source$)))
-(let (($x6300 (or $x5364 $x6262)))
-(let (($x6211 (fun_app$ ?x6005 ?v0!14)))
-(let (($x6870 (= $x6211 $x6300)))
-(let (($x6873 (or $x5105 $x6870)))
-(let ((@x6868 (monotonicity (rewrite (= (ite $x5364 true $x6262) $x6300)) (= (= $x6211 (ite $x5364 true $x6262)) $x6870))))
-(let ((@x6944 (monotonicity @x6868 (= (or $x5105 (= $x6211 (ite $x5364 true $x6262))) $x6873))))
-(let ((@x6946 (trans @x6944 (rewrite (= $x6873 $x6873)) (= (or $x5105 (= $x6211 (ite $x5364 true $x6262))) $x6873))))
-(let ((@x6947 (mp ((_ quant-inst v_b_Visited_G_1$ b_Source$ true ?v0!14) (or $x5105 (= $x6211 (ite $x5364 true $x6262)))) @x6946 $x6873)))
-(let ((@x6885 (mp (hypothesis $x2133) (symm (monotonicity @x6803 (= $x6211 $x2133)) (= $x2133 $x6211)) $x6211)))
-(let ((@x6923 (unit-resolution (def-axiom (or (not $x6870) (not $x6211) $x6300)) @x6885 (unit-resolution @x6947 @x3721 $x6870) $x6300)))
-(let (($x6603 (>= (+ ?x119 (* (- 1) ?x2136)) 0)))
-(let ((@x6948 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x6449 0)) $x6497)) (hypothesis $x6702) (not (= ?x6449 0)))))
-(let (($x6718 (= (or $x4439 (or $x6704 (= ?x6449 0))) (or $x4439 $x6704 (= ?x6449 0)))))
-(let ((@x5740 (mp ((_ quant-inst b_Source$ ?v0!14) (or $x4439 (or $x6704 (= ?x6449 0)))) (rewrite $x6718) (or $x4439 $x6704 (= ?x6449 0)))))
-(let ((@x6975 (unit-resolution (unit-resolution @x5740 @x3727 (or $x6704 (= ?x6449 0))) @x6948 $x6704)))
-(let ((@x6981 (mp @x6975 (monotonicity (commutativity (= $x6238 $x5364)) (= $x6704 (not $x5364))) (not $x5364))))
-(let ((@x6938 (unit-resolution (def-axiom (or (not $x6300) $x5364 $x6262)) @x6981 (hypothesis $x6300) $x6262)))
-(let ((@x6605 (rewrite (= (or $x3818 (or $x4244 $x6006 $x6603)) (or $x3818 $x4244 $x6006 $x6603)))))
-(let ((@x6664 (mp ((_ quant-inst ?v0!14 b_Source$) (or $x3818 (or $x4244 $x6006 $x6603))) @x6605 (or $x3818 $x4244 $x6006 $x6603))))
-(let ((@x6832 (unit-resolution ((_ th-lemma arith farkas 1 1) (or (>= ?x6449 0) $x6497)) (hypothesis $x6702) (>= ?x6449 0))))
-(let ((@x6833 ((_ th-lemma arith farkas 1 1 -1 -1 1) @x6832 (hypothesis $x6189) @x6842 (hypothesis $x6014) (unit-resolution @x6664 @x6970 (hypothesis $x5095) @x6938 $x6603) false)))
-(let ((@x6924 (unit-resolution (lemma @x6833 (or $x6497 (not $x6189) $x5623 (not $x6014) $x4244 (not $x6300))) @x6923 @x6879 @x6877 @x5742 (hypothesis $x5095) @x6893 false)))
-(let ((@x6199 (unit-resolution (lemma @x6924 (or $x2134 $x4244 $x3196 (not $x3279) $x3931 $x2137)) (unit-resolution (def-axiom (or $x2138 $x3646)) @x6196 $x3646) (unit-resolution (def-axiom (or $x2138 $x2133)) @x6196 $x2133) (unit-resolution (def-axiom (or $x4045 $x213)) @x5873 $x213) @x6065 @x5974 @x5493 false)))
-(let ((@x7353 (unit-resolution ((_ th-lemma arith farkas 1 1) (or $x3284 $x4951)) (unit-resolution (lemma @x6199 (or $x4045 $x2153 $x4138)) @x5873 @x7027 $x4138) $x4951)))
-(let ((@x7331 (unit-resolution ((_ th-lemma arith assign-bounds 1 1) (or $x6507 $x1522 (not $x4951))) @x7353 (unit-resolution (def-axiom (or $x4045 $x1525)) @x5873 $x1525) $x6507)))
-(let (($x6440 (= v_b_v_G_1$ ?v0!15)))
-(let (($x6441 (<= ?x6040 0)))
-(let (($x6477 (<= (+ ?x119 ?x3282) 0)))
-(let (($x4627 (= ?x3280 b_Source$)))
-(let ((?x5260 (+ ?x3281 (* (- 1) (fun_app$c v_b_SP_G_1$ (?v1!7 ?x3280))) (* (- 1) (b_G$ (pair$ (?v1!7 ?x3280) ?x3280))))))
-(let (($x5252 (<= (+ ?x3281 (* (- 1) (fun_app$c v_b_SP_G_1$ (?v1!7 ?x3280)))) 0)))
-(let (($x4638 (or $x5252 (not (fun_app$ v_b_Visited_G_1$ (?v1!7 ?x3280))) (not (= ?x5260 0)))))
-(let ((@x7029 (hypothesis $x4951)))
-(let ((@x7028 (hypothesis $x6237)))
-(let ((@x7030 (hypothesis (not $x5252))))
-(let (($x6656 (>= (fun_app$c v_b_SP_G_1$ (?v1!7 ?x3280)) 0)))
-(let ((@x6836 (unit-resolution ((_ th-lemma arith assign-bounds 1 1 1 1 1) (or $x6441 (not $x4951) (not $x6656) $x5252 $x2153 $x7034)) @x7030 @x7029 @x7028 @x7027 (unit-resolution ((_ quant-inst (?v1!7 ?x3280)) (or $x3809 $x6656)) @x5502 $x6656) $x6441)))
-(let (($x6469 (= (or (not $x3728) (or $x6440 (not $x6441))) (or (not $x3728) $x6440 (not $x6441)))))
-(let ((@x6472 (mp ((_ quant-inst v_b_v_G_1$ ?v0!15) (or (not $x3728) (or $x6440 (not $x6441)))) (rewrite $x6469) (or (not $x3728) $x6440 (not $x6441)))))
-(let ((@x7025 (unit-resolution (unit-resolution @x6472 @x3733 (or $x6440 (not $x6441))) (hypothesis $x6441) $x6440)))
-(let (($x6466 (= ?x6040 0)))
-(let (($x7038 (not $x6466)))
-(let (($x7031 (not (>= ?x6040 0))))
-(let ((@x7037 (unit-resolution ((_ th-lemma arith assign-bounds 1 1 1 1 1) (or $x7031 (not $x4951) (not $x6656) $x5252 $x2153 $x7034)) @x7030 @x7029 @x7028 @x7027 (unit-resolution ((_ quant-inst (?v1!7 ?x3280)) (or $x3809 $x6656)) @x5502 $x6656) $x7031)))
-(let ((@x6480 (rewrite (= (or $x4439 (or (not $x6440) $x6466)) (or $x4439 (not $x6440) $x6466)))))
-(let ((@x6481 (mp ((_ quant-inst v_b_v_G_1$ ?v0!15) (or $x4439 (or (not $x6440) $x6466))) @x6480 (or $x4439 (not $x6440) $x6466))))
-(let ((@x7043 (unit-resolution (unit-resolution @x6481 @x3727 (or (not $x6440) $x6466)) (unit-resolution ((_ th-lemma arith triangle-eq) (or $x7038 (>= ?x6040 0))) @x7037 $x7038) @x7025 false)))
-(let ((@x6866 (unit-resolution (lemma @x7043 (or (not $x6441) $x5252 (not $x4951) $x7034 $x2153)) @x6836 @x7030 @x7029 @x7028 @x7027 false)))
-(let ((@x6500 (unit-resolution (lemma @x6866 (or $x5252 (not $x4951) $x7034 $x2153)) @x7028 @x7029 @x7027 $x5252)))
-(let (($x5562 (= (or $x3834 (or $x4627 $x4633 (not $x4638))) (or $x3834 $x4627 $x4633 (not $x4638)))))
-(let ((@x5564 (mp ((_ quant-inst (?v1!7 v_b_v_G_1$)) (or $x3834 (or $x4627 $x4633 (not $x4638)))) (rewrite $x5562) (or $x3834 $x4627 $x4633 (not $x4638)))))
-(let ((@x6514 (unit-resolution (unit-resolution @x5564 @x4406 (hypothesis $x6507) (or $x4627 (not $x4638))) (unit-resolution (def-axiom (or $x4638 (not $x5252))) @x6500 $x4638) $x4627)))
-(let ((@x6521 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x119 ?x3281)) $x6477)) (symm (monotonicity @x6514 (= ?x3281 ?x119)) (= ?x119 ?x3281)) $x6477)))
-(let ((@x6529 (unit-resolution ((_ th-lemma arith assign-bounds 1 1 1 1 1) (or $x6441 (not $x4951) $x2153 $x7034 (not $x3478) (not $x6477))) @x7028 @x6523 @x7029 @x7027 @x6521 $x6441)))
-(let ((@x6534 (unit-resolution (unit-resolution @x6472 @x3733 (or $x6440 (not $x6441))) @x6529 $x6440)))
-(let ((@x6536 (unit-resolution ((_ th-lemma arith assign-bounds 1 -1 -1 1 -1) (or $x7031 (not $x4951) $x2153 $x7034 (not $x3478) (not $x6477))) @x7028 @x6523 @x7029 @x7027 @x6521 $x7031)))
-(let ((@x6538 (unit-resolution (unit-resolution @x6481 @x3727 (or (not $x6440) $x6466)) (unit-resolution ((_ th-lemma arith triangle-eq) (or $x7038 (>= ?x6040 0))) @x6536 $x7038) @x6534 false)))
-(let ((@x7332 (unit-resolution (lemma @x6538 (or $x7034 (not $x4951) $x2153 $x4633)) @x7353 @x7027 @x7331 $x7034)))
-(let ((@x7339 (unit-resolution (mp ((_ quant-inst ?v0!15) $x5496) @x5906 $x5652) @x4512 (hypothesis $x7159) $x5545)))
-(let ((@x7377 (unit-resolution @x7339 (unit-resolution (def-axiom (or $x5545 (not $x5984))) @x7154 (not $x5984)) (unit-resolution (def-axiom (or $x5545 (not $x6042))) @x7154 (not $x6042)) false)))
-(let ((@x7334 (unit-resolution (lemma @x7377 (or $x5552 $x3923 $x3931 $x2153)) (unit-resolution ((_ th-lemma arith triangle-eq) (or $x7159 $x6237)) @x7332 $x7159) @x5247 @x5974 @x7027 false)))
-(let (($x4282 (= ?x243 ?x119)))
-(let (($x4455 (<= (b_G$ (pair$ v_b_v_G_1$ b_Source$)) 0)))
-(let (($x4147 (>= ?x204 0)))
-(let (($x3479 (<= ?x119 0)))
-(let (($x4279 (<= (+ ?x119 ?x1520 (* (- 1) (b_G$ (pair$ v_b_v_G_1$ b_Source$)))) 0)))
-(let (($x4277 (<= (+ b_Infinity$ (* (- 1) (b_G$ (pair$ v_b_v_G_1$ b_Source$)))) 0)))
-(let (($x4281 (not (or $x4277 $x4279))))
-(let (($x4909 (not $x4282)))
-(let ((@x4883 (hypothesis $x913)))
-(let ((@x4907 (mp (hypothesis $x4282) (monotonicity (hypothesis $x120) (= $x4282 $x244)) $x244)))
-(let ((@x6051 (unit-resolution (lemma (unit-resolution @x4883 @x4907 false) (or $x4909 $x244 $x3213)) @x5456 (or $x4909 $x244))))
-(let ((@x5597 (mp ((_ quant-inst b_Source$) (or $x3931 (or $x4281 $x4282))) (rewrite (= (or $x3931 (or $x4281 $x4282)) (or $x3931 $x4281 $x4282))) (or $x3931 $x4281 $x4282))))
-(let ((@x5875 (unit-resolution (unit-resolution @x5597 @x6086 (or $x4281 $x4282)) (unit-resolution @x6051 @x4883 $x4909) $x4281)))
-(let ((@x5520 (unit-resolution (def-axiom (or (or $x4277 $x4279) (not $x4279))) @x5875 (not $x4279))))
-(let ((@x6090 (unit-resolution ((_ th-lemma arith assign-bounds 1 1 1) (or $x4455 (not $x3479) (not $x4147) $x4279)) @x5520 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x3213 $x3479)) @x5456 $x3479) (unit-resolution ((_ quant-inst v_b_v_G_1$) (or $x3809 $x4147)) @x5502 $x4147) $x4455)))
-(let (($x5519 (= (or (not $x3728) (or $x3279 (not $x4455))) (or (not $x3728) $x3279 (not $x4455)))))
-(let ((@x6055 (mp ((_ quant-inst v_b_v_G_1$ b_Source$) (or (not $x3728) (or $x3279 (not $x4455)))) (rewrite $x5519) (or (not $x3728) $x3279 (not $x4455)))))
-(let ((@x6223 (symm (unit-resolution @x6055 @x3733 @x6090 $x3279) (= b_Source$ v_b_v_G_1$))))
-(let ((@x5727 (trans (trans (monotonicity @x6223 (= ?x243 ?x3394)) @x6230 (= ?x243 ?x204)) (monotonicity (unit-resolution @x6055 @x3733 @x6090 $x3279) (= ?x204 ?x119)) $x4282)))
-(let ((@x5312 (lemma (unit-resolution @x4883 (trans @x5727 @x5456 $x244) false) (or $x244 $x3931))))
-(let ((@x8382 (unit-resolution (def-axiom (or $x4018 $x913 $x2154 $x4012)) (unit-resolution @x5312 @x8302 $x244) (unit-resolution (lemma @x7334 (or $x4045 $x2153)) @x8164 $x2153) (or $x4018 $x4012))))
-(let ((@x9064 (unit-resolution @x8382 (unit-resolution (def-axiom (or $x4021 $x4015)) @x10488 $x4015) $x4012)))
-(let ((@x10157 (unit-resolution (def-axiom (or $x4006 $x3039 $x4000)) (unit-resolution (def-axiom (or $x4009 $x4003)) @x9064 $x4003) (unit-resolution @x5143 @x10489 $x3034) $x4000)))
-(let ((@x8593 (hypothesis $x3988)))
-(let ((?x4618 (fun_app$c v_b_SP_G_1$ ?v0!20)))
-(let (($x4870 (<= (+ ?x4618 (* (- 1) (fun_app$c v_b_SP_G_1$ (?v1!7 ?v0!20)))) 0)))
-(let ((@x5730 (hypothesis $x2221)))
-(let (($x8567 (>= (+ (v_b_SP_G_2$ ?v0!20) (* (- 1) ?x4618)) 0)))
-(let ((?x2217 (v_b_SP_G_2$ ?v0!20)))
-(let (($x4625 (= ?x2217 ?x4618)))
-(let ((?x4660 (b_G$ (pair$ v_b_v_G_1$ ?v0!20))))
-(let ((?x4661 (* (- 1) ?x4660)))
-(let ((?x3395 (* (- 1) ?x3394)))
-(let ((?x8452 (+ ?x2217 ?x3395 ?x4661)))
-(let (($x8388 (<= ?x8452 0)))
-(let (($x8780 (>= ?x8452 0)))
-(let ((@x6097 (unit-resolution ((_ th-lemma arith farkas 1 1) (or $x8780 $x8388)) (hypothesis (not $x8388)) $x8780)))
-(let (($x4663 (<= (+ b_Infinity$ ?x4661) 0)))
-(let (($x4368 (fun_app$ v_b_Visited_G_2$ v_b_v_G_1$)))
-(let ((@x8557 (symm (monotonicity @x8214 (= $x4368 (fun_app$ ?x212 v_b_v_G_1$))) (= (fun_app$ ?x212 v_b_v_G_1$) $x4368))))
-(let (($x3413 (fun_app$ ?x212 v_b_v_G_1$)))
-(let (($x3709 (forall ((?v0 B_Vertex_bool_fun$) (?v1 B_Vertex$) (?v2 Bool) )(!(= (fun_app$ (fun_app$a (fun_app$b (fun_upd$ ?v0) ?v1) ?v2) ?v1) ?v2) :pattern ( (fun_app$a (fun_app$b (fun_upd$ ?v0) ?v1) ?v2) )))
-))
-(let (($x1092 (forall ((?v0 B_Vertex_bool_fun$) (?v1 B_Vertex$) (?v2 Bool) )(= (fun_app$ (fun_app$a (fun_app$b (fun_upd$ ?v0) ?v1) ?v2) ?v1) ?v2))
-))
-(let (($x1089 (= (fun_app$ (fun_app$a (fun_app$b (fun_upd$ ?2) ?1) ?0) ?1) ?0)))
-(let (($x49 (forall ((?v0 B_Vertex_bool_fun$) (?v1 B_Vertex$) (?v2 Bool) )(= (fun_app$ (fun_app$a (fun_app$b (fun_upd$ ?v0) ?v1) ?v2) ?v1) ?v2))
-))
-(let (($x48 (= (fun_app$ (fun_app$a (fun_app$b (fun_upd$ ?2) ?1) ?0) ?1) ?0)))
-(let ((@x1097 (mp (mp (asserted $x49) (rewrite* (= $x49 $x49)) $x49) (quant-intro (rewrite (= $x48 $x1089)) (= $x49 $x1092)) $x1092)))
-(let ((@x3714 (mp (mp~ @x1097 (nnf-pos (refl (~ $x1089 $x1089)) (~ $x1092 $x1092)) $x1092) (quant-intro (refl (= $x1089 $x1089)) (= $x1092 $x3709)) $x3709)))
-(let (($x4545 (or (not $x3709) $x3413)))
-(let ((@x6188 (monotonicity (rewrite (= (= $x3413 true) $x3413)) (= (or (not $x3709) (= $x3413 true)) $x4545))))
-(let ((@x5812 (trans @x6188 (rewrite (= $x4545 $x4545)) (= (or (not $x3709) (= $x3413 true)) $x4545))))
-(let ((@x8745 (unit-resolution (mp ((_ quant-inst v_b_Visited_G_1$ v_b_v_G_1$ true) (or (not $x3709) (= $x3413 true))) @x5812 $x4545) @x3714 $x3413)))
-(let ((@x6205 (hypothesis $x3968)))
-(let (($x4369 (not $x4368)))
-(let (($x9030 (or $x3973 $x4369 $x4663 $x8388)))
-(let (($x9031 (or $x3973 (or $x4369 $x4663 (>= (+ ?x4660 ?x3394 (* (- 1) ?x2217)) 0)))))
-(let (($x8458 (= (or $x4369 $x4663 (>= (+ ?x4660 ?x3394 (* (- 1) ?x2217)) 0)) (or $x4369 $x4663 $x8388))))
-(let (($x8517 (>= (+ ?x4660 ?x3394 (* (- 1) ?x2217)) 0)))
-(let ((@x8896 (rewrite (= (+ ?x4660 ?x3394 (* (- 1) ?x2217)) (+ (* (- 1) ?x2217) ?x3394 ?x4660)))))
-(let ((@x8448 (monotonicity @x8896 (= $x8517 (>= (+ (* (- 1) ?x2217) ?x3394 ?x4660) 0)))))
-(let ((@x8455 (trans @x8448 (rewrite (= (>= (+ (* (- 1) ?x2217) ?x3394 ?x4660) 0) $x8388)) (= $x8517 $x8388))))
-(let ((@x9127 (monotonicity (monotonicity @x8455 $x8458) (= $x9031 (or $x3973 (or $x4369 $x4663 $x8388))))))
-(let ((@x8184 (trans @x9127 (rewrite (= (or $x3973 (or $x4369 $x4663 $x8388)) $x9030)) (= $x9031 $x9030))))
-(let ((@x6333 (unit-resolution (mp ((_ quant-inst ?v0!20 v_b_v_G_1$) $x9031) @x8184 $x9030) @x6205 (mp @x8745 @x8557 $x4368) (hypothesis (not $x8388)) $x4663)))
-(let ((@x5997 (unit-resolution ((_ th-lemma arith assign-bounds 1 -1) (or $x6014 (not $x4147) (not $x3479))) (unit-resolution ((_ quant-inst v_b_v_G_1$) (or $x3809 $x4147)) @x5502 $x4147) (unit-resolution ((_ th-lemma arith triangle-eq) (or $x3213 $x3479)) @x5456 $x3479) $x6014)))
-(let (($x6242 (= ?x204 ?x3394)))
-(let ((@x9345 (mp (unit-resolution (mp ((_ quant-inst v_b_v_G_1$) $x4517) @x5481 $x5387) @x8302 @x6229 $x3329) (symm (commutativity (= $x6242 $x3329)) (= $x3329 $x6242)) $x6242)))
-(let ((@x8936 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x6242) (<= (+ ?x204 ?x3395) 0))) @x9345 (<= (+ ?x204 ?x3395) 0))))
-(let ((@x5629 (lemma ((_ th-lemma arith farkas 1 1 1 1 1 1) @x8936 @x5997 @x6523 @x6333 @x6097 @x5730 false) (or $x8388 $x2220 $x3973))))
-(let ((@x10145 (unit-resolution @x5629 (unit-resolution (def-axiom (or $x3985 $x3968)) @x8593 $x3968) @x5730 $x8388)))
-(let (($x8926 (<= (+ ?x2217 ?x3395) 0)))
-(let (($x8453 (= ?x8452 0)))
-(let ((?x2218 (* (- 1) ?x2217)))
-(let ((?x8793 (+ ?x204 ?x2218 ?x4660)))
-(let (($x8622 (<= ?x8793 0)))
-(let (($x8798 (= ?x8793 0)))
-(let (($x8551 (>= (+ ?x204 (* (- 1) ?x4618) ?x4660) 0)))
-(let (($x8822 (or $x4663 $x8551)))
-(let (($x8685 (not $x8822)))
-(let (($x8574 (or $x8685 $x4625)))
-(let (($x8550 (or $x3931 $x8685 $x4625)))
-(let (($x8571 (or $x3931 (or (not (or $x4663 (<= (+ ?x4618 ?x1520 ?x4661) 0))) $x4625))))
-(let ((@x9375 (monotonicity (rewrite (= (+ ?x4618 ?x1520 ?x4661) (+ ?x1520 ?x4618 ?x4661))) (= (<= (+ ?x4618 ?x1520 ?x4661) 0) (<= (+ ?x1520 ?x4618 ?x4661) 0)))))
-(let ((@x8823 (trans @x9375 (rewrite (= (<= (+ ?x1520 ?x4618 ?x4661) 0) $x8551)) (= (<= (+ ?x4618 ?x1520 ?x4661) 0) $x8551))))
-(let ((@x8684 (monotonicity @x8823 (= (or $x4663 (<= (+ ?x4618 ?x1520 ?x4661) 0)) $x8822))))
-(let ((@x8549 (monotonicity @x8684 (= (not (or $x4663 (<= (+ ?x4618 ?x1520 ?x4661) 0))) $x8685))))
-(let ((@x8576 (monotonicity @x8549 (= (or (not (or $x4663 (<= (+ ?x4618 ?x1520 ?x4661) 0))) $x4625) $x8574))))
-(let ((@x8764 (trans (monotonicity @x8576 (= $x8571 (or $x3931 $x8574))) (rewrite (= (or $x3931 $x8574) $x8550)) (= $x8571 $x8550))))
-(let ((@x10339 (unit-resolution (unit-resolution (mp ((_ quant-inst ?v0!20) $x8571) @x8764 $x8550) @x8302 $x8574) (hypothesis (not $x4625)) $x8685)))
-(let ((@x10165 (unit-resolution (def-axiom (or $x8822 (not $x4663))) (hypothesis $x8685) (not $x4663))))
-(let ((@x10166 (unit-resolution (def-axiom (or $x8822 (not $x8551))) (hypothesis $x8685) (not $x8551))))
-(let (($x8800 (or $x4663 $x8551 $x8798)))
-(let (($x8659 (or $x3923 $x4663 $x8551 $x8798)))
-(let (($x4665 (<= (+ ?x4618 ?x1520 ?x4661) 0)))
-(let (($x9296 (or $x3923 (or $x4663 $x4665 (= (+ ?x204 ?x4660 ?x2218) 0)))))
-(let ((@x8797 (monotonicity (rewrite (= (+ ?x204 ?x4660 ?x2218) ?x8793)) (= (= (+ ?x204 ?x4660 ?x2218) 0) $x8798))))
-(let ((@x8638 (monotonicity @x8823 @x8797 (= (or $x4663 $x4665 (= (+ ?x204 ?x4660 ?x2218) 0)) $x8800))))
-(let ((@x9312 (trans (monotonicity @x8638 (= $x9296 (or $x3923 $x8800))) (rewrite (= (or $x3923 $x8800) $x8659)) (= $x9296 $x8659))))
-(let ((@x10167 (unit-resolution (unit-resolution (mp ((_ quant-inst ?v0!20) $x9296) @x9312 $x8659) @x8165 $x8800) @x10166 @x10165 (hypothesis (not $x8798)) false)))
-(let ((@x10348 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x8798) $x8622)) (unit-resolution (lemma @x10167 (or $x8822 $x8798)) @x10339 $x8798) $x8622)))
-(let ((@x10388 (unit-resolution ((_ th-lemma arith assign-bounds 1 -1) (or (not $x8622) $x8780 (not $x3298))) @x8142 (or (not $x8622) $x8780))))
-(let ((@x10484 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x8453 (not $x8388) (not $x8780))) (hypothesis $x8388) (or $x8453 (not $x8780)))))
-(let ((@x11844 (hypothesis $x3977)))
-(let (($x8695 (not $x8453)))
-(let (($x8690 (or $x3982 $x8926 $x4369 $x8695)))
-(let (($x4741 (>= (+ ?x3394 ?x2218) 0)))
-(let (($x8692 (or $x3982 (or $x4741 $x4369 (not (= (+ ?x3394 ?x2218 ?x4660) 0))))))
-(let (($x9019 (= (or $x4741 $x4369 (not (= (+ ?x3394 ?x2218 ?x4660) 0))) (or $x8926 $x4369 $x8695))))
-(let ((@x8997 (monotonicity (rewrite (= (+ ?x3394 ?x2218 ?x4660) (+ ?x2218 ?x3394 ?x4660))) (= (= (+ ?x3394 ?x2218 ?x4660) 0) (= (+ ?x2218 ?x3394 ?x4660) 0)))))
-(let ((@x9034 (trans @x8997 (rewrite (= (= (+ ?x2218 ?x3394 ?x4660) 0) $x8453)) (= (= (+ ?x3394 ?x2218 ?x4660) 0) $x8453))))
-(let ((@x8397 (monotonicity (rewrite (= (+ ?x3394 ?x2218) (+ ?x2218 ?x3394))) (= $x4741 (>= (+ ?x2218 ?x3394) 0)))))
-(let ((@x9139 (trans @x8397 (rewrite (= (>= (+ ?x2218 ?x3394) 0) $x8926)) (= $x4741 $x8926))))
-(let ((@x9020 (monotonicity @x9139 (monotonicity @x9034 (= (not (= (+ ?x3394 ?x2218 ?x4660) 0)) $x8695)) $x9019)))
-(let ((@x8404 (trans (monotonicity @x9020 (= $x8692 (or $x3982 (or $x8926 $x4369 $x8695)))) (rewrite (= (or $x3982 (or $x8926 $x4369 $x8695)) $x8690)) (= $x8692 $x8690))))
-(let ((@x10486 (unit-resolution (mp ((_ quant-inst v_b_v_G_1$) $x8692) @x8404 $x8690) @x11844 (mp @x8745 @x8557 $x4368) (or $x8926 $x8695))))
-(let ((@x10481 (unit-resolution @x10486 (unit-resolution @x10484 (unit-resolution @x10388 @x10348 $x8780) $x8453) $x8926)))
-(let (($x6460 (not (<= ?x4660 0))))
-(let ((@x10539 (commutativity (= (= v_b_v_G_1$ ?v0!20) (= ?v0!20 v_b_v_G_1$)))))
-(let ((@x10627 (monotonicity (symm @x10539 (= (= ?v0!20 v_b_v_G_1$) (= v_b_v_G_1$ ?v0!20))) (= (not (= ?v0!20 v_b_v_G_1$)) (not (= v_b_v_G_1$ ?v0!20))))))
-(let (($x7719 (= ?v0!20 v_b_v_G_1$)))
-(let (($x10690 (not $x7719)))
-(let (($x10582 (or $x7719 (fun_app$ v_b_Visited_G_1$ ?v0!20))))
-(let (($x7724 (fun_app$ ?x212 ?v0!20)))
-(let (($x10917 (= $x7724 $x10582)))
-(let (($x10865 (or $x5105 $x10917)))
-(let (($x10888 (or $x5105 (= $x7724 (ite $x7719 true (fun_app$ v_b_Visited_G_1$ ?v0!20))))))
-(let (($x10747 (= (= $x7724 (ite $x7719 true (fun_app$ v_b_Visited_G_1$ ?v0!20))) $x10917)))
-(let ((@x9484 (rewrite (= (ite $x7719 true (fun_app$ v_b_Visited_G_1$ ?v0!20)) $x10582))))
-(let ((@x10687 (trans (monotonicity (monotonicity @x9484 $x10747) (= $x10888 $x10865)) (rewrite (= $x10865 $x10865)) (= $x10888 $x10865))))
-(let ((@x8210 (symm @x8214 (= ?x212 v_b_Visited_G_2$))))
-(let ((@x10510 (symm (monotonicity @x8210 (= $x7724 (fun_app$ v_b_Visited_G_2$ ?v0!20))) (= (fun_app$ v_b_Visited_G_2$ ?v0!20) $x7724))))
-(let ((@x10542 (monotonicity @x10510 (= (not (fun_app$ v_b_Visited_G_2$ ?v0!20)) (not $x7724)))))
-(let (($x4503 (fun_app$ v_b_Visited_G_2$ ?v0!20)))
-(let (($x4504 (not $x4503)))
-(let ((@x10611 (mp ((_ quant-inst ?v0!20) (or $x3948 (or $x4504 $x4625))) (rewrite (= (or $x3948 (or $x4504 $x4625)) (or $x3948 $x4504 $x4625))) (or $x3948 $x4504 $x4625))))
-(let ((@x10491 (unit-resolution (unit-resolution @x10611 @x10489 (or $x4504 $x4625)) (hypothesis (not $x4625)) $x4504)))
-(let ((@x10518 (unit-resolution (def-axiom (or (not $x10917) $x7724 (not $x10582))) (mp @x10491 @x10542 (not $x7724)) (unit-resolution (mp ((_ quant-inst v_b_Visited_G_1$ v_b_v_G_1$ true ?v0!20) $x10888) @x10687 $x10865) @x3721 $x10917) (not $x10582))))
-(let ((@x10563 (mp (unit-resolution (def-axiom (or $x10582 $x10690)) @x10518 $x10690) @x10627 (not (= v_b_v_G_1$ ?v0!20)))))
-(let (($x9114 (= (or (not $x3728) (or (= v_b_v_G_1$ ?v0!20) $x6460)) (or (not $x3728) (= v_b_v_G_1$ ?v0!20) $x6460))))
-(let ((@x9115 (mp ((_ quant-inst v_b_v_G_1$ ?v0!20) (or (not $x3728) (or (= v_b_v_G_1$ ?v0!20) $x6460))) (rewrite $x9114) (or (not $x3728) (= v_b_v_G_1$ ?v0!20) $x6460))))
-(let ((@x10566 (unit-resolution (unit-resolution @x9115 @x3733 (or (= v_b_v_G_1$ ?v0!20) $x6460)) @x10563 $x6460)))
-(let ((@x10568 (lemma ((_ th-lemma arith farkas -1 -1 1 1) @x8142 @x10566 @x10348 @x10481 false) (or $x4625 $x3982 (not $x8388)))))
-(let ((@x10170 (unit-resolution @x10568 (unit-resolution (def-axiom (or $x3985 $x3977)) @x8593 $x3977) @x10145 $x4625)))
-(let ((?x4866 (?v1!7 ?v0!20)))
-(let (($x8671 (fun_app$ v_b_Visited_G_2$ ?x4866)))
-(let (($x8672 (not $x8671)))
-(let ((@x11435 (symm (monotonicity @x8210 (= (fun_app$ ?x212 ?x4866) $x8671)) (= $x8671 (fun_app$ ?x212 ?x4866)))))
-(let (($x6693 (<= (+ b_Infinity$ (* (- 1) (b_G$ (pair$ ?x4866 ?v0!20)))) 0)))
-(let (($x11835 (not $x6693)))
-(let ((?x4874 (b_G$ (pair$ ?x4866 ?v0!20))))
-(let ((?x4875 (* (- 1) ?x4874)))
-(let ((?x4876 (+ ?x4618 (* (- 1) (fun_app$c v_b_SP_G_1$ ?x4866)) ?x4875)))
-(let (($x8645 (>= ?x4876 0)))
-(let (($x4877 (= ?x4876 0)))
-(let (($x4878 (not $x4877)))
-(let (($x4879 (or $x4870 (not (fun_app$ v_b_Visited_G_1$ ?x4866)) $x4878)))
-(let (($x4880 (not $x4879)))
-(let (($x4865 (<= (+ b_Infinity$ (* (- 1) ?x4618)) 0)))
-(let (($x8667 (not $x4865)))
-(let ((@x8893 (hypothesis $x8567)))
-(let ((@x8402 (lemma ((_ th-lemma arith farkas 1 -1 1) @x8893 (hypothesis $x4865) @x5730 false) (or $x8667 (not $x8567) $x2220))))
-(let ((@x9038 (rewrite (= (or $x3834 (or $x2215 $x4865 $x4880)) (or $x3834 $x2215 $x4865 $x4880)))))
-(let ((@x9039 (mp ((_ quant-inst ?v0!20) (or $x3834 (or $x2215 $x4865 $x4880))) @x9038 (or $x3834 $x2215 $x4865 $x4880))))
-(let ((@x9273 (unit-resolution (unit-resolution @x9039 @x4406 (hypothesis $x2216) (or $x4865 $x4880)) (unit-resolution @x8402 @x8893 @x5730 $x8667) $x4880)))
-(let ((@x11282 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x4878 $x8645)) (unit-resolution (def-axiom (or $x4879 $x4877)) @x9273 $x4877) $x8645)))
-(let ((?x4867 (fun_app$c v_b_SP_G_1$ ?x4866)))
-(let (($x5337 (>= ?x4867 0)))
-(let ((@x11717 (unit-resolution ((_ th-lemma arith assign-bounds -1 -1 -1 -1) (or $x11835 (not $x8645) $x2220 (not $x8567) (not $x5337))) (unit-resolution ((_ quant-inst (?v1!7 ?v0!20)) (or $x3809 $x5337)) @x5502 $x5337) @x5730 @x8893 @x11282 $x11835)))
-(let (($x9233 (<= ?x4876 0)))
-(let ((@x11182 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x4878 $x9233)) (unit-resolution (def-axiom (or $x4879 $x4877)) @x9273 $x4877) $x9233)))
-(let ((?x8643 (v_b_SP_G_2$ ?x4866)))
-(let ((?x9203 (* (- 1) ?x8643)))
-(let ((?x9103 (+ ?x2217 ?x4875 ?x9203)))
-(let (($x10503 (>= ?x9103 0)))
-(let (($x6233 (>= (+ ?x4867 ?x9203) 0)))
-(let ((@x11833 (unit-resolution ((_ th-lemma arith assign-bounds 1 1 1) (or $x10503 (not $x6233) (not $x8645) (not $x8567))) (hypothesis $x8645) @x8893 (unit-resolution ((_ quant-inst (?v1!7 ?v0!20)) (or $x3939 $x6233)) @x8305 $x6233) $x10503)))
-(let (($x10448 (<= (+ ?x2217 ?x9203) 0)))
-(let (($x11011 (= ?x9103 0)))
-(let (($x10912 (<= ?x9103 0)))
-(let (($x10744 (or $x8672 $x6693 $x10912)))
-(let (($x10746 (or $x3973 $x8672 $x6693 $x10912)))
-(let (($x10750 (or $x3973 (or $x8672 $x6693 (>= (+ ?x4874 ?x8643 ?x2218) 0)))))
-(let ((@x9876 (monotonicity (rewrite (= (+ ?x4874 ?x8643 ?x2218) (+ ?x2218 ?x4874 ?x8643))) (= (>= (+ ?x4874 ?x8643 ?x2218) 0) (>= (+ ?x2218 ?x4874 ?x8643) 0)))))
-(let ((@x10867 (trans @x9876 (rewrite (= (>= (+ ?x2218 ?x4874 ?x8643) 0) $x10912)) (= (>= (+ ?x4874 ?x8643 ?x2218) 0) $x10912))))
-(let ((@x10745 (monotonicity @x10867 (= (or $x8672 $x6693 (>= (+ ?x4874 ?x8643 ?x2218) 0)) $x10744))))
-(let ((@x10734 (trans (monotonicity @x10745 (= $x10750 (or $x3973 $x10744))) (rewrite (= (or $x3973 $x10744) $x10746)) (= $x10750 $x10746))))
-(let ((@x11838 (unit-resolution (unit-resolution (mp ((_ quant-inst ?v0!20 (?v1!7 ?v0!20)) $x10750) @x10734 $x10746) @x6205 $x10744) (hypothesis $x8671) (hypothesis $x11835) $x10912)))
-(let ((@x11843 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x11011 (not $x10912) (not $x10503))) @x11833 @x11838 $x11011)))
-(let (($x10804 (not $x11011)))
-(let (($x11040 (or $x10448 $x8672 $x10804)))
-(let (($x10301 (or $x3982 $x10448 $x8672 $x10804)))
-(let (($x6994 (>= (+ ?x8643 ?x2218) 0)))
-(let (($x10896 (or $x3982 (or $x6994 $x8672 (not (= (+ ?x8643 ?x2218 ?x4874) 0))))))
-(let ((@x11010 (monotonicity (rewrite (= (+ ?x8643 ?x2218 ?x4874) (+ ?x2218 ?x4874 ?x8643))) (= (= (+ ?x8643 ?x2218 ?x4874) 0) (= (+ ?x2218 ?x4874 ?x8643) 0)))))
-(let ((@x10803 (trans @x11010 (rewrite (= (= (+ ?x2218 ?x4874 ?x8643) 0) $x11011)) (= (= (+ ?x8643 ?x2218 ?x4874) 0) $x11011))))
-(let ((@x10440 (monotonicity (rewrite (= (+ ?x8643 ?x2218) (+ ?x2218 ?x8643))) (= $x6994 (>= (+ ?x2218 ?x8643) 0)))))
-(let ((@x10354 (trans @x10440 (rewrite (= (>= (+ ?x2218 ?x8643) 0) $x10448)) (= $x6994 $x10448))))
-(let ((@x10595 (monotonicity @x10354 (monotonicity @x10803 (= (not (= (+ ?x8643 ?x2218 ?x4874) 0)) $x10804)) (= (or $x6994 $x8672 (not (= (+ ?x8643 ?x2218 ?x4874) 0))) $x11040))))
-(let ((@x10685 (trans (monotonicity @x10595 (= $x10896 (or $x3982 $x11040))) (rewrite (= (or $x3982 $x11040) $x10301)) (= $x10896 $x10301))))
-(let ((@x11846 (unit-resolution (unit-resolution (mp ((_ quant-inst (?v1!7 ?v0!20)) $x10896) @x10685 $x10301) @x11844 $x11040) @x11843 (hypothesis $x8671) $x10448)))
-(let ((@x11850 (lemma ((_ th-lemma arith farkas -1 1 -1 1) @x11846 @x11833 (hypothesis $x9233) (hypothesis (not $x4870)) false) (or $x8672 (not $x9233) $x4870 $x3982 (not $x8645) (not $x8567) $x6693 $x3973))))
-(let ((@x11185 (unit-resolution @x11850 @x11182 (hypothesis (not $x4870)) @x11844 @x11282 @x8893 @x11717 @x6205 $x8672)))
-(let ((@x11550 (mp @x11185 (monotonicity @x11435 (= $x8672 (not (fun_app$ ?x212 ?x4866)))) (not (fun_app$ ?x212 ?x4866)))))
-(let (($x11789 (fun_app$ ?x212 ?x4866)))
-(let (($x4871 (fun_app$ v_b_Visited_G_1$ ?x4866)))
-(let (($x11792 (or (= ?x4866 v_b_v_G_1$) $x4871)))
-(let (($x11795 (= $x11789 $x11792)))
-(let (($x11638 (or $x5105 $x11795)))
-(let (($x11557 (= (or $x5105 (= $x11789 (ite (= ?x4866 v_b_v_G_1$) true $x4871))) $x11638)))
-(let ((@x11797 (monotonicity (rewrite (= (ite (= ?x4866 v_b_v_G_1$) true $x4871) $x11792)) (= (= $x11789 (ite (= ?x4866 v_b_v_G_1$) true $x4871)) $x11795))))
-(let ((@x11556 ((_ quant-inst v_b_Visited_G_1$ v_b_v_G_1$ true (?v1!7 ?v0!20)) (or $x5105 (= $x11789 (ite (= ?x4866 v_b_v_G_1$) true $x4871))))))
-(let ((@x11621 (mp @x11556 (trans (monotonicity @x11797 $x11557) (rewrite (= $x11638 $x11638)) $x11557) $x11638)))
-(let ((@x11379 (unit-resolution (def-axiom (or $x11792 (not $x4871))) (unit-resolution (def-axiom (or $x4879 $x4871)) @x9273 $x4871) $x11792)))
-(let ((@x11588 (unit-resolution (def-axiom (or (not $x11795) $x11789 (not $x11792))) @x11379 (or (not $x11795) $x11789))))
-(let ((@x11409 (unit-resolution (unit-resolution @x11588 (unit-resolution @x11621 @x3721 $x11795) $x11789) @x11550 false)))
-(let ((@x9681 (unit-resolution (lemma @x11409 (or (not $x8567) $x4870 $x3982 $x3973 $x2220 $x2215)) (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x4625) $x8567)) @x10170 $x8567) (unit-resolution (def-axiom (or $x3985 $x3977)) @x8593 $x3977) (unit-resolution (def-axiom (or $x3985 $x3968)) @x8593 $x3968) @x5730 (unit-resolution (def-axiom (or $x3985 $x2216)) @x8593 $x2216) $x4870)))
-(let ((@x9302 (unit-resolution @x8402 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x4625) $x8567)) @x10170 $x8567) @x5730 $x8667)))
-(let ((@x10155 (unit-resolution @x9039 @x4406 (unit-resolution (def-axiom (or $x3985 $x2216)) @x8593 $x2216) (or $x4865 $x4880))))
-(let ((@x10236 (unit-resolution (def-axiom (or $x4879 (not $x4870))) (unit-resolution @x10155 @x9302 $x4880) @x9681 false)))
-(let ((@x10357 (unit-resolution (lemma @x10236 (or $x3985 $x2220)) (unit-resolution (def-axiom (or $x3985 $x2221)) @x8593 $x2221) @x8593 false)))
-(let ((@x8697 (unit-resolution (def-axiom (or $x3994 $x3085 $x3988)) (lemma @x10357 $x3985) (unit-resolution (def-axiom (or $x3997 $x3991)) @x10157 $x3991) $x3085)))
-(let (($x2195 (not $x2194)))
-(let (($x4939 (<= (+ b_Infinity$ (* (- 1) (b_G$ (pair$ v_b_v_G_1$ ?v0!19)))) 0)))
-(let ((?x4936 (b_G$ (pair$ v_b_v_G_1$ ?v0!19))))
-(let ((?x4520 (fun_app$c v_b_SP_G_1$ ?v0!19)))
-(let ((?x4919 (* (- 1) ?x4520)))
-(let (($x7104 (>= (+ ?x204 ?x4919 ?x4936) 0)))
-(let (($x8037 (>= (+ ?x2191 (* (- 1) ?x4936)) 0)))
-(let (($x4552 (= ?v1!18 v_b_v_G_1$)))
-(let (($x4560 (fun_app$ v_b_Visited_G_1$ ?v1!18)))
-(let (($x4584 (not $x4560)))
-(let (($x3626 (not $x2202)))
-(let ((@x9184 (hypothesis $x3626)))
-(let (($x8491 (>= (+ ?x2198 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v1!18))) 0)))
-(let ((?x4539 (fun_app$c v_b_SP_G_1$ ?v1!18)))
-(let (($x4537 (= ?x2198 ?x4539)))
-(let ((@x8063 (mp ((_ quant-inst ?v1!18) (or $x3948 (or $x3065 $x4537))) (rewrite (= (or $x3948 (or $x3065 $x4537)) (or $x3948 $x3065 $x4537))) (or $x3948 $x3065 $x4537))))
-(let ((@x10071 (unit-resolution @x8063 @x10489 (unit-resolution (def-axiom (or $x3080 $x2189)) (hypothesis $x3085) $x2189) $x4537)))
-(let (($x9200 (<= (+ (v_b_SP_G_2$ ?v0!19) ?x4919) 0)))
-(let (($x9219 (or $x3939 $x9200)))
-(let ((@x6015 (monotonicity (rewrite (= (+ ?x4520 ?x2200) (+ ?x2200 ?x4520))) (= (>= (+ ?x4520 ?x2200) 0) (>= (+ ?x2200 ?x4520) 0)))))
-(let ((@x9261 (trans @x6015 (rewrite (= (>= (+ ?x2200 ?x4520) 0) $x9200)) (= (>= (+ ?x4520 ?x2200) 0) $x9200))))
-(let ((@x8768 (trans (monotonicity @x9261 (= (or $x3939 (>= (+ ?x4520 ?x2200) 0)) $x9219)) (rewrite (= $x9219 $x9219)) (= (or $x3939 (>= (+ ?x4520 ?x2200) 0)) $x9219))))
-(let ((@x9207 (unit-resolution (mp ((_ quant-inst ?v0!19) (or $x3939 (>= (+ ?x4520 ?x2200) 0))) @x8768 $x9219) @x8305 $x9200)))
-(let ((@x9209 ((_ th-lemma arith farkas 1 -1 -1 1) (hypothesis (>= (+ ?x2191 ?x4919 ?x4539) 0)) @x9207 @x9184 (hypothesis $x8491) false)))
-(let ((@x9157 (lemma @x9209 (or (not (>= (+ ?x2191 ?x4919 ?x4539) 0)) $x2202 (not $x8491)))))
-(let ((@x10062 (unit-resolution @x9157 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x4537) $x8491)) @x10071 $x8491) @x9184 (not (>= (+ ?x2191 ?x4919 ?x4539) 0)))))
-(let (($x8396 (>= (+ ?x2191 ?x4919 ?x4539) 0)))
-(let (($x7250 (or $x3826 $x4584 $x2194 $x8396)))
-(let (($x7254 (or $x3826 (or $x4584 $x2194 (>= (+ ?x2191 ?x4539 ?x4919) 0)))))
-(let (($x7281 (= (or $x4584 $x2194 (>= (+ ?x2191 ?x4539 ?x4919) 0)) (or $x4584 $x2194 $x8396))))
-(let ((@x7279 (monotonicity (rewrite (= (+ ?x2191 ?x4539 ?x4919) (+ ?x2191 ?x4919 ?x4539))) (= (>= (+ ?x2191 ?x4539 ?x4919) 0) $x8396))))
-(let ((@x7262 (monotonicity (monotonicity @x7279 $x7281) (= $x7254 (or $x3826 (or $x4584 $x2194 $x8396))))))
-(let ((@x7275 (trans @x7262 (rewrite (= (or $x3826 (or $x4584 $x2194 $x8396)) $x7250)) (= $x7254 $x7250))))
-(let ((@x10063 (unit-resolution (mp ((_ quant-inst ?v0!19 ?v1!18) $x7254) @x7275 $x7250) @x6172 (unit-resolution (def-axiom (or $x3080 $x2195)) (hypothesis $x3085) $x2195) (or $x4584 $x8396))))
-(let (($x8064 (or $x4552 $x4560)))
-(let (($x4569 (fun_app$ ?x212 ?v1!18)))
-(let (($x7915 (= $x4569 $x8064)))
-(let (($x5802 (or $x5105 $x7915)))
-(let ((@x7808 (monotonicity (rewrite (= (ite $x4552 true $x4560) $x8064)) (= (= $x4569 (ite $x4552 true $x4560)) $x7915))))
-(let ((@x8409 (monotonicity @x7808 (= (or $x5105 (= $x4569 (ite $x4552 true $x4560))) $x5802))))
-(let ((@x8439 (trans @x8409 (rewrite (= $x5802 $x5802)) (= (or $x5105 (= $x4569 (ite $x4552 true $x4560))) $x5802))))
-(let ((@x9247 (mp ((_ quant-inst v_b_Visited_G_1$ v_b_v_G_1$ true ?v1!18) (or $x5105 (= $x4569 (ite $x4552 true $x4560)))) @x8439 $x5802)))
-(let ((@x10467 (mp (unit-resolution (def-axiom (or $x3080 $x2189)) (hypothesis $x3085) $x2189) (symm (monotonicity @x8210 (= $x4569 $x2189)) (= $x2189 $x4569)) $x4569)))
-(let ((@x10247 (unit-resolution (def-axiom (or (not $x7915) (not $x4569) $x8064)) @x10467 (unit-resolution @x9247 @x3721 $x7915) $x8064)))
-(let ((@x10216 (unit-resolution (def-axiom (or (not $x8064) $x4552 $x4560)) @x10247 (unit-resolution @x10063 @x10062 $x4584) $x4552)))
-(let ((@x10847 (monotonicity @x10216 (= (pair$ ?v1!18 ?v0!19) (pair$ v_b_v_G_1$ ?v0!19)))))
-(let ((@x10848 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x2191 ?x4936)) $x8037)) (monotonicity @x10847 (= ?x2191 ?x4936)) $x8037)))
-(let (($x8038 (>= (+ ?x2198 ?x3395) 0)))
-(let ((@x10005 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x2198 ?x3394)) $x8038)) (monotonicity @x10216 (= ?x2198 ?x3394)) $x8038)))
-(let ((@x8468 ((_ th-lemma arith farkas -1 1 -1 -1 1 1) (hypothesis $x8038) @x8936 (hypothesis $x8037) (hypothesis $x7104) @x9207 @x9184 false)))
-(let ((@x9577 (unit-resolution (lemma @x8468 (or (not $x7104) (not $x8038) (not $x8037) $x2202)) @x10005 @x9184 @x10848 (not $x7104))))
-(let ((@x8883 ((_ th-lemma arith farkas -1 1 -1 -1 1) (hypothesis $x8038) @x8936 (hypothesis $x8037) (hypothesis (>= (+ ?x204 ?x2200 ?x4936) 0)) @x9184 false)))
-(let ((@x9326 (lemma @x8883 (or (not (>= (+ ?x204 ?x2200 ?x4936) 0)) (not $x8038) (not $x8037) $x2202))))
-(let ((@x9398 (unit-resolution @x9326 @x10848 @x9184 @x10005 (not (>= (+ ?x204 ?x2200 ?x4936) 0)))))
-(let ((?x7186 (+ ?x204 ?x2200 ?x4936)))
-(let (($x7258 (>= ?x7186 0)))
-(let ((@x8781 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x7186 0)) $x7258)) @x9398 (not (= ?x7186 0)))))
-(let (($x7111 (= ?x7186 0)))
-(let (($x7222 (or $x4939 $x7104 $x7111)))
-(let (($x7201 (or $x3923 $x4939 $x7104 $x7111)))
-(let (($x4941 (<= (+ ?x4520 ?x1520 (* (- 1) ?x4936)) 0)))
-(let (($x7208 (or $x3923 (or $x4939 $x4941 (= (+ ?x204 ?x4936 ?x2200) 0)))))
-(let ((@x7190 (monotonicity (rewrite (= (+ ?x204 ?x4936 ?x2200) ?x7186)) (= (= (+ ?x204 ?x4936 ?x2200) 0) $x7111))))
-(let ((@x7077 (rewrite (= (+ ?x4520 ?x1520 (* (- 1) ?x4936)) (+ ?x1520 ?x4520 (* (- 1) ?x4936))))))
-(let ((@x7001 (monotonicity @x7077 (= $x4941 (<= (+ ?x1520 ?x4520 (* (- 1) ?x4936)) 0)))))
-(let ((@x7110 (trans @x7001 (rewrite (= (<= (+ ?x1520 ?x4520 (* (- 1) ?x4936)) 0) $x7104)) (= $x4941 $x7104))))
-(let ((@x7200 (monotonicity @x7110 @x7190 (= (or $x4939 $x4941 (= (+ ?x204 ?x4936 ?x2200) 0)) $x7222))))
-(let ((@x7230 (trans (monotonicity @x7200 (= $x7208 (or $x3923 $x7222))) (rewrite (= (or $x3923 $x7222) $x7201)) (= $x7208 $x7201))))
-(let ((@x8782 (unit-resolution (unit-resolution (mp ((_ quant-inst ?v0!19) $x7208) @x7230 $x7201) @x8165 $x7222) @x8781 @x9577 $x4939)))
-(let ((@x7246 ((_ th-lemma arith farkas 1 -1 1) @x10848 @x8782 (unit-resolution (def-axiom (or $x3080 $x2195)) (hypothesis $x3085) $x2195) false)))
-(unit-resolution (lemma @x7246 (or $x3080 $x2202)) (unit-resolution (def-axiom (or $x3080 $x3626)) @x8697 $x3626) @x8697 false)))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))
-
+e3d9ca1db0784558fae8ee48f75145c34159be22 3044 0
+unsat
+((set-logic AUFLIA)
+(declare-fun ?v0!19 () B_Vertex$)
+(declare-fun ?v1!18 () B_Vertex$)
+(declare-fun ?v0!20 () B_Vertex$)
+(declare-fun ?v0!17 () B_Vertex$)
+(declare-fun ?v1!16 () B_Vertex$)
+(declare-fun ?v0!15 () B_Vertex$)
+(declare-fun ?v0!14 () B_Vertex$)
+(declare-fun ?v0!13 () B_Vertex$)
+(declare-fun ?v0!12 () B_Vertex$)
+(declare-fun ?v0!11 () B_Vertex$)
+(declare-fun ?v1!10 () B_Vertex$)
+(declare-fun ?v1!9 (B_Vertex$) B_Vertex$)
+(declare-fun ?v0!8 () B_Vertex$)
+(declare-fun ?v1!7 (B_Vertex$) B_Vertex$)
+(declare-fun ?v1!6 (B_Vertex$) B_Vertex$)
+(declare-fun ?v0!5 () B_Vertex$)
+(declare-fun ?v0!4 () B_Vertex$)
+(declare-fun ?v1!3 () B_Vertex$)
+(declare-fun ?v0!2 () B_Vertex$)
+(declare-fun ?v1!1 () B_Vertex$)
+(declare-fun ?v0!0 () B_Vertex$)
+(proof
+(let ((?x1893 (v_b_SP_G_2$ ?v0!19)))
+(let ((?x1894 (* (- 1) ?x1893)))
+(let ((?x1892 (v_b_SP_G_2$ ?v1!18)))
+(let ((?x1884 (pair$ ?v1!18 ?v0!19)))
+(let ((?x1885 (b_G$ ?x1884)))
+(let (($x1896 (>= (+ ?x1885 ?x1892 ?x1894) 0)))
+(let (($x1888 (<= (+ b_Infinity$ (* (- 1) ?x1885)) 0)))
+(let (($x1883 (fun_app$ v_b_Visited_G_2$ ?v1!18)))
+(let (($x2791 (not $x1883)))
+(let (($x2806 (or $x2791 $x1888 $x1896)))
+(let (($x2811 (not $x2806)))
+(let (($x3729 (forall ((?v1 B_Vertex$) )(!(let ((?x1911 (v_b_SP_G_2$ ?v0!20)))
+(let ((?x1912 (* (- 1) ?x1911)))
+(let ((?x273 (v_b_SP_G_2$ ?v1)))
+(let (($x2242 (= (+ ?x273 ?x1912 (b_G$ (pair$ ?v1 ?v0!20))) 0)))
+(let (($x291 (fun_app$ v_b_Visited_G_2$ ?v1)))
+(let (($x300 (not $x291)))
+(or (>= (+ ?x273 ?x1912) 0) $x300 (not $x2242)))))))) :pattern ( (v_b_SP_G_2$ ?v1) ) :pattern ( (fun_app$ v_b_Visited_G_2$ ?v1) ) :pattern ( (pair$ ?v1 ?v0!20) )))
+))
+(let (($x3734 (not $x3729)))
+(let (($x1914 (<= (+ b_Infinity$ (* (- 1) (v_b_SP_G_2$ ?v0!20))) 0)))
+(let (($x1909 (= ?v0!20 b_Source$)))
+(let (($x3720 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(!(let ((?x303 (v_b_SP_G_2$ ?v0)))
+(let ((?x1263 (* (- 1) ?x303)))
+(let ((?x273 (v_b_SP_G_2$ ?v1)))
+(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let (($x1282 (>= (+ ?x155 ?x273 ?x1263) 0)))
+(let (($x922 (<= (+ b_Infinity$ (* (- 1) ?x155)) 0)))
+(let (($x291 (fun_app$ v_b_Visited_G_2$ ?v1)))
+(let (($x300 (not $x291)))
+(or $x300 $x922 $x1282))))))))) :pattern ( (pair$ ?v1 ?v0) )))
+))
+(let (($x3725 (not $x3720)))
+(let (($x3737 (or $x3725 $x1909 $x1914 $x3734)))
+(let ((?x4393 (fun_app$c v_b_SP_G_1$ ?v0!20)))
+(let ((?x4418 (* (- 1) ?x4393)))
+(let ((?x1911 (v_b_SP_G_2$ ?v0!20)))
+(let ((?x4419 (+ ?x1911 ?x4418)))
+(let (($x5977 (>= ?x4419 0)))
+(let (($x4400 (= ?x1911 ?x4393)))
+(let ((?x4434 (pair$ v_b_v_G_1$ ?v0!20)))
+(let ((?x4435 (b_G$ ?x4434)))
+(let ((?x4436 (* (- 1) ?x4435)))
+(let ((?x3104 (v_b_SP_G_2$ v_b_v_G_1$)))
+(let ((?x3105 (* (- 1) ?x3104)))
+(let ((?x4546 (+ ?x1911 ?x3105 ?x4436)))
+(let (($x4569 (<= ?x4546 0)))
+(let (($x3740 (not $x3737)))
+(let ((@x8092 (hypothesis $x3740)))
+(let ((@x3222 (def-axiom (or $x3737 $x3720))))
+(let (($x4161 (>= ?x3104 0)))
+(let (($x3703 (forall ((?v0 B_Vertex$) )(!(let ((?x273 (v_b_SP_G_2$ ?v0)))
+(>= ?x273 0)) :pattern ( (v_b_SP_G_2$ ?v0) )))
+))
+(let (($x3743 (or $x2811 $x3740)))
+(let (($x3746 (not $x3743)))
+(let (($x3712 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(!(let (($x1262 (>= (+ (v_b_SP_G_2$ ?v1) (* (- 1) (v_b_SP_G_2$ ?v0))) 0)))
+(let (($x301 (fun_app$ v_b_Visited_G_2$ ?v0)))
+(let (($x2768 (not $x301)))
+(let (($x291 (fun_app$ v_b_Visited_G_2$ ?v1)))
+(or $x291 $x2768 $x1262))))) :pattern ( (v_b_SP_G_2$ ?v1) (v_b_SP_G_2$ ?v0) )))
+))
+(let (($x3717 (not $x3712)))
+(let (($x3749 (or $x3717 $x3746)))
+(let (($x3752 (not $x3749)))
+(let (($x1869 (>= (+ (v_b_SP_G_2$ ?v1!16) (* (- 1) (v_b_SP_G_2$ ?v0!17))) 0)))
+(let (($x1862 (fun_app$ v_b_Visited_G_2$ ?v0!17)))
+(let (($x2745 (not $x1862)))
+(let (($x1860 (fun_app$ v_b_Visited_G_2$ ?v1!16)))
+(let (($x2760 (or $x1860 $x2745 $x1869)))
+(let (($x2765 (not $x2760)))
+(let (($x3755 (or $x2765 $x3752)))
+(let (($x3758 (not $x3755)))
+(let (($x3708 (not $x3703)))
+(let (($x3761 (or $x3708 $x3758)))
+(let (($x3764 (not $x3761)))
+(let ((?x1846 (v_b_SP_G_2$ ?v0!15)))
+(let (($x1847 (>= ?x1846 0)))
+(let ((?x257 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
+(let (($x3904 (>= ?x257 0)))
+(let (($x3556 (forall ((?v0 B_Vertex$) )(!(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v0)))
+(>= ?x174 0)) :pattern ( (fun_app$c v_b_SP_G_1$ ?v0) )))
+))
+(let (($x1848 (not $x1847)))
+(let (($x3767 (or $x1848 $x3764)))
+(let (($x3770 (not $x3767)))
+(let ((?x296 (v_b_SP_G_2$ b_Source$)))
+(let (($x297 (= ?x296 0)))
+(let (($x773 (not $x297)))
+(let (($x3773 (or $x773 $x3770)))
+(let (($x3776 (not $x3773)))
+(let (($x3779 (or $x773 $x3776)))
+(let (($x3782 (not $x3779)))
+(let (($x3695 (forall ((?v0 B_Vertex$) )(!(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v0)))
+(let ((?x273 (v_b_SP_G_2$ ?v0)))
+(let (($x278 (= ?x273 ?x174)))
+(let (($x291 (fun_app$ v_b_Visited_G_2$ ?v0)))
+(let (($x300 (not $x291)))
+(or $x300 $x278)))))) :pattern ( (fun_app$ v_b_Visited_G_2$ ?v0) ) :pattern ( (v_b_SP_G_2$ ?v0) ) :pattern ( (fun_app$c v_b_SP_G_1$ ?v0) )))
+))
+(let (($x3700 (not $x3695)))
+(let (($x3785 (or $x3700 $x3782)))
+(let (($x3788 (not $x3785)))
+(let ((?x1827 (fun_app$c v_b_SP_G_1$ ?v0!14)))
+(let ((?x1826 (v_b_SP_G_2$ ?v0!14)))
+(let (($x1828 (= ?x1826 ?x1827)))
+(let (($x1829 (or (not (fun_app$ v_b_Visited_G_2$ ?v0!14)) $x1828)))
+(let (($x1830 (not $x1829)))
+(let (($x3791 (or $x1830 $x3788)))
+(let (($x3794 (not $x3791)))
+(let (($x3686 (forall ((?v0 B_Vertex$) )(!(>= (+ (fun_app$c v_b_SP_G_1$ ?v0) (* (- 1) (v_b_SP_G_2$ ?v0))) 0) :pattern ( (fun_app$c v_b_SP_G_1$ ?v0) ) :pattern ( (v_b_SP_G_2$ ?v0) )))
+))
+(let (($x3691 (not $x3686)))
+(let (($x3797 (or $x3691 $x3794)))
+(let (($x3800 (not $x3797)))
+(let ((?x1809 (v_b_SP_G_2$ ?v0!13)))
+(let ((?x1810 (* (- 1) ?x1809)))
+(let ((?x1808 (fun_app$c v_b_SP_G_1$ ?v0!13)))
+(let ((?x1811 (+ ?x1808 ?x1810)))
+(let (($x1812 (>= ?x1811 0)))
+(let (($x1813 (not $x1812)))
+(let (($x3803 (or $x1813 $x3800)))
+(let (($x3806 (not $x3803)))
+(let (($x3678 (forall ((?v0 B_Vertex$) )(!(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v0)))
+(let ((?x273 (v_b_SP_G_2$ ?v0)))
+(let (($x278 (= ?x273 ?x174)))
+(let ((?x257 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
+(let ((?x1173 (* (- 1) ?x257)))
+(let (($x1175 (<= (+ ?x174 ?x1173 (* (- 1) (b_G$ (pair$ v_b_v_G_1$ ?v0)))) 0)))
+(let (($x1169 (<= (+ b_Infinity$ (* (- 1) (b_G$ (pair$ v_b_v_G_1$ ?v0)))) 0)))
+(let (($x2717 (or $x1169 $x1175)))
+(let (($x2718 (not $x2717)))
+(or $x2718 $x278)))))))))) :pattern ( (pair$ v_b_v_G_1$ ?v0) ) :pattern ( (fun_app$c v_b_SP_G_1$ ?v0) ) :pattern ( (v_b_SP_G_2$ ?v0) )))
+))
+(let (($x3683 (not $x3678)))
+(let (($x3670 (forall ((?v0 B_Vertex$) )(!(let ((?x273 (v_b_SP_G_2$ ?v0)))
+(let ((?x1186 (* (- 1) ?x273)))
+(let ((?x268 (b_G$ (pair$ v_b_v_G_1$ ?v0))))
+(let ((?x257 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
+(let (($x1185 (= (+ ?x257 ?x268 ?x1186) 0)))
+(let (($x1175 (<= (+ (fun_app$c v_b_SP_G_1$ ?v0) (* (- 1) ?x257) (* (- 1) ?x268)) 0)))
+(let (($x1169 (<= (+ b_Infinity$ (* (- 1) ?x268)) 0)))
+(or $x1169 $x1175 $x1185)))))))) :pattern ( (pair$ v_b_v_G_1$ ?v0) ) :pattern ( (fun_app$c v_b_SP_G_1$ ?v0) ) :pattern ( (v_b_SP_G_2$ ?v0) )))
+))
+(let (($x3675 (not $x3670)))
+(let ((?x263 (fun_upd$ v_b_Visited_G_1$)))
+(let ((?x264 (fun_app$b ?x263 v_b_v_G_1$)))
+(let ((?x265 (fun_app$a ?x264 true)))
+(let (($x266 (= v_b_Visited_G_2$ ?x265)))
+(let (($x2935 (not $x266)))
+(let (($x3660 (forall ((?v0 B_Vertex$) )(!(let ((?x257 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
+(let ((?x1173 (* (- 1) ?x257)))
+(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v0)))
+(let (($x178 (fun_app$ v_b_Visited_G_1$ ?v0)))
+(or $x178 (>= (+ ?x174 ?x1173) 0)))))) :pattern ( (fun_app$ v_b_Visited_G_1$ ?v0) ) :pattern ( (fun_app$c v_b_SP_G_1$ ?v0) )))
+))
+(let (($x3665 (not $x3660)))
+(let ((?x1173 (* (- 1) ?x257)))
+(let ((?x1212 (+ b_Infinity$ ?x1173)))
+(let (($x1213 (<= ?x1212 0)))
+(let (($x255 (fun_app$ v_b_Visited_G_1$ v_b_v_G_1$)))
+(let ((?x1775 (fun_app$c v_b_SP_G_1$ ?v0!12)))
+(let ((?x1776 (* (- 1) ?x1775)))
+(let ((?x1777 (+ b_Infinity$ ?x1776)))
+(let (($x1778 (<= ?x1777 0)))
+(let (($x1773 (fun_app$ v_b_Visited_G_1$ ?v0!12)))
+(let (($x3809 (or $x1773 $x1778 $x255 $x1213 $x3665 $x2935 $x3675 $x3683 $x3806)))
+(let (($x3812 (not $x3809)))
+(let ((?x245 (fun_app$c v_b_SP_G_3$ b_Source$)))
+(let (($x246 (= ?x245 0)))
+(let (($x3622 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(!(let ((?x230 (fun_app$c v_b_SP_G_3$ ?v1)))
+(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let (($x1140 (>= (+ ?x155 ?x230 (* (- 1) (fun_app$c v_b_SP_G_3$ ?v0))) 0)))
+(let (($x922 (<= (+ b_Infinity$ (* (- 1) ?x155)) 0)))
+(let (($x1099 (<= (+ b_Infinity$ (* (- 1) ?x230)) 0)))
+(or $x1099 $x922 $x1140)))))) :pattern ( (pair$ ?v1 ?v0) )))
+))
+(let (($x3627 (not $x3622)))
+(let (($x3630 (or $x3627 $x246)))
+(let (($x3633 (not $x3630)))
+(let ((?x1734 (fun_app$c v_b_SP_G_3$ ?v0!11)))
+(let ((?x1735 (* (- 1) ?x1734)))
+(let ((?x1726 (pair$ ?v1!10 ?v0!11)))
+(let ((?x1727 (b_G$ ?x1726)))
+(let ((?x1721 (fun_app$c v_b_SP_G_3$ ?v1!10)))
+(let ((?x2206 (+ ?x1721 ?x1727 ?x1735)))
+(let (($x2209 (>= ?x2206 0)))
+(let (($x1730 (<= (+ b_Infinity$ (* (- 1) ?x1727)) 0)))
+(let (($x1724 (<= (+ b_Infinity$ (* (- 1) ?x1721)) 0)))
+(let (($x2645 (or $x1724 $x1730 $x2209)))
+(let (($x2650 (not $x2645)))
+(let (($x3636 (or $x2650 $x3633)))
+(let (($x3639 (not $x3636)))
+(let (($x3614 (forall ((?v0 B_Vertex$) )(!(let ((?x230 (fun_app$c v_b_SP_G_3$ ?v0)))
+(let ((?x2191 (+ ?x230 (* (- 1) (fun_app$c v_b_SP_G_3$ (?v1!9 ?v0))) (* (- 1) (b_G$ (pair$ (?v1!9 ?v0) ?v0))))))
+(let (($x2192 (= ?x2191 0)))
+(let (($x2176 (<= (+ ?x230 (* (- 1) (fun_app$c v_b_SP_G_3$ (?v1!9 ?v0)))) 0)))
+(let (($x2617 (not (or $x2176 (not $x2192)))))
+(let (($x1099 (<= (+ b_Infinity$ (* (- 1) ?x230)) 0)))
+(let (($x127 (= ?v0 b_Source$)))
+(or $x127 $x1099 $x2617)))))))) :pattern ( (fun_app$c v_b_SP_G_3$ ?v0) )))
+))
+(let (($x3619 (not $x3614)))
+(let (($x3642 (or $x3619 $x3639)))
+(let (($x3645 (not $x3642)))
+(let (($x3600 (forall ((?v1 B_Vertex$) )(!(let ((?x1661 (fun_app$c v_b_SP_G_3$ ?v0!8)))
+(let ((?x1662 (* (- 1) ?x1661)))
+(let ((?x230 (fun_app$c v_b_SP_G_3$ ?v1)))
+(let (($x2148 (= (+ ?x230 ?x1662 (b_G$ (pair$ ?v1 ?v0!8))) 0)))
+(or (>= (+ ?x230 ?x1662) 0) (not $x2148)))))) :pattern ( (fun_app$c v_b_SP_G_3$ ?v1) ) :pattern ( (pair$ ?v1 ?v0!8) )))
+))
+(let (($x3605 (not $x3600)))
+(let (($x1664 (<= (+ b_Infinity$ (* (- 1) (fun_app$c v_b_SP_G_3$ ?v0!8))) 0)))
+(let (($x1659 (= ?v0!8 b_Source$)))
+(let (($x3608 (or $x1659 $x1664 $x3605)))
+(let (($x3611 (not $x3608)))
+(let (($x3648 (or $x3611 $x3645)))
+(let (($x3651 (not $x3648)))
+(let (($x220 (= v_b_oldSP_G_1$ v_b_oldSP_G_0$)))
+(let (($x2709 (not $x220)))
+(let (($x217 (= v_b_SP_G_3$ v_b_SP_G_1$)))
+(let (($x2708 (not $x217)))
+(let (($x215 (= v_b_v_G_2$ v_b_v_G_0$)))
+(let (($x2707 (not $x215)))
+(let (($x212 (= v_b_Visited_G_3$ v_b_Visited_G_1$)))
+(let (($x2706 (not $x212)))
+(let (($x3590 (forall ((?v0 B_Vertex$) )(!(let (($x1002 (<= (+ b_Infinity$ (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0))) 0)))
+(let (($x178 (fun_app$ v_b_Visited_G_1$ ?v0)))
+(or $x178 $x1002))) :pattern ( (fun_app$ v_b_Visited_G_1$ ?v0) ) :pattern ( (fun_app$c v_b_SP_G_1$ ?v0) )))
+))
+(let (($x3595 (not $x3590)))
+(let (($x3654 (or $x3595 $x2706 $x2707 $x2708 $x2709 $x3651)))
+(let (($x3657 (not $x3654)))
+(let (($x3815 (or $x3657 $x3812)))
+(let (($x3818 (not $x3815)))
+(let (($x3581 (forall ((?v0 B_Vertex$) )(!(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v0)))
+(let ((?x2128 (+ ?x174 (* (- 1) (fun_app$c v_b_SP_G_1$ (?v1!7 ?v0))) (* (- 1) (b_G$ (pair$ (?v1!7 ?v0) ?v0))))))
+(let (($x2129 (= ?x2128 0)))
+(let (($x2113 (<= (+ ?x174 (* (- 1) (fun_app$c v_b_SP_G_1$ (?v1!7 ?v0)))) 0)))
+(let (($x2551 (not (or $x2113 (not (fun_app$ v_b_Visited_G_1$ (?v1!7 ?v0))) (not $x2129)))))
+(let (($x1002 (<= (+ b_Infinity$ (* (- 1) ?x174)) 0)))
+(let (($x127 (= ?v0 b_Source$)))
+(or $x127 $x1002 $x2551)))))))) :pattern ( (fun_app$c v_b_SP_G_1$ ?v0) )))
+))
+(let (($x3586 (not $x3581)))
+(let (($x3573 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(!(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v1)))
+(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let (($x990 (>= (+ ?x155 ?x174 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0))) 0)))
+(let (($x922 (<= (+ b_Infinity$ (* (- 1) ?x155)) 0)))
+(let (($x178 (fun_app$ v_b_Visited_G_1$ ?v1)))
+(let (($x179 (not $x178)))
+(or $x179 $x922 $x990))))))) :pattern ( (pair$ ?v1 ?v0) )))
+))
+(let (($x3578 (not $x3573)))
+(let (($x3565 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(!(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v1)))
+(let (($x1015 (>= (+ ?x174 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0))) 0)))
+(let (($x178 (fun_app$ v_b_Visited_G_1$ ?v1)))
+(or $x178 (not (fun_app$ v_b_Visited_G_1$ ?v0)) $x1015)))) :pattern ( (fun_app$ v_b_Visited_G_1$ ?v1) (fun_app$ v_b_Visited_G_1$ ?v0) )))
+))
+(let (($x3570 (not $x3565)))
+(let (($x3561 (not $x3556)))
+(let ((?x172 (fun_app$c v_b_SP_G_1$ b_Source$)))
+(let (($x173 (= ?x172 0)))
+(let (($x2952 (not $x173)))
+(let (($x3547 (forall ((?v0 B_Vertex$) )(!(let ((?x128 (v_b_SP_G_0$ ?v0)))
+(let ((?x2090 (+ ?x128 (* (- 1) (v_b_SP_G_0$ (?v1!6 ?v0))) (* (- 1) (b_G$ (pair$ (?v1!6 ?v0) ?v0))))))
+(let (($x2091 (= ?x2090 0)))
+(let (($x2075 (<= (+ ?x128 (* (- 1) (v_b_SP_G_0$ (?v1!6 ?v0)))) 0)))
+(let (($x2478 (not (or $x2075 (not (v_b_Visited_G_0$ (?v1!6 ?v0))) (not $x2091)))))
+(let (($x947 (<= (+ b_Infinity$ (* (- 1) ?x128)) 0)))
+(let (($x127 (= ?v0 b_Source$)))
+(or $x127 $x947 $x2478)))))))) :pattern ( (v_b_SP_G_0$ ?v0) )))
+))
+(let (($x3552 (not $x3547)))
+(let (($x3821 (or $x3552 $x2952 $x3561 $x3570 $x3578 $x3586 $x3818)))
+(let (($x3824 (not $x3821)))
+(let (($x3533 (forall ((?v1 B_Vertex$) )(!(let ((?x1540 (v_b_SP_G_0$ ?v0!5)))
+(let ((?x1541 (* (- 1) ?x1540)))
+(let ((?x128 (v_b_SP_G_0$ ?v1)))
+(let (($x136 (v_b_Visited_G_0$ ?v1)))
+(let (($x137 (not $x136)))
+(or (>= (+ ?x128 ?x1541) 0) $x137 (not (= (+ ?x128 ?x1541 (b_G$ (pair$ ?v1 ?v0!5))) 0)))))))) :pattern ( (v_b_SP_G_0$ ?v1) ) :pattern ( (v_b_Visited_G_0$ ?v1) ) :pattern ( (pair$ ?v1 ?v0!5) )))
+))
+(let (($x3538 (not $x3533)))
+(let ((?x1540 (v_b_SP_G_0$ ?v0!5)))
+(let ((?x1541 (* (- 1) ?x1540)))
+(let ((?x1542 (+ b_Infinity$ ?x1541)))
+(let (($x1543 (<= ?x1542 0)))
+(let (($x1538 (= ?v0!5 b_Source$)))
+(let (($x3541 (or $x1538 $x1543 $x3538)))
+(let (($x1539 (not $x1538)))
+(let ((@x6246 (unit-resolution (def-axiom (or $x3541 $x1539)) (hypothesis (not $x3541)) $x1539)))
+(let (($x5625 (= b_Infinity$ ?x1540)))
+(let (($x6457 (not $x5625)))
+(let (($x1544 (not $x1543)))
+(let ((@x6514 (unit-resolution (def-axiom (or $x3541 $x1544)) (hypothesis (not $x3541)) $x1544)))
+(let ((@x5778 (symm (commutativity (= $x5625 (= ?x1540 b_Infinity$))) (= (= ?x1540 b_Infinity$) $x5625))))
+(let (($x5616 (= ?x1540 b_Infinity$)))
+(let (($x3493 (forall ((?v0 B_Vertex$) )(!(let (($x127 (= ?v0 b_Source$)))
+(or $x127 (= (v_b_SP_G_0$ ?v0) b_Infinity$))) :pattern ( (v_b_SP_G_0$ ?v0) )))
+))
+(let (($x360 (forall ((?v0 B_Vertex$) )(let (($x127 (= ?v0 b_Source$)))
+(or $x127 (= (v_b_SP_G_0$ ?v0) b_Infinity$))))
+))
+(let (($x127 (= ?0 b_Source$)))
+(let (($x357 (or $x127 (= (v_b_SP_G_0$ ?0) b_Infinity$))))
+(let (($x138 (forall ((?v0 B_Vertex$) )(let (($x136 (v_b_Visited_G_0$ ?v0)))
+(not $x136)))
+))
+(let (($x354 (forall ((?v0 B_Vertex$) )(let (($x127 (= ?v0 b_Source$)))
+(let (($x132 (not $x127)))
+(or $x132 (= (v_b_SP_G_0$ ?v0) 0)))))
+))
+(let (($x890 (and $x354 $x360 $x138)))
+(let (($x1329 (forall ((?v0 B_Vertex$) )(let (($x1323 (exists ((?v1 B_Vertex$) )(let ((?x303 (v_b_SP_G_2$ ?v0)))
+(let ((?x1263 (* (- 1) ?x303)))
+(let ((?x273 (v_b_SP_G_2$ ?v1)))
+(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let (($x1306 (= (+ ?x155 ?x273 ?x1263) 0)))
+(let (($x291 (fun_app$ v_b_Visited_G_2$ ?v1)))
+(let (($x1262 (>= (+ ?x273 ?x1263) 0)))
+(let (($x1309 (not $x1262)))
+(and $x1309 $x291 $x1306))))))))))
+))
+(let (($x127 (= ?v0 b_Source$)))
+(let (($x132 (not $x127)))
+(let (($x1300 (and $x132 (not (<= (+ b_Infinity$ (* (- 1) (v_b_SP_G_2$ ?v0))) 0)))))
+(or (not $x1300) $x1323))))))
+))
+(let (($x1289 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x303 (v_b_SP_G_2$ ?v0)))
+(let ((?x1263 (* (- 1) ?x303)))
+(let ((?x273 (v_b_SP_G_2$ ?v1)))
+(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let (($x1282 (>= (+ ?x155 ?x273 ?x1263) 0)))
+(let (($x922 (<= (+ b_Infinity$ (* (- 1) ?x155)) 0)))
+(let (($x923 (not $x922)))
+(let (($x291 (fun_app$ v_b_Visited_G_2$ ?v1)))
+(let (($x1276 (and $x291 $x923)))
+(let (($x1279 (not $x1276)))
+(or $x1279 $x1282))))))))))))
+))
+(let (($x1292 (not $x1289)))
+(let (($x1332 (or $x1292 $x1329)))
+(let (($x1335 (and $x1289 $x1332)))
+(let (($x1270 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let (($x1262 (>= (+ (v_b_SP_G_2$ ?v1) (* (- 1) (v_b_SP_G_2$ ?v0))) 0)))
+(let (($x301 (fun_app$ v_b_Visited_G_2$ ?v0)))
+(let (($x291 (fun_app$ v_b_Visited_G_2$ ?v1)))
+(let (($x300 (not $x291)))
+(let (($x302 (and $x300 $x301)))
+(let (($x664 (not $x302)))
+(or $x664 $x1262))))))))
+))
+(let (($x1273 (not $x1270)))
+(let (($x1338 (or $x1273 $x1335)))
+(let (($x1341 (and $x1270 $x1338)))
+(let (($x1256 (forall ((?v0 B_Vertex$) )(let ((?x273 (v_b_SP_G_2$ ?v0)))
+(>= ?x273 0)))
+))
+(let (($x1259 (not $x1256)))
+(let (($x1344 (or $x1259 $x1341)))
+(let (($x1347 (and $x1256 $x1344)))
+(let (($x1350 (or $x773 $x1347)))
+(let (($x1353 (and $x297 $x1350)))
+(let (($x652 (forall ((?v0 B_Vertex$) )(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v0)))
+(let ((?x273 (v_b_SP_G_2$ ?v0)))
+(let (($x278 (= ?x273 ?x174)))
+(let (($x291 (fun_app$ v_b_Visited_G_2$ ?v0)))
+(let (($x300 (not $x291)))
+(or $x300 $x278)))))))
+))
+(let (($x785 (not $x652)))
+(let (($x1356 (or $x785 $x1353)))
+(let (($x1359 (and $x652 $x1356)))
+(let (($x1247 (forall ((?v0 B_Vertex$) )(>= (+ (fun_app$c v_b_SP_G_1$ ?v0) (* (- 1) (v_b_SP_G_2$ ?v0))) 0))
+))
+(let (($x1250 (not $x1247)))
+(let (($x1362 (or $x1250 $x1359)))
+(let (($x1365 (and $x1247 $x1362)))
+(let (($x1199 (forall ((?v0 B_Vertex$) )(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v0)))
+(let ((?x273 (v_b_SP_G_2$ ?v0)))
+(let (($x278 (= ?x273 ?x174)))
+(let ((?x257 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
+(let ((?x1173 (* (- 1) ?x257)))
+(let (($x1175 (<= (+ ?x174 ?x1173 (* (- 1) (b_G$ (pair$ v_b_v_G_1$ ?v0)))) 0)))
+(let (($x1169 (<= (+ b_Infinity$ (* (- 1) (b_G$ (pair$ v_b_v_G_1$ ?v0)))) 0)))
+(let (($x1179 (and (not $x1169) (not $x1175))))
+(or $x1179 $x278))))))))))
+))
+(let (($x1193 (forall ((?v0 B_Vertex$) )(let ((?x273 (v_b_SP_G_2$ ?v0)))
+(let ((?x1186 (* (- 1) ?x273)))
+(let ((?x268 (b_G$ (pair$ v_b_v_G_1$ ?v0))))
+(let ((?x257 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
+(let (($x1185 (= (+ ?x257 ?x268 ?x1186) 0)))
+(let (($x1175 (<= (+ (fun_app$c v_b_SP_G_1$ ?v0) (* (- 1) ?x257) (* (- 1) ?x268)) 0)))
+(let (($x1179 (and (not (<= (+ b_Infinity$ (* (- 1) ?x268)) 0)) (not $x1175))))
+(let (($x1182 (not $x1179)))
+(or $x1182 $x1185))))))))))
+))
+(let (($x1209 (forall ((?v0 B_Vertex$) )(let ((?x257 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
+(let ((?x1173 (* (- 1) ?x257)))
+(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v0)))
+(let (($x178 (fun_app$ v_b_Visited_G_1$ ?v0)))
+(or $x178 (>= (+ ?x174 ?x1173) 0)))))))
+))
+(let (($x1214 (not $x1213)))
+(let (($x256 (not $x255)))
+(let (($x1080 (exists ((?v0 B_Vertex$) )(let (($x1002 (<= (+ b_Infinity$ (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0))) 0)))
+(let (($x1003 (not $x1002)))
+(let (($x178 (fun_app$ v_b_Visited_G_1$ ?v0)))
+(let (($x179 (not $x178)))
+(and $x179 $x1003))))))
+))
+(let (($x1235 (and $x1080 $x256 $x1214 $x1209 $x266 $x1193 $x1199)))
+(let (($x1240 (not $x1235)))
+(let (($x1368 (or $x1240 $x1365)))
+(let (($x1146 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x230 (fun_app$c v_b_SP_G_3$ ?v1)))
+(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let (($x1140 (>= (+ ?x155 ?x230 (* (- 1) (fun_app$c v_b_SP_G_3$ ?v0))) 0)))
+(let (($x922 (<= (+ b_Infinity$ (* (- 1) ?x155)) 0)))
+(let (($x923 (not $x922)))
+(let (($x1099 (<= (+ b_Infinity$ (* (- 1) ?x230)) 0)))
+(let (($x1100 (not $x1099)))
+(let (($x1134 (and $x1100 $x923)))
+(let (($x1137 (not $x1134)))
+(or $x1137 $x1140)))))))))))
+))
+(let (($x1149 (not $x1146)))
+(let (($x1152 (or $x1149 $x246)))
+(let (($x1155 (and $x1146 $x1152)))
+(let (($x1128 (forall ((?v0 B_Vertex$) )(let (($x1122 (exists ((?v1 B_Vertex$) )(let ((?x230 (fun_app$c v_b_SP_G_3$ ?v1)))
+(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(and (not (>= (+ ?x230 (* (- 1) (fun_app$c v_b_SP_G_3$ ?v0))) 0)) (= (+ ?x155 ?x230 (* (- 1) (fun_app$c v_b_SP_G_3$ ?v0))) 0)))))
+))
+(let (($x1099 (<= (+ b_Infinity$ (* (- 1) (fun_app$c v_b_SP_G_3$ ?v0))) 0)))
+(let (($x1100 (not $x1099)))
+(let (($x127 (= ?v0 b_Source$)))
+(let (($x132 (not $x127)))
+(let (($x1103 (and $x132 $x1100)))
+(let (($x1106 (not $x1103)))
+(or $x1106 $x1122)))))))))
+))
+(let (($x1131 (not $x1128)))
+(let (($x1158 (or $x1131 $x1155)))
+(let (($x1161 (and $x1128 $x1158)))
+(let (($x1083 (not $x1080)))
+(let (($x1089 (and $x1083 $x212 $x215 $x217 $x220)))
+(let (($x1094 (not $x1089)))
+(let (($x1164 (or $x1094 $x1161)))
+(let (($x1371 (and $x1164 $x1368)))
+(let (($x1037 (forall ((?v0 B_Vertex$) )(let (($x1031 (exists ((?v1 B_Vertex$) )(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v1)))
+(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let (($x1012 (= (+ ?x155 ?x174 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0))) 0)))
+(let (($x178 (fun_app$ v_b_Visited_G_1$ ?v1)))
+(let (($x1015 (>= (+ ?x174 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0))) 0)))
+(let (($x1017 (not $x1015)))
+(and $x1017 $x178 $x1012))))))))
+))
+(let (($x1002 (<= (+ b_Infinity$ (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0))) 0)))
+(let (($x1003 (not $x1002)))
+(let (($x127 (= ?v0 b_Source$)))
+(let (($x132 (not $x127)))
+(let (($x1006 (and $x132 $x1003)))
+(let (($x1009 (not $x1006)))
+(or $x1009 $x1031)))))))))
+))
+(let (($x997 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v1)))
+(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let (($x990 (>= (+ ?x155 ?x174 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0))) 0)))
+(let (($x922 (<= (+ b_Infinity$ (* (- 1) ?x155)) 0)))
+(let (($x923 (not $x922)))
+(let (($x178 (fun_app$ v_b_Visited_G_1$ ?v1)))
+(let (($x983 (and $x178 $x923)))
+(let (($x986 (not $x983)))
+(or $x986 $x990))))))))))
+))
+(let (($x1045 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v1)))
+(let (($x1015 (>= (+ ?x174 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0))) 0)))
+(let (($x180 (fun_app$ v_b_Visited_G_1$ ?v0)))
+(let (($x178 (fun_app$ v_b_Visited_G_1$ ?v1)))
+(let (($x179 (not $x178)))
+(let (($x181 (and $x179 $x180)))
+(let (($x403 (not $x181)))
+(or $x403 $x1015)))))))))
+))
+(let (($x1051 (forall ((?v0 B_Vertex$) )(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v0)))
+(>= ?x174 0)))
+))
+(let (($x980 (forall ((?v0 B_Vertex$) )(let (($x974 (exists ((?v1 B_Vertex$) )(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let ((?x128 (v_b_SP_G_0$ ?v1)))
+(let (($x957 (= (+ ?x128 (* (- 1) (v_b_SP_G_0$ ?v0)) ?x155) 0)))
+(let (($x136 (v_b_Visited_G_0$ ?v1)))
+(let (($x907 (>= (+ ?x128 (* (- 1) (v_b_SP_G_0$ ?v0))) 0)))
+(let (($x960 (not $x907)))
+(and $x960 $x136 $x957))))))))
+))
+(let (($x127 (= ?v0 b_Source$)))
+(let (($x132 (not $x127)))
+(let (($x951 (and $x132 (not (<= (+ b_Infinity$ (* (- 1) (v_b_SP_G_0$ ?v0))) 0)))))
+(let (($x954 (not $x951)))
+(or $x954 $x974)))))))
+))
+(let (($x1069 (and $x980 $x173 $x1051 $x1045 $x997 $x1037)))
+(let (($x1074 (not $x1069)))
+(let (($x1374 (or $x1074 $x1371)))
+(let (($x1377 (and $x980 $x1374)))
+(let (($x939 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let ((?x128 (v_b_SP_G_0$ ?v1)))
+(let (($x933 (>= (+ ?x128 (* (- 1) (v_b_SP_G_0$ ?v0)) ?x155) 0)))
+(let (($x922 (<= (+ b_Infinity$ (* (- 1) ?x155)) 0)))
+(let (($x923 (not $x922)))
+(let (($x136 (v_b_Visited_G_0$ ?v1)))
+(let (($x926 (and $x136 $x923)))
+(let (($x929 (not $x926)))
+(or $x929 $x933))))))))))
+))
+(let (($x942 (not $x939)))
+(let (($x1380 (or $x942 $x1377)))
+(let (($x1383 (and $x939 $x1380)))
+(let (($x914 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let (($x907 (>= (+ (v_b_SP_G_0$ ?v1) (* (- 1) (v_b_SP_G_0$ ?v0))) 0)))
+(let (($x148 (v_b_Visited_G_0$ ?v0)))
+(let (($x136 (v_b_Visited_G_0$ ?v1)))
+(let (($x137 (not $x136)))
+(let (($x149 (and $x137 $x148)))
+(let (($x382 (not $x149)))
+(or $x382 $x907))))))))
+))
+(let (($x917 (not $x914)))
+(let (($x1386 (or $x917 $x1383)))
+(let (($x1389 (and $x914 $x1386)))
+(let (($x899 (forall ((?v0 B_Vertex$) )(let ((?x128 (v_b_SP_G_0$ ?v0)))
+(>= ?x128 0)))
+))
+(let (($x902 (not $x899)))
+(let (($x1392 (or $x902 $x1389)))
+(let (($x1395 (and $x899 $x1392)))
+(let ((?x144 (v_b_SP_G_0$ b_Source$)))
+(let (($x145 (= ?x144 0)))
+(let (($x869 (not $x145)))
+(let (($x1398 (or $x869 $x1395)))
+(let (($x1401 (and $x145 $x1398)))
+(let (($x1407 (not (or (not $x890) $x1401))))
+(let (($x320 (forall ((?v0 B_Vertex$) )(let (($x318 (exists ((?v1 B_Vertex$) )(let (($x291 (fun_app$ v_b_Visited_G_2$ ?v1)))
+(let (($x316 (and $x291 (= (v_b_SP_G_2$ ?v0) (+ (v_b_SP_G_2$ ?v1) (b_G$ (pair$ ?v1 ?v0)))))))
+(let ((?x303 (v_b_SP_G_2$ ?v0)))
+(let ((?x273 (v_b_SP_G_2$ ?v1)))
+(let (($x314 (< ?x273 ?x303)))
+(and $x314 $x316)))))))
+))
+(let (($x127 (= ?v0 b_Source$)))
+(let (($x132 (not $x127)))
+(let (($x313 (and $x132 (< (v_b_SP_G_2$ ?v0) b_Infinity$))))
+(=> $x313 $x318))))))
+))
+(let (($x321 (and $x320 false)))
+(let (($x322 (=> $x321 true)))
+(let (($x323 (and $x320 $x322)))
+(let (($x311 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let ((?x273 (v_b_SP_G_2$ ?v1)))
+(let ((?x308 (+ ?x273 ?x155)))
+(let ((?x303 (v_b_SP_G_2$ ?v0)))
+(let (($x156 (< ?x155 b_Infinity$)))
+(let (($x291 (fun_app$ v_b_Visited_G_2$ ?v1)))
+(let (($x307 (and $x291 $x156)))
+(=> $x307 (<= ?x303 ?x308))))))))))
+))
+(let (($x324 (=> $x311 $x323)))
+(let (($x306 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x273 (v_b_SP_G_2$ ?v1)))
+(let ((?x303 (v_b_SP_G_2$ ?v0)))
+(let (($x304 (<= ?x303 ?x273)))
+(let (($x301 (fun_app$ v_b_Visited_G_2$ ?v0)))
+(let (($x291 (fun_app$ v_b_Visited_G_2$ ?v1)))
+(let (($x300 (not $x291)))
+(let (($x302 (and $x300 $x301)))
+(=> $x302 $x304)))))))))
+))
+(let (($x326 (=> $x306 (and $x311 $x324))))
+(let (($x299 (forall ((?v0 B_Vertex$) )(let ((?x273 (v_b_SP_G_2$ ?v0)))
+(<= 0 ?x273)))
+))
+(let (($x328 (=> $x299 (and $x306 $x326))))
+(let (($x330 (=> $x297 (and $x299 $x328))))
+(let (($x293 (forall ((?v0 B_Vertex$) )(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v0)))
+(let ((?x273 (v_b_SP_G_2$ ?v0)))
+(let (($x278 (= ?x273 ?x174)))
+(let (($x291 (fun_app$ v_b_Visited_G_2$ ?v0)))
+(=> $x291 $x278))))))
+))
+(let (($x295 (and $x293 (and true true))))
+(let (($x332 (=> $x295 (and $x297 $x330))))
+(let (($x290 (forall ((?v0 B_Vertex$) )(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v0)))
+(let ((?x273 (v_b_SP_G_2$ ?v0)))
+(<= ?x273 ?x174))))
+))
+(let (($x334 (=> $x290 (and $x293 $x332))))
+(let (($x280 (forall ((?v0 B_Vertex$) )(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v0)))
+(let ((?x273 (v_b_SP_G_2$ ?v0)))
+(let (($x278 (= ?x273 ?x174)))
+(let ((?x268 (b_G$ (pair$ v_b_v_G_1$ ?v0))))
+(let ((?x257 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
+(let ((?x270 (+ ?x257 ?x268)))
+(let (($x272 (and (< ?x268 b_Infinity$) (< ?x270 ?x174))))
+(let (($x277 (not $x272)))
+(=> $x277 $x278))))))))))
+))
+(let (($x276 (forall ((?v0 B_Vertex$) )(let ((?x268 (b_G$ (pair$ v_b_v_G_1$ ?v0))))
+(let ((?x257 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
+(let ((?x270 (+ ?x257 ?x268)))
+(let ((?x273 (v_b_SP_G_2$ ?v0)))
+(let (($x274 (= ?x273 ?x270)))
+(let (($x272 (and (< ?x268 b_Infinity$) (< ?x270 (fun_app$c v_b_SP_G_1$ ?v0)))))
+(=> $x272 $x274))))))))
+))
+(let (($x261 (forall ((?v0 B_Vertex$) )(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v0)))
+(let ((?x257 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
+(let (($x259 (<= ?x257 ?x174)))
+(let (($x178 (fun_app$ v_b_Visited_G_1$ ?v0)))
+(let (($x179 (not $x178)))
+(=> $x179 $x259)))))))
+))
+(let (($x258 (< ?x257 b_Infinity$)))
+(let (($x209 (exists ((?v0 B_Vertex$) )(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v0)))
+(let (($x191 (< ?x174 b_Infinity$)))
+(let (($x178 (fun_app$ v_b_Visited_G_1$ ?v0)))
+(let (($x179 (not $x178)))
+(and $x179 $x191))))))
+))
+(let (($x286 (and $x209 (and $x256 (and $x258 (and $x261 (and $x266 (and $x276 $x280))))))))
+(let (($x287 (and true $x286)))
+(let (($x288 (and true $x287)))
+(let (($x336 (=> $x288 (and $x290 $x334))))
+(let (($x248 (and $x246 (=> $x246 true))))
+(let (($x244 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let ((?x230 (fun_app$c v_b_SP_G_3$ ?v1)))
+(let ((?x235 (+ ?x230 ?x155)))
+(let ((?x233 (fun_app$c v_b_SP_G_3$ ?v0)))
+(let (($x156 (< ?x155 b_Infinity$)))
+(let (($x231 (< ?x230 b_Infinity$)))
+(let (($x241 (and $x231 $x156)))
+(=> $x241 (<= ?x233 ?x235))))))))))
+))
+(let (($x249 (=> $x244 $x248)))
+(let (($x240 (forall ((?v0 B_Vertex$) )(let (($x238 (exists ((?v1 B_Vertex$) )(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let ((?x230 (fun_app$c v_b_SP_G_3$ ?v1)))
+(let ((?x235 (+ ?x230 ?x155)))
+(let ((?x233 (fun_app$c v_b_SP_G_3$ ?v0)))
+(let (($x234 (< ?x230 ?x233)))
+(and $x234 (= ?x233 ?x235))))))))
+))
+(let ((?x230 (fun_app$c v_b_SP_G_3$ ?v0)))
+(let (($x231 (< ?x230 b_Infinity$)))
+(let (($x127 (= ?v0 b_Source$)))
+(let (($x132 (not $x127)))
+(let (($x232 (and $x132 $x231)))
+(=> $x232 $x238))))))))
+))
+(let (($x251 (=> $x240 (and $x244 $x249))))
+(let (($x225 (and true (and $x212 (and $x215 (and $x217 (and $x220 true)))))))
+(let (($x226 (and true $x225)))
+(let (($x210 (not $x209)))
+(let (($x228 (and true (and $x210 $x226))))
+(let (($x229 (and true $x228)))
+(let (($x253 (=> $x229 (and $x240 $x251))))
+(let (($x199 (forall ((?v0 B_Vertex$) )(let (($x197 (exists ((?v1 B_Vertex$) )(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v1)))
+(let ((?x187 (+ ?x174 ?x155)))
+(let ((?x182 (fun_app$c v_b_SP_G_1$ ?v0)))
+(let (($x178 (fun_app$ v_b_Visited_G_1$ ?v1)))
+(let (($x193 (< ?x174 ?x182)))
+(and $x193 (and $x178 (= ?x182 ?x187))))))))))
+))
+(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v0)))
+(let (($x191 (< ?x174 b_Infinity$)))
+(let (($x127 (= ?v0 b_Source$)))
+(let (($x132 (not $x127)))
+(let (($x192 (and $x132 $x191)))
+(=> $x192 $x197))))))))
+))
+(let (($x200 (and $x199 true)))
+(let (($x190 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v1)))
+(let ((?x187 (+ ?x174 ?x155)))
+(let ((?x182 (fun_app$c v_b_SP_G_1$ ?v0)))
+(let (($x156 (< ?x155 b_Infinity$)))
+(let (($x178 (fun_app$ v_b_Visited_G_1$ ?v1)))
+(let (($x186 (and $x178 $x156)))
+(=> $x186 (<= ?x182 ?x187))))))))))
+))
+(let (($x185 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v1)))
+(let ((?x182 (fun_app$c v_b_SP_G_1$ ?v0)))
+(let (($x183 (<= ?x182 ?x174)))
+(let (($x180 (fun_app$ v_b_Visited_G_1$ ?v0)))
+(let (($x178 (fun_app$ v_b_Visited_G_1$ ?v1)))
+(let (($x179 (not $x178)))
+(let (($x181 (and $x179 $x180)))
+(=> $x181 $x183)))))))))
+))
+(let (($x176 (forall ((?v0 B_Vertex$) )(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v0)))
+(<= 0 ?x174)))
+))
+(let (($x205 (and true (and $x173 (and $x176 (and $x185 (and $x190 $x200)))))))
+(let (($x206 (and true $x205)))
+(let (($x170 (forall ((?v0 B_Vertex$) )(let (($x168 (exists ((?v1 B_Vertex$) )(let (($x136 (v_b_Visited_G_0$ ?v1)))
+(let (($x166 (and $x136 (= (v_b_SP_G_0$ ?v0) (+ (v_b_SP_G_0$ ?v1) (b_G$ (pair$ ?v1 ?v0)))))))
+(and (< (v_b_SP_G_0$ ?v1) (v_b_SP_G_0$ ?v0)) $x166))))
+))
+(let (($x127 (= ?v0 b_Source$)))
+(let (($x132 (not $x127)))
+(let (($x163 (and $x132 (< (v_b_SP_G_0$ ?v0) b_Infinity$))))
+(=> $x163 $x168))))))
+))
+(let (($x338 (=> (and $x170 $x206) (and $x253 $x336))))
+(let (($x161 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x150 (v_b_SP_G_0$ ?v0)))
+(let (($x159 (<= ?x150 (+ (v_b_SP_G_0$ ?v1) (b_G$ (pair$ ?v1 ?v0))))))
+(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let (($x156 (< ?x155 b_Infinity$)))
+(let (($x136 (v_b_Visited_G_0$ ?v1)))
+(let (($x157 (and $x136 $x156)))
+(=> $x157 $x159))))))))
+))
+(let (($x340 (=> $x161 (and $x170 $x338))))
+(let (($x153 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x128 (v_b_SP_G_0$ ?v1)))
+(let ((?x150 (v_b_SP_G_0$ ?v0)))
+(let (($x151 (<= ?x150 ?x128)))
+(let (($x148 (v_b_Visited_G_0$ ?v0)))
+(let (($x136 (v_b_Visited_G_0$ ?v1)))
+(let (($x137 (not $x136)))
+(let (($x149 (and $x137 $x148)))
+(=> $x149 $x151)))))))))
+))
+(let (($x342 (=> $x153 (and $x161 $x340))))
+(let (($x147 (forall ((?v0 B_Vertex$) )(let ((?x128 (v_b_SP_G_0$ ?v0)))
+(<= 0 ?x128)))
+))
+(let (($x344 (=> $x147 (and $x153 $x342))))
+(let (($x346 (=> $x145 (and $x147 $x344))))
+(let (($x135 (forall ((?v0 B_Vertex$) )(let (($x127 (= ?v0 b_Source$)))
+(let (($x132 (not $x127)))
+(=> $x132 (= (v_b_SP_G_0$ ?v0) b_Infinity$)))))
+))
+(let (($x131 (forall ((?v0 B_Vertex$) )(let (($x127 (= ?v0 b_Source$)))
+(=> $x127 (= (v_b_SP_G_0$ ?v0) 0))))
+))
+(let (($x142 (and true (and $x131 (and $x135 (and $x138 true))))))
+(let (($x143 (and true $x142)))
+(let (($x348 (=> $x143 (and $x145 $x346))))
+(let (($x349 (not $x348)))
+(let (($x710 (forall ((?v0 B_Vertex$) )(let (($x698 (exists ((?v1 B_Vertex$) )(let ((?x273 (v_b_SP_G_2$ ?v1)))
+(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let ((?x671 (+ ?x155 ?x273)))
+(let ((?x303 (v_b_SP_G_2$ ?v0)))
+(let (($x689 (= ?x303 ?x671)))
+(let (($x291 (fun_app$ v_b_Visited_G_2$ ?v1)))
+(let (($x692 (and $x291 $x689)))
+(let (($x314 (< ?x273 ?x303)))
+(and $x314 $x692))))))))))
+))
+(let (($x127 (= ?v0 b_Source$)))
+(let (($x132 (not $x127)))
+(let (($x313 (and $x132 (< (v_b_SP_G_2$ ?v0) b_Infinity$))))
+(or (not $x313) $x698))))))
+))
+(let (($x686 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x273 (v_b_SP_G_2$ ?v1)))
+(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let ((?x671 (+ ?x155 ?x273)))
+(let ((?x303 (v_b_SP_G_2$ ?v0)))
+(let (($x674 (<= ?x303 ?x671)))
+(or (not (and (fun_app$ v_b_Visited_G_2$ ?v1) (< ?x155 b_Infinity$))) $x674)))))))
+))
+(let (($x738 (or (not $x686) $x710)))
+(let (($x743 (and $x686 $x738)))
+(let (($x668 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x273 (v_b_SP_G_2$ ?v1)))
+(let ((?x303 (v_b_SP_G_2$ ?v0)))
+(let (($x304 (<= ?x303 ?x273)))
+(let (($x301 (fun_app$ v_b_Visited_G_2$ ?v0)))
+(let (($x291 (fun_app$ v_b_Visited_G_2$ ?v1)))
+(let (($x300 (not $x291)))
+(let (($x302 (and $x300 $x301)))
+(let (($x664 (not $x302)))
+(or $x664 $x304))))))))))
+))
+(let (($x750 (or (not $x668) $x743)))
+(let (($x755 (and $x668 $x750)))
+(let (($x762 (or (not $x299) $x755)))
+(let (($x767 (and $x299 $x762)))
+(let (($x774 (or $x773 $x767)))
+(let (($x779 (and $x297 $x774)))
+(let (($x786 (or $x785 $x779)))
+(let (($x791 (and $x652 $x786)))
+(let (($x798 (or (not $x290) $x791)))
+(let (($x803 (and $x290 $x798)))
+(let (($x617 (forall ((?v0 B_Vertex$) )(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v0)))
+(let ((?x273 (v_b_SP_G_2$ ?v0)))
+(let (($x278 (= ?x273 ?x174)))
+(let ((?x268 (b_G$ (pair$ v_b_v_G_1$ ?v0))))
+(let ((?x257 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
+(let ((?x270 (+ ?x257 ?x268)))
+(let (($x272 (and (< ?x268 b_Infinity$) (< ?x270 ?x174))))
+(or $x272 $x278)))))))))
+))
+(let (($x611 (forall ((?v0 B_Vertex$) )(let ((?x268 (b_G$ (pair$ v_b_v_G_1$ ?v0))))
+(let ((?x257 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
+(let ((?x270 (+ ?x257 ?x268)))
+(let ((?x273 (v_b_SP_G_2$ ?v0)))
+(let (($x274 (= ?x273 ?x270)))
+(let (($x272 (and (< ?x268 b_Infinity$) (< ?x270 (fun_app$c v_b_SP_G_1$ ?v0)))))
+(let (($x277 (not $x272)))
+(or $x277 $x274)))))))))
+))
+(let (($x620 (and $x611 $x617)))
+(let (($x623 (and $x266 $x620)))
+(let (($x605 (forall ((?v0 B_Vertex$) )(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v0)))
+(let ((?x257 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
+(let (($x259 (<= ?x257 ?x174)))
+(let (($x178 (fun_app$ v_b_Visited_G_1$ ?v0)))
+(or $x178 $x259))))))
+))
+(let (($x626 (and $x605 $x623)))
+(let (($x629 (and $x258 $x626)))
+(let (($x632 (and $x256 $x629)))
+(let (($x635 (and $x209 $x632)))
+(let (($x810 (or (not $x635) $x803)))
+(let (($x557 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x230 (fun_app$c v_b_SP_G_3$ ?v1)))
+(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let ((?x521 (+ ?x155 ?x230)))
+(let ((?x233 (fun_app$c v_b_SP_G_3$ ?v0)))
+(let (($x545 (<= ?x233 ?x521)))
+(or (not (and (< ?x230 b_Infinity$) (< ?x155 b_Infinity$))) $x545)))))))
+))
+(let (($x573 (or (not $x557) $x246)))
+(let (($x578 (and $x557 $x573)))
+(let (($x542 (forall ((?v0 B_Vertex$) )(let (($x530 (exists ((?v1 B_Vertex$) )(let ((?x230 (fun_app$c v_b_SP_G_3$ ?v1)))
+(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let ((?x521 (+ ?x155 ?x230)))
+(let ((?x233 (fun_app$c v_b_SP_G_3$ ?v0)))
+(let (($x524 (= ?x233 ?x521)))
+(let (($x234 (< ?x230 ?x233)))
+(and $x234 $x524))))))))
+))
+(let ((?x230 (fun_app$c v_b_SP_G_3$ ?v0)))
+(let (($x231 (< ?x230 b_Infinity$)))
+(let (($x127 (= ?v0 b_Source$)))
+(let (($x132 (not $x127)))
+(let (($x232 (and $x132 $x231)))
+(or (not $x232) $x530))))))))
+))
+(let (($x585 (or (not $x542) $x578)))
+(let (($x590 (and $x542 $x585)))
+(let (($x597 (or (not (and $x210 (and $x212 (and $x215 (and $x217 $x220))))) $x590)))
+(let (($x815 (and $x597 $x810)))
+(let (($x449 (forall ((?v0 B_Vertex$) )(let (($x437 (exists ((?v1 B_Vertex$) )(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v1)))
+(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let ((?x410 (+ ?x155 ?x174)))
+(let ((?x182 (fun_app$c v_b_SP_G_1$ ?v0)))
+(let (($x428 (= ?x182 ?x410)))
+(let (($x178 (fun_app$ v_b_Visited_G_1$ ?v1)))
+(let (($x431 (and $x178 $x428)))
+(let (($x193 (< ?x174 ?x182)))
+(and $x193 $x431))))))))))
+))
+(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v0)))
+(let (($x191 (< ?x174 b_Infinity$)))
+(let (($x127 (= ?v0 b_Source$)))
+(let (($x132 (not $x127)))
+(let (($x192 (and $x132 $x191)))
+(or (not $x192) $x437))))))))
+))
+(let (($x425 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v1)))
+(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let ((?x410 (+ ?x155 ?x174)))
+(let ((?x182 (fun_app$c v_b_SP_G_1$ ?v0)))
+(let (($x413 (<= ?x182 ?x410)))
+(or (not (and (fun_app$ v_b_Visited_G_1$ ?v1) (< ?x155 b_Infinity$))) $x413)))))))
+))
+(let (($x459 (and $x425 $x449)))
+(let (($x407 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v1)))
+(let ((?x182 (fun_app$c v_b_SP_G_1$ ?v0)))
+(let (($x183 (<= ?x182 ?x174)))
+(let (($x180 (fun_app$ v_b_Visited_G_1$ ?v0)))
+(let (($x178 (fun_app$ v_b_Visited_G_1$ ?v1)))
+(let (($x179 (not $x178)))
+(let (($x181 (and $x179 $x180)))
+(let (($x403 (not $x181)))
+(or $x403 $x183))))))))))
+))
+(let (($x462 (and $x407 $x459)))
+(let (($x465 (and $x176 $x462)))
+(let (($x468 (and $x173 $x465)))
+(let (($x400 (forall ((?v0 B_Vertex$) )(let (($x168 (exists ((?v1 B_Vertex$) )(let (($x136 (v_b_Visited_G_0$ ?v1)))
+(let (($x166 (and $x136 (= (v_b_SP_G_0$ ?v0) (+ (v_b_SP_G_0$ ?v1) (b_G$ (pair$ ?v1 ?v0)))))))
+(and (< (v_b_SP_G_0$ ?v1) (v_b_SP_G_0$ ?v0)) $x166))))
+))
+(let (($x127 (= ?v0 b_Source$)))
+(let (($x132 (not $x127)))
+(let (($x163 (and $x132 (< (v_b_SP_G_0$ ?v0) b_Infinity$))))
+(or (not $x163) $x168))))))
+))
+(let (($x482 (and $x400 $x468)))
+(let (($x822 (or (not $x482) $x815)))
+(let (($x827 (and $x400 $x822)))
+(let (($x393 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x150 (v_b_SP_G_0$ ?v0)))
+(let (($x159 (<= ?x150 (+ (v_b_SP_G_0$ ?v1) (b_G$ (pair$ ?v1 ?v0))))))
+(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let (($x156 (< ?x155 b_Infinity$)))
+(let (($x136 (v_b_Visited_G_0$ ?v1)))
+(let (($x157 (and $x136 $x156)))
+(or (not $x157) $x159))))))))
+))
+(let (($x834 (or (not $x393) $x827)))
+(let (($x839 (and $x393 $x834)))
+(let (($x386 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x128 (v_b_SP_G_0$ ?v1)))
+(let ((?x150 (v_b_SP_G_0$ ?v0)))
+(let (($x151 (<= ?x150 ?x128)))
+(let (($x148 (v_b_Visited_G_0$ ?v0)))
+(let (($x136 (v_b_Visited_G_0$ ?v1)))
+(let (($x137 (not $x136)))
+(let (($x149 (and $x137 $x148)))
+(let (($x382 (not $x149)))
+(or $x382 $x151))))))))))
+))
+(let (($x846 (or (not $x386) $x839)))
+(let (($x851 (and $x386 $x846)))
+(let (($x858 (or (not $x147) $x851)))
+(let (($x863 (and $x147 $x858)))
+(let (($x870 (or $x869 $x863)))
+(let (($x875 (and $x145 $x870)))
+(let (($x882 (or (not (and $x354 (and $x360 $x138))) $x875)))
+(let (($x1323 (exists ((?v1 B_Vertex$) )(let ((?x303 (v_b_SP_G_2$ ?0)))
+(let ((?x1263 (* (- 1) ?x303)))
+(let ((?x273 (v_b_SP_G_2$ ?v1)))
+(let ((?x155 (b_G$ (pair$ ?v1 ?0))))
+(let (($x1306 (= (+ ?x155 ?x273 ?x1263) 0)))
+(let (($x291 (fun_app$ v_b_Visited_G_2$ ?v1)))
+(let (($x1262 (>= (+ ?x273 ?x1263) 0)))
+(let (($x1309 (not $x1262)))
+(and $x1309 $x291 $x1306))))))))))
+))
+(let (($x132 (not $x127)))
+(let (($x1300 (and $x132 (not (<= (+ b_Infinity$ (* (- 1) (v_b_SP_G_2$ ?0))) 0)))))
+(let (($x698 (exists ((?v1 B_Vertex$) )(let ((?x273 (v_b_SP_G_2$ ?v1)))
+(let ((?x155 (b_G$ (pair$ ?v1 ?0))))
+(let ((?x671 (+ ?x155 ?x273)))
+(let ((?x303 (v_b_SP_G_2$ ?0)))
+(let (($x689 (= ?x303 ?x671)))
+(let (($x291 (fun_app$ v_b_Visited_G_2$ ?v1)))
+(let (($x692 (and $x291 $x689)))
+(let (($x314 (< ?x273 ?x303)))
+(and $x314 $x692))))))))))
+))
+(let (($x705 (or (not (and $x132 (< (v_b_SP_G_2$ ?0) b_Infinity$))) $x698)))
+(let ((?x303 (v_b_SP_G_2$ ?1)))
+(let ((?x1263 (* (- 1) ?x303)))
+(let ((?x273 (v_b_SP_G_2$ ?0)))
+(let ((?x155 (b_G$ (pair$ ?0 ?1))))
+(let (($x1306 (= (+ ?x155 ?x273 ?x1263) 0)))
+(let (($x291 (fun_app$ v_b_Visited_G_2$ ?0)))
+(let (($x1262 (>= (+ ?x273 ?x1263) 0)))
+(let (($x1309 (not $x1262)))
+(let (($x1318 (and $x1309 $x291 $x1306)))
+(let ((?x671 (+ ?x155 ?x273)))
+(let (($x689 (= ?x303 ?x671)))
+(let (($x692 (and $x291 $x689)))
+(let (($x314 (< ?x273 ?x303)))
+(let (($x695 (and $x314 $x692)))
+(let ((@x1317 (monotonicity (rewrite (= $x314 $x1309)) (monotonicity (rewrite (= $x689 $x1306)) (= $x692 (and $x291 $x1306))) (= $x695 (and $x1309 (and $x291 $x1306))))))
+(let ((@x1322 (trans @x1317 (rewrite (= (and $x1309 (and $x291 $x1306)) $x1318)) (= $x695 $x1318))))
+(let (($x1298 (= (< ?x273 b_Infinity$) (not (<= (+ b_Infinity$ (* (- 1) ?x273)) 0)))))
+(let ((@x1302 (monotonicity (rewrite $x1298) (= (and $x132 (< ?x273 b_Infinity$)) $x1300))))
+(let ((@x1305 (monotonicity @x1302 (= (not (and $x132 (< ?x273 b_Infinity$))) (not $x1300)))))
+(let ((@x1328 (monotonicity @x1305 (quant-intro @x1322 (= $x698 $x1323)) (= $x705 (or (not $x1300) $x1323)))))
+(let (($x1282 (>= (+ ?x155 ?x273 ?x1263) 0)))
+(let (($x922 (<= (+ b_Infinity$ (* (- 1) ?x155)) 0)))
+(let (($x923 (not $x922)))
+(let (($x1276 (and $x291 $x923)))
+(let (($x1279 (not $x1276)))
+(let (($x1286 (or $x1279 $x1282)))
+(let (($x674 (<= ?x303 ?x671)))
+(let (($x681 (or (not (and $x291 (< ?x155 b_Infinity$))) $x674)))
+(let ((@x925 (rewrite (= (< ?x155 b_Infinity$) $x923))))
+(let ((@x1281 (monotonicity (monotonicity @x925 (= (and $x291 (< ?x155 b_Infinity$)) $x1276)) (= (not (and $x291 (< ?x155 b_Infinity$))) $x1279))))
+(let ((@x1291 (quant-intro (monotonicity @x1281 (rewrite (= $x674 $x1282)) (= $x681 $x1286)) (= $x686 $x1289))))
+(let ((@x1334 (monotonicity (monotonicity @x1291 (= (not $x686) $x1292)) (quant-intro @x1328 (= $x710 $x1329)) (= $x738 $x1332))))
+(let (($x301 (fun_app$ v_b_Visited_G_2$ ?1)))
+(let (($x300 (not $x291)))
+(let (($x302 (and $x300 $x301)))
+(let (($x664 (not $x302)))
+(let (($x1267 (or $x664 $x1262)))
+(let (($x304 (<= ?x303 ?x273)))
+(let (($x665 (or $x664 $x304)))
+(let ((@x1272 (quant-intro (monotonicity (rewrite (= $x304 $x1262)) (= $x665 $x1267)) (= $x668 $x1270))))
+(let ((@x1340 (monotonicity (monotonicity @x1272 (= (not $x668) $x1273)) (monotonicity @x1291 @x1334 (= $x743 $x1335)) (= $x750 $x1338))))
+(let ((@x1258 (quant-intro (rewrite (= (<= 0 ?x273) (>= ?x273 0))) (= $x299 $x1256))))
+(let ((@x1346 (monotonicity (monotonicity @x1258 (= (not $x299) $x1259)) (monotonicity @x1272 @x1340 (= $x755 $x1341)) (= $x762 $x1344))))
+(let ((@x1352 (monotonicity (monotonicity @x1258 @x1346 (= $x767 $x1347)) (= $x774 $x1350))))
+(let ((@x1361 (monotonicity (monotonicity (monotonicity @x1352 (= $x779 $x1353)) (= $x786 $x1356)) (= $x791 $x1359))))
+(let (($x1243 (>= (+ (fun_app$c v_b_SP_G_1$ ?0) (* (- 1) ?x273)) 0)))
+(let ((@x1249 (quant-intro (rewrite (= (<= ?x273 (fun_app$c v_b_SP_G_1$ ?0)) $x1243)) (= $x290 $x1247))))
+(let ((@x1364 (monotonicity (monotonicity @x1249 (= (not $x290) $x1250)) @x1361 (= $x798 $x1362))))
+(let (($x1232 (and $x1080 (and $x256 (and $x1214 (and $x1209 (and $x266 (and $x1193 $x1199))))))))
+(let (($x1230 (= $x632 (and $x256 (and $x1214 (and $x1209 (and $x266 (and $x1193 $x1199))))))))
+(let ((?x174 (fun_app$c v_b_SP_G_1$ ?0)))
+(let (($x278 (= ?x273 ?x174)))
+(let (($x1175 (<= (+ ?x174 ?x1173 (* (- 1) (b_G$ (pair$ v_b_v_G_1$ ?0)))) 0)))
+(let (($x1169 (<= (+ b_Infinity$ (* (- 1) (b_G$ (pair$ v_b_v_G_1$ ?0)))) 0)))
+(let (($x1179 (and (not $x1169) (not $x1175))))
+(let (($x1196 (or $x1179 $x278)))
+(let (($x272 (and (< (b_G$ (pair$ v_b_v_G_1$ ?0)) b_Infinity$) (< (+ ?x257 (b_G$ (pair$ v_b_v_G_1$ ?0))) ?x174))))
+(let (($x614 (or $x272 $x278)))
+(let ((@x1178 (rewrite (= (< (+ ?x257 (b_G$ (pair$ v_b_v_G_1$ ?0))) ?x174) (not $x1175)))))
+(let ((@x1172 (rewrite (= (< (b_G$ (pair$ v_b_v_G_1$ ?0)) b_Infinity$) (not $x1169)))))
+(let ((@x1198 (monotonicity (monotonicity @x1172 @x1178 (= $x272 $x1179)) (= $x614 $x1196))))
+(let (($x1185 (= (+ ?x257 (b_G$ (pair$ v_b_v_G_1$ ?0)) (* (- 1) ?x273)) 0)))
+(let (($x1182 (not $x1179)))
+(let (($x1190 (or $x1182 $x1185)))
+(let ((?x268 (b_G$ (pair$ v_b_v_G_1$ ?0))))
+(let ((?x270 (+ ?x257 ?x268)))
+(let (($x274 (= ?x273 ?x270)))
+(let (($x277 (not $x272)))
+(let (($x608 (or $x277 $x274)))
+(let ((@x1184 (monotonicity (monotonicity @x1172 @x1178 (= $x272 $x1179)) (= $x277 $x1182))))
+(let ((@x1195 (quant-intro (monotonicity @x1184 (rewrite (= $x274 $x1185)) (= $x608 $x1190)) (= $x611 $x1193))))
+(let ((@x1219 (monotonicity @x1195 (quant-intro @x1198 (= $x617 $x1199)) (= $x620 (and $x1193 $x1199)))))
+(let (($x178 (fun_app$ v_b_Visited_G_1$ ?0)))
+(let (($x1206 (or $x178 (>= (+ ?x174 ?x1173) 0))))
+(let (($x259 (<= ?x257 ?x174)))
+(let (($x602 (or $x178 $x259)))
+(let ((@x1208 (monotonicity (rewrite (= $x259 (>= (+ ?x174 ?x1173) 0))) (= $x602 $x1206))))
+(let ((@x1225 (monotonicity (quant-intro @x1208 (= $x605 $x1209)) (monotonicity @x1219 (= $x623 (and $x266 (and $x1193 $x1199)))) (= $x626 (and $x1209 (and $x266 (and $x1193 $x1199)))))))
+(let ((@x1228 (monotonicity (rewrite (= $x258 $x1214)) @x1225 (= $x629 (and $x1214 (and $x1209 (and $x266 (and $x1193 $x1199))))))))
+(let (($x1002 (<= (+ b_Infinity$ (* (- 1) ?x174)) 0)))
+(let (($x1003 (not $x1002)))
+(let (($x179 (not $x178)))
+(let (($x1077 (and $x179 $x1003)))
+(let ((@x1079 (monotonicity (rewrite (= (< ?x174 b_Infinity$) $x1003)) (= (and $x179 (< ?x174 b_Infinity$)) $x1077))))
+(let ((@x1234 (monotonicity (quant-intro @x1079 (= $x209 $x1080)) (monotonicity @x1228 $x1230) (= $x635 $x1232))))
+(let ((@x1242 (monotonicity (trans @x1234 (rewrite (= $x1232 $x1235)) (= $x635 $x1235)) (= (not $x635) $x1240))))
+(let ((@x1370 (monotonicity @x1242 (monotonicity @x1249 @x1364 (= $x803 $x1365)) (= $x810 $x1368))))
+(let ((?x230 (fun_app$c v_b_SP_G_3$ ?0)))
+(let (($x1140 (>= (+ ?x155 ?x230 (* (- 1) (fun_app$c v_b_SP_G_3$ ?1))) 0)))
+(let (($x1099 (<= (+ b_Infinity$ (* (- 1) ?x230)) 0)))
+(let (($x1100 (not $x1099)))
+(let (($x1134 (and $x1100 $x923)))
+(let (($x1137 (not $x1134)))
+(let (($x1143 (or $x1137 $x1140)))
+(let ((?x521 (+ ?x155 ?x230)))
+(let ((?x233 (fun_app$c v_b_SP_G_3$ ?1)))
+(let (($x545 (<= ?x233 ?x521)))
+(let (($x552 (or (not (and (< ?x230 b_Infinity$) (< ?x155 b_Infinity$))) $x545)))
+(let ((@x1136 (monotonicity (rewrite (= (< ?x230 b_Infinity$) $x1100)) @x925 (= (and (< ?x230 b_Infinity$) (< ?x155 b_Infinity$)) $x1134))))
+(let ((@x1139 (monotonicity @x1136 (= (not (and (< ?x230 b_Infinity$) (< ?x155 b_Infinity$))) $x1137))))
+(let ((@x1148 (quant-intro (monotonicity @x1139 (rewrite (= $x545 $x1140)) (= $x552 $x1143)) (= $x557 $x1146))))
+(let ((@x1154 (monotonicity (monotonicity @x1148 (= (not $x557) $x1149)) (= $x573 $x1152))))
+(let (($x1122 (exists ((?v1 B_Vertex$) )(let ((?x230 (fun_app$c v_b_SP_G_3$ ?v1)))
+(let ((?x155 (b_G$ (pair$ ?v1 ?0))))
+(and (not (>= (+ ?x230 (* (- 1) (fun_app$c v_b_SP_G_3$ ?0))) 0)) (= (+ ?x155 ?x230 (* (- 1) (fun_app$c v_b_SP_G_3$ ?0))) 0)))))
+))
+(let (($x1103 (and $x132 $x1100)))
+(let (($x1106 (not $x1103)))
+(let (($x1125 (or $x1106 $x1122)))
+(let (($x530 (exists ((?v1 B_Vertex$) )(let ((?x230 (fun_app$c v_b_SP_G_3$ ?v1)))
+(let ((?x155 (b_G$ (pair$ ?v1 ?0))))
+(let ((?x521 (+ ?x155 ?x230)))
+(let ((?x233 (fun_app$c v_b_SP_G_3$ ?0)))
+(let (($x524 (= ?x233 ?x521)))
+(let (($x234 (< ?x230 ?x233)))
+(and $x234 $x524))))))))
+))
+(let (($x537 (or (not (and $x132 (< ?x230 b_Infinity$))) $x530)))
+(let (($x1119 (and (not (>= (+ ?x230 (* (- 1) ?x233)) 0)) (= (+ ?x155 ?x230 (* (- 1) ?x233)) 0))))
+(let (($x524 (= ?x233 ?x521)))
+(let (($x234 (< ?x230 ?x233)))
+(let (($x527 (and $x234 $x524)))
+(let ((@x1121 (monotonicity (rewrite (= $x234 (not (>= (+ ?x230 (* (- 1) ?x233)) 0)))) (rewrite (= $x524 (= (+ ?x155 ?x230 (* (- 1) ?x233)) 0))) (= $x527 $x1119))))
+(let ((@x1105 (monotonicity (rewrite (= (< ?x230 b_Infinity$) $x1100)) (= (and $x132 (< ?x230 b_Infinity$)) $x1103))))
+(let ((@x1127 (monotonicity (monotonicity @x1105 (= (not (and $x132 (< ?x230 b_Infinity$))) $x1106)) (quant-intro @x1121 (= $x530 $x1122)) (= $x537 $x1125))))
+(let ((@x1133 (monotonicity (quant-intro @x1127 (= $x542 $x1128)) (= (not $x542) $x1131))))
+(let ((@x1160 (monotonicity @x1133 (monotonicity @x1148 @x1154 (= $x578 $x1155)) (= $x585 $x1158))))
+(let ((@x1091 (rewrite (= (and $x1083 (and $x212 (and $x215 (and $x217 $x220)))) $x1089))))
+(let (($x493 (and $x212 (and $x215 (and $x217 $x220)))))
+(let (($x507 (and $x210 $x493)))
+(let ((@x1088 (monotonicity (monotonicity (quant-intro @x1079 (= $x209 $x1080)) (= $x210 $x1083)) (= $x507 (and $x1083 $x493)))))
+(let ((@x1096 (monotonicity (trans @x1088 @x1091 (= $x507 $x1089)) (= (not $x507) $x1094))))
+(let ((@x1166 (monotonicity @x1096 (monotonicity (quant-intro @x1127 (= $x542 $x1128)) @x1160 (= $x590 $x1161)) (= $x597 $x1164))))
+(let (($x1070 (= (and $x980 (and $x173 (and $x1051 (and $x1045 (and $x997 $x1037))))) $x1069)))
+(let (($x1067 (= $x482 (and $x980 (and $x173 (and $x1051 (and $x1045 (and $x997 $x1037))))))))
+(let (($x1031 (exists ((?v1 B_Vertex$) )(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v1)))
+(let ((?x155 (b_G$ (pair$ ?v1 ?0))))
+(let (($x1012 (= (+ ?x155 ?x174 (* (- 1) (fun_app$c v_b_SP_G_1$ ?0))) 0)))
+(let (($x178 (fun_app$ v_b_Visited_G_1$ ?v1)))
+(let (($x1015 (>= (+ ?x174 (* (- 1) (fun_app$c v_b_SP_G_1$ ?0))) 0)))
+(let (($x1017 (not $x1015)))
+(and $x1017 $x178 $x1012))))))))
+))
+(let (($x1006 (and $x132 $x1003)))
+(let (($x1009 (not $x1006)))
+(let (($x1034 (or $x1009 $x1031)))
+(let (($x437 (exists ((?v1 B_Vertex$) )(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v1)))
+(let ((?x155 (b_G$ (pair$ ?v1 ?0))))
+(let ((?x410 (+ ?x155 ?x174)))
+(let ((?x182 (fun_app$c v_b_SP_G_1$ ?0)))
+(let (($x428 (= ?x182 ?x410)))
+(let (($x178 (fun_app$ v_b_Visited_G_1$ ?v1)))
+(let (($x431 (and $x178 $x428)))
+(let (($x193 (< ?x174 ?x182)))
+(and $x193 $x431))))))))))
+))
+(let (($x444 (or (not (and $x132 (< ?x174 b_Infinity$))) $x437)))
+(let (($x1012 (= (+ ?x155 ?x174 (* (- 1) (fun_app$c v_b_SP_G_1$ ?1))) 0)))
+(let (($x1015 (>= (+ ?x174 (* (- 1) (fun_app$c v_b_SP_G_1$ ?1))) 0)))
+(let (($x1017 (not $x1015)))
+(let (($x1026 (and $x1017 $x178 $x1012)))
+(let ((?x410 (+ ?x155 ?x174)))
+(let ((?x182 (fun_app$c v_b_SP_G_1$ ?1)))
+(let (($x428 (= ?x182 ?x410)))
+(let (($x431 (and $x178 $x428)))
+(let (($x193 (< ?x174 ?x182)))
+(let (($x434 (and $x193 $x431)))
+(let ((@x1025 (monotonicity (rewrite (= $x193 $x1017)) (monotonicity (rewrite (= $x428 $x1012)) (= $x431 (and $x178 $x1012))) (= $x434 (and $x1017 (and $x178 $x1012))))))
+(let ((@x1030 (trans @x1025 (rewrite (= (and $x1017 (and $x178 $x1012)) $x1026)) (= $x434 $x1026))))
+(let ((@x1008 (monotonicity (rewrite (= (< ?x174 b_Infinity$) $x1003)) (= (and $x132 (< ?x174 b_Infinity$)) $x1006))))
+(let ((@x1036 (monotonicity (monotonicity @x1008 (= (not (and $x132 (< ?x174 b_Infinity$))) $x1009)) (quant-intro @x1030 (= $x437 $x1031)) (= $x444 $x1034))))
+(let (($x990 (>= (+ ?x155 ?x174 (* (- 1) ?x182)) 0)))
+(let (($x983 (and $x178 $x923)))
+(let (($x986 (not $x983)))
+(let (($x994 (or $x986 $x990)))
+(let (($x413 (<= ?x182 ?x410)))
+(let (($x420 (or (not (and $x178 (< ?x155 b_Infinity$))) $x413)))
+(let ((@x988 (monotonicity (monotonicity @x925 (= (and $x178 (< ?x155 b_Infinity$)) $x983)) (= (not (and $x178 (< ?x155 b_Infinity$))) $x986))))
+(let ((@x999 (quant-intro (monotonicity @x988 (rewrite (= $x413 $x990)) (= $x420 $x994)) (= $x425 $x997))))
+(let ((@x1056 (monotonicity @x999 (quant-intro @x1036 (= $x449 $x1037)) (= $x459 (and $x997 $x1037)))))
+(let (($x180 (fun_app$ v_b_Visited_G_1$ ?1)))
+(let (($x181 (and $x179 $x180)))
+(let (($x403 (not $x181)))
+(let (($x1042 (or $x403 $x1015)))
+(let (($x183 (<= ?x182 ?x174)))
+(let (($x404 (or $x403 $x183)))
+(let ((@x1047 (quant-intro (monotonicity (rewrite (= $x183 $x1015)) (= $x404 $x1042)) (= $x407 $x1045))))
+(let ((@x1053 (quant-intro (rewrite (= (<= 0 ?x174) (>= ?x174 0))) (= $x176 $x1051))))
+(let ((@x1062 (monotonicity @x1053 (monotonicity @x1047 @x1056 (= $x462 (and $x1045 (and $x997 $x1037)))) (= $x465 (and $x1051 (and $x1045 (and $x997 $x1037)))))))
+(let ((@x1065 (monotonicity @x1062 (= $x468 (and $x173 (and $x1051 (and $x1045 (and $x997 $x1037))))))))
+(let (($x974 (exists ((?v1 B_Vertex$) )(let ((?x155 (b_G$ (pair$ ?v1 ?0))))
+(let ((?x128 (v_b_SP_G_0$ ?v1)))
+(let (($x957 (= (+ ?x128 (* (- 1) (v_b_SP_G_0$ ?0)) ?x155) 0)))
+(let (($x136 (v_b_Visited_G_0$ ?v1)))
+(let (($x907 (>= (+ ?x128 (* (- 1) (v_b_SP_G_0$ ?0))) 0)))
+(let (($x960 (not $x907)))
+(and $x960 $x136 $x957))))))))
+))
+(let (($x951 (and $x132 (not (<= (+ b_Infinity$ (* (- 1) (v_b_SP_G_0$ ?0))) 0)))))
+(let (($x954 (not $x951)))
+(let (($x977 (or $x954 $x974)))
+(let (($x168 (exists ((?v1 B_Vertex$) )(let (($x136 (v_b_Visited_G_0$ ?v1)))
+(let (($x166 (and $x136 (= (v_b_SP_G_0$ ?0) (+ (v_b_SP_G_0$ ?v1) (b_G$ (pair$ ?v1 ?0)))))))
+(and (< (v_b_SP_G_0$ ?v1) (v_b_SP_G_0$ ?0)) $x166))))
+))
+(let (($x397 (or (not (and $x132 (< (v_b_SP_G_0$ ?0) b_Infinity$))) $x168)))
+(let (($x957 (= (+ (v_b_SP_G_0$ ?0) (* (- 1) (v_b_SP_G_0$ ?1)) ?x155) 0)))
+(let (($x136 (v_b_Visited_G_0$ ?0)))
+(let (($x907 (>= (+ (v_b_SP_G_0$ ?0) (* (- 1) (v_b_SP_G_0$ ?1))) 0)))
+(let (($x960 (not $x907)))
+(let (($x969 (and $x960 $x136 $x957)))
+(let (($x167 (and (< (v_b_SP_G_0$ ?0) (v_b_SP_G_0$ ?1)) (and $x136 (= (v_b_SP_G_0$ ?1) (+ (v_b_SP_G_0$ ?0) ?x155))))))
+(let (($x964 (= (and $x136 (= (v_b_SP_G_0$ ?1) (+ (v_b_SP_G_0$ ?0) ?x155))) (and $x136 $x957))))
+(let ((@x959 (rewrite (= (= (v_b_SP_G_0$ ?1) (+ (v_b_SP_G_0$ ?0) ?x155)) $x957))))
+(let ((@x968 (monotonicity (rewrite (= (< (v_b_SP_G_0$ ?0) (v_b_SP_G_0$ ?1)) $x960)) (monotonicity @x959 $x964) (= $x167 (and $x960 (and $x136 $x957))))))
+(let ((@x973 (trans @x968 (rewrite (= (and $x960 (and $x136 $x957)) $x969)) (= $x167 $x969))))
+(let (($x949 (= (< (v_b_SP_G_0$ ?0) b_Infinity$) (not (<= (+ b_Infinity$ (* (- 1) (v_b_SP_G_0$ ?0))) 0)))))
+(let ((@x953 (monotonicity (rewrite $x949) (= (and $x132 (< (v_b_SP_G_0$ ?0) b_Infinity$)) $x951))))
+(let ((@x956 (monotonicity @x953 (= (not (and $x132 (< (v_b_SP_G_0$ ?0) b_Infinity$))) $x954))))
+(let ((@x982 (quant-intro (monotonicity @x956 (quant-intro @x973 (= $x168 $x974)) (= $x397 $x977)) (= $x400 $x980))))
+(let ((@x1076 (monotonicity (trans (monotonicity @x982 @x1065 $x1067) (rewrite $x1070) (= $x482 $x1069)) (= (not $x482) $x1074))))
+(let ((@x1376 (monotonicity @x1076 (monotonicity @x1166 @x1370 (= $x815 $x1371)) (= $x822 $x1374))))
+(let (($x933 (>= (+ (v_b_SP_G_0$ ?0) (* (- 1) (v_b_SP_G_0$ ?1)) ?x155) 0)))
+(let (($x926 (and $x136 $x923)))
+(let (($x929 (not $x926)))
+(let (($x936 (or $x929 $x933)))
+(let ((?x150 (v_b_SP_G_0$ ?1)))
+(let (($x159 (<= ?x150 (+ (v_b_SP_G_0$ ?0) ?x155))))
+(let (($x390 (or (not (and $x136 (< ?x155 b_Infinity$))) $x159)))
+(let ((@x931 (monotonicity (monotonicity @x925 (= (and $x136 (< ?x155 b_Infinity$)) $x926)) (= (not (and $x136 (< ?x155 b_Infinity$))) $x929))))
+(let ((@x941 (quant-intro (monotonicity @x931 (rewrite (= $x159 $x933)) (= $x390 $x936)) (= $x393 $x939))))
+(let ((@x1382 (monotonicity (monotonicity @x941 (= (not $x393) $x942)) (monotonicity @x982 @x1376 (= $x827 $x1377)) (= $x834 $x1380))))
+(let (($x148 (v_b_Visited_G_0$ ?1)))
+(let (($x137 (not $x136)))
+(let (($x149 (and $x137 $x148)))
+(let (($x382 (not $x149)))
+(let (($x911 (or $x382 $x907)))
+(let ((?x128 (v_b_SP_G_0$ ?0)))
+(let (($x151 (<= ?x150 ?x128)))
+(let (($x383 (or $x382 $x151)))
+(let ((@x916 (quant-intro (monotonicity (rewrite (= $x151 $x907)) (= $x383 $x911)) (= $x386 $x914))))
+(let ((@x1388 (monotonicity (monotonicity @x916 (= (not $x386) $x917)) (monotonicity @x941 @x1382 (= $x839 $x1383)) (= $x846 $x1386))))
+(let ((@x901 (quant-intro (rewrite (= (<= 0 ?x128) (>= ?x128 0))) (= $x147 $x899))))
+(let ((@x1394 (monotonicity (monotonicity @x901 (= (not $x147) $x902)) (monotonicity @x916 @x1388 (= $x851 $x1389)) (= $x858 $x1392))))
+(let ((@x1400 (monotonicity (monotonicity @x901 @x1394 (= $x863 $x1395)) (= $x870 $x1398))))
+(let ((@x895 (monotonicity (rewrite (= (and $x354 (and $x360 $x138)) $x890)) (= (not (and $x354 (and $x360 $x138))) (not $x890)))))
+(let ((@x1406 (monotonicity @x895 (monotonicity @x1400 (= $x875 $x1401)) (= $x882 (or (not $x890) $x1401)))))
+(let (($x318 (exists ((?v1 B_Vertex$) )(let (($x291 (fun_app$ v_b_Visited_G_2$ ?v1)))
+(let (($x316 (and $x291 (= (v_b_SP_G_2$ ?0) (+ (v_b_SP_G_2$ ?v1) (b_G$ (pair$ ?v1 ?0)))))))
+(let ((?x303 (v_b_SP_G_2$ ?0)))
+(let ((?x273 (v_b_SP_G_2$ ?v1)))
+(let (($x314 (< ?x273 ?x303)))
+(and $x314 $x316)))))))
+))
+(let (($x313 (and $x132 (< ?x273 b_Infinity$))))
+(let (($x319 (=> $x313 $x318)))
+(let ((@x691 (monotonicity (rewrite (= (+ ?x273 ?x155) ?x671)) (= (= ?x303 (+ ?x273 ?x155)) $x689))))
+(let ((@x697 (monotonicity (monotonicity @x691 (= (and $x291 (= ?x303 (+ ?x273 ?x155))) $x692)) (= (and $x314 (and $x291 (= ?x303 (+ ?x273 ?x155)))) $x695))))
+(let ((@x703 (monotonicity (quant-intro @x697 (= $x318 $x698)) (= $x319 (=> $x313 $x698)))))
+(let ((@x712 (quant-intro (trans @x703 (rewrite (= (=> $x313 $x698) $x705)) (= $x319 $x705)) (= $x320 $x710))))
+(let ((@x719 (trans (monotonicity @x712 (= $x321 (and $x710 false))) (rewrite (= (and $x710 false) false)) (= $x321 false))))
+(let ((@x726 (trans (monotonicity @x719 (= $x322 (=> false true))) (rewrite (= (=> false true) true)) (= $x322 true))))
+(let ((@x733 (trans (monotonicity @x712 @x726 (= $x323 (and $x710 true))) (rewrite (= (and $x710 true) $x710)) (= $x323 $x710))))
+(let (($x156 (< ?x155 b_Infinity$)))
+(let (($x307 (and $x291 $x156)))
+(let (($x310 (=> $x307 (<= ?x303 (+ ?x273 ?x155)))))
+(let ((@x676 (monotonicity (rewrite (= (+ ?x273 ?x155) ?x671)) (= (<= ?x303 (+ ?x273 ?x155)) $x674))))
+(let ((@x685 (trans (monotonicity @x676 (= $x310 (=> $x307 $x674))) (rewrite (= (=> $x307 $x674) $x681)) (= $x310 $x681))))
+(let ((@x736 (monotonicity (quant-intro @x685 (= $x311 $x686)) @x733 (= $x324 (=> $x686 $x710)))))
+(let ((@x745 (monotonicity (quant-intro @x685 (= $x311 $x686)) (trans @x736 (rewrite (= (=> $x686 $x710) $x738)) (= $x324 $x738)) (= (and $x311 $x324) $x743))))
+(let ((@x748 (monotonicity (quant-intro (rewrite (= (=> $x302 $x304) $x665)) (= $x306 $x668)) @x745 (= $x326 (=> $x668 $x743)))))
+(let ((@x757 (monotonicity (quant-intro (rewrite (= (=> $x302 $x304) $x665)) (= $x306 $x668)) (trans @x748 (rewrite (= (=> $x668 $x743) $x750)) (= $x326 $x750)) (= (and $x306 $x326) $x755))))
+(let ((@x766 (trans (monotonicity @x757 (= $x328 (=> $x299 $x755))) (rewrite (= (=> $x299 $x755) $x762)) (= $x328 $x762))))
+(let ((@x772 (monotonicity (monotonicity @x766 (= (and $x299 $x328) $x767)) (= $x330 (=> $x297 $x767)))))
+(let ((@x781 (monotonicity (trans @x772 (rewrite (= (=> $x297 $x767) $x774)) (= $x330 $x774)) (= (and $x297 $x330) $x779))))
+(let ((@x654 (quant-intro (rewrite (= (=> $x291 $x278) (or $x300 $x278))) (= $x293 $x652))))
+(let ((@x659 (monotonicity @x654 (rewrite (= (and true true) true)) (= $x295 (and $x652 true)))))
+(let ((@x784 (monotonicity (trans @x659 (rewrite (= (and $x652 true) $x652)) (= $x295 $x652)) @x781 (= $x332 (=> $x652 $x779)))))
+(let ((@x793 (monotonicity @x654 (trans @x784 (rewrite (= (=> $x652 $x779) $x786)) (= $x332 $x786)) (= (and $x293 $x332) $x791))))
+(let ((@x802 (trans (monotonicity @x793 (= $x334 (=> $x290 $x791))) (rewrite (= (=> $x290 $x791) $x798)) (= $x334 $x798))))
+(let (($x633 (= (and $x256 (and $x258 (and $x261 (and $x266 (and $x276 $x280))))) $x632)))
+(let ((@x622 (monotonicity (quant-intro (rewrite (= (=> $x272 $x274) $x608)) (= $x276 $x611)) (quant-intro (rewrite (= (=> $x277 $x278) $x614)) (= $x280 $x617)) (= (and $x276 $x280) $x620))))
+(let ((@x628 (monotonicity (quant-intro (rewrite (= (=> $x179 $x259) $x602)) (= $x261 $x605)) (monotonicity @x622 (= (and $x266 (and $x276 $x280)) $x623)) (= (and $x261 (and $x266 (and $x276 $x280))) $x626))))
+(let ((@x631 (monotonicity @x628 (= (and $x258 (and $x261 (and $x266 (and $x276 $x280)))) $x629))))
+(let ((@x640 (monotonicity (monotonicity (monotonicity @x631 $x633) (= $x286 $x635)) (= $x287 (and true $x635)))))
+(let ((@x646 (monotonicity (trans @x640 (rewrite (= (and true $x635) $x635)) (= $x287 $x635)) (= $x288 (and true $x635)))))
+(let ((@x808 (monotonicity (trans @x646 (rewrite (= (and true $x635) $x635)) (= $x288 $x635)) (monotonicity @x802 (= (and $x290 $x334) $x803)) (= $x336 (=> $x635 $x803)))))
+(let ((@x564 (monotonicity (rewrite (= (=> $x246 true) true)) (= $x248 (and $x246 true)))))
+(let (($x231 (< ?x230 b_Infinity$)))
+(let (($x241 (and $x231 $x156)))
+(let (($x243 (=> $x241 (<= ?x233 (+ ?x230 ?x155)))))
+(let ((@x547 (monotonicity (rewrite (= (+ ?x230 ?x155) ?x521)) (= (<= ?x233 (+ ?x230 ?x155)) $x545))))
+(let ((@x556 (trans (monotonicity @x547 (= $x243 (=> $x241 $x545))) (rewrite (= (=> $x241 $x545) $x552)) (= $x243 $x552))))
+(let ((@x571 (monotonicity (quant-intro @x556 (= $x244 $x557)) (trans @x564 (rewrite (= (and $x246 true) $x246)) (= $x248 $x246)) (= $x249 (=> $x557 $x246)))))
+(let ((@x580 (monotonicity (quant-intro @x556 (= $x244 $x557)) (trans @x571 (rewrite (= (=> $x557 $x246) $x573)) (= $x249 $x573)) (= (and $x244 $x249) $x578))))
+(let (($x238 (exists ((?v1 B_Vertex$) )(let ((?x155 (b_G$ (pair$ ?v1 ?0))))
+(let ((?x230 (fun_app$c v_b_SP_G_3$ ?v1)))
+(let ((?x235 (+ ?x230 ?x155)))
+(let ((?x233 (fun_app$c v_b_SP_G_3$ ?0)))
+(let (($x234 (< ?x230 ?x233)))
+(and $x234 (= ?x233 ?x235))))))))
+))
+(let (($x232 (and $x132 $x231)))
+(let (($x239 (=> $x232 $x238)))
+(let ((@x526 (monotonicity (rewrite (= (+ ?x230 ?x155) ?x521)) (= (= ?x233 (+ ?x230 ?x155)) $x524))))
+(let ((@x532 (quant-intro (monotonicity @x526 (= (and $x234 (= ?x233 (+ ?x230 ?x155))) $x527)) (= $x238 $x530))))
+(let ((@x541 (trans (monotonicity @x532 (= $x239 (=> $x232 $x530))) (rewrite (= (=> $x232 $x530) $x537)) (= $x239 $x537))))
+(let ((@x583 (monotonicity (quant-intro @x541 (= $x240 $x542)) @x580 (= $x251 (=> $x542 $x578)))))
+(let ((@x592 (monotonicity (quant-intro @x541 (= $x240 $x542)) (trans @x583 (rewrite (= (=> $x542 $x578) $x585)) (= $x251 $x585)) (= (and $x240 $x251) $x590))))
+(let (($x491 (= (and $x215 (and $x217 (and $x220 true))) (and $x215 (and $x217 $x220)))))
+(let ((@x489 (monotonicity (rewrite (= (and $x220 true) $x220)) (= (and $x217 (and $x220 true)) (and $x217 $x220)))))
+(let ((@x495 (monotonicity (monotonicity @x489 $x491) (= (and $x212 (and $x215 (and $x217 (and $x220 true)))) $x493))))
+(let ((@x502 (trans (monotonicity @x495 (= $x225 (and true $x493))) (rewrite (= (and true $x493) $x493)) (= $x225 $x493))))
+(let ((@x506 (trans (monotonicity @x502 (= $x226 (and true $x493))) (rewrite (= (and true $x493) $x493)) (= $x226 $x493))))
+(let ((@x512 (monotonicity (monotonicity @x506 (= (and $x210 $x226) $x507)) (= $x228 (and true $x507)))))
+(let ((@x518 (monotonicity (trans @x512 (rewrite (= (and true $x507) $x507)) (= $x228 $x507)) (= $x229 (and true $x507)))))
+(let ((@x595 (monotonicity (trans @x518 (rewrite (= (and true $x507) $x507)) (= $x229 $x507)) @x592 (= $x253 (=> $x507 $x590)))))
+(let ((@x817 (monotonicity (trans @x595 (rewrite (= (=> $x507 $x590) $x597)) (= $x253 $x597)) (trans @x808 (rewrite (= (=> $x635 $x803) $x810)) (= $x336 $x810)) (= (and $x253 $x336) $x815))))
+(let (($x197 (exists ((?v1 B_Vertex$) )(let ((?x155 (b_G$ (pair$ ?v1 ?0))))
+(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v1)))
+(let ((?x187 (+ ?x174 ?x155)))
+(let ((?x182 (fun_app$c v_b_SP_G_1$ ?0)))
+(let (($x178 (fun_app$ v_b_Visited_G_1$ ?v1)))
+(let (($x193 (< ?x174 ?x182)))
+(and $x193 (and $x178 (= ?x182 ?x187))))))))))
+))
+(let (($x191 (< ?x174 b_Infinity$)))
+(let (($x192 (and $x132 $x191)))
+(let (($x198 (=> $x192 $x197)))
+(let ((@x430 (monotonicity (rewrite (= (+ ?x174 ?x155) ?x410)) (= (= ?x182 (+ ?x174 ?x155)) $x428))))
+(let ((@x436 (monotonicity (monotonicity @x430 (= (and $x178 (= ?x182 (+ ?x174 ?x155))) $x431)) (= (and $x193 (and $x178 (= ?x182 (+ ?x174 ?x155)))) $x434))))
+(let ((@x442 (monotonicity (quant-intro @x436 (= $x197 $x437)) (= $x198 (=> $x192 $x437)))))
+(let ((@x451 (quant-intro (trans @x442 (rewrite (= (=> $x192 $x437) $x444)) (= $x198 $x444)) (= $x199 $x449))))
+(let ((@x458 (trans (monotonicity @x451 (= $x200 (and $x449 true))) (rewrite (= (and $x449 true) $x449)) (= $x200 $x449))))
+(let (($x186 (and $x178 $x156)))
+(let (($x189 (=> $x186 (<= ?x182 (+ ?x174 ?x155)))))
+(let ((@x415 (monotonicity (rewrite (= (+ ?x174 ?x155) ?x410)) (= (<= ?x182 (+ ?x174 ?x155)) $x413))))
+(let ((@x424 (trans (monotonicity @x415 (= $x189 (=> $x186 $x413))) (rewrite (= (=> $x186 $x413) $x420)) (= $x189 $x420))))
+(let ((@x461 (monotonicity (quant-intro @x424 (= $x190 $x425)) @x458 (= (and $x190 $x200) $x459))))
+(let ((@x464 (monotonicity (quant-intro (rewrite (= (=> $x181 $x183) $x404)) (= $x185 $x407)) @x461 (= (and $x185 (and $x190 $x200)) $x462))))
+(let ((@x470 (monotonicity (monotonicity @x464 (= (and $x176 (and $x185 (and $x190 $x200))) $x465)) (= (and $x173 (and $x176 (and $x185 (and $x190 $x200)))) $x468))))
+(let ((@x477 (trans (monotonicity @x470 (= $x205 (and true $x468))) (rewrite (= (and true $x468) $x468)) (= $x205 $x468))))
+(let ((@x481 (trans (monotonicity @x477 (= $x206 (and true $x468))) (rewrite (= (and true $x468) $x468)) (= $x206 $x468))))
+(let ((@x402 (quant-intro (rewrite (= (=> (and $x132 (< ?x128 b_Infinity$)) $x168) $x397)) (= $x170 $x400))))
+(let ((@x820 (monotonicity (monotonicity @x402 @x481 (= (and $x170 $x206) $x482)) @x817 (= $x338 (=> $x482 $x815)))))
+(let ((@x829 (monotonicity @x402 (trans @x820 (rewrite (= (=> $x482 $x815) $x822)) (= $x338 $x822)) (= (and $x170 $x338) $x827))))
+(let ((@x395 (quant-intro (rewrite (= (=> (and $x136 $x156) $x159) $x390)) (= $x161 $x393))))
+(let ((@x838 (trans (monotonicity @x395 @x829 (= $x340 (=> $x393 $x827))) (rewrite (= (=> $x393 $x827) $x834)) (= $x340 $x834))))
+(let ((@x844 (monotonicity (quant-intro (rewrite (= (=> $x149 $x151) $x383)) (= $x153 $x386)) (monotonicity @x395 @x838 (= (and $x161 $x340) $x839)) (= $x342 (=> $x386 $x839)))))
+(let ((@x853 (monotonicity (quant-intro (rewrite (= (=> $x149 $x151) $x383)) (= $x153 $x386)) (trans @x844 (rewrite (= (=> $x386 $x839) $x846)) (= $x342 $x846)) (= (and $x153 $x342) $x851))))
+(let ((@x862 (trans (monotonicity @x853 (= $x344 (=> $x147 $x851))) (rewrite (= (=> $x147 $x851) $x858)) (= $x344 $x858))))
+(let ((@x868 (monotonicity (monotonicity @x862 (= (and $x147 $x344) $x863)) (= $x346 (=> $x145 $x863)))))
+(let ((@x877 (monotonicity (trans @x868 (rewrite (= (=> $x145 $x863) $x870)) (= $x346 $x870)) (= (and $x145 $x346) $x875))))
+(let (($x368 (and $x354 (and $x360 $x138))))
+(let (($x371 (and true $x368)))
+(let ((@x362 (quant-intro (rewrite (= (=> $x132 (= ?x128 b_Infinity$)) $x357)) (= $x135 $x360))))
+(let ((@x367 (monotonicity @x362 (rewrite (= (and $x138 true) $x138)) (= (and $x135 (and $x138 true)) (and $x360 $x138)))))
+(let ((@x356 (quant-intro (rewrite (= (=> $x127 (= ?x128 0)) (or $x132 (= ?x128 0)))) (= $x131 $x354))))
+(let ((@x370 (monotonicity @x356 @x367 (= (and $x131 (and $x135 (and $x138 true))) $x368))))
+(let ((@x377 (trans (monotonicity @x370 (= $x142 $x371)) (rewrite (= $x371 $x368)) (= $x142 $x368))))
+(let ((@x381 (trans (monotonicity @x377 (= $x143 $x371)) (rewrite (= $x371 $x368)) (= $x143 $x368))))
+(let ((@x886 (trans (monotonicity @x381 @x877 (= $x348 (=> $x368 $x875))) (rewrite (= (=> $x368 $x875) $x882)) (= $x348 $x882))))
+(let ((@x1411 (trans (monotonicity @x886 (= $x349 (not $x882))) (monotonicity @x1406 (= (not $x882) $x1407)) (= $x349 $x1407))))
+(let ((@x1413 (not-or-elim (mp (asserted $x349) @x1411 $x1407) $x890)))
+(let ((@x1463 (mp~ (and-elim @x1413 $x360) (nnf-pos (refl (~ $x357 $x357)) (~ $x360 $x360)) $x360)))
+(let ((@x3498 (mp @x1463 (quant-intro (refl (= $x357 $x357)) (= $x360 $x3493)) $x3493)))
+(let ((@x6489 (rewrite (= (or (not $x3493) (or $x1538 $x5616)) (or (not $x3493) $x1538 $x5616)))))
+(let ((@x5602 (mp ((_ quant-inst ?v0!5) (or (not $x3493) (or $x1538 $x5616))) @x6489 (or (not $x3493) $x1538 $x5616))))
+(let ((@x5777 (unit-resolution (hypothesis $x6457) (mp (unit-resolution @x5602 @x3498 (hypothesis $x1539) $x5616) @x5778 $x5625) false)))
+(let ((@x5735 (unit-resolution (lemma @x5777 (or $x5625 $x1538)) (unit-resolution ((_ th-lemma arith triangle-eq) (or $x6457 $x1543)) @x6514 $x6457) @x6246 false)))
+(let (($x3544 (not $x3541)))
+(let (($x3827 (or $x3544 $x3824)))
+(let (($x3830 (not $x3827)))
+(let (($x3524 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(!(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let ((?x128 (v_b_SP_G_0$ ?v1)))
+(let (($x933 (>= (+ ?x128 (* (- 1) (v_b_SP_G_0$ ?v0)) ?x155) 0)))
+(let (($x922 (<= (+ b_Infinity$ (* (- 1) ?x155)) 0)))
+(let (($x136 (v_b_Visited_G_0$ ?v1)))
+(let (($x137 (not $x136)))
+(or $x137 $x922 $x933))))))) :pattern ( (pair$ ?v1 ?v0) )))
+))
+(let (($x3529 (not $x3524)))
+(let (($x3833 (or $x3529 $x3830)))
+(let (($x3836 (not $x3833)))
+(let ((?x1522 (v_b_SP_G_0$ ?v0!4)))
+(let ((?x1523 (* (- 1) ?x1522)))
+(let ((?x1521 (v_b_SP_G_0$ ?v1!3)))
+(let ((?x1513 (pair$ ?v1!3 ?v0!4)))
+(let ((?x1514 (b_G$ ?x1513)))
+(let ((?x2045 (+ ?x1514 ?x1521 ?x1523)))
+(let (($x2048 (>= ?x2045 0)))
+(let (($x1517 (<= (+ b_Infinity$ (* (- 1) ?x1514)) 0)))
+(let (($x1512 (v_b_Visited_G_0$ ?v1!3)))
+(let (($x2394 (not $x1512)))
+(let (($x2409 (or $x2394 $x1517 $x2048)))
+(let (($x3500 (forall ((?v0 B_Vertex$) )(!(let (($x136 (v_b_Visited_G_0$ ?v0)))
+(not $x136)) :pattern ( (v_b_Visited_G_0$ ?v0) )))
+))
+(let ((@x1468 (mp~ (and-elim @x1413 $x138) (nnf-pos (refl (~ $x137 $x137)) (~ $x138 $x138)) $x138)))
+(let ((@x3505 (mp @x1468 (quant-intro (refl (= $x137 $x137)) (= $x138 $x3500)) $x3500)))
+(let ((@x3073 (unit-resolution ((_ quant-inst ?v1!3) (or (not $x3500) $x2394)) @x3505 (hypothesis $x1512) false)))
+(let (($x2414 (not $x2409)))
+(let (($x3839 (or $x2414 $x3836)))
+(let (($x3842 (not $x3839)))
+(let (($x3515 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(!(let (($x907 (>= (+ (v_b_SP_G_0$ ?v1) (* (- 1) (v_b_SP_G_0$ ?v0))) 0)))
+(let (($x136 (v_b_Visited_G_0$ ?v1)))
+(or $x136 (not (v_b_Visited_G_0$ ?v0)) $x907))) :pattern ( (v_b_Visited_G_0$ ?v1) (v_b_Visited_G_0$ ?v0) )))
+))
+(let (($x3520 (not $x3515)))
+(let (($x3845 (or $x3520 $x3842)))
+(let (($x3848 (not $x3845)))
+(let (($x1498 (>= (+ (v_b_SP_G_0$ ?v1!1) (* (- 1) (v_b_SP_G_0$ ?v0!2))) 0)))
+(let (($x1491 (v_b_Visited_G_0$ ?v0!2)))
+(let (($x2348 (not $x1491)))
+(let (($x1489 (v_b_Visited_G_0$ ?v1!1)))
+(let (($x2363 (or $x1489 $x2348 $x1498)))
+(let (($x2368 (not $x2363)))
+(let (($x3851 (or $x2368 $x3848)))
+(let (($x3854 (not $x3851)))
+(let (($x3506 (forall ((?v0 B_Vertex$) )(!(let ((?x128 (v_b_SP_G_0$ ?v0)))
+(>= ?x128 0)) :pattern ( (v_b_SP_G_0$ ?v0) )))
+))
+(let (($x3511 (not $x3506)))
+(let (($x3857 (or $x3511 $x3854)))
+(let (($x3860 (not $x3857)))
+(let ((?x1475 (v_b_SP_G_0$ ?v0!0)))
+(let (($x1476 (>= ?x1475 0)))
+(let (($x1477 (not $x1476)))
+(let ((@x5848 (hypothesis $x1477)))
+(let (($x5440 (<= ?x1475 0)))
+(let (($x86 (<= b_Infinity$ 0)))
+(let (($x87 (not $x86)))
+(let ((@x90 (mp (asserted (< 0 b_Infinity$)) (rewrite (= (< 0 b_Infinity$) $x87)) $x87)))
+(let (($x5734 (= b_Infinity$ ?x1475)))
+(let ((@x4994 (symm (commutativity (= $x5734 (= ?x1475 b_Infinity$))) (= (= ?x1475 b_Infinity$) $x5734))))
+(let (($x5461 (= ?x1475 b_Infinity$)))
+(let (($x5589 (= ?v0!0 b_Source$)))
+(let (($x4695 (not $x5589)))
+(let ((@x5096 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x1475 0)) $x1476)) @x5848 (not (= ?x1475 0)))))
+(let (($x3487 (forall ((?v0 B_Vertex$) )(!(let (($x127 (= ?v0 b_Source$)))
+(let (($x132 (not $x127)))
+(or $x132 (= (v_b_SP_G_0$ ?v0) 0)))) :pattern ( (v_b_SP_G_0$ ?v0) )))
+))
+(let ((@x3491 (quant-intro (refl (= (or $x132 (= ?x128 0)) (or $x132 (= ?x128 0)))) (= $x354 $x3487))))
+(let ((@x1457 (nnf-pos (refl (~ (or $x132 (= ?x128 0)) (or $x132 (= ?x128 0)))) (~ $x354 $x354))))
+(let ((@x3492 (mp (mp~ (and-elim @x1413 $x354) @x1457 $x354) @x3491 $x3487)))
+(let (($x5571 (= (or (not $x3487) (or $x4695 (= ?x1475 0))) (or (not $x3487) $x4695 (= ?x1475 0)))))
+(let ((@x5058 (mp ((_ quant-inst ?v0!0) (or (not $x3487) (or $x4695 (= ?x1475 0)))) (rewrite $x5571) (or (not $x3487) $x4695 (= ?x1475 0)))))
+(let ((@x5156 (rewrite (= (or (not $x3493) (or $x5589 $x5461)) (or (not $x3493) $x5589 $x5461)))))
+(let ((@x5542 (mp ((_ quant-inst ?v0!0) (or (not $x3493) (or $x5589 $x5461))) @x5156 (or (not $x3493) $x5589 $x5461))))
+(let ((@x5003 (mp (unit-resolution @x5542 @x3498 (unit-resolution @x5058 @x3492 @x5096 $x4695) $x5461) @x4994 $x5734)))
+(let ((@x5457 ((_ th-lemma arith triangle-eq) (or (not $x5734) (<= (+ b_Infinity$ (* (- 1) ?x1475)) 0)))))
+(let ((@x5462 (unit-resolution @x5457 @x5003 (<= (+ b_Infinity$ (* (- 1) ?x1475)) 0))))
+(let ((@x5446 (lemma ((_ th-lemma arith farkas 1 -1 1) (hypothesis $x5440) @x5462 @x90 false) (or (not $x5440) $x1476))))
+(let ((@x6353 (unit-resolution @x5446 (unit-resolution ((_ th-lemma arith farkas 1 1) (or $x5440 $x1476)) @x5848 $x5440) @x5848 false)))
+(let (($x3863 (or $x1477 $x3860)))
+(let (($x3866 (not $x3863)))
+(let (($x3869 (or $x869 $x3866)))
+(let (($x3872 (not $x3869)))
+(let (($x5983 (not $x3487)))
+(let (($x3194 (or $x5983 $x145)))
+(let ((@x5448 (monotonicity (rewrite (= (= b_Source$ b_Source$) true)) (= (not (= b_Source$ b_Source$)) (not true)))))
+(let ((@x5820 (trans @x5448 (rewrite (= (not true) false)) (= (not (= b_Source$ b_Source$)) false))))
+(let ((@x5657 (monotonicity @x5820 (= (or (not (= b_Source$ b_Source$)) $x145) (or false $x145)))))
+(let ((@x5707 (trans @x5657 (rewrite (= (or false $x145) $x145)) (= (or (not (= b_Source$ b_Source$)) $x145) $x145))))
+(let ((@x5373 (monotonicity @x5707 (= (or $x5983 (or (not (= b_Source$ b_Source$)) $x145)) $x3194))))
+(let ((@x5431 (trans @x5373 (rewrite (= $x3194 $x3194)) (= (or $x5983 (or (not (= b_Source$ b_Source$)) $x145)) $x3194))))
+(let ((@x5763 (mp ((_ quant-inst b_Source$) (or $x5983 (or (not (= b_Source$ b_Source$)) $x145))) @x5431 $x3194)))
+(let (($x3875 (or $x869 $x3872)))
+(let (($x2848 (forall ((?v1 B_Vertex$) )(let ((?x1911 (v_b_SP_G_2$ ?v0!20)))
+(let ((?x1912 (* (- 1) ?x1911)))
+(let ((?x273 (v_b_SP_G_2$ ?v1)))
+(let (($x2242 (= (+ ?x273 ?x1912 (b_G$ (pair$ ?v1 ?v0!20))) 0)))
+(let (($x291 (fun_app$ v_b_Visited_G_2$ ?v1)))
+(let (($x300 (not $x291)))
+(or (>= (+ ?x273 ?x1912) 0) $x300 (not $x2242)))))))))
+))
+(let (($x2833 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x303 (v_b_SP_G_2$ ?v0)))
+(let ((?x1263 (* (- 1) ?x303)))
+(let ((?x273 (v_b_SP_G_2$ ?v1)))
+(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let (($x1282 (>= (+ ?x155 ?x273 ?x1263) 0)))
+(let (($x922 (<= (+ b_Infinity$ (* (- 1) ?x155)) 0)))
+(let (($x291 (fun_app$ v_b_Visited_G_2$ ?v1)))
+(let (($x300 (not $x291)))
+(or $x300 $x922 $x1282))))))))))
+))
+(let (($x2857 (not (or (not $x2833) $x1909 $x1914 (not $x2848)))))
+(let (($x2862 (or $x2811 $x2857)))
+(let (($x2788 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let (($x1262 (>= (+ (v_b_SP_G_2$ ?v1) (* (- 1) (v_b_SP_G_2$ ?v0))) 0)))
+(let (($x301 (fun_app$ v_b_Visited_G_2$ ?v0)))
+(let (($x2768 (not $x301)))
+(let (($x291 (fun_app$ v_b_Visited_G_2$ ?v1)))
+(or $x291 $x2768 $x1262))))))
+))
+(let (($x2871 (not (or (not $x2788) (not $x2862)))))
+(let (($x2876 (or $x2765 $x2871)))
+(let (($x2884 (not (or $x1259 (not $x2876)))))
+(let (($x2889 (or $x1848 $x2884)))
+(let (($x2897 (not (or $x773 (not $x2889)))))
+(let (($x2902 (or $x773 $x2897)))
+(let (($x2910 (not (or $x785 (not $x2902)))))
+(let (($x2915 (or $x1830 $x2910)))
+(let (($x2923 (not (or $x1250 (not $x2915)))))
+(let (($x2928 (or $x1813 $x2923)))
+(let (($x2742 (forall ((?v0 B_Vertex$) )(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v0)))
+(let ((?x273 (v_b_SP_G_2$ ?v0)))
+(let (($x278 (= ?x273 ?x174)))
+(let ((?x257 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
+(let ((?x1173 (* (- 1) ?x257)))
+(let (($x1175 (<= (+ ?x174 ?x1173 (* (- 1) (b_G$ (pair$ v_b_v_G_1$ ?v0)))) 0)))
+(let (($x1169 (<= (+ b_Infinity$ (* (- 1) (b_G$ (pair$ v_b_v_G_1$ ?v0)))) 0)))
+(let (($x2717 (or $x1169 $x1175)))
+(let (($x2718 (not $x2717)))
+(or $x2718 $x278)))))))))))
+))
+(let (($x2736 (forall ((?v0 B_Vertex$) )(let ((?x273 (v_b_SP_G_2$ ?v0)))
+(let ((?x1186 (* (- 1) ?x273)))
+(let ((?x268 (b_G$ (pair$ v_b_v_G_1$ ?v0))))
+(let ((?x257 (fun_app$c v_b_SP_G_1$ v_b_v_G_1$)))
+(let (($x1185 (= (+ ?x257 ?x268 ?x1186) 0)))
+(let (($x1175 (<= (+ (fun_app$c v_b_SP_G_1$ ?v0) (* (- 1) ?x257) (* (- 1) ?x268)) 0)))
+(let (($x1169 (<= (+ b_Infinity$ (* (- 1) ?x268)) 0)))
+(or $x1169 $x1175 $x1185)))))))))
+))
+(let (($x2939 (or $x1773 $x1778 $x255 $x1213 (not $x1209) $x2935 (not $x2736) (not $x2742) (not $x2928))))
+(let (($x2940 (not $x2939)))
+(let (($x2672 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x230 (fun_app$c v_b_SP_G_3$ ?v1)))
+(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let (($x1140 (>= (+ ?x155 ?x230 (* (- 1) (fun_app$c v_b_SP_G_3$ ?v0))) 0)))
+(let (($x922 (<= (+ b_Infinity$ (* (- 1) ?x155)) 0)))
+(let (($x1099 (<= (+ b_Infinity$ (* (- 1) ?x230)) 0)))
+(or $x1099 $x922 $x1140)))))))
+))
+(let (($x2680 (not (or (not $x2672) $x246))))
+(let (($x2685 (or $x2650 $x2680)))
+(let (($x2628 (forall ((?v0 B_Vertex$) )(let ((?x230 (fun_app$c v_b_SP_G_3$ ?v0)))
+(let ((?x2191 (+ ?x230 (* (- 1) (fun_app$c v_b_SP_G_3$ (?v1!9 ?v0))) (* (- 1) (b_G$ (pair$ (?v1!9 ?v0) ?v0))))))
+(let (($x2192 (= ?x2191 0)))
+(let (($x2176 (<= (+ ?x230 (* (- 1) (fun_app$c v_b_SP_G_3$ (?v1!9 ?v0)))) 0)))
+(let (($x2617 (not (or $x2176 (not $x2192)))))
+(let (($x1099 (<= (+ b_Infinity$ (* (- 1) ?x230)) 0)))
+(let (($x127 (= ?v0 b_Source$)))
+(or $x127 $x1099 $x2617)))))))))
+))
+(let (($x2694 (not (or (not $x2628) (not $x2685)))))
+(let (($x2591 (forall ((?v1 B_Vertex$) )(let ((?x1661 (fun_app$c v_b_SP_G_3$ ?v0!8)))
+(let ((?x1662 (* (- 1) ?x1661)))
+(let ((?x230 (fun_app$c v_b_SP_G_3$ ?v1)))
+(let (($x2148 (= (+ ?x230 ?x1662 (b_G$ (pair$ ?v1 ?v0!8))) 0)))
+(or (>= (+ ?x230 ?x1662) 0) (not $x2148)))))))
+))
+(let (($x2599 (not (or $x1659 $x1664 (not $x2591)))))
+(let (($x2699 (or $x2599 $x2694)))
+(let (($x2576 (forall ((?v0 B_Vertex$) )(let (($x1002 (<= (+ b_Infinity$ (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0))) 0)))
+(let (($x178 (fun_app$ v_b_Visited_G_1$ ?v0)))
+(or $x178 $x1002))))
+))
+(let (($x2712 (not (or (not $x2576) $x2706 $x2707 $x2708 $x2709 (not $x2699)))))
+(let (($x2945 (or $x2712 $x2940)))
+(let (($x2562 (forall ((?v0 B_Vertex$) )(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v0)))
+(let ((?x2128 (+ ?x174 (* (- 1) (fun_app$c v_b_SP_G_1$ (?v1!7 ?v0))) (* (- 1) (b_G$ (pair$ (?v1!7 ?v0) ?v0))))))
+(let (($x2129 (= ?x2128 0)))
+(let (($x2113 (<= (+ ?x174 (* (- 1) (fun_app$c v_b_SP_G_1$ (?v1!7 ?v0)))) 0)))
+(let (($x2551 (not (or $x2113 (not (fun_app$ v_b_Visited_G_1$ (?v1!7 ?v0))) (not $x2129)))))
+(let (($x1002 (<= (+ b_Infinity$ (* (- 1) ?x174)) 0)))
+(let (($x127 (= ?v0 b_Source$)))
+(or $x127 $x1002 $x2551)))))))))
+))
+(let (($x2534 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v1)))
+(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let (($x990 (>= (+ ?x155 ?x174 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0))) 0)))
+(let (($x922 (<= (+ b_Infinity$ (* (- 1) ?x155)) 0)))
+(let (($x178 (fun_app$ v_b_Visited_G_1$ ?v1)))
+(let (($x179 (not $x178)))
+(or $x179 $x922 $x990))))))))
+))
+(let (($x2512 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v1)))
+(let (($x1015 (>= (+ ?x174 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0))) 0)))
+(let (($x178 (fun_app$ v_b_Visited_G_1$ ?v1)))
+(or $x178 (not (fun_app$ v_b_Visited_G_1$ ?v0)) $x1015)))))
+))
+(let (($x2489 (forall ((?v0 B_Vertex$) )(let ((?x128 (v_b_SP_G_0$ ?v0)))
+(let ((?x2090 (+ ?x128 (* (- 1) (v_b_SP_G_0$ (?v1!6 ?v0))) (* (- 1) (b_G$ (pair$ (?v1!6 ?v0) ?v0))))))
+(let (($x2091 (= ?x2090 0)))
+(let (($x2075 (<= (+ ?x128 (* (- 1) (v_b_SP_G_0$ (?v1!6 ?v0)))) 0)))
+(let (($x2478 (not (or $x2075 (not (v_b_Visited_G_0$ (?v1!6 ?v0))) (not $x2091)))))
+(let (($x947 (<= (+ b_Infinity$ (* (- 1) ?x128)) 0)))
+(let (($x127 (= ?v0 b_Source$)))
+(or $x127 $x947 $x2478)))))))))
+))
+(let (($x2958 (or (not $x2489) $x2952 (not $x1051) (not $x2512) (not $x2534) (not $x2562) (not $x2945))))
+(let (($x2959 (not $x2958)))
+(let (($x2451 (forall ((?v1 B_Vertex$) )(let ((?x1540 (v_b_SP_G_0$ ?v0!5)))
+(let ((?x1541 (* (- 1) ?x1540)))
+(let ((?x128 (v_b_SP_G_0$ ?v1)))
+(let (($x136 (v_b_Visited_G_0$ ?v1)))
+(let (($x137 (not $x136)))
+(or (>= (+ ?x128 ?x1541) 0) $x137 (not (= (+ ?x128 ?x1541 (b_G$ (pair$ ?v1 ?v0!5))) 0)))))))))
+))
+(let (($x2459 (not (or $x1538 $x1543 (not $x2451)))))
+(let (($x2964 (or $x2459 $x2959)))
+(let (($x2436 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x155 (b_G$ (pair$ ?v1 ?v0))))
+(let ((?x128 (v_b_SP_G_0$ ?v1)))
+(let (($x933 (>= (+ ?x128 (* (- 1) (v_b_SP_G_0$ ?v0)) ?x155) 0)))
+(let (($x922 (<= (+ b_Infinity$ (* (- 1) ?x155)) 0)))
+(let (($x136 (v_b_Visited_G_0$ ?v1)))
+(let (($x137 (not $x136)))
+(or $x137 $x922 $x933))))))))
+))
+(let (($x2973 (not (or (not $x2436) (not $x2964)))))
+(let (($x2978 (or $x2414 $x2973)))
+(let (($x2391 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let (($x907 (>= (+ (v_b_SP_G_0$ ?v1) (* (- 1) (v_b_SP_G_0$ ?v0))) 0)))
+(let (($x136 (v_b_Visited_G_0$ ?v1)))
+(or $x136 (not (v_b_Visited_G_0$ ?v0)) $x907))))
+))
+(let (($x2987 (not (or (not $x2391) (not $x2978)))))
+(let (($x2992 (or $x2368 $x2987)))
+(let (($x3000 (not (or $x902 (not $x2992)))))
+(let (($x3005 (or $x1477 $x3000)))
+(let (($x3013 (not (or $x869 (not $x3005)))))
+(let (($x3018 (or $x869 $x3013)))
+(let (($x2837 (or (>= (+ ?x273 (* (- 1) ?x1911)) 0) $x300 (not (= (+ ?x273 (* (- 1) ?x1911) (b_G$ (pair$ ?0 ?v0!20))) 0)))))
+(let ((@x3736 (monotonicity (quant-intro (refl (= $x2837 $x2837)) (= $x2848 $x3729)) (= (not $x2848) $x3734))))
+(let ((@x3724 (quant-intro (refl (= (or $x300 $x922 $x1282) (or $x300 $x922 $x1282))) (= $x2833 $x3720))))
+(let ((@x3739 (monotonicity (monotonicity @x3724 (= (not $x2833) $x3725)) @x3736 (= (or (not $x2833) $x1909 $x1914 (not $x2848)) $x3737))))
+(let ((@x3748 (monotonicity (monotonicity (monotonicity @x3739 (= $x2857 $x3740)) (= $x2862 $x3743)) (= (not $x2862) $x3746))))
+(let ((@x3716 (quant-intro (refl (= (or $x291 (not $x301) $x1262) (or $x291 (not $x301) $x1262))) (= $x2788 $x3712))))
+(let ((@x3751 (monotonicity (monotonicity @x3716 (= (not $x2788) $x3717)) @x3748 (= (or (not $x2788) (not $x2862)) $x3749))))
+(let ((@x3760 (monotonicity (monotonicity (monotonicity @x3751 (= $x2871 $x3752)) (= $x2876 $x3755)) (= (not $x2876) $x3758))))
+(let ((@x3707 (quant-intro (refl (= (>= ?x273 0) (>= ?x273 0))) (= $x1256 $x3703))))
+(let ((@x3763 (monotonicity (monotonicity @x3707 (= $x1259 $x3708)) @x3760 (= (or $x1259 (not $x2876)) $x3761))))
+(let ((@x3772 (monotonicity (monotonicity (monotonicity @x3763 (= $x2884 $x3764)) (= $x2889 $x3767)) (= (not $x2889) $x3770))))
+(let ((@x3778 (monotonicity (monotonicity @x3772 (= (or $x773 (not $x2889)) $x3773)) (= $x2897 $x3776))))
+(let ((@x3784 (monotonicity (monotonicity @x3778 (= $x2902 $x3779)) (= (not $x2902) $x3782))))
+(let ((@x3699 (quant-intro (refl (= (or $x300 $x278) (or $x300 $x278))) (= $x652 $x3695))))
+(let ((@x3787 (monotonicity (monotonicity @x3699 (= $x785 $x3700)) @x3784 (= (or $x785 (not $x2902)) $x3785))))
+(let ((@x3796 (monotonicity (monotonicity (monotonicity @x3787 (= $x2910 $x3788)) (= $x2915 $x3791)) (= (not $x2915) $x3794))))
+(let ((@x3693 (monotonicity (quant-intro (refl (= $x1243 $x1243)) (= $x1247 $x3686)) (= $x1250 $x3691))))
+(let ((@x3802 (monotonicity (monotonicity @x3693 @x3796 (= (or $x1250 (not $x2915)) $x3797)) (= $x2923 $x3800))))
+(let ((@x3808 (monotonicity (monotonicity @x3802 (= $x2928 $x3803)) (= (not $x2928) $x3806))))
+(let ((@x3680 (refl (= (or (not (or $x1169 $x1175)) $x278) (or (not (or $x1169 $x1175)) $x278)))))
+(let ((@x3685 (monotonicity (quant-intro @x3680 (= $x2742 $x3678)) (= (not $x2742) $x3683))))
+(let ((@x3674 (quant-intro (refl (= (or $x1169 $x1175 $x1185) (or $x1169 $x1175 $x1185))) (= $x2736 $x3670))))
+(let ((@x3667 (monotonicity (quant-intro (refl (= $x1206 $x1206)) (= $x1209 $x3660)) (= (not $x1209) $x3665))))
+(let ((@x3811 (monotonicity @x3667 (monotonicity @x3674 (= (not $x2736) $x3675)) @x3685 @x3808 (= $x2939 $x3809))))
+(let ((@x3626 (quant-intro (refl (= (or $x1099 $x922 $x1140) (or $x1099 $x922 $x1140))) (= $x2672 $x3622))))
+(let ((@x3632 (monotonicity (monotonicity @x3626 (= (not $x2672) $x3627)) (= (or (not $x2672) $x246) $x3630))))
+(let ((@x3641 (monotonicity (monotonicity (monotonicity @x3632 (= $x2680 $x3633)) (= $x2685 $x3636)) (= (not $x2685) $x3639))))
+(let ((?x2191 (+ ?x230 (* (- 1) (fun_app$c v_b_SP_G_3$ (?v1!9 ?0))) (* (- 1) (b_G$ (pair$ (?v1!9 ?0) ?0))))))
+(let (($x2192 (= ?x2191 0)))
+(let (($x2176 (<= (+ ?x230 (* (- 1) (fun_app$c v_b_SP_G_3$ (?v1!9 ?0)))) 0)))
+(let (($x2617 (not (or $x2176 (not $x2192)))))
+(let (($x2623 (or $x127 $x1099 $x2617)))
+(let ((@x3621 (monotonicity (quant-intro (refl (= $x2623 $x2623)) (= $x2628 $x3614)) (= (not $x2628) $x3619))))
+(let ((@x3647 (monotonicity (monotonicity @x3621 @x3641 (= (or (not $x2628) (not $x2685)) $x3642)) (= $x2694 $x3645))))
+(let ((?x1661 (fun_app$c v_b_SP_G_3$ ?v0!8)))
+(let ((?x1662 (* (- 1) ?x1661)))
+(let (($x2148 (= (+ ?x230 ?x1662 (b_G$ (pair$ ?0 ?v0!8))) 0)))
+(let (($x2580 (or (>= (+ ?x230 ?x1662) 0) (not $x2148))))
+(let ((@x3607 (monotonicity (quant-intro (refl (= $x2580 $x2580)) (= $x2591 $x3600)) (= (not $x2591) $x3605))))
+(let ((@x3613 (monotonicity (monotonicity @x3607 (= (or $x1659 $x1664 (not $x2591)) $x3608)) (= $x2599 $x3611))))
+(let ((@x3653 (monotonicity (monotonicity @x3613 @x3647 (= $x2699 $x3648)) (= (not $x2699) $x3651))))
+(let ((@x3594 (quant-intro (refl (= (or $x178 $x1002) (or $x178 $x1002))) (= $x2576 $x3590))))
+(let ((@x3656 (monotonicity (monotonicity @x3594 (= (not $x2576) $x3595)) @x3653 (= (or (not $x2576) $x2706 $x2707 $x2708 $x2709 (not $x2699)) $x3654))))
+(let ((@x3817 (monotonicity (monotonicity @x3656 (= $x2712 $x3657)) (monotonicity @x3811 (= $x2940 $x3812)) (= $x2945 $x3815))))
+(let ((?x2128 (+ ?x174 (* (- 1) (fun_app$c v_b_SP_G_1$ (?v1!7 ?0))) (* (- 1) (b_G$ (pair$ (?v1!7 ?0) ?0))))))
+(let (($x2129 (= ?x2128 0)))
+(let (($x2113 (<= (+ ?x174 (* (- 1) (fun_app$c v_b_SP_G_1$ (?v1!7 ?0)))) 0)))
+(let (($x2551 (not (or $x2113 (not (fun_app$ v_b_Visited_G_1$ (?v1!7 ?0))) (not $x2129)))))
+(let (($x2557 (or $x127 $x1002 $x2551)))
+(let ((@x3588 (monotonicity (quant-intro (refl (= $x2557 $x2557)) (= $x2562 $x3581)) (= (not $x2562) $x3586))))
+(let ((@x3577 (quant-intro (refl (= (or $x179 $x922 $x990) (or $x179 $x922 $x990))) (= $x2534 $x3573))))
+(let ((@x3569 (quant-intro (refl (= (or $x178 (not $x180) $x1015) (or $x178 (not $x180) $x1015))) (= $x2512 $x3565))))
+(let ((@x3560 (quant-intro (refl (= (>= ?x174 0) (>= ?x174 0))) (= $x1051 $x3556))))
+(let ((?x2090 (+ ?x128 (* (- 1) (v_b_SP_G_0$ (?v1!6 ?0))) (* (- 1) (b_G$ (pair$ (?v1!6 ?0) ?0))))))
+(let (($x2091 (= ?x2090 0)))
+(let (($x2075 (<= (+ ?x128 (* (- 1) (v_b_SP_G_0$ (?v1!6 ?0)))) 0)))
+(let (($x2478 (not (or $x2075 (not (v_b_Visited_G_0$ (?v1!6 ?0))) (not $x2091)))))
+(let (($x947 (<= (+ b_Infinity$ (* (- 1) ?x128)) 0)))
+(let (($x2484 (or $x127 $x947 $x2478)))
+(let ((@x3554 (monotonicity (quant-intro (refl (= $x2484 $x2484)) (= $x2489 $x3547)) (= (not $x2489) $x3552))))
+(let ((@x3823 (monotonicity @x3554 (monotonicity @x3560 (= (not $x1051) $x3561)) (monotonicity @x3569 (= (not $x2512) $x3570)) (monotonicity @x3577 (= (not $x2534) $x3578)) @x3588 (monotonicity @x3817 (= (not $x2945) $x3818)) (= $x2958 $x3821))))
+(let (($x2440 (or (>= (+ ?x128 ?x1541) 0) $x137 (not (= (+ ?x128 ?x1541 (b_G$ (pair$ ?0 ?v0!5))) 0)))))
+(let ((@x3540 (monotonicity (quant-intro (refl (= $x2440 $x2440)) (= $x2451 $x3533)) (= (not $x2451) $x3538))))
+(let ((@x3546 (monotonicity (monotonicity @x3540 (= (or $x1538 $x1543 (not $x2451)) $x3541)) (= $x2459 $x3544))))
+(let ((@x3829 (monotonicity @x3546 (monotonicity @x3823 (= $x2959 $x3824)) (= $x2964 $x3827))))
+(let ((@x3528 (quant-intro (refl (= (or $x137 $x922 $x933) (or $x137 $x922 $x933))) (= $x2436 $x3524))))
+(let ((@x3835 (monotonicity (monotonicity @x3528 (= (not $x2436) $x3529)) (monotonicity @x3829 (= (not $x2964) $x3830)) (= (or (not $x2436) (not $x2964)) $x3833))))
+(let ((@x3844 (monotonicity (monotonicity (monotonicity @x3835 (= $x2973 $x3836)) (= $x2978 $x3839)) (= (not $x2978) $x3842))))
+(let ((@x3519 (quant-intro (refl (= (or $x136 (not $x148) $x907) (or $x136 (not $x148) $x907))) (= $x2391 $x3515))))
+(let ((@x3847 (monotonicity (monotonicity @x3519 (= (not $x2391) $x3520)) @x3844 (= (or (not $x2391) (not $x2978)) $x3845))))
+(let ((@x3856 (monotonicity (monotonicity (monotonicity @x3847 (= $x2987 $x3848)) (= $x2992 $x3851)) (= (not $x2992) $x3854))))
+(let ((@x3510 (quant-intro (refl (= (>= ?x128 0) (>= ?x128 0))) (= $x899 $x3506))))
+(let ((@x3859 (monotonicity (monotonicity @x3510 (= $x902 $x3511)) @x3856 (= (or $x902 (not $x2992)) $x3857))))
+(let ((@x3868 (monotonicity (monotonicity (monotonicity @x3859 (= $x3000 $x3860)) (= $x3005 $x3863)) (= (not $x3005) $x3866))))
+(let ((@x3874 (monotonicity (monotonicity @x3868 (= (or $x869 (not $x3005)) $x3869)) (= $x3013 $x3872))))
+(let (($x2251 (forall ((?v1 B_Vertex$) )(let ((?x1911 (v_b_SP_G_2$ ?v0!20)))
+(let ((?x1912 (* (- 1) ?x1911)))
+(let ((?x273 (v_b_SP_G_2$ ?v1)))
+(let (($x2242 (= (+ ?x273 ?x1912 (b_G$ (pair$ ?v1 ?v0!20))) 0)))
+(let (($x291 (fun_app$ v_b_Visited_G_2$ ?v1)))
+(let (($x2245 (and (not (>= (+ ?x273 ?x1912) 0)) $x291 $x2242)))
+(not $x2245))))))))
+))
+(let (($x1915 (not $x1914)))
+(let (($x1910 (not $x1909)))
+(let (($x2260 (and $x1289 $x1910 $x1915 $x2251)))
+(let (($x1891 (not (and $x1883 (not $x1888)))))
+(let (($x1897 (or $x1891 $x1896)))
+(let (($x1898 (not $x1897)))
+(let (($x2265 (or $x1898 $x2260)))
+(let (($x2268 (and $x1270 $x2265)))
+(let (($x1864 (not (and (not $x1860) $x1862))))
+(let (($x1870 (or $x1864 $x1869)))
+(let (($x1871 (not $x1870)))
+(let (($x2271 (or $x1871 $x2268)))
+(let (($x2274 (and $x1256 $x2271)))
+(let (($x2277 (or $x1848 $x2274)))
+(let (($x2280 (and $x297 $x2277)))
+(let (($x2283 (or $x773 $x2280)))
+(let (($x2286 (and $x652 $x2283)))
+(let (($x2289 (or $x1830 $x2286)))
+(let (($x2292 (and $x1247 $x2289)))
+(let (($x2295 (or $x1813 $x2292)))
+(let (($x1779 (not $x1778)))
+(let (($x1774 (not $x1773)))
+(let (($x2301 (and $x1774 $x1779 $x256 $x1214 $x1209 $x266 $x1193 $x1199 $x2295)))
+(let (($x1749 (not $x246)))
+(let (($x1752 (and $x1146 $x1749)))
+(let (($x1733 (not (and (not $x1724) (not $x1730)))))
+(let (($x2212 (or $x1733 $x2209)))
+(let (($x2215 (not $x2212)))
+(let (($x2218 (or $x2215 $x1752)))
+(let (($x2203 (forall ((?v0 B_Vertex$) )(let ((?x230 (fun_app$c v_b_SP_G_3$ ?v0)))
+(let ((?x2191 (+ ?x230 (* (- 1) (fun_app$c v_b_SP_G_3$ (?v1!9 ?v0))) (* (- 1) (b_G$ (pair$ (?v1!9 ?v0) ?v0))))))
+(let (($x2192 (= ?x2191 0)))
+(let (($x2176 (<= (+ ?x230 (* (- 1) (fun_app$c v_b_SP_G_3$ (?v1!9 ?v0)))) 0)))
+(let (($x2197 (and (not $x2176) $x2192)))
+(let (($x1099 (<= (+ b_Infinity$ (* (- 1) ?x230)) 0)))
+(let (($x1100 (not $x1099)))
+(let (($x127 (= ?v0 b_Source$)))
+(let (($x132 (not $x127)))
+(let (($x1103 (and $x132 $x1100)))
+(let (($x1106 (not $x1103)))
+(or $x1106 $x2197)))))))))))))
+))
+(let (($x2221 (and $x2203 $x2218)))
+(let (($x2157 (forall ((?v1 B_Vertex$) )(let ((?x1661 (fun_app$c v_b_SP_G_3$ ?v0!8)))
+(let ((?x1662 (* (- 1) ?x1661)))
+(let ((?x230 (fun_app$c v_b_SP_G_3$ ?v1)))
+(let (($x2148 (= (+ ?x230 ?x1662 (b_G$ (pair$ ?v1 ?v0!8))) 0)))
+(let (($x2151 (and (not (>= (+ ?x230 ?x1662) 0)) $x2148)))
+(not $x2151)))))))
+))
+(let (($x1665 (not $x1664)))
+(let (($x1660 (not $x1659)))
+(let (($x2163 (and $x1660 $x1665 $x2157)))
+(let (($x2224 (or $x2163 $x2221)))
+(let (($x1641 (forall ((?v0 B_Vertex$) )(let (($x1002 (<= (+ b_Infinity$ (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0))) 0)))
+(let (($x1003 (not $x1002)))
+(let (($x178 (fun_app$ v_b_Visited_G_1$ ?v0)))
+(let (($x179 (not $x178)))
+(let (($x1077 (and $x179 $x1003)))
+(not $x1077)))))))
+))
+(let (($x2230 (and $x1641 $x212 $x215 $x217 $x220 $x2224)))
+(let (($x2306 (or $x2230 $x2301)))
+(let (($x2140 (forall ((?v0 B_Vertex$) )(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v0)))
+(let ((?x2128 (+ ?x174 (* (- 1) (fun_app$c v_b_SP_G_1$ (?v1!7 ?v0))) (* (- 1) (b_G$ (pair$ (?v1!7 ?v0) ?v0))))))
+(let (($x2129 (= ?x2128 0)))
+(let ((?x1613 (?v1!7 ?v0)))
+(let (($x1618 (fun_app$ v_b_Visited_G_1$ ?x1613)))
+(let (($x2134 (and (not (<= (+ ?x174 (* (- 1) (fun_app$c v_b_SP_G_1$ ?x1613))) 0)) $x1618 $x2129)))
+(let (($x1002 (<= (+ b_Infinity$ (* (- 1) ?x174)) 0)))
+(let (($x1003 (not $x1002)))
+(let (($x127 (= ?v0 b_Source$)))
+(let (($x132 (not $x127)))
+(let (($x1006 (and $x132 $x1003)))
+(let (($x1009 (not $x1006)))
+(or $x1009 $x2134))))))))))))))
+))
+(let (($x2102 (forall ((?v0 B_Vertex$) )(let ((?x128 (v_b_SP_G_0$ ?v0)))
+(let ((?x2090 (+ ?x128 (* (- 1) (v_b_SP_G_0$ (?v1!6 ?v0))) (* (- 1) (b_G$ (pair$ (?v1!6 ?v0) ?v0))))))
+(let (($x2091 (= ?x2090 0)))
+(let ((?x1578 (?v1!6 ?v0)))
+(let (($x1583 (v_b_Visited_G_0$ ?x1578)))
+(let (($x2096 (and (not (<= (+ ?x128 (* (- 1) (v_b_SP_G_0$ ?x1578))) 0)) $x1583 $x2091)))
+(let (($x127 (= ?v0 b_Source$)))
+(let (($x132 (not $x127)))
+(let (($x951 (and $x132 (not (<= (+ b_Infinity$ (* (- 1) ?x128)) 0)))))
+(let (($x954 (not $x951)))
+(or $x954 $x2096))))))))))))
+))
+(let (($x2315 (and $x2102 $x173 $x1051 $x1045 $x997 $x2140 $x2306)))
+(let (($x1567 (forall ((?v1 B_Vertex$) )(let ((?x1540 (v_b_SP_G_0$ ?v0!5)))
+(let ((?x1541 (* (- 1) ?x1540)))
+(let ((?x128 (v_b_SP_G_0$ ?v1)))
+(let (($x136 (v_b_Visited_G_0$ ?v1)))
+(let (($x1554 (and (not (>= (+ ?x128 ?x1541) 0)) $x136 (= (+ ?x128 ?x1541 (b_G$ (pair$ ?v1 ?v0!5))) 0))))
+(not $x1554)))))))
+))
+(let (($x2062 (and $x1539 $x1544 $x1567)))
+(let (($x2320 (or $x2062 $x2315)))
+(let (($x2323 (and $x939 $x2320)))
+(let (($x1520 (not (and $x1512 (not $x1517)))))
+(let (($x2051 (or $x1520 $x2048)))
+(let (($x2054 (not $x2051)))
+(let (($x2326 (or $x2054 $x2323)))
+(let (($x2329 (and $x914 $x2326)))
+(let (($x1493 (not (and (not $x1489) $x1491))))
+(let (($x1499 (or $x1493 $x1498)))
+(let (($x1500 (not $x1499)))
+(let (($x2332 (or $x1500 $x2329)))
+(let (($x2335 (and $x899 $x2332)))
+(let (($x2338 (or $x1477 $x2335)))
+(let (($x2341 (and $x145 $x2338)))
+(let (($x2344 (or $x869 $x2341)))
+(let ((@x2942 (rewrite (= (and $x1774 $x1779 $x256 $x1214 $x1209 $x266 $x2736 $x2742 $x2928) $x2940))))
+(let (($x2242 (= (+ ?x273 (* (- 1) ?x1911) (b_G$ (pair$ ?0 ?v0!20))) 0)))
+(let (($x2245 (and (not (>= (+ ?x273 (* (- 1) ?x1911)) 0)) $x291 $x2242)))
+(let (($x2248 (not $x2245)))
+(let ((@x2843 (monotonicity (rewrite (= $x2245 (not $x2837))) (= $x2248 (not (not $x2837))))))
+(let ((@x2850 (quant-intro (trans @x2843 (rewrite (= (not (not $x2837)) $x2837)) (= $x2248 $x2837)) (= $x2251 $x2848))))
+(let ((@x2820 (monotonicity (rewrite (= $x1276 (not (or $x300 $x922)))) (= $x1279 (not (not (or $x300 $x922)))))))
+(let ((@x2824 (trans @x2820 (rewrite (= (not (not (or $x300 $x922))) (or $x300 $x922))) (= $x1279 (or $x300 $x922)))))
+(let ((@x2832 (trans (monotonicity @x2824 (= $x1286 (or (or $x300 $x922) $x1282))) (rewrite (= (or (or $x300 $x922) $x1282) (or $x300 $x922 $x1282))) (= $x1286 (or $x300 $x922 $x1282)))))
+(let ((@x2853 (monotonicity (quant-intro @x2832 (= $x1289 $x2833)) @x2850 (= $x2260 (and $x2833 $x1910 $x1915 $x2848)))))
+(let ((@x2861 (trans @x2853 (rewrite (= (and $x2833 $x1910 $x1915 $x2848) $x2857)) (= $x2260 $x2857))))
+(let ((@x2798 (monotonicity (rewrite (= (and $x1883 (not $x1888)) (not (or $x2791 $x1888)))) (= $x1891 (not (not (or $x2791 $x1888)))))))
+(let ((@x2802 (trans @x2798 (rewrite (= (not (not (or $x2791 $x1888))) (or $x2791 $x1888))) (= $x1891 (or $x2791 $x1888)))))
+(let ((@x2810 (trans (monotonicity @x2802 (= $x1897 (or (or $x2791 $x1888) $x1896))) (rewrite (= (or (or $x2791 $x1888) $x1896) $x2806)) (= $x1897 $x2806))))
+(let ((@x2864 (monotonicity (monotonicity @x2810 (= $x1898 $x2811)) @x2861 (= $x2265 $x2862))))
+(let ((@x2785 (rewrite (= (or (or $x291 (not $x301)) $x1262) (or $x291 (not $x301) $x1262)))))
+(let ((@x2777 (rewrite (= (not (not (or $x291 (not $x301)))) (or $x291 (not $x301))))))
+(let ((@x2775 (monotonicity (rewrite (= $x302 (not (or $x291 (not $x301))))) (= $x664 (not (not (or $x291 (not $x301))))))))
+(let ((@x2782 (monotonicity (trans @x2775 @x2777 (= $x664 (or $x291 (not $x301)))) (= $x1267 (or (or $x291 (not $x301)) $x1262)))))
+(let ((@x2790 (quant-intro (trans @x2782 @x2785 (= $x1267 (or $x291 (not $x301) $x1262))) (= $x1270 $x2788))))
+(let ((@x2875 (trans (monotonicity @x2790 @x2864 (= $x2268 (and $x2788 $x2862))) (rewrite (= (and $x2788 $x2862) $x2871)) (= $x2268 $x2871))))
+(let ((@x2752 (monotonicity (rewrite (= (and (not $x1860) $x1862) (not (or $x1860 $x2745)))) (= $x1864 (not (not (or $x1860 $x2745)))))))
+(let ((@x2756 (trans @x2752 (rewrite (= (not (not (or $x1860 $x2745))) (or $x1860 $x2745))) (= $x1864 (or $x1860 $x2745)))))
+(let ((@x2764 (trans (monotonicity @x2756 (= $x1870 (or (or $x1860 $x2745) $x1869))) (rewrite (= (or (or $x1860 $x2745) $x1869) $x2760)) (= $x1870 $x2760))))
+(let ((@x2878 (monotonicity (monotonicity @x2764 (= $x1871 $x2765)) @x2875 (= $x2271 $x2876))))
+(let ((@x2888 (trans (monotonicity @x2878 (= $x2274 (and $x1256 $x2876))) (rewrite (= (and $x1256 $x2876) $x2884)) (= $x2274 $x2884))))
+(let ((@x2894 (monotonicity (monotonicity @x2888 (= $x2277 $x2889)) (= $x2280 (and $x297 $x2889)))))
+(let ((@x2904 (monotonicity (trans @x2894 (rewrite (= (and $x297 $x2889) $x2897)) (= $x2280 $x2897)) (= $x2283 $x2902))))
+(let ((@x2914 (trans (monotonicity @x2904 (= $x2286 (and $x652 $x2902))) (rewrite (= (and $x652 $x2902) $x2910)) (= $x2286 $x2910))))
+(let ((@x2920 (monotonicity (monotonicity @x2914 (= $x2289 $x2915)) (= $x2292 (and $x1247 $x2915)))))
+(let ((@x2930 (monotonicity (trans @x2920 (rewrite (= (and $x1247 $x2915) $x2923)) (= $x2292 $x2923)) (= $x2295 $x2928))))
+(let ((@x2741 (monotonicity (rewrite (= $x1179 (not (or $x1169 $x1175)))) (= $x1196 (or (not (or $x1169 $x1175)) $x278)))))
+(let ((@x2723 (monotonicity (rewrite (= $x1179 (not (or $x1169 $x1175)))) (= $x1182 (not (not (or $x1169 $x1175)))))))
+(let ((@x2727 (trans @x2723 (rewrite (= (not (not (or $x1169 $x1175))) (or $x1169 $x1175))) (= $x1182 (or $x1169 $x1175)))))
+(let ((@x2735 (trans (monotonicity @x2727 (= $x1190 (or (or $x1169 $x1175) $x1185))) (rewrite (= (or (or $x1169 $x1175) $x1185) (or $x1169 $x1175 $x1185))) (= $x1190 (or $x1169 $x1175 $x1185)))))
+(let ((@x2933 (monotonicity (quant-intro @x2735 (= $x1193 $x2736)) (quant-intro @x2741 (= $x1199 $x2742)) @x2930 (= $x2301 (and $x1774 $x1779 $x256 $x1214 $x1209 $x266 $x2736 $x2742 $x2928)))))
+(let ((@x2659 (monotonicity (rewrite (= $x1134 (not (or $x1099 $x922)))) (= $x1137 (not (not (or $x1099 $x922)))))))
+(let ((@x2663 (trans @x2659 (rewrite (= (not (not (or $x1099 $x922))) (or $x1099 $x922))) (= $x1137 (or $x1099 $x922)))))
+(let ((@x2671 (trans (monotonicity @x2663 (= $x1143 (or (or $x1099 $x922) $x1140))) (rewrite (= (or (or $x1099 $x922) $x1140) (or $x1099 $x922 $x1140))) (= $x1143 (or $x1099 $x922 $x1140)))))
+(let ((@x2677 (monotonicity (quant-intro @x2671 (= $x1146 $x2672)) (= $x1752 (and $x2672 $x1749)))))
+(let ((@x2637 (monotonicity (rewrite (= (and (not $x1724) (not $x1730)) (not (or $x1724 $x1730)))) (= $x1733 (not (not (or $x1724 $x1730)))))))
+(let ((@x2641 (trans @x2637 (rewrite (= (not (not (or $x1724 $x1730))) (or $x1724 $x1730))) (= $x1733 (or $x1724 $x1730)))))
+(let ((@x2649 (trans (monotonicity @x2641 (= $x2212 (or (or $x1724 $x1730) $x2209))) (rewrite (= (or (or $x1724 $x1730) $x2209) $x2645)) (= $x2212 $x2645))))
+(let ((@x2687 (monotonicity (monotonicity @x2649 (= $x2215 $x2650)) (trans @x2677 (rewrite (= (and $x2672 $x1749) $x2680)) (= $x1752 $x2680)) (= $x2218 $x2685))))
+(let ((@x2610 (monotonicity (rewrite (= $x1103 (not (or $x127 $x1099)))) (= $x1106 (not (not (or $x127 $x1099)))))))
+(let ((@x2614 (trans @x2610 (rewrite (= (not (not (or $x127 $x1099))) (or $x127 $x1099))) (= $x1106 (or $x127 $x1099)))))
+(let ((@x2622 (monotonicity @x2614 (rewrite (= (and (not $x2176) $x2192) $x2617)) (= (or $x1106 (and (not $x2176) $x2192)) (or (or $x127 $x1099) $x2617)))))
+(let ((@x2627 (trans @x2622 (rewrite (= (or (or $x127 $x1099) $x2617) $x2623)) (= (or $x1106 (and (not $x2176) $x2192)) $x2623))))
+(let ((@x2690 (monotonicity (quant-intro @x2627 (= $x2203 $x2628)) @x2687 (= $x2221 (and $x2628 $x2685)))))
+(let (($x2151 (and (not (>= (+ ?x230 ?x1662) 0)) $x2148)))
+(let (($x2154 (not $x2151)))
+(let ((@x2586 (monotonicity (rewrite (= $x2151 (not $x2580))) (= $x2154 (not (not $x2580))))))
+(let ((@x2593 (quant-intro (trans @x2586 (rewrite (= (not (not $x2580)) $x2580)) (= $x2154 $x2580)) (= $x2157 $x2591))))
+(let ((@x2603 (trans (monotonicity @x2593 (= $x2163 (and $x1660 $x1665 $x2591))) (rewrite (= (and $x1660 $x1665 $x2591) $x2599)) (= $x2163 $x2599))))
+(let ((@x2701 (monotonicity @x2603 (trans @x2690 (rewrite (= (and $x2628 $x2685) $x2694)) (= $x2221 $x2694)) (= $x2224 $x2699))))
+(let ((@x2571 (monotonicity (rewrite (= $x1077 (not (or $x178 $x1002)))) (= (not $x1077) (not (not (or $x178 $x1002)))))))
+(let ((@x2575 (trans @x2571 (rewrite (= (not (not (or $x178 $x1002))) (or $x178 $x1002))) (= (not $x1077) (or $x178 $x1002)))))
+(let ((@x2704 (monotonicity (quant-intro @x2575 (= $x1641 $x2576)) @x2701 (= $x2230 (and $x2576 $x212 $x215 $x217 $x220 $x2699)))))
+(let ((@x2716 (trans @x2704 (rewrite (= (and $x2576 $x212 $x215 $x217 $x220 $x2699) $x2712)) (= $x2230 $x2712))))
+(let ((?x1613 (?v1!7 ?0)))
+(let (($x1618 (fun_app$ v_b_Visited_G_1$ ?x1613)))
+(let (($x2134 (and (not $x2113) $x1618 $x2129)))
+(let (($x2137 (or $x1009 $x2134)))
+(let ((@x2543 (monotonicity (rewrite (= $x1006 (not (or $x127 $x1002)))) (= $x1009 (not (not (or $x127 $x1002)))))))
+(let ((@x2547 (trans @x2543 (rewrite (= (not (not (or $x127 $x1002))) (or $x127 $x1002))) (= $x1009 (or $x127 $x1002)))))
+(let ((@x2556 (monotonicity @x2547 (rewrite (= $x2134 $x2551)) (= $x2137 (or (or $x127 $x1002) $x2551)))))
+(let ((@x2561 (trans @x2556 (rewrite (= (or (or $x127 $x1002) $x2551) $x2557)) (= $x2137 $x2557))))
+(let ((@x2521 (monotonicity (rewrite (= $x983 (not (or $x179 $x922)))) (= $x986 (not (not (or $x179 $x922)))))))
+(let ((@x2525 (trans @x2521 (rewrite (= (not (not (or $x179 $x922))) (or $x179 $x922))) (= $x986 (or $x179 $x922)))))
+(let ((@x2533 (trans (monotonicity @x2525 (= $x994 (or (or $x179 $x922) $x990))) (rewrite (= (or (or $x179 $x922) $x990) (or $x179 $x922 $x990))) (= $x994 (or $x179 $x922 $x990)))))
+(let ((@x2509 (rewrite (= (or (or $x178 (not $x180)) $x1015) (or $x178 (not $x180) $x1015)))))
+(let ((@x2501 (rewrite (= (not (not (or $x178 (not $x180)))) (or $x178 (not $x180))))))
+(let ((@x2499 (monotonicity (rewrite (= $x181 (not (or $x178 (not $x180))))) (= $x403 (not (not (or $x178 (not $x180))))))))
+(let ((@x2506 (monotonicity (trans @x2499 @x2501 (= $x403 (or $x178 (not $x180)))) (= $x1042 (or (or $x178 (not $x180)) $x1015)))))
+(let ((@x2514 (quant-intro (trans @x2506 @x2509 (= $x1042 (or $x178 (not $x180) $x1015))) (= $x1045 $x2512))))
+(let ((?x1578 (?v1!6 ?0)))
+(let (($x1583 (v_b_Visited_G_0$ ?x1578)))
+(let (($x2096 (and (not $x2075) $x1583 $x2091)))
+(let (($x2099 (or $x954 $x2096)))
+(let ((@x2470 (monotonicity (rewrite (= $x951 (not (or $x127 $x947)))) (= $x954 (not (not (or $x127 $x947)))))))
+(let ((@x2474 (trans @x2470 (rewrite (= (not (not (or $x127 $x947))) (or $x127 $x947))) (= $x954 (or $x127 $x947)))))
+(let ((@x2483 (monotonicity @x2474 (rewrite (= $x2096 $x2478)) (= $x2099 (or (or $x127 $x947) $x2478)))))
+(let ((@x2488 (trans @x2483 (rewrite (= (or (or $x127 $x947) $x2478) $x2484)) (= $x2099 $x2484))))
+(let ((@x2950 (monotonicity (quant-intro @x2488 (= $x2102 $x2489)) @x2514 (quant-intro @x2533 (= $x997 $x2534)) (quant-intro @x2561 (= $x2140 $x2562)) (monotonicity @x2716 (trans @x2933 @x2942 (= $x2301 $x2940)) (= $x2306 $x2945)) (= $x2315 (and $x2489 $x173 $x1051 $x2512 $x2534 $x2562 $x2945)))))
+(let ((@x2963 (trans @x2950 (rewrite (= (and $x2489 $x173 $x1051 $x2512 $x2534 $x2562 $x2945) $x2959)) (= $x2315 $x2959))))
+(let (($x1554 (and (not (>= (+ ?x128 ?x1541) 0)) $x136 (= (+ ?x128 ?x1541 (b_G$ (pair$ ?0 ?v0!5))) 0))))
+(let (($x1564 (not $x1554)))
+(let ((@x2446 (monotonicity (rewrite (= $x1554 (not $x2440))) (= $x1564 (not (not $x2440))))))
+(let ((@x2453 (quant-intro (trans @x2446 (rewrite (= (not (not $x2440)) $x2440)) (= $x1564 $x2440)) (= $x1567 $x2451))))
+(let ((@x2463 (trans (monotonicity @x2453 (= $x2062 (and $x1539 $x1544 $x2451))) (rewrite (= (and $x1539 $x1544 $x2451) $x2459)) (= $x2062 $x2459))))
+(let ((@x2423 (monotonicity (rewrite (= $x926 (not (or $x137 $x922)))) (= $x929 (not (not (or $x137 $x922)))))))
+(let ((@x2427 (trans @x2423 (rewrite (= (not (not (or $x137 $x922))) (or $x137 $x922))) (= $x929 (or $x137 $x922)))))
+(let ((@x2435 (trans (monotonicity @x2427 (= $x936 (or (or $x137 $x922) $x933))) (rewrite (= (or (or $x137 $x922) $x933) (or $x137 $x922 $x933))) (= $x936 (or $x137 $x922 $x933)))))
+(let ((@x2969 (monotonicity (quant-intro @x2435 (= $x939 $x2436)) (monotonicity @x2463 @x2963 (= $x2320 $x2964)) (= $x2323 (and $x2436 $x2964)))))
+(let ((@x2401 (monotonicity (rewrite (= (and $x1512 (not $x1517)) (not (or $x2394 $x1517)))) (= $x1520 (not (not (or $x2394 $x1517)))))))
+(let ((@x2405 (trans @x2401 (rewrite (= (not (not (or $x2394 $x1517))) (or $x2394 $x1517))) (= $x1520 (or $x2394 $x1517)))))
+(let ((@x2413 (trans (monotonicity @x2405 (= $x2051 (or (or $x2394 $x1517) $x2048))) (rewrite (= (or (or $x2394 $x1517) $x2048) $x2409)) (= $x2051 $x2409))))
+(let ((@x2980 (monotonicity (monotonicity @x2413 (= $x2054 $x2414)) (trans @x2969 (rewrite (= (and $x2436 $x2964) $x2973)) (= $x2323 $x2973)) (= $x2326 $x2978))))
+(let ((@x2388 (rewrite (= (or (or $x136 (not $x148)) $x907) (or $x136 (not $x148) $x907)))))
+(let ((@x2380 (rewrite (= (not (not (or $x136 (not $x148)))) (or $x136 (not $x148))))))
+(let ((@x2378 (monotonicity (rewrite (= $x149 (not (or $x136 (not $x148))))) (= $x382 (not (not (or $x136 (not $x148))))))))
+(let ((@x2385 (monotonicity (trans @x2378 @x2380 (= $x382 (or $x136 (not $x148)))) (= $x911 (or (or $x136 (not $x148)) $x907)))))
+(let ((@x2393 (quant-intro (trans @x2385 @x2388 (= $x911 (or $x136 (not $x148) $x907))) (= $x914 $x2391))))
+(let ((@x2991 (trans (monotonicity @x2393 @x2980 (= $x2329 (and $x2391 $x2978))) (rewrite (= (and $x2391 $x2978) $x2987)) (= $x2329 $x2987))))
+(let ((@x2355 (monotonicity (rewrite (= (and (not $x1489) $x1491) (not (or $x1489 $x2348)))) (= $x1493 (not (not (or $x1489 $x2348)))))))
+(let ((@x2359 (trans @x2355 (rewrite (= (not (not (or $x1489 $x2348))) (or $x1489 $x2348))) (= $x1493 (or $x1489 $x2348)))))
+(let ((@x2367 (trans (monotonicity @x2359 (= $x1499 (or (or $x1489 $x2348) $x1498))) (rewrite (= (or (or $x1489 $x2348) $x1498) $x2363)) (= $x1499 $x2363))))
+(let ((@x2994 (monotonicity (monotonicity @x2367 (= $x1500 $x2368)) @x2991 (= $x2332 $x2992))))
+(let ((@x3004 (trans (monotonicity @x2994 (= $x2335 (and $x899 $x2992))) (rewrite (= (and $x899 $x2992) $x3000)) (= $x2335 $x3000))))
+(let ((@x3010 (monotonicity (monotonicity @x3004 (= $x2338 $x3005)) (= $x2341 (and $x145 $x3005)))))
+(let ((@x3020 (monotonicity (trans @x3010 (rewrite (= (and $x145 $x3005) $x3013)) (= $x2341 $x3013)) (= $x2344 $x3018))))
+(let (($x1938 (forall ((?v1 B_Vertex$) )(let ((?x1911 (v_b_SP_G_2$ ?v0!20)))
+(let ((?x1912 (* (- 1) ?x1911)))
+(let ((?x273 (v_b_SP_G_2$ ?v1)))
+(let (($x291 (fun_app$ v_b_Visited_G_2$ ?v1)))
+(let (($x1925 (and (not (>= (+ ?x273 ?x1912) 0)) $x291 (= (+ (b_G$ (pair$ ?v1 ?v0!20)) ?x273 ?x1912) 0))))
+(not $x1925)))))))
+))
+(let (($x1932 (not (not (and $x1910 $x1915)))))
+(let (($x1942 (and $x1932 $x1938)))
+(let (($x1947 (and $x1289 $x1942)))
+(let (($x1951 (or $x1898 $x1947)))
+(let (($x1955 (and $x1270 $x1951)))
+(let (($x1959 (or $x1871 $x1955)))
+(let (($x1963 (and $x1256 $x1959)))
+(let (($x1967 (or $x1848 $x1963)))
+(let (($x1842 (not $x773)))
+(let (($x1971 (and $x1842 $x1967)))
+(let (($x1975 (or $x773 $x1971)))
+(let (($x1979 (and $x652 $x1975)))
+(let (($x1983 (or $x1830 $x1979)))
+(let (($x1987 (and $x1247 $x1983)))
+(let (($x1991 (or $x1813 $x1987)))
+(let (($x1801 (and (and $x1774 $x1779) $x256 $x1214 $x1209 $x266 $x1193 $x1199)))
+(let (($x1995 (and $x1801 $x1991)))
+(let (($x1739 (not (or $x1733 (>= (+ ?x1727 ?x1721 ?x1735) 0)))))
+(let (($x1756 (or $x1739 $x1752)))
+(let (($x1713 (forall ((?v0 B_Vertex$) )(let ((?x230 (fun_app$c v_b_SP_G_3$ ?v0)))
+(let ((?x1097 (* (- 1) ?x230)))
+(let ((?x1699 (fun_app$c v_b_SP_G_3$ (?v1!9 ?v0))))
+(let ((?x1704 (b_G$ (pair$ (?v1!9 ?v0) ?v0))))
+(let (($x1706 (= (+ ?x1704 ?x1699 ?x1097) 0)))
+(let (($x1707 (and (not (>= (+ ?x1699 ?x1097) 0)) $x1706)))
+(let (($x1099 (<= (+ b_Infinity$ ?x1097) 0)))
+(let (($x1100 (not $x1099)))
+(let (($x127 (= ?v0 b_Source$)))
+(let (($x132 (not $x127)))
+(let (($x1103 (and $x132 $x1100)))
+(let (($x1106 (not $x1103)))
+(or $x1106 $x1707))))))))))))))
+))
+(let (($x1760 (and $x1713 $x1756)))
+(let (($x1687 (forall ((?v1 B_Vertex$) )(let ((?x1661 (fun_app$c v_b_SP_G_3$ ?v0!8)))
+(let ((?x1662 (* (- 1) ?x1661)))
+(let ((?x230 (fun_app$c v_b_SP_G_3$ ?v1)))
+(let (($x1675 (and (not (>= (+ ?x230 ?x1662) 0)) (= (+ (b_G$ (pair$ ?v1 ?v0!8)) ?x230 ?x1662) 0))))
+(not $x1675))))))
+))
+(let (($x1681 (not (not (and $x1660 $x1665)))))
+(let (($x1691 (and $x1681 $x1687)))
+(let (($x1764 (or $x1691 $x1760)))
+(let (($x1652 (and $x1641 $x212 $x215 $x217 $x220)))
+(let (($x1768 (and $x1652 $x1764)))
+(let (($x1999 (or $x1768 $x1995)))
+(let (($x1629 (forall ((?v0 B_Vertex$) )(let ((?x174 (fun_app$c v_b_SP_G_1$ ?v0)))
+(let ((?x1000 (* (- 1) ?x174)))
+(let ((?x1613 (?v1!7 ?v0)))
+(let ((?x1614 (fun_app$c v_b_SP_G_1$ ?x1613)))
+(let ((?x1620 (b_G$ (pair$ ?x1613 ?v0))))
+(let (($x1622 (= (+ ?x1620 ?x1614 ?x1000) 0)))
+(let (($x1618 (fun_app$ v_b_Visited_G_1$ ?x1613)))
+(let (($x1623 (and (not (>= (+ ?x1614 ?x1000) 0)) $x1618 $x1622)))
+(let (($x1002 (<= (+ b_Infinity$ ?x1000) 0)))
+(let (($x1003 (not $x1002)))
+(let (($x127 (= ?v0 b_Source$)))
+(let (($x132 (not $x127)))
+(let (($x1006 (and $x132 $x1003)))
+(let (($x1009 (not $x1006)))
+(or $x1009 $x1623))))))))))))))))
+))
+(let (($x1594 (forall ((?v0 B_Vertex$) )(let ((?x1585 (b_G$ (pair$ (?v1!6 ?v0) ?v0))))
+(let ((?x128 (v_b_SP_G_0$ ?v0)))
+(let ((?x945 (* (- 1) ?x128)))
+(let ((?x1578 (?v1!6 ?v0)))
+(let ((?x1579 (v_b_SP_G_0$ ?x1578)))
+(let (($x1587 (= (+ ?x1579 ?x945 ?x1585) 0)))
+(let (($x1583 (v_b_Visited_G_0$ ?x1578)))
+(let (($x1588 (and (not (>= (+ ?x1579 ?x945) 0)) $x1583 $x1587)))
+(let (($x127 (= ?v0 b_Source$)))
+(let (($x132 (not $x127)))
+(let (($x951 (and $x132 (not (<= (+ b_Infinity$ ?x945) 0)))))
+(let (($x954 (not $x951)))
+(or $x954 $x1588))))))))))))))
+))
+(let (($x1632 (and $x1594 $x173 $x1051 $x1045 $x997 $x1629)))
+(let (($x2003 (and $x1632 $x1999)))
+(let (($x1561 (not (not (and $x1539 $x1544)))))
+(let (($x1571 (and $x1561 $x1567)))
+(let (($x2007 (or $x1571 $x2003)))
+(let (($x2011 (and $x939 $x2007)))
+(let (($x1527 (not (or $x1520 (>= (+ ?x1521 ?x1523 ?x1514) 0)))))
+(let (($x2015 (or $x1527 $x2011)))
+(let (($x2019 (and $x914 $x2015)))
+(let (($x2023 (or $x1500 $x2019)))
+(let (($x2027 (and $x899 $x2023)))
+(let (($x2031 (or $x1477 $x2027)))
+(let (($x1471 (not $x869)))
+(let (($x2035 (and $x1471 $x2031)))
+(let (($x2039 (or $x869 $x2035)))
+(let (($x1925 (and (not (>= (+ ?x273 (* (- 1) ?x1911)) 0)) $x291 (= (+ (b_G$ (pair$ ?0 ?v0!20)) ?x273 (* (- 1) ?x1911)) 0))))
+(let (($x1935 (not $x1925)))
+(let (($x2243 (= (= (+ (b_G$ (pair$ ?0 ?v0!20)) ?x273 (* (- 1) ?x1911)) 0) $x2242)))
+(let (($x2240 (= (+ (b_G$ (pair$ ?0 ?v0!20)) ?x273 (* (- 1) ?x1911)) (+ ?x273 (* (- 1) ?x1911) (b_G$ (pair$ ?0 ?v0!20))))))
+(let ((@x2250 (monotonicity (monotonicity (monotonicity (rewrite $x2240) $x2243) (= $x1925 $x2245)) (= $x1935 $x2248))))
+(let ((@x2256 (monotonicity (rewrite (= $x1932 (and $x1910 $x1915))) (quant-intro @x2250 (= $x1938 $x2251)) (= $x1942 (and (and $x1910 $x1915) $x2251)))))
+(let ((@x2264 (trans (monotonicity @x2256 (= $x1947 (and $x1289 (and (and $x1910 $x1915) $x2251)))) (rewrite (= (and $x1289 (and (and $x1910 $x1915) $x2251)) $x2260)) (= $x1947 $x2260))))
+(let ((@x2273 (monotonicity (monotonicity (monotonicity @x2264 (= $x1951 $x2265)) (= $x1955 $x2268)) (= $x1959 $x2271))))
+(let ((@x2282 (monotonicity (rewrite (= $x1842 $x297)) (monotonicity (monotonicity @x2273 (= $x1963 $x2274)) (= $x1967 $x2277)) (= $x1971 $x2280))))
+(let ((@x2291 (monotonicity (monotonicity (monotonicity @x2282 (= $x1975 $x2283)) (= $x1979 $x2286)) (= $x1983 $x2289))))
+(let ((@x2300 (monotonicity (monotonicity (monotonicity @x2291 (= $x1987 $x2292)) (= $x1991 $x2295)) (= $x1995 (and $x1801 $x2295)))))
+(let ((@x2211 (monotonicity (rewrite (= (+ ?x1727 ?x1721 ?x1735) ?x2206)) (= (>= (+ ?x1727 ?x1721 ?x1735) 0) $x2209))))
+(let ((@x2214 (monotonicity @x2211 (= (or $x1733 (>= (+ ?x1727 ?x1721 ?x1735) 0)) $x2212))))
+(let (($x2197 (and (not $x2176) $x2192)))
+(let (($x2200 (or $x1106 $x2197)))
+(let ((?x1097 (* (- 1) ?x230)))
+(let ((?x1699 (fun_app$c v_b_SP_G_3$ (?v1!9 ?0))))
+(let ((?x1704 (b_G$ (pair$ (?v1!9 ?0) ?0))))
+(let (($x1706 (= (+ ?x1704 ?x1699 ?x1097) 0)))
+(let (($x1707 (and (not (>= (+ ?x1699 ?x1097) 0)) $x1706)))
+(let (($x1710 (or $x1106 $x1707)))
+(let ((@x2189 (monotonicity (rewrite (= (+ ?x1704 ?x1699 ?x1097) (+ ?x1097 ?x1699 ?x1704))) (= $x1706 (= (+ ?x1097 ?x1699 ?x1704) 0)))))
+(let ((@x2196 (trans @x2189 (rewrite (= (= (+ ?x1097 ?x1699 ?x1704) 0) $x2192)) (= $x1706 $x2192))))
+(let ((@x2173 (monotonicity (rewrite (= (+ ?x1699 ?x1097) (+ ?x1097 ?x1699))) (= (>= (+ ?x1699 ?x1097) 0) (>= (+ ?x1097 ?x1699) 0)))))
+(let ((@x2180 (trans @x2173 (rewrite (= (>= (+ ?x1097 ?x1699) 0) $x2176)) (= (>= (+ ?x1699 ?x1097) 0) $x2176))))
+(let ((@x2199 (monotonicity (monotonicity @x2180 (= (not (>= (+ ?x1699 ?x1097) 0)) (not $x2176))) @x2196 (= $x1707 $x2197))))
+(let ((@x2223 (monotonicity (quant-intro (monotonicity @x2199 (= $x1710 $x2200)) (= $x1713 $x2203)) (monotonicity (monotonicity @x2214 (= $x1739 $x2215)) (= $x1756 $x2218)) (= $x1760 $x2221))))
+(let (($x1675 (and (not (>= (+ ?x230 ?x1662) 0)) (= (+ (b_G$ (pair$ ?0 ?v0!8)) ?x230 ?x1662) 0))))
+(let (($x1684 (not $x1675)))
+(let (($x2146 (= (+ (b_G$ (pair$ ?0 ?v0!8)) ?x230 ?x1662) (+ ?x230 ?x1662 (b_G$ (pair$ ?0 ?v0!8))))))
+(let ((@x2150 (monotonicity (rewrite $x2146) (= (= (+ (b_G$ (pair$ ?0 ?v0!8)) ?x230 ?x1662) 0) $x2148))))
+(let ((@x2159 (quant-intro (monotonicity (monotonicity @x2150 (= $x1675 $x2151)) (= $x1684 $x2154)) (= $x1687 $x2157))))
+(let ((@x2162 (monotonicity (rewrite (= $x1681 (and $x1660 $x1665))) @x2159 (= $x1691 (and (and $x1660 $x1665) $x2157)))))
+(let ((@x2167 (trans @x2162 (rewrite (= (and (and $x1660 $x1665) $x2157) $x2163)) (= $x1691 $x2163))))
+(let ((@x2229 (monotonicity (monotonicity @x2167 @x2223 (= $x1764 $x2224)) (= $x1768 (and $x1652 $x2224)))))
+(let ((@x2308 (monotonicity (trans @x2229 (rewrite (= (and $x1652 $x2224) $x2230)) (= $x1768 $x2230)) (trans @x2300 (rewrite (= (and $x1801 $x2295) $x2301)) (= $x1995 $x2301)) (= $x1999 $x2306))))
+(let ((?x1000 (* (- 1) ?x174)))
+(let ((?x1614 (fun_app$c v_b_SP_G_1$ ?x1613)))
+(let ((?x1620 (b_G$ (pair$ ?x1613 ?0))))
+(let (($x1622 (= (+ ?x1620 ?x1614 ?x1000) 0)))
+(let (($x1623 (and (not (>= (+ ?x1614 ?x1000) 0)) $x1618 $x1622)))
+(let (($x1626 (or $x1009 $x1623)))
+(let ((@x2126 (monotonicity (rewrite (= (+ ?x1620 ?x1614 ?x1000) (+ ?x1000 ?x1614 ?x1620))) (= $x1622 (= (+ ?x1000 ?x1614 ?x1620) 0)))))
+(let ((@x2133 (trans @x2126 (rewrite (= (= (+ ?x1000 ?x1614 ?x1620) 0) $x2129)) (= $x1622 $x2129))))
+(let ((@x2110 (monotonicity (rewrite (= (+ ?x1614 ?x1000) (+ ?x1000 ?x1614))) (= (>= (+ ?x1614 ?x1000) 0) (>= (+ ?x1000 ?x1614) 0)))))
+(let ((@x2117 (trans @x2110 (rewrite (= (>= (+ ?x1000 ?x1614) 0) $x2113)) (= (>= (+ ?x1614 ?x1000) 0) $x2113))))
+(let ((@x2136 (monotonicity (monotonicity @x2117 (= (not (>= (+ ?x1614 ?x1000) 0)) (not $x2113))) @x2133 (= $x1623 $x2134))))
+(let (($x1587 (= (+ (v_b_SP_G_0$ ?x1578) (* (- 1) ?x128) (b_G$ (pair$ ?x1578 ?0))) 0)))
+(let (($x1588 (and (not (>= (+ (v_b_SP_G_0$ ?x1578) (* (- 1) ?x128)) 0)) $x1583 $x1587)))
+(let (($x1591 (or $x954 $x1588)))
+(let (($x2086 (= (+ (* (- 1) ?x128) (v_b_SP_G_0$ ?x1578) (b_G$ (pair$ ?x1578 ?0))) 0)))
+(let (($x2084 (= (+ (v_b_SP_G_0$ ?x1578) (* (- 1) ?x128) (b_G$ (pair$ ?x1578 ?0))) (+ (* (- 1) ?x128) (v_b_SP_G_0$ ?x1578) (b_G$ (pair$ ?x1578 ?0))))))
+(let ((@x2095 (trans (monotonicity (rewrite $x2084) (= $x1587 $x2086)) (rewrite (= $x2086 $x2091)) (= $x1587 $x2091))))
+(let (($x2081 (= (not (>= (+ (v_b_SP_G_0$ ?x1578) (* (- 1) ?x128)) 0)) (not $x2075))))
+(let (($x1581 (>= (+ (v_b_SP_G_0$ ?x1578) (* (- 1) ?x128)) 0)))
+(let (($x2068 (= (+ (v_b_SP_G_0$ ?x1578) (* (- 1) ?x128)) (+ (* (- 1) ?x128) (v_b_SP_G_0$ ?x1578)))))
+(let ((@x2072 (monotonicity (rewrite $x2068) (= $x1581 (>= (+ (* (- 1) ?x128) (v_b_SP_G_0$ ?x1578)) 0)))))
+(let ((@x2079 (trans @x2072 (rewrite (= (>= (+ (* (- 1) ?x128) (v_b_SP_G_0$ ?x1578)) 0) $x2075)) (= $x1581 $x2075))))
+(let ((@x2101 (monotonicity (monotonicity (monotonicity @x2079 $x2081) @x2095 (= $x1588 $x2096)) (= $x1591 $x2099))))
+(let ((@x2311 (monotonicity (quant-intro @x2101 (= $x1594 $x2102)) (quant-intro (monotonicity @x2136 (= $x1626 $x2137)) (= $x1629 $x2140)) (= $x1632 (and $x2102 $x173 $x1051 $x1045 $x997 $x2140)))))
+(let ((@x2314 (monotonicity @x2311 @x2308 (= $x2003 (and (and $x2102 $x173 $x1051 $x1045 $x997 $x2140) $x2306)))))
+(let ((@x2319 (trans @x2314 (rewrite (= (and (and $x2102 $x173 $x1051 $x1045 $x997 $x2140) $x2306) $x2315)) (= $x2003 $x2315))))
+(let ((@x2061 (monotonicity (rewrite (= $x1561 (and $x1539 $x1544))) (= $x1571 (and (and $x1539 $x1544) $x1567)))))
+(let ((@x2066 (trans @x2061 (rewrite (= (and (and $x1539 $x1544) $x1567) $x2062)) (= $x1571 $x2062))))
+(let ((@x2325 (monotonicity (monotonicity @x2066 @x2319 (= $x2007 $x2320)) (= $x2011 $x2323))))
+(let ((@x2050 (monotonicity (rewrite (= (+ ?x1521 ?x1523 ?x1514) ?x2045)) (= (>= (+ ?x1521 ?x1523 ?x1514) 0) $x2048))))
+(let ((@x2053 (monotonicity @x2050 (= (or $x1520 (>= (+ ?x1521 ?x1523 ?x1514) 0)) $x2051))))
+(let ((@x2328 (monotonicity (monotonicity @x2053 (= $x1527 $x2054)) @x2325 (= $x2015 $x2326))))
+(let ((@x2337 (monotonicity (monotonicity (monotonicity @x2328 (= $x2019 $x2329)) (= $x2023 $x2332)) (= $x2027 $x2335))))
+(let ((@x2343 (monotonicity (rewrite (= $x1471 $x145)) (monotonicity @x2337 (= $x2031 $x2338)) (= $x2035 $x2341))))
+(let (($x1926 (exists ((?v1 B_Vertex$) )(let ((?x1911 (v_b_SP_G_2$ ?v0!20)))
+(let ((?x1912 (* (- 1) ?x1911)))
+(let ((?x273 (v_b_SP_G_2$ ?v1)))
+(let (($x291 (fun_app$ v_b_Visited_G_2$ ?v1)))
+(and (not (>= (+ ?x273 ?x1912) 0)) $x291 (= (+ (b_G$ (pair$ ?v1 ?v0!20)) ?x273 ?x1912) 0)))))))
+))
+(let ((@x1944 (nnf-neg (refl (~ $x1932 $x1932)) (nnf-neg (refl (~ $x1935 $x1935)) (~ (not $x1926) $x1938)) (~ (not (or (not (and $x1910 $x1915)) $x1926)) $x1942))))
+(let ((@x1946 (trans (sk (~ (not $x1329) (not (or (not (and $x1910 $x1915)) $x1926)))) @x1944 (~ (not $x1329) $x1942))))
+(let ((@x1907 (nnf-neg (nnf-pos (refl (~ $x1286 $x1286)) (~ $x1289 $x1289)) (~ (not $x1292) $x1289))))
+(let ((@x1954 (nnf-neg (sk (~ $x1292 $x1898)) (nnf-neg @x1907 @x1946 (~ (not $x1332) $x1947)) (~ (not $x1335) $x1951))))
+(let ((@x1880 (nnf-neg (nnf-pos (refl (~ $x1267 $x1267)) (~ $x1270 $x1270)) (~ (not $x1273) $x1270))))
+(let ((@x1962 (nnf-neg (sk (~ $x1273 $x1871)) (nnf-neg @x1880 @x1954 (~ (not $x1338) $x1955)) (~ (not $x1341) $x1959))))
+(let ((@x1857 (nnf-neg (nnf-pos (refl (~ (>= ?x273 0) (>= ?x273 0))) (~ $x1256 $x1256)) (~ (not $x1259) $x1256))))
+(let ((@x1970 (nnf-neg (sk (~ $x1259 $x1848)) (nnf-neg @x1857 @x1962 (~ (not $x1344) $x1963)) (~ (not $x1347) $x1967))))
+(let ((@x1978 (nnf-neg (refl (~ $x773 $x773)) (nnf-neg (refl (~ $x1842 $x1842)) @x1970 (~ (not $x1350) $x1971)) (~ (not $x1353) $x1975))))
+(let ((@x1839 (nnf-neg (nnf-pos (refl (~ (or $x300 $x278) (or $x300 $x278))) (~ $x652 $x652)) (~ (not $x785) $x652))))
+(let ((@x1986 (nnf-neg (sk (~ $x785 $x1830)) (nnf-neg @x1839 @x1978 (~ (not $x1356) $x1979)) (~ (not $x1359) $x1983))))
+(let ((@x1822 (nnf-neg (nnf-pos (refl (~ $x1243 $x1243)) (~ $x1247 $x1247)) (~ (not $x1250) $x1247))))
+(let ((@x1994 (nnf-neg (sk (~ $x1250 $x1813)) (nnf-neg @x1822 @x1986 (~ (not $x1362) $x1987)) (~ (not $x1365) $x1991))))
+(let ((@x1803 (monotonicity (sk (~ $x1080 (and $x1774 $x1779))) (refl (~ $x256 $x256)) (refl (~ $x1214 $x1214)) (nnf-pos (refl (~ $x1206 $x1206)) (~ $x1209 $x1209)) (refl (~ $x266 $x266)) (nnf-pos (refl (~ $x1190 $x1190)) (~ $x1193 $x1193)) (nnf-pos (refl (~ $x1196 $x1196)) (~ $x1199 $x1199)) (~ $x1235 $x1801))))
+(let ((@x1998 (nnf-neg (nnf-neg @x1803 (~ (not $x1240) $x1801)) @x1994 (~ (not $x1368) $x1995))))
+(let ((@x1748 (nnf-neg (nnf-pos (refl (~ $x1143 $x1143)) (~ $x1146 $x1146)) (~ (not $x1149) $x1146))))
+(let ((@x1759 (nnf-neg (sk (~ $x1149 $x1739)) (nnf-neg @x1748 (refl (~ $x1749 $x1749)) (~ (not $x1152) $x1752)) (~ (not $x1155) $x1756))))
+(let ((@x1715 (nnf-pos (monotonicity (refl (~ $x1106 $x1106)) (sk (~ $x1122 $x1707)) (~ $x1125 $x1710)) (~ $x1128 $x1713))))
+(let ((@x1763 (nnf-neg (nnf-neg @x1715 (~ (not $x1131) $x1713)) @x1759 (~ (not $x1158) $x1760))))
+(let (($x1676 (exists ((?v1 B_Vertex$) )(let ((?x1661 (fun_app$c v_b_SP_G_3$ ?v0!8)))
+(let ((?x1662 (* (- 1) ?x1661)))
+(let ((?x230 (fun_app$c v_b_SP_G_3$ ?v1)))
+(and (not (>= (+ ?x230 ?x1662) 0)) (= (+ (b_G$ (pair$ ?v1 ?v0!8)) ?x230 ?x1662) 0))))))
+))
+(let ((@x1693 (nnf-neg (refl (~ $x1681 $x1681)) (nnf-neg (refl (~ $x1684 $x1684)) (~ (not $x1676) $x1687)) (~ (not (or (not (and $x1660 $x1665)) $x1676)) $x1691))))
+(let ((@x1695 (trans (sk (~ $x1131 (not (or (not (and $x1660 $x1665)) $x1676)))) @x1693 (~ $x1131 $x1691))))
+(let ((@x1654 (monotonicity (nnf-neg (refl (~ (not $x1077) (not $x1077))) (~ $x1083 $x1641)) (refl (~ $x212 $x212)) (refl (~ $x215 $x215)) (refl (~ $x217 $x217)) (refl (~ $x220 $x220)) (~ $x1089 $x1652))))
+(let ((@x1771 (nnf-neg (nnf-neg @x1654 (~ (not $x1094) $x1652)) (nnf-neg @x1695 @x1763 (~ (not $x1161) $x1764)) (~ (not $x1164) $x1768))))
+(let ((@x1631 (nnf-pos (monotonicity (refl (~ $x1009 $x1009)) (sk (~ $x1031 $x1623)) (~ $x1034 $x1626)) (~ $x1037 $x1629))))
+(let ((@x1596 (nnf-pos (monotonicity (refl (~ $x954 $x954)) (sk (~ $x974 $x1588)) (~ $x977 $x1591)) (~ $x980 $x1594))))
+(let ((@x1634 (monotonicity @x1596 (refl (~ $x173 $x173)) (nnf-pos (refl (~ (>= ?x174 0) (>= ?x174 0))) (~ $x1051 $x1051)) (nnf-pos (refl (~ $x1042 $x1042)) (~ $x1045 $x1045)) (nnf-pos (refl (~ $x994 $x994)) (~ $x997 $x997)) @x1631 (~ $x1069 $x1632))))
+(let ((@x2006 (nnf-neg (nnf-neg @x1634 (~ (not $x1074) $x1632)) (nnf-neg @x1771 @x1998 (~ (not $x1371) $x1999)) (~ (not $x1374) $x2003))))
+(let (($x1555 (exists ((?v1 B_Vertex$) )(let ((?x1540 (v_b_SP_G_0$ ?v0!5)))
+(let ((?x1541 (* (- 1) ?x1540)))
+(let ((?x128 (v_b_SP_G_0$ ?v1)))
+(let (($x136 (v_b_Visited_G_0$ ?v1)))
+(and (not (>= (+ ?x128 ?x1541) 0)) $x136 (= (+ ?x128 ?x1541 (b_G$ (pair$ ?v1 ?v0!5))) 0)))))))
+))
+(let ((@x1573 (nnf-neg (refl (~ $x1561 $x1561)) (nnf-neg (refl (~ $x1564 $x1564)) (~ (not $x1555) $x1567)) (~ (not (or (not (and $x1539 $x1544)) $x1555)) $x1571))))
+(let ((@x1575 (trans (sk (~ (not $x980) (not (or (not (and $x1539 $x1544)) $x1555)))) @x1573 (~ (not $x980) $x1571))))
+(let ((@x1536 (nnf-neg (nnf-pos (refl (~ $x936 $x936)) (~ $x939 $x939)) (~ (not $x942) $x939))))
+(let ((@x2014 (nnf-neg @x1536 (nnf-neg @x1575 @x2006 (~ (not $x1377) $x2007)) (~ (not $x1380) $x2011))))
+(let ((@x1509 (nnf-neg (nnf-pos (refl (~ $x911 $x911)) (~ $x914 $x914)) (~ (not $x917) $x914))))
+(let ((@x2022 (nnf-neg @x1509 (nnf-neg (sk (~ $x942 $x1527)) @x2014 (~ (not $x1383) $x2015)) (~ (not $x1386) $x2019))))
+(let ((@x1486 (nnf-neg (nnf-pos (refl (~ (>= ?x128 0) (>= ?x128 0))) (~ $x899 $x899)) (~ (not $x902) $x899))))
+(let ((@x2030 (nnf-neg @x1486 (nnf-neg (sk (~ $x917 $x1500)) @x2022 (~ (not $x1389) $x2023)) (~ (not $x1392) $x2027))))
+(let ((@x2038 (nnf-neg (refl (~ $x1471 $x1471)) (nnf-neg (sk (~ $x902 $x1477)) @x2030 (~ (not $x1395) $x2031)) (~ (not $x1398) $x2035))))
+(let ((@x2042 (mp~ (not-or-elim (mp (asserted $x349) @x1411 $x1407) (not $x1401)) (nnf-neg (refl (~ $x869 $x869)) @x2038 (~ (not $x1401) $x2039)) $x2039)))
+(let ((@x3878 (mp (mp (mp @x2042 (monotonicity @x2343 (= $x2039 $x2344)) $x2344) @x3020 $x3018) (monotonicity @x3874 (= $x3018 $x3875)) $x3875)))
+(let ((@x4209 (unit-resolution @x3878 (lemma (unit-resolution @x5763 @x3492 (hypothesis $x869) false) $x145) $x3872)))
+(let ((@x4211 (unit-resolution (def-axiom (or $x3866 $x1477 $x3860)) (unit-resolution (def-axiom (or $x3869 $x3863)) @x4209 $x3863) (lemma @x6353 $x1476) $x3860)))
+(let ((@x6165 (unit-resolution ((_ quant-inst ?v0!2) (or (not $x3500) $x2348)) @x3505 (hypothesis $x1491) false)))
+(let ((@x4215 (unit-resolution (def-axiom (or $x3854 $x2368 $x3848)) (unit-resolution (def-axiom (or $x2363 $x1491)) (lemma @x6165 $x2348) $x2363) (unit-resolution (def-axiom (or $x3857 $x3851)) @x4211 $x3851) $x3848)))
+(let ((@x4217 (unit-resolution (def-axiom (or $x3842 $x2414 $x3836)) (unit-resolution (def-axiom (or $x3845 $x3839)) @x4215 $x3839) (unit-resolution (def-axiom (or $x2409 $x1512)) (lemma @x3073 $x2394) $x2409) $x3836)))
+(let ((@x4219 (unit-resolution (def-axiom (or $x3830 $x3544 $x3824)) (unit-resolution (def-axiom (or $x3833 $x3827)) @x4217 $x3827) (lemma @x5735 $x3541) $x3824)))
+(let ((@x5955 (unit-resolution (def-axiom (or $x3821 $x3556)) @x4219 $x3556)))
+(let (($x4373 (or $x3561 $x3904)))
+(let ((@x4363 ((_ quant-inst v_b_v_G_1$) $x4373)))
+(let ((@x5049 (unit-resolution @x4363 @x5955 $x3904)))
+(let ((?x5210 (pair$ v_b_v_G_1$ ?v0!15)))
+(let ((?x5018 (b_G$ ?x5210)))
+(let ((?x4456 (* (- 1) ?x1846)))
+(let ((?x6267 (+ ?x257 ?x4456 ?x5018)))
+(let (($x5853 (<= ?x6267 0)))
+(let (($x6128 (= ?x6267 0)))
+(let (($x6822 (>= (+ ?x257 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0!15)) ?x5018) 0)))
+(let (($x4911 (<= (+ b_Infinity$ (* (- 1) ?x5018)) 0)))
+(let (($x6706 (or $x4911 $x6822)))
+(let (($x6711 (not $x6706)))
+(let ((@x5703 (hypothesis $x1848)))
+(let (($x5745 (or (not (>= (+ ?x1846 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0!15))) 0)) $x1847)))
+(let ((?x4480 (fun_app$c v_b_SP_G_1$ ?v0!15)))
+(let (($x5850 (>= ?x4480 0)))
+(let ((@x5698 ((_ th-lemma arith farkas -1 1 1) @x5703 (hypothesis (>= (+ ?x1846 (* (- 1) ?x4480)) 0)) (unit-resolution ((_ quant-inst ?v0!15) (or $x3561 $x5850)) @x5955 $x5850) false)))
+(let ((@x6183 (unit-resolution (lemma @x5698 $x5745) @x5703 (not (>= (+ ?x1846 (* (- 1) ?x4480)) 0)))))
+(let ((@x6242 ((_ th-lemma arith triangle-eq) (or (not (= ?x1846 ?x4480)) (>= (+ ?x1846 (* (- 1) ?x4480)) 0)))))
+(let ((@x4529 (unit-resolution (def-axiom (or $x3821 $x173)) @x4219 $x173)))
+(let ((@x5142 (hypothesis $x3657)))
+(let ((@x4265 (unit-resolution (def-axiom (or $x3654 $x217)) @x5142 $x217)))
+(let ((?x5667 (fun_app$c v_b_SP_G_1$ ?v1!10)))
+(let ((?x5152 (fun_app$c v_b_SP_G_1$ ?v0!11)))
+(let ((?x5630 (* (- 1) ?x5152)))
+(let (($x4072 (>= (+ ?x1727 ?x5630 ?x5667) 0)))
+(let (($x5699 (fun_app$ v_b_Visited_G_1$ ?v1!10)))
+(let (($x1725 (not $x1724)))
+(let ((@x4170 (hypothesis $x2650)))
+(let (($x4150 (>= (+ ?x1721 (* (- 1) ?x5667)) 0)))
+(let ((@x4195 (monotonicity (symm (hypothesis $x217) (= v_b_SP_G_1$ v_b_SP_G_3$)) (= ?x5667 ?x1721))))
+(let ((@x4203 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x1721 ?x5667)) $x4150)) (symm @x4195 (= ?x1721 ?x5667)) $x4150)))
+(let (($x4167 (or (not (<= (+ b_Infinity$ (* (- 1) ?x5667)) 0)) (not $x4150) $x1724)))
+(let ((@x4163 ((_ th-lemma arith farkas 1 -1 1) (hypothesis $x4150) (hypothesis (<= (+ b_Infinity$ (* (- 1) ?x5667)) 0)) (hypothesis $x1725) false)))
+(let ((@x4204 (unit-resolution (lemma @x4163 $x4167) @x4203 (unit-resolution (def-axiom (or $x2645 $x1725)) @x4170 $x1725) (not (<= (+ b_Infinity$ (* (- 1) ?x5667)) 0)))))
+(let (($x6045 (<= (+ b_Infinity$ (* (- 1) ?x5667)) 0)))
+(let (($x5247 (or $x5699 $x6045)))
+(let ((@x3048 (mp ((_ quant-inst ?v1!10) (or $x3595 $x5247)) (rewrite (= (or $x3595 $x5247) (or $x3595 $x5699 $x6045))) (or $x3595 $x5699 $x6045))))
+(let ((@x4206 (unit-resolution (unit-resolution @x3048 (hypothesis $x3590) $x5247) @x4204 $x5699)))
+(let ((@x4223 (unit-resolution (def-axiom (or $x3821 $x3573)) @x4219 $x3573)))
+(let (($x5758 (not $x5699)))
+(let (($x4064 (or $x3578 $x5758 $x1730 $x4072)))
+(let (($x5845 (or $x5758 $x1730 (>= (+ ?x1727 ?x5667 ?x5630) 0))))
+(let (($x4065 (or $x3578 $x5845)))
+(let ((@x4061 (monotonicity (rewrite (= (+ ?x1727 ?x5667 ?x5630) (+ ?x1727 ?x5630 ?x5667))) (= (>= (+ ?x1727 ?x5667 ?x5630) 0) $x4072))))
+(let ((@x4102 (monotonicity (monotonicity @x4061 (= $x5845 (or $x5758 $x1730 $x4072))) (= $x4065 (or $x3578 (or $x5758 $x1730 $x4072))))))
+(let ((@x4106 (trans @x4102 (rewrite (= (or $x3578 (or $x5758 $x1730 $x4072)) $x4064)) (= $x4065 $x4064))))
+(let ((@x4225 (unit-resolution (mp ((_ quant-inst ?v0!11 ?v1!10) $x4065) @x4106 $x4064) @x4223 (unit-resolution (def-axiom (or $x2645 (not $x1730))) @x4170 (not $x1730)) (or $x5758 $x4072))))
+(let ((@x4228 (monotonicity (symm (hypothesis $x217) (= v_b_SP_G_1$ v_b_SP_G_3$)) (= ?x5152 ?x1734))))
+(let ((@x4234 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x1734 ?x5152)) (<= (+ ?x1734 ?x5630) 0))) (symm @x4228 (= ?x1734 ?x5152)) (<= (+ ?x1734 ?x5630) 0))))
+(let ((@x4235 ((_ th-lemma arith farkas -1 -1 1 1) @x4234 (unit-resolution (def-axiom (or $x2645 (not $x2209))) @x4170 (not $x2209)) @x4203 (unit-resolution @x4225 @x4206 $x4072) false)))
+(let ((@x4885 (unit-resolution (lemma @x4235 (or $x2645 $x3595 $x2708)) @x4265 (unit-resolution (def-axiom (or $x3654 $x3590)) @x5142 $x3590) $x2645)))
+(let (($x4595 (<= (+ ?x1661 (* (- 1) (fun_app$c v_b_SP_G_3$ (?v1!7 ?v0!8)))) 0)))
+(let ((?x3922 (?v1!7 ?v0!8)))
+(let ((?x3910 (fun_app$c v_b_SP_G_1$ ?x3922)))
+(let ((?x3989 (* (- 1) ?x3910)))
+(let ((?x3142 (fun_app$c v_b_SP_G_1$ ?v0!8)))
+(let (($x3936 (<= (+ ?x3142 ?x3989) 0)))
+(let (($x4266 (not $x3936)))
+(let ((?x3945 (pair$ ?x3922 ?v0!8)))
+(let ((?x3946 (b_G$ ?x3945)))
+(let ((?x3031 (* (- 1) ?x3946)))
+(let ((?x3056 (+ ?x3142 ?x3989 ?x3031)))
+(let (($x3032 (= ?x3056 0)))
+(let (($x3033 (not $x3032)))
+(let (($x3034 (or $x3936 (not (fun_app$ v_b_Visited_G_1$ ?x3922)) $x3033)))
+(let (($x3049 (not $x3034)))
+(let ((@x3978 (hypothesis $x1665)))
+(let ((?x3144 (* (- 1) ?x3142)))
+(let ((?x3984 (+ ?x1661 ?x3144)))
+(let (($x3969 (>= ?x3984 0)))
+(let ((@x4544 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x1661 ?x3142)) $x3969)) (monotonicity @x4265 (= ?x1661 ?x3142)) $x3969)))
+(let ((@x3973 ((_ th-lemma arith farkas 1 -1 1) (hypothesis $x3969) (hypothesis (<= (+ b_Infinity$ ?x3144) 0)) @x3978 false)))
+(let ((@x4027 (lemma @x3973 (or (not (<= (+ b_Infinity$ ?x3144) 0)) (not $x3969) $x1664))))
+(let ((@x4552 (unit-resolution @x4027 @x4544 @x3978 (not (<= (+ b_Infinity$ ?x3144) 0)))))
+(let ((@x3425 (def-axiom (or $x3630 $x1749))))
+(let ((@x4543 (unit-resolution @x3425 (trans (monotonicity @x4265 (= ?x245 ?x172)) @x4529 $x246) $x3630)))
+(let ((@x3134 (def-axiom (or $x3639 $x2650 $x3633))))
+(let ((@x3138 (def-axiom (or $x3642 $x3636))))
+(let ((@x3120 (def-axiom (or $x3651 $x3611 $x3645))))
+(let ((@x4905 (unit-resolution @x3120 (unit-resolution @x3138 (unit-resolution @x3134 @x4543 @x4885 $x3639) $x3642) (unit-resolution (def-axiom (or $x3654 $x3648)) @x5142 $x3648) $x3611)))
+(let ((@x4545 (unit-resolution (def-axiom (or $x3821 $x3581)) @x4219 $x3581)))
+(let (($x4738 (= (or $x3586 (or $x1659 (<= (+ b_Infinity$ ?x3144) 0) $x3049)) (or $x3586 $x1659 (<= (+ b_Infinity$ ?x3144) 0) $x3049))))
+(let ((@x4737 ((_ quant-inst ?v0!8) (or $x3586 (or $x1659 (<= (+ b_Infinity$ ?x3144) 0) $x3049)))))
+(let ((@x5209 (mp @x4737 (rewrite $x4738) (or $x3586 $x1659 (<= (+ b_Infinity$ ?x3144) 0) $x3049))))
+(let ((@x4406 (unit-resolution @x5209 @x4545 (unit-resolution (def-axiom (or $x3608 $x1660)) @x4905 $x1660) @x4552 $x3049)))
+(let ((?x3126 (fun_app$c v_b_SP_G_3$ ?x3922)))
+(let ((?x4327 (+ ?x3126 ?x3989)))
+(let (($x4402 (<= ?x4327 0)))
+(let ((@x4541 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x3126 ?x3910)) $x4402)) (monotonicity @x4265 (= ?x3126 ?x3910)) $x4402)))
+(let ((@x4852 ((_ th-lemma arith farkas 1 -1 -1 1) (hypothesis $x3969) (hypothesis $x4595) (hypothesis $x4402) (hypothesis $x4266) false)))
+(let ((@x4542 (unit-resolution (lemma @x4852 (or (not $x4595) (not $x3969) (not $x4402) $x3936)) @x4544 @x4541 (unit-resolution (def-axiom (or $x3034 $x4266)) @x4406 $x4266) (not $x4595))))
+(let ((?x5182 (* (- 1) ?x3126)))
+(let ((?x4179 (+ ?x1661 ?x5182 ?x3031)))
+(let (($x5089 (= ?x4179 0)))
+(let (($x3918 (>= ?x4179 0)))
+(let (($x5284 (>= ?x3056 0)))
+(let ((@x4264 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x3033 $x5284)) (unit-resolution (def-axiom (or $x3034 $x3032)) @x4406 $x3032) $x5284)))
+(let ((@x5267 (unit-resolution ((_ th-lemma arith assign-bounds -1 -1 1) (or $x3918 (not $x5284) (not $x3969) (not $x4402))) @x4264 @x4544 @x4541 $x3918)))
+(let (($x3917 (<= ?x4179 0)))
+(let (($x4407 (>= ?x4327 0)))
+(let ((@x4549 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x3126 ?x3910)) $x4407)) (monotonicity @x4265 (= ?x3126 ?x3910)) $x4407)))
+(let (($x3979 (<= ?x3984 0)))
+(let ((@x6239 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x1661 ?x3142)) $x3979)) (monotonicity @x4265 (= ?x1661 ?x3142)) $x3979)))
+(let (($x5179 (<= ?x3056 0)))
+(let ((@x3960 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x3033 $x5179)) (unit-resolution (def-axiom (or $x3034 $x3032)) @x4406 $x3032) $x5179)))
+(let ((@x4631 (unit-resolution ((_ th-lemma arith assign-bounds -1 -1 1) (or $x3917 (not $x5179) (not $x3979) (not $x4407))) @x3960 @x6239 @x4549 $x3917)))
+(let ((@x4760 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x5089 (not $x3917) (not $x3918))) @x4631 @x5267 $x5089)))
+(let (($x4746 (not $x5089)))
+(let (($x4181 (or $x4595 $x4746)))
+(let (($x3184 (or $x3605 $x4595 $x4746)))
+(let (($x5980 (>= (+ ?x3126 ?x1662) 0)))
+(let (($x5913 (or $x5980 (not (= (+ ?x3126 ?x1662 ?x3946) 0)))))
+(let (($x3976 (or $x3605 $x5913)))
+(let ((@x4178 (monotonicity (rewrite (= (+ ?x3126 ?x1662 ?x3946) (+ ?x1662 ?x3126 ?x3946))) (= (= (+ ?x3126 ?x1662 ?x3946) 0) (= (+ ?x1662 ?x3126 ?x3946) 0)))))
+(let ((@x4745 (trans @x4178 (rewrite (= (= (+ ?x1662 ?x3126 ?x3946) 0) $x5089)) (= (= (+ ?x3126 ?x1662 ?x3946) 0) $x5089))))
+(let ((@x5181 (monotonicity (rewrite (= (+ ?x3126 ?x1662) (+ ?x1662 ?x3126))) (= $x5980 (>= (+ ?x1662 ?x3126) 0)))))
+(let ((@x4634 (trans @x5181 (rewrite (= (>= (+ ?x1662 ?x3126) 0) $x4595)) (= $x5980 $x4595))))
+(let ((@x4184 (monotonicity @x4634 (monotonicity @x4745 (= (not (= (+ ?x3126 ?x1662 ?x3946) 0)) $x4746)) (= $x5913 $x4181))))
+(let ((@x3916 (trans (monotonicity @x4184 (= $x3976 (or $x3605 $x4181))) (rewrite (= (or $x3605 $x4181) $x3184)) (= $x3976 $x3184))))
+(let ((@x5060 (unit-resolution (mp ((_ quant-inst (?v1!7 ?v0!8)) $x3976) @x3916 $x3184) (unit-resolution (def-axiom (or $x3608 $x3600)) @x4905 $x3600) $x4181)))
+(let ((@x6153 (unit-resolution (lemma (unit-resolution @x5060 @x4760 @x4542 false) (or $x3654 $x1664)) @x5142 $x1664)))
+(let ((@x6273 (unit-resolution @x3120 (unit-resolution (def-axiom (or $x3608 $x1665)) @x6153 $x3608) (unit-resolution (def-axiom (or $x3654 $x3648)) @x5142 $x3648) $x3645)))
+(let ((@x5939 (unit-resolution @x3425 (unit-resolution @x3134 (unit-resolution @x3138 @x6273 $x3636) @x4885 $x3633) $x1749)))
+(let ((@x5914 (unit-resolution @x5939 (trans (monotonicity @x4265 (= ?x245 ?x172)) @x4529 $x246) false)))
+(let ((@x6386 (unit-resolution (def-axiom (or $x3818 $x3657 $x3812)) (unit-resolution (def-axiom (or $x3821 $x3815)) @x4219 $x3815) $x3815)))
+(let ((@x6181 (unit-resolution @x6386 (lemma @x5914 $x3654) $x3812)))
+(let ((@x5944 (unit-resolution (def-axiom (or $x3809 $x3678)) @x6181 $x3678)))
+(let (($x4481 (= ?x1846 ?x4480)))
+(let (($x3188 (or $x3683 $x6711 $x4481)))
+(let (($x5285 (or (not (or $x4911 (<= (+ ?x4480 ?x1173 (* (- 1) ?x5018)) 0))) $x4481)))
+(let (($x6363 (or $x3683 $x5285)))
+(let (($x5370 (<= (+ ?x4480 ?x1173 (* (- 1) ?x5018)) 0)))
+(let ((@x4465 (rewrite (= (+ ?x4480 ?x1173 (* (- 1) ?x5018)) (+ ?x1173 ?x4480 (* (- 1) ?x5018))))))
+(let ((@x6818 (monotonicity @x4465 (= $x5370 (<= (+ ?x1173 ?x4480 (* (- 1) ?x5018)) 0)))))
+(let ((@x6705 (trans @x6818 (rewrite (= (<= (+ ?x1173 ?x4480 (* (- 1) ?x5018)) 0) $x6822)) (= $x5370 $x6822))))
+(let ((@x5840 (monotonicity (monotonicity @x6705 (= (or $x4911 $x5370) $x6706)) (= (not (or $x4911 $x5370)) $x6711))))
+(let ((@x6545 (monotonicity (monotonicity @x5840 (= $x5285 (or $x6711 $x4481))) (= $x6363 (or $x3683 (or $x6711 $x4481))))))
+(let ((@x4811 (trans @x6545 (rewrite (= (or $x3683 (or $x6711 $x4481)) $x3188)) (= $x6363 $x3188))))
+(let ((@x6726 (unit-resolution (mp ((_ quant-inst ?v0!15) $x6363) @x4811 $x3188) @x5944 (unit-resolution @x6242 @x6183 (not $x4481)) $x6711)))
+(let ((@x6470 (unit-resolution (def-axiom (or $x6706 (not $x4911))) (hypothesis $x6711) (not $x4911))))
+(let ((@x6494 (unit-resolution (def-axiom (or $x6706 (not $x6822))) (hypothesis $x6711) (not $x6822))))
+(let (($x6511 (or $x4911 $x6822 $x6128)))
+(let ((@x6588 (unit-resolution (def-axiom (or $x3809 $x3670)) @x6181 $x3670)))
+(let (($x6235 (or $x3675 $x4911 $x6822 $x6128)))
+(let (($x6510 (or $x4911 $x5370 (= (+ ?x257 ?x5018 ?x4456) 0))))
+(let (($x6263 (or $x3675 $x6510)))
+(let ((@x6480 (monotonicity (rewrite (= (+ ?x257 ?x5018 ?x4456) ?x6267)) (= (= (+ ?x257 ?x5018 ?x4456) 0) $x6128))))
+(let ((@x4472 (monotonicity (monotonicity @x6705 @x6480 (= $x6510 $x6511)) (= $x6263 (or $x3675 $x6511)))))
+(let ((@x5852 (mp ((_ quant-inst ?v0!15) $x6263) (trans @x4472 (rewrite (= (or $x3675 $x6511) $x6235)) (= $x6263 $x6235)) $x6235)))
+(let ((@x6501 (unit-resolution (unit-resolution @x5852 @x6588 $x6511) @x6494 @x6470 (hypothesis (not $x6128)) false)))
+(let ((@x4608 (lemma @x6501 (or $x6706 $x6128))))
+(let ((@x6959 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x6128) $x5853)) (unit-resolution @x4608 @x6726 $x6128) $x5853)))
+(let (($x6603 (>= ?x5018 0)))
+(let (($x6582 (<= ?x5018 0)))
+(let (($x6583 (not $x6582)))
+(let (($x6156 (= v_b_v_G_1$ ?v0!15)))
+(let (($x5538 (not $x6156)))
+(let ((@x7337 (symm (commutativity (= $x6156 (= ?v0!15 v_b_v_G_1$))) (= (= ?v0!15 v_b_v_G_1$) $x6156))))
+(let (($x6631 (= ?v0!15 v_b_v_G_1$)))
+(let (($x7483 (not $x6631)))
+(let (($x6269 (fun_app$ v_b_Visited_G_1$ ?v0!15)))
+(let (($x7698 (or $x6631 $x6269)))
+(let (($x6630 (fun_app$ ?x265 ?v0!15)))
+(let (($x7702 (= $x6630 $x7698)))
+(let (($x3468 (forall ((?v0 B_Vertex_bool_fun$) (?v1 B_Vertex$) (?v2 Bool) (?v3 B_Vertex$) )(!(let (($x67 (fun_app$ (fun_app$a (fun_app$b (fun_upd$ ?v0) ?v1) ?v2) ?v3)))
+(= $x67 (ite (= ?v3 ?v1) ?v2 (fun_app$ ?v0 ?v3)))) :pattern ( (fun_app$ (fun_app$a (fun_app$b (fun_upd$ ?v0) ?v1) ?v2) ?v3) )))
+))
+(let (($x77 (forall ((?v0 B_Vertex_bool_fun$) (?v1 B_Vertex$) (?v2 Bool) (?v3 B_Vertex$) )(let (($x67 (fun_app$ (fun_app$a (fun_app$b (fun_upd$ ?v0) ?v1) ?v2) ?v3)))
+(= $x67 (ite (= ?v3 ?v1) ?v2 (fun_app$ ?v0 ?v3)))))
+))
+(let (($x67 (fun_app$ (fun_app$a (fun_app$b (fun_upd$ ?3) ?2) ?1) ?0)))
+(let (($x74 (= $x67 (ite (= ?0 ?2) ?1 (fun_app$ ?3 ?0)))))
+(let (($x72 (forall ((?v0 B_Vertex_bool_fun$) (?v1 B_Vertex$) (?v2 Bool) (?v3 B_Vertex$) )(let (($x67 (fun_app$ (fun_app$a (fun_app$b (fun_upd$ ?v0) ?v1) ?v2) ?v3)))
+(= $x67 (ite (= ?v3 ?v1) ?v2 (fun_app$ ?v0 ?v3)))))
+))
+(let ((@x76 (rewrite (= (= $x67 (ite (= ?0 ?2) ?1 (fun_app$ ?3 ?0))) $x74))))
+(let ((@x1443 (mp~ (mp (asserted $x72) (quant-intro @x76 (= $x72 $x77)) $x77) (nnf-pos (refl (~ $x74 $x74)) (~ $x77 $x77)) $x77)))
+(let ((@x3473 (mp @x1443 (quant-intro (refl (= $x74 $x74)) (= $x77 $x3468)) $x3468)))
+(let (($x4114 (not $x3468)))
+(let (($x6435 (or $x4114 $x7702)))
+(let ((@x5925 (monotonicity (rewrite (= (ite $x6631 true $x6269) $x7698)) (= (= $x6630 (ite $x6631 true $x6269)) $x7702))))
+(let ((@x6213 (monotonicity @x5925 (= (or $x4114 (= $x6630 (ite $x6631 true $x6269))) $x6435))))
+(let ((@x7487 (trans @x6213 (rewrite (= $x6435 $x6435)) (= (or $x4114 (= $x6630 (ite $x6631 true $x6269))) $x6435))))
+(let ((@x7488 (mp ((_ quant-inst v_b_Visited_G_1$ v_b_v_G_1$ true ?v0!15) (or $x4114 (= $x6630 (ite $x6631 true $x6269)))) @x7487 $x6435)))
+(let ((@x5875 (symm (unit-resolution (def-axiom (or $x3809 $x266)) @x6181 $x266) (= ?x265 v_b_Visited_G_2$))))
+(let ((@x7321 (symm (monotonicity @x5875 (= $x6630 (fun_app$ v_b_Visited_G_2$ ?v0!15))) (= (fun_app$ v_b_Visited_G_2$ ?v0!15) $x6630))))
+(let ((@x7322 (monotonicity @x7321 (= (not (fun_app$ v_b_Visited_G_2$ ?v0!15)) (not $x6630)))))
+(let (($x4415 (fun_app$ v_b_Visited_G_2$ ?v0!15)))
+(let (($x4479 (not $x4415)))
+(let ((?x5054 (b_G$ (pair$ v_b_v_G_1$ ?v0!13))))
+(let ((?x4706 (+ ?x257 ?x1810 ?x5054)))
+(let (($x4687 (= ?x4706 0)))
+(let (($x5187 (>= (+ ?x257 (* (- 1) ?x1808) ?x5054) 0)))
+(let (($x5051 (<= (+ b_Infinity$ (* (- 1) ?x5054)) 0)))
+(let (($x5186 (or $x5051 $x5187)))
+(let (($x5221 (not $x5186)))
+(let ((@x5744 (monotonicity (commutativity (= (= ?x1808 ?x1809) (= ?x1809 ?x1808))) (= (not (= ?x1808 ?x1809)) (not (= ?x1809 ?x1808))))))
+(let (($x5690 (not (= ?x1808 ?x1809))))
+(let ((@x5726 (mp (unit-resolution ((_ th-lemma arith triangle-eq) (or $x5690 $x1812)) (hypothesis $x1813) $x5690) @x5744 (not (= ?x1809 ?x1808)))))
+(let (($x5270 (= ?x1809 ?x1808)))
+(let (($x5230 (or $x5221 $x5270)))
+(let ((@x4739 (hypothesis $x3678)))
+(let (($x5327 (or $x3683 $x5221 $x5270)))
+(let (($x5333 (or (not (or $x5051 (<= (+ ?x1808 ?x1173 (* (- 1) ?x5054)) 0))) $x5270)))
+(let (($x5268 (or $x3683 $x5333)))
+(let (($x5095 (<= (+ ?x1808 ?x1173 (* (- 1) ?x5054)) 0)))
+(let ((@x5120 (rewrite (= (+ ?x1808 ?x1173 (* (- 1) ?x5054)) (+ ?x1173 ?x1808 (* (- 1) ?x5054))))))
+(let ((@x5127 (monotonicity @x5120 (= $x5095 (<= (+ ?x1173 ?x1808 (* (- 1) ?x5054)) 0)))))
+(let ((@x4705 (trans @x5127 (rewrite (= (<= (+ ?x1173 ?x1808 (* (- 1) ?x5054)) 0) $x5187)) (= $x5095 $x5187))))
+(let ((@x5229 (monotonicity (monotonicity @x4705 (= (or $x5051 $x5095) $x5186)) (= (not (or $x5051 $x5095)) $x5221))))
+(let ((@x5269 (monotonicity (monotonicity @x5229 (= $x5333 $x5230)) (= $x5268 (or $x3683 $x5230)))))
+(let ((@x5432 (mp ((_ quant-inst ?v0!13) $x5268) (trans @x5269 (rewrite (= (or $x3683 $x5230) $x5327)) (= $x5268 $x5327)) $x5327)))
+(let ((@x5729 (unit-resolution (def-axiom (or $x5186 (not $x5051))) (unit-resolution (unit-resolution @x5432 @x4739 $x5230) @x5726 $x5221) (not $x5051))))
+(let ((@x5749 (unit-resolution (def-axiom (or $x5186 (not $x5187))) (unit-resolution (unit-resolution @x5432 @x4739 $x5230) @x5726 $x5221) (not $x5187))))
+(let (($x5211 (or $x5051 $x5187 $x4687)))
+(let ((@x5807 (hypothesis $x3670)))
+(let (($x5189 (or $x3675 $x5051 $x5187 $x4687)))
+(let (($x5102 (or $x5051 $x5095 (= (+ ?x257 ?x5054 ?x1810) 0))))
+(let (($x5163 (or $x3675 $x5102)))
+(let ((@x5164 (monotonicity (rewrite (= (+ ?x257 ?x5054 ?x1810) ?x4706)) (= (= (+ ?x257 ?x5054 ?x1810) 0) $x4687))))
+(let ((@x5215 (monotonicity (monotonicity @x4705 @x5164 (= $x5102 $x5211)) (= $x5163 (or $x3675 $x5211)))))
+(let ((@x5376 (mp ((_ quant-inst ?v0!13) $x5163) (trans @x5215 (rewrite (= (or $x3675 $x5211) $x5189)) (= $x5163 $x5189)) $x5189)))
+(let ((@x5714 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x4687) (>= ?x4706 0))) (unit-resolution (unit-resolution @x5376 @x5807 $x5211) @x5749 @x5729 $x4687) (>= ?x4706 0))))
+(let ((@x5723 (unit-resolution ((_ th-lemma arith farkas 1 1) (or (<= ?x1811 0) $x1812)) (hypothesis $x1813) (<= ?x1811 0))))
+(let ((@x6888 (unit-resolution (lemma ((_ th-lemma arith farkas 1 -1 1) @x5723 @x5749 @x5714 false) (or $x1812 $x3675 $x3683)) @x6588 @x5944 $x1812)))
+(let ((@x6891 (unit-resolution (def-axiom (or $x3806 $x1813 $x3800)) @x6888 (unit-resolution (def-axiom (or $x3809 $x3803)) @x6181 $x3803) $x3800)))
+(let (($x6050 (= ?v0!14 v_b_v_G_1$)))
+(let (($x5678 (fun_app$ v_b_Visited_G_1$ ?v0!14)))
+(let (($x4963 (or $x6050 $x5678)))
+(let (($x6049 (fun_app$ ?x265 ?v0!14)))
+(let (($x6452 (= $x6049 $x4963)))
+(let (($x5869 (or $x4114 $x6452)))
+(let ((@x6355 (monotonicity (rewrite (= (ite $x6050 true $x5678) $x4963)) (= (= $x6049 (ite $x6050 true $x5678)) $x6452))))
+(let ((@x5854 (monotonicity @x6355 (= (or $x4114 (= $x6049 (ite $x6050 true $x5678))) $x5869))))
+(let ((@x6366 (trans @x5854 (rewrite (= $x5869 $x5869)) (= (or $x4114 (= $x6049 (ite $x6050 true $x5678))) $x5869))))
+(let ((@x6233 (mp ((_ quant-inst v_b_Visited_G_1$ v_b_v_G_1$ true ?v0!14) (or $x4114 (= $x6049 (ite $x6050 true $x5678)))) @x6366 $x5869)))
+(let ((@x6372 (symm (monotonicity @x5875 (= $x6049 (fun_app$ v_b_Visited_G_2$ ?v0!14))) (= (fun_app$ v_b_Visited_G_2$ ?v0!14) $x6049))))
+(let (($x1824 (fun_app$ v_b_Visited_G_2$ ?v0!14)))
+(let ((@x4837 (mp (unit-resolution (def-axiom (or $x1829 $x1824)) (hypothesis $x1830) $x1824) @x6372 $x6049)))
+(let ((@x5037 (unit-resolution (def-axiom (or (not $x6452) (not $x6049) $x4963)) @x4837 (unit-resolution @x6233 @x3473 $x6452) $x4963)))
+(let (($x4290 (not $x5678)))
+(let ((?x5658 (* (- 1) ?x1827)))
+(let ((?x4907 (+ ?x257 ?x5658)))
+(let (($x6523 (>= ?x4907 0)))
+(let (($x6556 (not $x6523)))
+(let (($x4887 (>= (+ ?x257 ?x5658 (b_G$ (pair$ v_b_v_G_1$ ?v0!14))) 0)))
+(let (($x4812 (not $x4887)))
+(let (($x4783 (<= (+ b_Infinity$ (* (- 1) (b_G$ (pair$ v_b_v_G_1$ ?v0!14)))) 0)))
+(let (($x5110 (or $x4783 $x4887)))
+(let (($x5079 (not $x5110)))
+(let ((@x5065 (unit-resolution (def-axiom (or $x1829 (not $x1828))) (hypothesis $x1830) (not $x1828))))
+(let (($x4844 (or $x3683 $x5079 $x1828)))
+(let (($x4891 (<= (+ ?x1827 ?x1173 (* (- 1) (b_G$ (pair$ v_b_v_G_1$ ?v0!14)))) 0)))
+(let (($x5552 (or (not (or $x4783 $x4891)) $x1828)))
+(let (($x4766 (or $x3683 $x5552)))
+(let (($x4493 (<= (+ ?x1173 ?x1827 (* (- 1) (b_G$ (pair$ v_b_v_G_1$ ?v0!14)))) 0)))
+(let (($x5019 (= (+ ?x1827 ?x1173 (* (- 1) (b_G$ (pair$ v_b_v_G_1$ ?v0!14)))) (+ ?x1173 ?x1827 (* (- 1) (b_G$ (pair$ v_b_v_G_1$ ?v0!14)))))))
+(let ((@x5288 (trans (monotonicity (rewrite $x5019) (= $x4891 $x4493)) (rewrite (= $x4493 $x4887)) (= $x4891 $x4887))))
+(let ((@x5082 (monotonicity (monotonicity @x5288 (= (or $x4783 $x4891) $x5110)) (= (not (or $x4783 $x4891)) $x5079))))
+(let ((@x5868 (monotonicity (monotonicity @x5082 (= $x5552 (or $x5079 $x1828))) (= $x4766 (or $x3683 (or $x5079 $x1828))))))
+(let ((@x5811 (trans @x5868 (rewrite (= (or $x3683 (or $x5079 $x1828)) $x4844)) (= $x4766 $x4844))))
+(let ((@x6433 (unit-resolution (def-axiom (or $x5110 $x4812)) (unit-resolution (mp ((_ quant-inst ?v0!14) $x4766) @x5811 $x4844) @x5944 @x5065 $x5079) $x4812)))
+(let ((?x6047 (pair$ v_b_v_G_1$ ?v0!14)))
+(let ((?x6491 (b_G$ ?x6047)))
+(let (($x5826 (>= ?x6491 0)))
+(let ((@x6283 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x6491 0)) $x5826)) (hypothesis (not $x5826)) (not (= ?x6491 0)))))
+(let (($x5742 (= v_b_v_G_1$ ?v0!14)))
+(let (($x5751 (<= ?x6491 0)))
+(let ((@x6302 (unit-resolution ((_ th-lemma arith farkas 1 1) (or $x5826 $x5751)) (hypothesis (not $x5826)) $x5751)))
+(let (($x5738 (or $x5742 (not $x5751))))
+(let (($x3480 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(!(let (($x84 (= ?v0 ?v1)))
+(or $x84 (not (<= (b_G$ (pair$ ?v0 ?v1)) 0)))) :pattern ( (pair$ ?v0 ?v1) )))
+))
+(let (($x120 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let (($x84 (= ?v0 ?v1)))
+(or $x84 (not (<= (b_G$ (pair$ ?v0 ?v1)) 0)))))
+))
+(let (($x84 (= ?1 ?0)))
+(let (($x117 (or $x84 (not (<= (b_G$ (pair$ ?1 ?0)) 0)))))
+(let (($x105 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x29 (pair$ ?v0 ?v1)))
+(let ((?x85 (b_G$ ?x29)))
+(let (($x102 (< 0 ?x85)))
+(=> (not (= ?v0 ?v1)) $x102)))))
+))
+(let (($x110 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let ((?x29 (pair$ ?v0 ?v1)))
+(let ((?x85 (b_G$ ?x29)))
+(let (($x102 (< 0 ?x85)))
+(let (($x84 (= ?v0 ?v1)))
+(or $x84 $x102))))))
+))
+(let ((?x29 (pair$ ?1 ?0)))
+(let ((?x85 (b_G$ ?x29)))
+(let (($x102 (< 0 ?x85)))
+(let ((@x119 (monotonicity (rewrite (= $x102 (not (<= ?x85 0)))) (= (or $x84 $x102) $x117))))
+(let ((@x112 (quant-intro (rewrite (= (=> (not $x84) $x102) (or $x84 $x102))) (= $x105 $x110))))
+(let ((@x125 (mp (asserted $x105) (trans @x112 (quant-intro @x119 (= $x110 $x120)) (= $x105 $x120)) $x120)))
+(let ((@x3485 (mp (mp~ @x125 (nnf-pos (refl (~ $x117 $x117)) (~ $x120 $x120)) $x120) (quant-intro (refl (= $x117 $x117)) (= $x120 $x3480)) $x3480)))
+(let ((@x5780 (mp ((_ quant-inst v_b_v_G_1$ ?v0!14) (or (not $x3480) $x5738)) (rewrite (= (or (not $x3480) $x5738) (or (not $x3480) $x5742 (not $x5751)))) (or (not $x3480) $x5742 (not $x5751)))))
+(let (($x5739 (= ?x6491 0)))
+(let (($x5781 (or (not $x5742) $x5739)))
+(let (($x3474 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(!(or (not (= ?v0 ?v1)) (= (b_G$ (pair$ ?v0 ?v1)) 0)) :pattern ( (pair$ ?v0 ?v1) )))
+))
+(let (($x99 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(or (not (= ?v0 ?v1)) (= (b_G$ (pair$ ?v0 ?v1)) 0)))
+))
+(let ((@x3476 (refl (= (or (not $x84) (= ?x85 0)) (or (not $x84) (= ?x85 0))))))
+(let ((@x1447 (refl (~ (or (not $x84) (= ?x85 0)) (or (not $x84) (= ?x85 0))))))
+(let (($x93 (forall ((?v0 B_Vertex$) (?v1 B_Vertex$) )(let (($x84 (= ?v0 ?v1)))
+(=> $x84 (= (b_G$ (pair$ ?v0 ?v1)) 0))))
+))
+(let ((@x98 (rewrite (= (=> $x84 (= ?x85 0)) (or (not $x84) (= ?x85 0))))))
+(let ((@x1448 (mp~ (mp (asserted $x93) (quant-intro @x98 (= $x93 $x99)) $x99) (nnf-pos @x1447 (~ $x99 $x99)) $x99)))
+(let ((@x3479 (mp @x1448 (quant-intro @x3476 (= $x99 $x3474)) $x3474)))
+(let ((@x5817 (mp ((_ quant-inst v_b_v_G_1$ ?v0!14) (or (not $x3474) $x5781)) (rewrite (= (or (not $x3474) $x5781) (or (not $x3474) (not $x5742) $x5739))) (or (not $x3474) (not $x5742) $x5739))))
+(let ((@x6306 (unit-resolution (unit-resolution @x5817 @x3479 $x5781) (unit-resolution (unit-resolution @x5780 @x3485 $x5738) @x6302 $x5742) @x6283 false)))
+(let ((@x6555 ((_ th-lemma arith farkas 1 -1 1) (lemma @x6306 $x5826) (hypothesis $x4812) (hypothesis $x6523) false)))
+(let ((@x6225 (unit-resolution (def-axiom (or $x3809 $x256)) @x6181 $x256)))
+(let ((@x5748 (unit-resolution (def-axiom (or $x3821 $x3565)) @x4219 $x3565)))
+(let ((@x6018 (rewrite (= (or $x3570 (or $x255 $x4290 $x6523)) (or $x3570 $x255 $x4290 $x6523)))))
+(let ((@x6055 (mp ((_ quant-inst ?v0!14 v_b_v_G_1$) (or $x3570 (or $x255 $x4290 $x6523))) @x6018 (or $x3570 $x255 $x4290 $x6523))))
+(let ((@x6222 (unit-resolution @x6055 @x5748 @x6225 (hypothesis $x5678) (hypothesis $x6556) false)))
+(let ((@x5057 (unit-resolution (lemma @x6222 (or $x4290 $x6523)) (unit-resolution (lemma @x6555 (or $x6556 $x4887)) @x6433 $x6556) $x4290)))
+(let ((@x6293 (monotonicity (unit-resolution (def-axiom (or (not $x4963) $x6050 $x5678)) @x5057 @x5037 $x6050) (= ?x1827 ?x257))))
+(let (($x3052 (= ?x3104 ?x257)))
+(let ((?x3130 (pair$ v_b_v_G_1$ v_b_v_G_1$)))
+(let ((?x3096 (b_G$ ?x3130)))
+(let (($x3079 (>= ?x3096 0)))
+(let (($x3088 (<= (+ b_Infinity$ (* (- 1) ?x3096)) 0)))
+(let (($x4242 (or $x3088 $x3079)))
+(let (($x4785 (= ?x3096 0)))
+(let (($x3151 (not $x3474)))
+(let (($x4816 (or $x3151 $x4785)))
+(let ((@x4770 (monotonicity (rewrite (= (= v_b_v_G_1$ v_b_v_G_1$) true)) (= (not (= v_b_v_G_1$ v_b_v_G_1$)) (not true)))))
+(let ((@x4775 (trans @x4770 (rewrite (= (not true) false)) (= (not (= v_b_v_G_1$ v_b_v_G_1$)) false))))
+(let ((@x4767 (monotonicity @x4775 (= (or (not (= v_b_v_G_1$ v_b_v_G_1$)) $x4785) (or false $x4785)))))
+(let ((@x4773 (trans @x4767 (rewrite (= (or false $x4785) $x4785)) (= (or (not (= v_b_v_G_1$ v_b_v_G_1$)) $x4785) $x4785))))
+(let ((@x4820 (monotonicity @x4773 (= (or $x3151 (or (not (= v_b_v_G_1$ v_b_v_G_1$)) $x4785)) $x4816))))
+(let ((@x4821 (trans @x4820 (rewrite (= $x4816 $x4816)) (= (or $x3151 (or (not (= v_b_v_G_1$ v_b_v_G_1$)) $x4785)) $x4816))))
+(let ((@x4822 (mp ((_ quant-inst v_b_v_G_1$ v_b_v_G_1$) (or $x3151 (or (not (= v_b_v_G_1$ v_b_v_G_1$)) $x4785))) @x4821 $x4816)))
+(let ((@x4849 (lemma (unit-resolution @x4822 @x3479 (hypothesis (not $x4785)) false) $x4785)))
+(let ((@x6019 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x4785) $x3079)) @x4849 $x3079)))
+(let ((@x4316 (def-axiom (or $x4242 (not $x3079)))))
+(let (($x4245 (not $x4242)))
+(let (($x3975 (or $x3683 $x4245 $x3052)))
+(let (($x3053 (or (not (or $x3088 (<= (+ ?x257 ?x1173 (* (- 1) ?x3096)) 0))) $x3052)))
+(let (($x3958 (or $x3683 $x3053)))
+(let (($x3103 (<= (+ ?x257 ?x1173 (* (- 1) ?x3096)) 0)))
+(let ((@x4023 (monotonicity (rewrite (= (+ ?x257 ?x1173 (* (- 1) ?x3096)) (* (- 1) ?x3096))) (= $x3103 (<= (* (- 1) ?x3096) 0)))))
+(let ((@x4044 (trans @x4023 (rewrite (= (<= (* (- 1) ?x3096) 0) $x3079)) (= $x3103 $x3079))))
+(let ((@x4247 (monotonicity (monotonicity @x4044 (= (or $x3088 $x3103) $x4242)) (= (not (or $x3088 $x3103)) $x4245))))
+(let ((@x4254 (monotonicity (monotonicity @x4247 (= $x3053 (or $x4245 $x3052))) (= $x3958 (or $x3683 (or $x4245 $x3052))))))
+(let ((@x4258 (trans @x4254 (rewrite (= (or $x3683 (or $x4245 $x3052)) $x3975)) (= $x3958 $x3975))))
+(let ((@x4259 (mp ((_ quant-inst v_b_v_G_1$) $x3958) @x4258 $x3975)))
+(let ((@x6268 (monotonicity (unit-resolution (def-axiom (or (not $x4963) $x6050 $x5678)) @x5057 @x5037 $x6050) (= ?x1826 ?x3104))))
+(let ((@x6107 (trans @x6268 (unit-resolution @x4259 @x5944 (unit-resolution @x4316 @x6019 $x4242) $x3052) (= ?x1826 ?x257))))
+(let ((@x6162 (unit-resolution @x5065 (trans @x6107 (symm @x6293 (= ?x257 ?x1827)) $x1828) false)))
+(let ((@x7615 (unit-resolution (def-axiom (or $x3794 $x1830 $x3788)) (lemma @x6162 $x1829) (unit-resolution (def-axiom (or $x3797 $x3791)) @x6891 $x3791) $x3788)))
+(let ((@x7616 (unit-resolution (def-axiom (or $x3785 $x3695)) @x7615 $x3695)))
+(let ((@x7443 (mp ((_ quant-inst ?v0!15) (or $x3700 (or $x4479 $x4481))) (rewrite (= (or $x3700 (or $x4479 $x4481)) (or $x3700 $x4479 $x4481))) (or $x3700 $x4479 $x4481))))
+(let ((@x7323 (mp (unit-resolution @x7443 @x7616 (unit-resolution @x6242 @x6183 (not $x4481)) $x4479) @x7322 (not $x6630))))
+(let ((@x7334 (unit-resolution (def-axiom (or (not $x7702) $x6630 (not $x7698))) @x7323 (unit-resolution @x7488 @x3473 $x7702) (not $x7698))))
+(let ((@x7344 (mp (unit-resolution (def-axiom (or $x7698 $x7483)) @x7334 $x7483) (monotonicity @x7337 (= $x7483 $x5538)) $x5538)))
+(let (($x5470 (or $x6156 $x6583)))
+(let ((@x6577 (mp ((_ quant-inst v_b_v_G_1$ ?v0!15) (or (not $x3480) $x5470)) (rewrite (= (or (not $x3480) $x5470) (or (not $x3480) $x6156 $x6583))) (or (not $x3480) $x6156 $x6583))))
+(let ((@x7345 (unit-resolution ((_ th-lemma arith farkas 1 1) (or $x6603 $x6582)) (unit-resolution (unit-resolution @x6577 @x3485 $x5470) @x7344 $x6583) $x6603)))
+(let (($x4153 (<= ?x296 0)))
+(let ((?x4058 (* (- 1) ?x296)))
+(let ((?x4124 (+ ?x172 ?x4058)))
+(let (($x4125 (>= ?x4124 0)))
+(let ((@x6892 (unit-resolution (def-axiom (or $x3797 $x3686)) @x6891 $x3686)))
+(let (($x4878 (or $x3691 $x4125)))
+(let ((@x4880 ((_ quant-inst b_Source$) $x4878)))
+(let (($x3198 (<= ?x172 0)))
+(let ((@x4532 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x2952 $x3198)) @x4529 $x3198)))
+(let ((@x6899 (unit-resolution ((_ th-lemma arith assign-bounds -1 1) (or $x4153 (not $x3198) (not $x4125))) @x4532 (or $x4153 (not $x4125)))))
+(let ((@x6900 (unit-resolution @x6899 (unit-resolution @x4880 @x6892 $x4125) $x4153)))
+(let (($x3887 (= v_b_v_G_1$ b_Source$)))
+(let (($x5313 (not $x3887)))
+(let ((@x5202 (hypothesis $x773)))
+(let ((?x4565 (pair$ b_Source$ b_Source$)))
+(let ((?x4566 (b_G$ ?x4565)))
+(let ((?x4567 (* (- 1) ?x4566)))
+(let ((?x4041 (pair$ v_b_v_G_1$ b_Source$)))
+(let ((?x4042 (b_G$ ?x4041)))
+(let ((@x4671 (monotonicity (symm (hypothesis $x3887) (= b_Source$ v_b_v_G_1$)) (= ?x4565 ?x4041))))
+(let ((@x4659 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x4042 ?x4566)) (>= (+ ?x4042 ?x4567) 0))) (monotonicity (symm @x4671 (= ?x4041 ?x4565)) (= ?x4042 ?x4566)) (>= (+ ?x4042 ?x4567) 0))))
+(let ((?x4049 (* (- 1) ?x4042)))
+(let ((?x5672 (+ ?x3096 ?x4049)))
+(let (($x5674 (>= ?x5672 0)))
+(let ((@x4664 (monotonicity (monotonicity (hypothesis $x3887) (= ?x3130 ?x4041)) (= ?x3096 ?x4042))))
+(let (($x4315 (not $x3079)))
+(let ((@x4728 (trans (monotonicity (hypothesis $x3887) (= ?x257 ?x172)) @x4529 (= ?x257 0))))
+(let ((@x4830 (monotonicity (monotonicity (hypothesis $x3887) (= ?x3104 ?x296)) @x4728 (= $x3052 $x297))))
+(let ((@x4736 (mp @x5202 (monotonicity (symm @x4830 (= $x297 $x3052)) (= $x773 (not $x3052))) (not $x3052))))
+(let ((@x5369 (unit-resolution @x4316 (unit-resolution (unit-resolution @x4259 @x4739 (or $x4245 $x3052)) @x4736 $x4245) $x4315)))
+(let (($x4601 (= ?x4566 0)))
+(let (($x4613 (or $x3151 $x4601)))
+(let ((@x4604 (monotonicity @x5820 (= (or (not (= b_Source$ b_Source$)) $x4601) (or false $x4601)))))
+(let ((@x4630 (trans @x4604 (rewrite (= (or false $x4601) $x4601)) (= (or (not (= b_Source$ b_Source$)) $x4601) $x4601))))
+(let ((@x4617 (monotonicity @x4630 (= (or $x3151 (or (not (= b_Source$ b_Source$)) $x4601)) $x4613))))
+(let ((@x4620 (trans @x4617 (rewrite (= $x4613 $x4613)) (= (or $x3151 (or (not (= b_Source$ b_Source$)) $x4601)) $x4613))))
+(let ((@x4621 (mp ((_ quant-inst b_Source$ b_Source$) (or $x3151 (or (not (= b_Source$ b_Source$)) $x4601))) @x4620 $x4613)))
+(let ((@x5180 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x4601) (>= ?x4566 0))) (unit-resolution @x4621 @x3479 $x4601) (>= ?x4566 0))))
+(let ((@x5283 ((_ th-lemma arith farkas 1 -1 1 1) @x5180 @x5369 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x3096 ?x4042)) $x5674)) @x4664 $x5674) @x4659 false)))
+(let (($x5310 (<= ?x4042 0)))
+(let ((?x4076 (+ ?x257 ?x4058 ?x4042)))
+(let (($x4096 (<= ?x4076 0)))
+(let (($x4079 (= ?x4076 0)))
+(let (($x4053 (<= (+ ?x172 ?x1173 ?x4049) 0)))
+(let (($x4051 (<= (+ b_Infinity$ ?x4049) 0)))
+(let (($x4054 (or $x4051 $x4053)))
+(let (($x4055 (not $x4054)))
+(let ((@x5609 (symm (monotonicity @x4529 (= (= ?x296 ?x172) $x297)) (= $x297 (= ?x296 ?x172)))))
+(let ((@x5618 (mp @x5202 (monotonicity @x5609 (= $x773 (not (= ?x296 ?x172)))) (not (= ?x296 ?x172)))))
+(let (($x4056 (= ?x296 ?x172)))
+(let (($x4057 (or $x4055 $x4056)))
+(let (($x4295 (or $x3683 $x4055 $x4056)))
+(let ((@x4884 (mp ((_ quant-inst b_Source$) (or $x3683 $x4057)) (rewrite (= (or $x3683 $x4057) $x4295)) $x4295)))
+(let ((@x5791 (unit-resolution (def-axiom (or $x4054 (not $x4051))) (hypothesis $x4055) (not $x4051))))
+(let ((@x5806 (unit-resolution (def-axiom (or $x4054 (not $x4053))) (hypothesis $x4055) (not $x4053))))
+(let (($x4082 (or $x4051 $x4053 $x4079)))
+(let (($x4085 (or $x3675 $x4051 $x4053 $x4079)))
+(let (($x4075 (or $x4051 $x4053 (= (+ ?x257 ?x4042 ?x4058) 0))))
+(let (($x4086 (or $x3675 $x4075)))
+(let ((@x4081 (monotonicity (rewrite (= (+ ?x257 ?x4042 ?x4058) ?x4076)) (= (= (+ ?x257 ?x4042 ?x4058) 0) $x4079))))
+(let ((@x4090 (monotonicity (monotonicity @x4081 (= $x4075 $x4082)) (= $x4086 (or $x3675 $x4082)))))
+(let ((@x4095 (mp ((_ quant-inst b_Source$) $x4086) (trans @x4090 (rewrite (= (or $x3675 $x4082) $x4085)) (= $x4086 $x4085)) $x4085)))
+(let ((@x5789 (unit-resolution (unit-resolution @x4095 @x5807 $x4082) @x5806 @x5791 (hypothesis (not $x4079)) false)))
+(let ((@x5623 (unit-resolution (lemma @x5789 (or $x4054 $x4079 $x3675)) (unit-resolution (unit-resolution @x4884 @x4739 $x4057) @x5618 $x4055) @x5807 $x4079)))
+(let ((@x5923 (hypothesis $x4096)))
+(let ((@x5933 ((_ th-lemma arith farkas -1 1 -1 1) (hypothesis $x3904) (hypothesis $x4153) (hypothesis (not $x5310)) @x5923 false)))
+(let ((@x5938 (lemma @x5933 (or $x5310 (not $x3904) (not $x4153) (not $x4096)))))
+(let ((@x5596 (unit-resolution @x5938 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x4079) $x4096)) @x5623 $x4096) (hypothesis $x4153) @x5049 $x5310)))
+(let (($x5886 (= (or (not $x3480) (or $x3887 (not $x5310))) (or (not $x3480) $x3887 (not $x5310)))))
+(let ((@x5952 (mp ((_ quant-inst v_b_v_G_1$ b_Source$) (or (not $x3480) (or $x3887 (not $x5310)))) (rewrite $x5886) (or (not $x3480) $x3887 (not $x5310)))))
+(let ((@x5597 (unit-resolution @x5952 @x3485 @x5596 (unit-resolution (lemma @x5283 (or $x5313 $x3683 $x297)) @x5202 @x4739 $x5313) false)))
+(let ((@x6788 (unit-resolution (lemma @x5597 (or $x297 (not $x4153) $x3675 $x3683)) @x6900 @x6588 @x5944 $x297)))
+(let ((@x7810 (unit-resolution (def-axiom (or $x3782 $x773 $x3776)) (unit-resolution (def-axiom (or $x3785 $x3779)) @x7615 $x3779) @x6788 $x3776)))
+(let ((@x3347 (def-axiom (or $x3770 $x1848 $x3764))))
+(let ((@x9293 (unit-resolution @x3347 (unit-resolution (def-axiom (or $x3773 $x3767)) @x7810 $x3767) $x3767)))
+(let ((@x9294 (unit-resolution @x9293 (lemma ((_ th-lemma arith farkas 1 1 -1 1) @x5703 @x7345 @x6959 @x5049 false) $x1847) $x3764)))
+(let ((@x3367 (def-axiom (or $x3761 $x3703))))
+(let (($x4335 (or $x3708 $x4161)))
+(let ((@x4337 ((_ quant-inst v_b_v_G_1$) $x4335)))
+(let (($x4126 (fun_app$ v_b_Visited_G_2$ v_b_v_G_1$)))
+(let (($x3136 (fun_app$ ?x265 v_b_v_G_1$)))
+(let (($x3461 (forall ((?v0 B_Vertex_bool_fun$) (?v1 B_Vertex$) (?v2 Bool) )(!(= (fun_app$ (fun_app$a (fun_app$b (fun_upd$ ?v0) ?v1) ?v2) ?v1) ?v2) :pattern ( (fun_app$a (fun_app$b (fun_upd$ ?v0) ?v1) ?v2) )))
+))
+(let (($x57 (forall ((?v0 B_Vertex_bool_fun$) (?v1 B_Vertex$) (?v2 Bool) )(= (fun_app$ (fun_app$a (fun_app$b (fun_upd$ ?v0) ?v1) ?v2) ?v1) ?v2))
+))
+(let (($x54 (= (fun_app$ (fun_app$a (fun_app$b (fun_upd$ ?2) ?1) ?0) ?1) ?0)))
+(let (($x52 (forall ((?v0 B_Vertex_bool_fun$) (?v1 B_Vertex$) (?v2 Bool) )(= (fun_app$ (fun_app$a (fun_app$b (fun_upd$ ?v0) ?v1) ?v2) ?v1) ?v2))
+))
+(let (($x51 (= (fun_app$ (fun_app$a (fun_app$b (fun_upd$ ?2) ?1) ?0) ?1) ?0)))
+(let ((@x62 (mp (asserted $x52) (quant-intro (rewrite (= $x51 $x54)) (= $x52 $x57)) $x57)))
+(let ((@x3466 (mp (mp~ @x62 (nnf-pos (refl (~ $x54 $x54)) (~ $x57 $x57)) $x57) (quant-intro (refl (= $x54 $x54)) (= $x57 $x3461)) $x3461)))
+(let (($x6140 (or (not $x3461) $x3136)))
+(let ((@x6106 (monotonicity (rewrite (= (= $x3136 true) $x3136)) (= (or (not $x3461) (= $x3136 true)) $x6140))))
+(let ((@x5837 (trans @x6106 (rewrite (= $x6140 $x6140)) (= (or (not $x3461) (= $x3136 true)) $x6140))))
+(let ((@x5928 (mp ((_ quant-inst v_b_Visited_G_1$ v_b_v_G_1$ true) (or (not $x3461) (= $x3136 true))) @x5837 $x6140)))
+(let ((@x7482 (mp (unit-resolution @x5928 @x3466 $x3136) (monotonicity @x5875 (= $x3136 $x4126)) $x4126)))
+(let (($x4570 (>= ?x4546 0)))
+(let ((@x5420 (unit-resolution ((_ th-lemma arith farkas 1 1) (or $x4570 $x4569)) (hypothesis (not $x4569)) $x4570)))
+(let (($x4438 (<= (+ b_Infinity$ ?x4436) 0)))
+(let (($x4127 (not $x4126)))
+(let (($x5352 (or $x3725 $x4127 $x4438 $x4569)))
+(let (($x5336 (>= (+ ?x4435 ?x3104 (* (- 1) ?x1911)) 0)))
+(let (($x5339 (or $x4127 $x4438 $x5336)))
+(let (($x5353 (or $x3725 $x5339)))
+(let ((@x5341 (rewrite (= (+ ?x4435 ?x3104 (* (- 1) ?x1911)) (+ (* (- 1) ?x1911) ?x3104 ?x4435)))))
+(let ((@x5344 (monotonicity @x5341 (= $x5336 (>= (+ (* (- 1) ?x1911) ?x3104 ?x4435) 0)))))
+(let ((@x5348 (trans @x5344 (rewrite (= (>= (+ (* (- 1) ?x1911) ?x3104 ?x4435) 0) $x4569)) (= $x5336 $x4569))))
+(let ((@x5357 (monotonicity (monotonicity @x5348 (= $x5339 (or $x4127 $x4438 $x4569))) (= $x5353 (or $x3725 (or $x4127 $x4438 $x4569))))))
+(let ((@x5361 (trans @x5357 (rewrite (= (or $x3725 (or $x4127 $x4438 $x4569)) $x5352)) (= $x5353 $x5352))))
+(let ((@x5424 (unit-resolution (mp ((_ quant-inst ?v0!20 v_b_v_G_1$) $x5353) @x5361 $x5352) (hypothesis $x3720) (hypothesis $x4126) (hypothesis (not $x4569)) $x4438)))
+(let ((@x5428 (lemma ((_ th-lemma arith farkas 1 1 1 1) @x5424 (hypothesis $x4161) @x5420 (hypothesis $x1915) false) (or $x4569 (not $x4161) $x1914 $x3725 $x4127))))
+(let ((@x7692 (unit-resolution (unit-resolution @x5428 @x7482 (or $x4569 (not $x4161) $x1914 $x3725)) (unit-resolution @x4337 (unit-resolution @x3367 @x9294 $x3703) $x4161) (or $x4569 $x1914 $x3725))))
+(let ((@x7751 (unit-resolution @x7692 (unit-resolution (def-axiom (or $x3737 $x1915)) @x8092 $x1915) (unit-resolution @x3222 @x8092 $x3720) $x4569)))
+(let (($x5386 (= v_b_v_G_1$ ?v0!20)))
+(let (($x5390 (not $x5386)))
+(let ((@x9325 (symm (commutativity (= $x5386 (= ?v0!20 v_b_v_G_1$))) (= (= ?v0!20 v_b_v_G_1$) $x5386))))
+(let (($x5240 (= ?v0!20 v_b_v_G_1$)))
+(let (($x9145 (not $x5240)))
+(let (($x4609 (fun_app$ v_b_Visited_G_1$ ?v0!20)))
+(let (($x9130 (or $x5240 $x4609)))
+(let (($x5237 (fun_app$ ?x265 ?v0!20)))
+(let (($x9133 (= $x5237 $x9130)))
+(let (($x9136 (or $x4114 $x9133)))
+(let ((@x9135 (monotonicity (rewrite (= (ite $x5240 true $x4609) $x9130)) (= (= $x5237 (ite $x5240 true $x4609)) $x9133))))
+(let ((@x9140 (monotonicity @x9135 (= (or $x4114 (= $x5237 (ite $x5240 true $x4609))) $x9136))))
+(let ((@x9143 (trans @x9140 (rewrite (= $x9136 $x9136)) (= (or $x4114 (= $x5237 (ite $x5240 true $x4609))) $x9136))))
+(let ((@x9144 (mp ((_ quant-inst v_b_Visited_G_1$ v_b_v_G_1$ true ?v0!20) (or $x4114 (= $x5237 (ite $x5240 true $x4609)))) @x9143 $x9136)))
+(let ((@x9316 (symm (monotonicity @x5875 (= $x5237 (fun_app$ v_b_Visited_G_2$ ?v0!20))) (= (fun_app$ v_b_Visited_G_2$ ?v0!20) $x5237))))
+(let ((@x9318 (monotonicity @x9316 (= (not (fun_app$ v_b_Visited_G_2$ ?v0!20)) (not $x5237)))))
+(let (($x4278 (fun_app$ v_b_Visited_G_2$ ?v0!20)))
+(let (($x4279 (not $x4278)))
+(let (($x4403 (or $x4279 $x4400)))
+(let ((@x8012 (mp ((_ quant-inst ?v0!20) (or $x3700 $x4403)) (rewrite (= (or $x3700 $x4403) (or $x3700 $x4279 $x4400))) (or $x3700 $x4279 $x4400))))
+(let ((@x9292 (unit-resolution (unit-resolution @x8012 @x7616 $x4403) (hypothesis (not $x4400)) $x4279)))
+(let ((@x9320 (unit-resolution (def-axiom (or (not $x9133) $x5237 (not $x9130))) (mp @x9292 @x9318 (not $x5237)) (unit-resolution @x9144 @x3473 $x9133) (not $x9130))))
+(let ((@x9328 (mp (unit-resolution (def-axiom (or $x9130 $x9145)) @x9320 $x9145) (monotonicity @x9325 (= $x9145 $x5390)) $x5390)))
+(let (($x5387 (<= ?x4435 0)))
+(let (($x5391 (= ?x4435 0)))
+(let ((?x3106 (+ ?x257 ?x3096 ?x3105)))
+(let (($x4239 (<= ?x3106 0)))
+(let ((?x3884 (+ ?x257 ?x3105)))
+(let (($x3885 (<= ?x3884 0)))
+(let (($x6004 (= ?x257 ?x3104)))
+(let ((@x7828 (mp (unit-resolution @x4259 @x5944 (unit-resolution @x4316 @x6019 $x4242) $x3052) (symm (commutativity (= $x6004 $x3052)) (= $x3052 $x6004)) $x6004)))
+(let (($x4177 (<= ?x3096 0)))
+(let ((@x6933 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x4785) $x4177)) @x4849 $x4177)))
+(let ((@x7838 (unit-resolution ((_ th-lemma arith assign-bounds 1 1) (or $x4239 (not $x3885) (not $x4177))) @x6933 (or $x4239 (not $x3885)))))
+(let ((@x7839 (unit-resolution @x7838 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x6004) $x3885)) @x7828 $x3885) $x4239)))
+(let (($x3044 (>= ?x3106 0)))
+(let (($x3886 (>= ?x3884 0)))
+(let (($x5927 (or $x3691 $x3886)))
+(let ((@x5941 ((_ quant-inst v_b_v_G_1$) $x5927)))
+(let ((@x6925 (unit-resolution @x5941 @x6892 $x3886)))
+(let ((@x6929 (unit-resolution ((_ th-lemma arith assign-bounds -1 -1) (or $x3044 $x4315 (not $x3886))) @x6019 (or $x3044 (not $x3886)))))
+(let ((@x6930 (unit-resolution @x6929 @x6925 $x3044)))
+(let ((?x4381 (+ ?x1911 ?x3105)))
+(let (($x7049 (<= ?x4381 0)))
+(let (($x7135 (= ?x4546 0)))
+(let ((?x1912 (* (- 1) ?x1911)))
+(let ((?x4487 (+ ?x257 ?x1912 ?x4435)))
+(let (($x4507 (<= ?x4487 0)))
+(let (($x5673 (= ?x4487 0)))
+(let (($x6827 (>= (+ ?x257 ?x4418 ?x4435) 0)))
+(let (($x6723 (or $x4438 $x6827)))
+(let (($x6684 (not $x6723)))
+(let (($x6831 (or $x6684 $x4400)))
+(let (($x6789 (or $x3683 $x6684 $x4400)))
+(let (($x4443 (or (not (or $x4438 (<= (+ ?x4393 ?x1173 ?x4436) 0))) $x4400)))
+(let (($x6790 (or $x3683 $x4443)))
+(let ((@x6945 (monotonicity (rewrite (= (+ ?x4393 ?x1173 ?x4436) (+ ?x1173 ?x4393 ?x4436))) (= (<= (+ ?x4393 ?x1173 ?x4436) 0) (<= (+ ?x1173 ?x4393 ?x4436) 0)))))
+(let ((@x6725 (trans @x6945 (rewrite (= (<= (+ ?x1173 ?x4393 ?x4436) 0) $x6827)) (= (<= (+ ?x4393 ?x1173 ?x4436) 0) $x6827))))
+(let ((@x6730 (monotonicity @x6725 (= (or $x4438 (<= (+ ?x4393 ?x1173 ?x4436) 0)) $x6723))))
+(let ((@x6830 (monotonicity @x6730 (= (not (or $x4438 (<= (+ ?x4393 ?x1173 ?x4436) 0))) $x6684))))
+(let ((@x6829 (monotonicity (monotonicity @x6830 (= $x4443 $x6831)) (= $x6790 (or $x3683 $x6831)))))
+(let ((@x6824 (mp ((_ quant-inst ?v0!20) $x6790) (trans @x6829 (rewrite (= (or $x3683 $x6831) $x6789)) (= $x6790 $x6789)) $x6789)))
+(let ((@x9281 (unit-resolution (unit-resolution @x6824 @x5944 $x6831) (hypothesis (not $x4400)) $x6684)))
+(let ((@x7436 (unit-resolution (def-axiom (or $x6723 (not $x4438))) (hypothesis $x6684) (not $x4438))))
+(let ((@x7494 (unit-resolution (def-axiom (or $x6723 (not $x6827))) (hypothesis $x6684) (not $x6827))))
+(let (($x6621 (or $x4438 $x6827 $x5673)))
+(let (($x6987 (or $x3675 $x4438 $x6827 $x5673)))
+(let (($x4440 (<= (+ ?x4393 ?x1173 ?x4436) 0)))
+(let (($x4486 (or $x4438 $x4440 (= (+ ?x257 ?x4435 ?x1912) 0))))
+(let (($x6624 (or $x3675 $x4486)))
+(let ((@x5324 (monotonicity (rewrite (= (+ ?x257 ?x4435 ?x1912) ?x4487)) (= (= (+ ?x257 ?x4435 ?x1912) 0) $x5673))))
+(let ((@x6996 (monotonicity (monotonicity @x6725 @x5324 (= $x4486 $x6621)) (= $x6624 (or $x3675 $x6621)))))
+(let ((@x7057 (mp ((_ quant-inst ?v0!20) $x6624) (trans @x6996 (rewrite (= (or $x3675 $x6621) $x6987)) (= $x6624 $x6987)) $x6987)))
+(let ((@x7649 (unit-resolution (unit-resolution @x7057 @x6588 $x6621) @x7494 @x7436 (hypothesis (not $x5673)) false)))
+(let ((@x7699 (lemma @x7649 (or $x6723 $x5673))))
+(let ((@x9285 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x5673) $x4507)) (unit-resolution @x7699 @x9281 $x5673) $x4507)))
+(let ((@x9287 (unit-resolution ((_ th-lemma arith assign-bounds 1 -1) (or (not $x4507) $x4570 (not $x3886))) @x6925 (or (not $x4507) $x4570))))
+(let ((@x7251 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x7135 (not $x4569) (not $x4570))) (hypothesis $x4569) (or $x7135 (not $x4570)))))
+(let (($x7151 (not $x7135)))
+(let (($x7157 (or $x3734 $x7049 $x4127 $x7151)))
+(let (($x4516 (>= (+ ?x3104 ?x1912) 0)))
+(let (($x4528 (or $x4516 $x4127 (not (= (+ ?x3104 ?x1912 ?x4435) 0)))))
+(let (($x7317 (or $x3734 $x4528)))
+(let ((@x7137 (monotonicity (rewrite (= (+ ?x3104 ?x1912 ?x4435) (+ ?x1912 ?x3104 ?x4435))) (= (= (+ ?x3104 ?x1912 ?x4435) 0) (= (+ ?x1912 ?x3104 ?x4435) 0)))))
+(let ((@x7149 (trans @x7137 (rewrite (= (= (+ ?x1912 ?x3104 ?x4435) 0) $x7135)) (= (= (+ ?x3104 ?x1912 ?x4435) 0) $x7135))))
+(let ((@x7063 (monotonicity (rewrite (= (+ ?x3104 ?x1912) (+ ?x1912 ?x3104))) (= $x4516 (>= (+ ?x1912 ?x3104) 0)))))
+(let ((@x7144 (trans @x7063 (rewrite (= (>= (+ ?x1912 ?x3104) 0) $x7049)) (= $x4516 $x7049))))
+(let ((@x7156 (monotonicity @x7144 (monotonicity @x7149 (= (not (= (+ ?x3104 ?x1912 ?x4435) 0)) $x7151)) (= $x4528 (or $x7049 $x4127 $x7151)))))
+(let ((@x7313 (trans (monotonicity @x7156 (= $x7317 (or $x3734 (or $x7049 $x4127 $x7151)))) (rewrite (= (or $x3734 (or $x7049 $x4127 $x7151)) $x7157)) (= $x7317 $x7157))))
+(let ((@x7502 (unit-resolution (mp ((_ quant-inst v_b_v_G_1$) $x7317) @x7313 $x7157) (hypothesis $x3729) @x7482 (or $x7049 $x7151))))
+(let ((@x9290 (unit-resolution @x7502 (unit-resolution @x7251 (unit-resolution @x9287 @x9285 $x4570) $x7135) $x7049)))
+(let (($x4382 (>= ?x4381 0)))
+(let (($x6813 (= ?v1!16 v_b_v_G_1$)))
+(let (($x7202 (= v_b_v_G_1$ ?v1!16)))
+(let ((?x6481 (pair$ v_b_v_G_1$ ?v1!16)))
+(let ((?x6374 (b_G$ ?x6481)))
+(let (($x7203 (<= ?x6374 0)))
+(let ((?x1866 (v_b_SP_G_2$ ?v0!17)))
+(let ((?x6890 (+ ?x1866 ?x3105)))
+(let (($x6886 (<= ?x6890 0)))
+(let ((?x4496 (fun_app$c v_b_SP_G_1$ ?v0!17)))
+(let ((?x6307 (* (- 1) ?x4496)))
+(let ((?x5972 (+ ?x257 ?x6307)))
+(let (($x7220 (>= ?x5972 0)))
+(let (($x3187 (fun_app$ v_b_Visited_G_1$ ?v0!17)))
+(let (($x4478 (= ?v0!17 v_b_v_G_1$)))
+(let (($x4499 (or $x4478 $x3187)))
+(let (($x4471 (fun_app$ ?x265 ?v0!17)))
+(let (($x4593 (= $x4471 $x4499)))
+(let (($x4712 (or $x4114 $x4593)))
+(let ((@x4495 (monotonicity (rewrite (= (ite $x4478 true $x3187) $x4499)) (= (= $x4471 (ite $x4478 true $x3187)) $x4593))))
+(let ((@x5371 (monotonicity @x4495 (= (or $x4114 (= $x4471 (ite $x4478 true $x3187))) $x4712))))
+(let ((@x5958 (trans @x5371 (rewrite (= $x4712 $x4712)) (= (or $x4114 (= $x4471 (ite $x4478 true $x3187))) $x4712))))
+(let ((@x6125 (mp ((_ quant-inst v_b_Visited_G_1$ v_b_v_G_1$ true ?v0!17) (or $x4114 (= $x4471 (ite $x4478 true $x3187)))) @x5958 $x4712)))
+(let ((@x8166 (mp (unit-resolution (def-axiom (or $x2760 $x1862)) (hypothesis $x2765) $x1862) (symm (monotonicity @x5875 (= $x4471 $x1862)) (= $x1862 $x4471)) $x4471)))
+(let ((@x8237 (unit-resolution (def-axiom (or (not $x4593) (not $x4471) $x4499)) @x8166 (unit-resolution @x6125 @x3473 $x4593) $x4499)))
+(let (($x6485 (not $x4478)))
+(let (($x8046 (<= (+ ?x257 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v1!16))) 0)))
+(let (($x6814 (fun_app$ v_b_Visited_G_1$ ?v1!16)))
+(let (($x8334 (or $x6813 $x6814)))
+(let (($x6812 (fun_app$ ?x265 ?v1!16)))
+(let (($x7683 (= $x6812 $x8334)))
+(let (($x6622 (or $x4114 $x7683)))
+(let ((@x6719 (monotonicity (rewrite (= (ite $x6813 true $x6814) $x8334)) (= (= $x6812 (ite $x6813 true $x6814)) $x7683))))
+(let ((@x8777 (monotonicity @x6719 (= (or $x4114 (= $x6812 (ite $x6813 true $x6814))) $x6622))))
+(let ((@x8650 (trans @x8777 (rewrite (= $x6622 $x6622)) (= (or $x4114 (= $x6812 (ite $x6813 true $x6814))) $x6622))))
+(let ((@x8651 (mp ((_ quant-inst v_b_Visited_G_1$ v_b_v_G_1$ true ?v1!16) (or $x4114 (= $x6812 (ite $x6813 true $x6814)))) @x8650 $x6622)))
+(let ((@x8121 (monotonicity (symm (monotonicity @x5875 (= $x6812 $x1860)) (= $x1860 $x6812)) (= (not $x1860) (not $x6812)))))
+(let (($x1861 (not $x1860)))
+(let ((@x7803 (hypothesis $x2765)))
+(let ((@x8141 (mp (unit-resolution (def-axiom (or $x2760 $x1861)) @x7803 $x1861) @x8121 (not $x6812))))
+(let ((@x8147 (unit-resolution (def-axiom (or (not $x7683) $x6812 (not $x8334))) @x8141 (unit-resolution @x8651 @x3473 $x7683) (not $x8334))))
+(let (($x8156 (or $x6814 $x8046)))
+(let (($x8160 (or $x3665 $x6814 $x8046)))
+(let (($x6666 (>= (+ (fun_app$c v_b_SP_G_1$ ?v1!16) ?x1173) 0)))
+(let (($x6673 (or $x6814 $x6666)))
+(let (($x8163 (or $x3665 $x6673)))
+(let ((@x7990 (rewrite (= (>= (+ ?x1173 (fun_app$c v_b_SP_G_1$ ?v1!16)) 0) $x8046))))
+(let (($x8213 (= (+ (fun_app$c v_b_SP_G_1$ ?v1!16) ?x1173) (+ ?x1173 (fun_app$c v_b_SP_G_1$ ?v1!16)))))
+(let ((@x8047 (monotonicity (rewrite $x8213) (= $x6666 (>= (+ ?x1173 (fun_app$c v_b_SP_G_1$ ?v1!16)) 0)))))
+(let ((@x8089 (monotonicity (monotonicity (trans @x8047 @x7990 (= $x6666 $x8046)) (= $x6673 $x8156)) (= $x8163 (or $x3665 $x8156)))))
+(let ((@x8093 (mp ((_ quant-inst ?v1!16) $x8163) (trans @x8089 (rewrite (= (or $x3665 $x8156) $x8160)) (= $x8163 $x8160)) $x8160)))
+(let ((@x8217 (unit-resolution @x8093 (unit-resolution (def-axiom (or $x3809 $x3660)) @x6181 $x3660) $x8156)))
+(let ((@x8239 (unit-resolution @x8217 (unit-resolution (def-axiom (or $x8334 (not $x6814))) @x8147 (not $x6814)) $x8046)))
+(let (($x3386 (not $x1869)))
+(let ((@x3390 (def-axiom (or $x2760 $x3386))))
+(let ((@x8240 (unit-resolution @x3390 @x7803 $x3386)))
+(let ((?x6009 (pair$ v_b_v_G_1$ ?v0!17)))
+(let ((?x6010 (b_G$ ?x6009)))
+(let ((?x1867 (* (- 1) ?x1866)))
+(let ((?x6187 (+ ?x257 ?x1867 ?x6010)))
+(let ((@x8743 (monotonicity (monotonicity (hypothesis $x4478) (= ?x6009 ?x3130)) (= ?x6010 ?x3096))))
+(let (($x6889 (= ?x1866 ?x3104)))
+(let ((@x6922 (hypothesis $x4478)))
+(let ((@x6921 (unit-resolution (hypothesis (not $x6889)) (monotonicity @x6922 $x6889) false)))
+(let ((@x6939 (lemma @x6921 (or $x6485 $x6889))))
+(let ((@x6214 ((_ th-lemma arith triangle-eq) (or (not $x6889) $x6886))))
+(let (($x7675 (>= ?x6890 0)))
+(let ((@x8362 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x6889) $x7675)) (unit-resolution @x6939 @x6922 $x6889) $x7675)))
+(let ((@x7970 ((_ th-lemma arith eq-propagate 1 1 1 1 -1 -1) @x8362 (unit-resolution @x6214 (unit-resolution @x6939 @x6922 $x6889) $x6886) @x6019 @x6933 @x6930 @x7839 (= ?x6010 ?x6187))))
+(let ((@x8765 (trans (trans (symm @x7970 (= ?x6187 ?x6010)) @x8743 (= ?x6187 ?x3096)) @x4849 (= ?x6187 0))))
+(let (($x6564 (>= ?x6187 0)))
+(let (($x7274 (not $x6564)))
+(let ((@x7271 (hypothesis $x3386)))
+(let ((?x1865 (v_b_SP_G_2$ ?v1!16)))
+(let ((?x6126 (* (- 1) ?x1865)))
+(let ((?x6400 (+ ?x257 ?x6126 ?x6374)))
+(let (($x6319 (<= ?x6400 0)))
+(let (($x8008 (= ?x6400 0)))
+(let (($x6238 (<= (+ b_Infinity$ (* (- 1) ?x6374)) 0)))
+(let (($x8646 (not $x6238)))
+(let (($x7241 (>= (+ ?x257 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v1!16)) ?x6374) 0)))
+(let (($x7239 (or $x6238 $x7241)))
+(let (($x4416 (not $x7239)))
+(let ((?x6234 (fun_app$c v_b_SP_G_1$ ?v1!16)))
+(let (($x6378 (= ?x1865 ?x6234)))
+(let (($x8565 (not $x6378)))
+(let (($x8664 (>= (+ ?x1865 (* (- 1) ?x6234)) 0)))
+(let (($x8549 (not $x8664)))
+(let ((@x8517 ((_ th-lemma arith assign-bounds -1 -1 -1 -1 1) (or $x8549 (not $x8046) $x1869 (not $x6886) (not $x4177) (not $x3044)))))
+(let ((@x8321 (unit-resolution @x8517 (unit-resolution @x6214 (unit-resolution @x6939 @x6922 $x6889) $x6886) @x6933 @x6930 @x7271 (hypothesis $x8046) $x8549)))
+(let (($x8358 (or $x4416 $x6378)))
+(let (($x8640 (or $x3683 $x4416 $x6378)))
+(let (($x6219 (or (not (or $x6238 (<= (+ ?x6234 ?x1173 (* (- 1) ?x6374)) 0))) $x6378)))
+(let (($x8252 (or $x3683 $x6219)))
+(let (($x6539 (<= (+ ?x6234 ?x1173 (* (- 1) ?x6374)) 0)))
+(let ((@x7664 (rewrite (= (+ ?x6234 ?x1173 (* (- 1) ?x6374)) (+ ?x1173 ?x6234 (* (- 1) ?x6374))))))
+(let ((@x7697 (monotonicity @x7664 (= $x6539 (<= (+ ?x1173 ?x6234 (* (- 1) ?x6374)) 0)))))
+(let ((@x4371 (trans @x7697 (rewrite (= (<= (+ ?x1173 ?x6234 (* (- 1) ?x6374)) 0) $x7241)) (= $x6539 $x7241))))
+(let ((@x8352 (monotonicity (monotonicity @x4371 (= (or $x6238 $x6539) $x7239)) (= (not (or $x6238 $x6539)) $x4416))))
+(let ((@x8173 (monotonicity (monotonicity @x8352 (= $x6219 $x8358)) (= $x8252 (or $x3683 $x8358)))))
+(let ((@x8649 (mp ((_ quant-inst ?v1!16) $x8252) (trans @x8173 (rewrite (= (or $x3683 $x8358) $x8640)) (= $x8252 $x8640)) $x8640)))
+(let ((@x8632 (unit-resolution (unit-resolution @x8649 @x5944 $x8358) (unit-resolution ((_ th-lemma arith triangle-eq) (or $x8565 $x8664)) @x8321 $x8565) $x4416)))
+(let (($x8029 (or $x6238 $x7241 $x8008)))
+(let (($x8118 (or $x3675 $x6238 $x7241 $x8008)))
+(let (($x6399 (or $x6238 $x6539 (= (+ ?x257 ?x6374 ?x6126) 0))))
+(let (($x8113 (or $x3675 $x6399)))
+(let ((@x8010 (monotonicity (rewrite (= (+ ?x257 ?x6374 ?x6126) ?x6400)) (= (= (+ ?x257 ?x6374 ?x6126) 0) $x8008))))
+(let ((@x5909 (monotonicity (monotonicity @x4371 @x8010 (= $x6399 $x8029)) (= $x8113 (or $x3675 $x8029)))))
+(let ((@x7712 (mp ((_ quant-inst ?v1!16) $x8113) (trans @x5909 (rewrite (= (or $x3675 $x8029) $x8118)) (= $x8113 $x8118)) $x8118)))
+(let ((@x8635 (unit-resolution (unit-resolution @x7712 @x6588 $x8029) (unit-resolution (def-axiom (or $x7239 (not $x7241))) @x8632 (not $x7241)) (unit-resolution (def-axiom (or $x7239 $x8646)) @x8632 $x8646) $x8008)))
+(let ((@x7288 (monotonicity (commutativity (= (= v_b_v_G_1$ ?v0!17) $x4478)) (= (not (= v_b_v_G_1$ ?v0!17)) $x6485))))
+(let (($x7176 (= v_b_v_G_1$ ?v0!17)))
+(let (($x7180 (not $x7176)))
+(let (($x7177 (<= ?x6010 0)))
+(let (($x7178 (not $x7177)))
+(let (($x7206 (not $x7203)))
+(let ((@x7267 (monotonicity (symm (commutativity (= $x7202 $x6813)) (= $x6813 $x7202)) (= (not $x6813) (not $x7202)))))
+(let (($x7207 (or $x7202 $x7206)))
+(let ((@x7215 (mp ((_ quant-inst v_b_v_G_1$ ?v1!16) (or (not $x3480) $x7207)) (rewrite (= (or (not $x3480) $x7207) (or (not $x3480) $x7202 $x7206))) (or (not $x3480) $x7202 $x7206))))
+(let ((@x7270 (unit-resolution (unit-resolution @x7215 @x3485 $x7207) (mp (hypothesis (not $x6813)) @x7267 (not $x7202)) $x7206)))
+(let ((@x7278 (unit-resolution ((_ th-lemma arith assign-bounds 1 1 1 1) (or $x7178 $x7274 $x1869 $x7203 (not $x6319))) (hypothesis $x6319) (hypothesis $x6564) @x7271 @x7270 $x7178)))
+(let ((@x7282 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x6010 0)) $x7177)) @x7278 (not (= ?x6010 0)))))
+(let (($x7181 (= ?x6010 0)))
+(let (($x7188 (or $x7180 $x7181)))
+(let ((@x7196 (mp ((_ quant-inst v_b_v_G_1$ ?v0!17) (or $x3151 $x7188)) (rewrite (= (or $x3151 $x7188) (or $x3151 $x7180 $x7181))) (or $x3151 $x7180 $x7181))))
+(let ((@x7289 (mp (unit-resolution (unit-resolution @x7196 @x3479 $x7188) @x7282 $x7180) @x7288 $x6485)))
+(let ((@x5812 (def-axiom (or (not $x4499) $x4478 $x3187))))
+(let (($x7229 (= (or $x3570 (or $x255 (not $x3187) $x7220)) (or $x3570 $x255 (not $x3187) $x7220))))
+(let ((@x7231 (mp ((_ quant-inst ?v0!17 v_b_v_G_1$) (or $x3570 (or $x255 (not $x3187) $x7220))) (rewrite $x7229) (or $x3570 $x255 (not $x3187) $x7220))))
+(let ((@x7291 (unit-resolution @x7231 @x5748 @x6225 (unit-resolution @x5812 @x7289 (hypothesis $x4499) $x3187) $x7220)))
+(let (($x6327 (<= (+ ?x1866 ?x6307) 0)))
+(let (($x6088 (or $x3691 $x6327)))
+(let ((@x6464 (monotonicity (rewrite (= (+ ?x4496 ?x1867) (+ ?x1867 ?x4496))) (= (>= (+ ?x4496 ?x1867) 0) (>= (+ ?x1867 ?x4496) 0)))))
+(let ((@x5905 (trans @x6464 (rewrite (= (>= (+ ?x1867 ?x4496) 0) $x6327)) (= (>= (+ ?x4496 ?x1867) 0) $x6327))))
+(let ((@x5843 (trans (monotonicity @x5905 (= (or $x3691 (>= (+ ?x4496 ?x1867) 0)) $x6088)) (rewrite (= $x6088 $x6088)) (= (or $x3691 (>= (+ ?x4496 ?x1867) 0)) $x6088))))
+(let ((@x7292 (unit-resolution (mp ((_ quant-inst ?v0!17) (or $x3691 (>= (+ ?x4496 ?x1867) 0))) @x5843 $x6088) @x6892 $x6327)))
+(let ((@x7295 (lemma ((_ th-lemma arith farkas 1 1 1 1 1) @x7292 @x7271 @x7270 (hypothesis $x6319) @x7291 false) (or (not $x6319) $x1869 (not $x4499) $x7274 $x6813))))
+(let ((@x8734 (unit-resolution @x7295 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x8008) $x6319)) @x8635 $x6319) (hypothesis $x4499) (hypothesis (not $x6813)) @x7271 $x7274)))
+(let ((@x8324 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x6187 0)) $x6564)) @x8734 (not (= ?x6187 0)))))
+(let ((@x8494 (lemma (unit-resolution @x8324 @x8765 false) (or $x6485 (not $x4499) $x6813 $x1869 (not $x8046)))))
+(let ((@x8211 (unit-resolution @x8494 @x8237 (unit-resolution (def-axiom (or $x8334 (not $x6813))) @x8147 (not $x6813)) @x8240 @x8239 $x6485)))
+(let ((@x8909 (unit-resolution @x7231 @x5748 @x6225 (hypothesis $x3187) (hypothesis (not $x7220)) false)))
+(let ((@x8256 (unit-resolution (lemma @x8909 (or (not $x3187) $x7220)) (unit-resolution @x5812 @x8211 @x8237 $x3187) $x7220)))
+(let ((@x8314 (unit-resolution ((_ th-lemma arith assign-bounds 1 -1 1 -1) (or $x6886 (not $x7220) (not $x6327) $x4315 (not $x4239))) @x7292 @x7839 @x8256 @x6019 $x6886)))
+(let ((@x8385 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x8565 $x8664)) (unit-resolution @x8517 @x8314 @x6933 @x6930 @x8240 @x8239 $x8549) $x8565)))
+(let ((@x8386 (unit-resolution (def-axiom (or $x7239 $x8646)) (unit-resolution (unit-resolution @x8649 @x5944 $x8358) @x8385 $x4416) $x8646)))
+(let (($x8654 (not $x7241)))
+(let ((@x8390 (unit-resolution (def-axiom (or $x7239 $x8654)) (unit-resolution (unit-resolution @x8649 @x5944 $x8358) @x8385 $x4416) $x8654)))
+(let ((@x8410 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x8008) $x6319)) (unit-resolution (unit-resolution @x7712 @x6588 $x8029) @x8390 @x8386 $x8008) $x6319)))
+(let ((@x8411 ((_ th-lemma arith assign-bounds 1 1 1 1 1) (or $x7203 (not $x6319) $x1869 (not $x6886) (not $x4177) (not $x3044)))))
+(let ((@x8413 (unit-resolution @x7215 @x3485 (unit-resolution @x8411 @x8410 @x6933 @x6930 @x8240 @x8314 $x7203) $x7202)))
+(let ((@x8417 (unit-resolution (unit-resolution (def-axiom (or $x8334 (not $x6813))) @x8147 (not $x6813)) (symm @x8413 $x6813) false)))
+(let ((@x3365 (def-axiom (or $x3758 $x2765 $x3752))))
+(let ((@x9296 (unit-resolution @x3365 (lemma @x8417 $x2760) (unit-resolution (def-axiom (or $x3761 $x3755)) @x9294 $x3755) $x3752)))
+(let ((@x8225 (rewrite (= (or $x3717 (or $x4278 $x4127 $x4382)) (or $x3717 $x4278 $x4127 $x4382)))))
+(let ((@x8229 (mp ((_ quant-inst v_b_v_G_1$ ?v0!20) (or $x3717 (or $x4278 $x4127 $x4382))) @x8225 (or $x3717 $x4278 $x4127 $x4382))))
+(let ((@x9299 (unit-resolution @x8229 (unit-resolution (def-axiom (or $x3749 $x3712)) @x9296 $x3712) @x7482 (or $x4278 $x4382))))
+(let (($x4508 (>= ?x4487 0)))
+(let ((@x9304 (unit-resolution ((_ th-lemma arith assign-bounds 1 -1) (or $x4508 (not $x4569) (not $x3886))) @x6925 (or $x4508 (not $x4569)))))
+(let ((@x9306 ((_ th-lemma arith eq-propagate -1 -1 -1 -1 -1 -1 1 1) (unit-resolution @x9304 (hypothesis $x4569) $x4508) @x9285 (unit-resolution @x9299 @x9292 $x4382) @x9290 @x6019 @x6933 @x6930 @x7839 $x5391)))
+(let (($x5388 (not $x5387)))
+(let (($x5389 (or $x5386 $x5388)))
+(let ((@x7598 (mp ((_ quant-inst v_b_v_G_1$ ?v0!20) (or (not $x3480) $x5389)) (rewrite (= (or (not $x3480) $x5389) (or (not $x3480) $x5386 $x5388))) (or (not $x3480) $x5386 $x5388))))
+(let ((@x9311 (unit-resolution (unit-resolution @x7598 @x3485 $x5389) (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x5391) $x5387)) @x9306 $x5387) $x5386)))
+(let ((@x8045 (unit-resolution (lemma (unit-resolution @x9311 @x9328 false) (or $x4400 $x3734 (not $x4569))) (unit-resolution (def-axiom (or $x3737 $x3729)) @x8092 $x3729) @x7751 $x4400)))
+(let ((@x8812 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x4400) $x5977)) @x8045 $x5977)))
+(let ((?x4641 (?v1!7 ?v0!20)))
+(let ((?x4648 (pair$ ?x4641 ?v0!20)))
+(let ((?x4649 (b_G$ ?x4648)))
+(let ((?x4650 (* (- 1) ?x4649)))
+(let ((?x4642 (fun_app$c v_b_SP_G_1$ ?x4641)))
+(let ((?x4643 (* (- 1) ?x4642)))
+(let ((?x4651 (+ ?x4393 ?x4643 ?x4650)))
+(let (($x4391 (>= ?x4651 0)))
+(let (($x4652 (= ?x4651 0)))
+(let (($x4653 (not $x4652)))
+(let (($x4646 (fun_app$ v_b_Visited_G_1$ ?x4641)))
+(let (($x4647 (not $x4646)))
+(let ((?x4644 (+ ?x4393 ?x4643)))
+(let (($x4645 (<= ?x4644 0)))
+(let (($x4654 (or $x4645 $x4647 $x4653)))
+(let (($x4655 (not $x4654)))
+(let (($x4640 (<= (+ b_Infinity$ ?x4418) 0)))
+(let (($x7886 (not $x4640)))
+(let ((@x8816 (unit-resolution ((_ th-lemma arith assign-bounds 1 -1) (or (not $x5977) $x1914 $x7886)) @x8812 (unit-resolution (def-axiom (or $x3737 $x1915)) @x8092 $x1915) $x7886)))
+(let ((@x7414 (rewrite (= (or $x3586 (or $x1909 $x4640 $x4655)) (or $x3586 $x1909 $x4640 $x4655)))))
+(let ((@x7415 (mp ((_ quant-inst ?v0!20) (or $x3586 (or $x1909 $x4640 $x4655))) @x7414 (or $x3586 $x1909 $x4640 $x4655))))
+(let ((@x8817 (unit-resolution @x7415 @x4545 (unit-resolution (def-axiom (or $x3737 $x1910)) @x8092 $x1910) (or $x4640 $x4655))))
+(let ((@x8826 (unit-resolution @x8817 @x8816 $x4655)))
+(let ((@x6085 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x4653 $x4391)) (unit-resolution (def-axiom (or $x4654 $x4652)) @x8826 $x4652) $x4391)))
+(let (($x7707 (<= ?x4651 0)))
+(let ((@x8177 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x4653 $x7707)) (unit-resolution (def-axiom (or $x4654 $x4652)) @x8826 $x4652) $x7707)))
+(let (($x4689 (fun_app$ v_b_Visited_G_2$ ?x4641)))
+(let ((@x6032 (monotonicity (symm (hypothesis $x266) (= ?x265 v_b_Visited_G_2$)) (= (fun_app$ ?x265 ?x4641) $x4689))))
+(let ((@x6036 (monotonicity (symm @x6032 (= $x4689 (fun_app$ ?x265 ?x4641))) (= (not $x4689) (not (fun_app$ ?x265 ?x4641))))))
+(let (($x5978 (fun_app$ ?x265 ?x4641)))
+(let (($x5985 (= ?x4641 v_b_v_G_1$)))
+(let (($x5988 (or $x5985 $x4646)))
+(let (($x5991 (= $x5978 $x5988)))
+(let (($x5994 (or $x4114 $x5991)))
+(let ((@x5993 (monotonicity (rewrite (= (ite $x5985 true $x4646) $x5988)) (= (= $x5978 (ite $x5985 true $x4646)) $x5991))))
+(let ((@x5998 (monotonicity @x5993 (= (or $x4114 (= $x5978 (ite $x5985 true $x4646))) $x5994))))
+(let ((@x6001 (trans @x5998 (rewrite (= $x5994 $x5994)) (= (or $x4114 (= $x5978 (ite $x5985 true $x4646))) $x5994))))
+(let ((@x6002 (mp ((_ quant-inst v_b_Visited_G_1$ v_b_v_G_1$ true (?v1!7 ?v0!20)) (or $x4114 (= $x5978 (ite $x5985 true $x4646)))) @x6001 $x5994)))
+(let ((@x6025 (unit-resolution (def-axiom (or (not $x5991) $x5978 (not $x5988))) (unit-resolution (def-axiom (or $x5988 $x4647)) (hypothesis $x4646) $x5988) (or (not $x5991) $x5978))))
+(let ((@x6038 (unit-resolution (unit-resolution @x6025 (unit-resolution @x6002 @x3473 $x5991) $x5978) (mp (hypothesis (not $x4689)) @x6036 (not $x5978)) false)))
+(let ((@x8986 (unit-resolution (lemma @x6038 (or $x4689 $x2935 $x4647)) (unit-resolution (def-axiom (or $x3809 $x266)) @x6181 $x266) (or $x4689 $x4647))))
+(let ((@x8987 (unit-resolution @x8986 (unit-resolution (def-axiom (or $x4654 $x4646)) @x8826 $x4646) $x4689)))
+(let ((?x4697 (v_b_SP_G_2$ ?x4641)))
+(let ((?x4700 (* (- 1) ?x4697)))
+(let ((?x4868 (+ ?x1911 ?x4700)))
+(let (($x9248 (<= ?x4868 0)))
+(let (($x8507 (not $x9248)))
+(let ((?x4701 (+ ?x4642 ?x4700)))
+(let (($x4708 (>= ?x4701 0)))
+(let ((@x8348 (unit-resolution ((_ th-lemma arith assign-bounds -1 -1 -1) (or $x8507 (not $x4708) $x4645 (not $x5977))) @x8812 (unit-resolution ((_ quant-inst (?v1!7 ?v0!20)) (or $x3691 $x4708)) @x6892 $x4708) (unit-resolution (def-axiom (or $x4654 (not $x4645))) @x8826 (not $x4645)) $x8507)))
+(let ((?x8311 (+ ?x1911 ?x4650 ?x4700)))
+(let (($x8266 (>= ?x8311 0)))
+(let ((@x10143 (unit-resolution ((_ th-lemma arith assign-bounds -1 -1 -1) (or $x8266 (not $x4391) (not $x4708) (not $x5977))) (unit-resolution ((_ quant-inst (?v1!7 ?v0!20)) (or $x3691 $x4708)) @x6892 $x4708) (hypothesis $x4391) (hypothesis $x5977) $x8266)))
+(let (($x8534 (<= ?x8311 0)))
+(let (($x5038 (<= ?x4701 0)))
+(let (($x5863 (= ?x4642 ?x4697)))
+(let ((@x10149 (symm (commutativity (= $x5863 (= ?x4697 ?x4642))) (= (= ?x4697 ?x4642) $x5863))))
+(let (($x4698 (= ?x4697 ?x4642)))
+(let ((@x7939 (rewrite (= (or $x3700 (or (not $x4689) $x4698)) (or $x3700 (not $x4689) $x4698)))))
+(let ((@x7943 (mp ((_ quant-inst (?v1!7 ?v0!20)) (or $x3700 (or (not $x4689) $x4698))) @x7939 (or $x3700 (not $x4689) $x4698))))
+(let ((@x7980 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x5863) $x5038)) (mp (unit-resolution @x7943 @x7616 (hypothesis $x4689) $x4698) @x10149 $x5863) $x5038)))
+(let (($x8014 (<= ?x4419 0)))
+(let (($x8221 (or $x3691 $x8014)))
+(let ((@x8001 (monotonicity (rewrite (= (+ ?x4393 ?x1912) (+ ?x1912 ?x4393))) (= (>= (+ ?x4393 ?x1912) 0) (>= (+ ?x1912 ?x4393) 0)))))
+(let ((@x8035 (trans @x8001 (rewrite (= (>= (+ ?x1912 ?x4393) 0) $x8014)) (= (>= (+ ?x4393 ?x1912) 0) $x8014))))
+(let ((@x8178 (trans (monotonicity @x8035 (= (or $x3691 (>= (+ ?x4393 ?x1912) 0)) $x8221)) (rewrite (= $x8221 $x8221)) (= (or $x3691 (>= (+ ?x4393 ?x1912) 0)) $x8221))))
+(let ((@x8659 (unit-resolution (mp ((_ quant-inst ?v0!20) (or $x3691 (>= (+ ?x4393 ?x1912) 0))) @x8178 $x8221) @x6892 $x8014)))
+(let ((@x8083 (unit-resolution ((_ th-lemma arith assign-bounds -1 -1 -1) (or $x8534 (not $x7707) (not $x5038) (not $x8014))) @x8659 (hypothesis $x7707) @x7980 $x8534)))
+(let (($x9251 (= ?x8311 0)))
+(let (($x8749 (not $x9251)))
+(let (($x4690 (not $x4689)))
+(let (($x8567 (or $x3734 $x9248 $x4690 $x8749)))
+(let (($x4857 (>= (+ ?x4697 ?x1912) 0)))
+(let (($x4861 (or $x4857 $x4690 (not (= (+ ?x4697 ?x1912 ?x4649) 0)))))
+(let (($x8927 (or $x3734 $x4861)))
+(let ((@x8955 (monotonicity (rewrite (= (+ ?x4697 ?x1912 ?x4649) (+ ?x1912 ?x4649 ?x4697))) (= (= (+ ?x4697 ?x1912 ?x4649) 0) (= (+ ?x1912 ?x4649 ?x4697) 0)))))
+(let ((@x8627 (trans @x8955 (rewrite (= (= (+ ?x1912 ?x4649 ?x4697) 0) $x9251)) (= (= (+ ?x4697 ?x1912 ?x4649) 0) $x9251))))
+(let ((@x8965 (monotonicity (rewrite (= (+ ?x4697 ?x1912) (+ ?x1912 ?x4697))) (= $x4857 (>= (+ ?x1912 ?x4697) 0)))))
+(let ((@x8985 (trans @x8965 (rewrite (= (>= (+ ?x1912 ?x4697) 0) $x9248)) (= $x4857 $x9248))))
+(let ((@x9087 (monotonicity @x8985 (monotonicity @x8627 (= (not (= (+ ?x4697 ?x1912 ?x4649) 0)) $x8749)) (= $x4861 (or $x9248 $x4690 $x8749)))))
+(let ((@x8874 (trans (monotonicity @x9087 (= $x8927 (or $x3734 (or $x9248 $x4690 $x8749)))) (rewrite (= (or $x3734 (or $x9248 $x4690 $x8749)) $x8567)) (= $x8927 $x8567))))
+(let ((@x8397 (unit-resolution (mp ((_ quant-inst (?v1!7 ?v0!20)) $x8927) @x8874 $x8567) (hypothesis $x3729) (hypothesis $x4689) (or $x9248 $x8749))))
+(let ((@x5592 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x9251 (not $x8534) (not $x8266))) (unit-resolution @x8397 (hypothesis $x8507) $x8749) @x8083 @x10143 false)))
+(let ((@x8013 (unit-resolution (lemma @x5592 (or $x9248 $x3734 $x4690 (not $x7707) (not $x4391) (not $x5977))) @x8348 (unit-resolution (def-axiom (or $x3737 $x3729)) @x8092 $x3729) @x8987 @x8177 @x6085 @x8812 false)))
+(let ((@x3278 (def-axiom (or $x3746 $x2811 $x3740))))
+(let ((@x8433 (unit-resolution @x3278 (unit-resolution (def-axiom (or $x3749 $x3743)) @x9296 $x3743) $x3743)))
+(let (($x3378 (not $x1896)))
+(let ((@x3380 (def-axiom (or $x2806 $x3378))))
+(let ((@x8434 (unit-resolution @x3380 (unit-resolution @x8433 (lemma @x8013 $x3737) $x2811) $x3378)))
+(let ((?x6619 (fun_app$c v_b_SP_G_1$ ?v1!18)))
+(let (($x6615 (= ?x1892 ?x6619)))
+(let (($x7618 (not $x6615)))
+(let ((@x7591 (hypothesis $x2811)))
+(let ((@x7607 (unit-resolution (def-axiom (or $x2806 $x1883)) @x7591 $x1883)))
+(let ((@x7571 (hypothesis $x3378)))
+(let (($x1889 (not $x1888)))
+(let ((@x7592 (unit-resolution (def-axiom (or $x2806 $x1889)) @x7591 $x1889)))
+(let ((?x7110 (pair$ v_b_v_G_1$ ?v0!19)))
+(let ((?x7111 (b_G$ ?x7110)))
+(let ((?x7100 (* (- 1) ?x7111)))
+(let ((?x7554 (+ ?x1885 ?x7100)))
+(let (($x7556 (>= ?x7554 0)))
+(let (($x7003 (= ?x1885 ?x7111)))
+(let (($x7243 (= ?v1!18 v_b_v_G_1$)))
+(let (($x7246 (fun_app$ v_b_Visited_G_1$ ?v1!18)))
+(let (($x6211 (not $x7246)))
+(let (($x7248 (>= (+ ?x1885 ?x6619 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0!19))) 0)))
+(let (($x7499 (not $x7248)))
+(let ((?x6721 (* (- 1) ?x6619)))
+(let ((?x5600 (+ ?x1892 ?x6721)))
+(let (($x7353 (>= ?x5600 0)))
+(let ((@x8658 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x7618 $x7353)) (hypothesis $x6615) $x7353)))
+(let (($x7076 (<= (+ ?x1893 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0!19))) 0)))
+(let (($x7084 (or $x3691 $x7076)))
+(let (($x7081 (= (or $x3691 (>= (+ (fun_app$c v_b_SP_G_1$ ?v0!19) ?x1894) 0)) $x7084)))
+(let ((@x7078 (rewrite (= (>= (+ ?x1894 (fun_app$c v_b_SP_G_1$ ?v0!19)) 0) $x7076))))
+(let (($x7048 (>= (+ (fun_app$c v_b_SP_G_1$ ?v0!19) ?x1894) 0)))
+(let (($x7069 (= (+ (fun_app$c v_b_SP_G_1$ ?v0!19) ?x1894) (+ ?x1894 (fun_app$c v_b_SP_G_1$ ?v0!19)))))
+(let ((@x7073 (monotonicity (rewrite $x7069) (= $x7048 (>= (+ ?x1894 (fun_app$c v_b_SP_G_1$ ?v0!19)) 0)))))
+(let ((@x7090 (trans (monotonicity (trans @x7073 @x7078 (= $x7048 $x7076)) $x7081) (rewrite (= $x7084 $x7084)) $x7081)))
+(let ((@x7496 (unit-resolution (mp ((_ quant-inst ?v0!19) (or $x3691 $x7048)) @x7090 $x7084) @x6892 $x7076)))
+(let ((@x7501 (lemma ((_ th-lemma arith farkas 1 -1 -1 1) (hypothesis $x7248) @x7571 @x7496 (hypothesis $x7353) false) (or $x7499 $x1896 (not $x7353)))))
+(let ((@x6992 (rewrite (= (or $x3578 (or $x6211 $x1888 $x7248)) (or $x3578 $x6211 $x1888 $x7248)))))
+(let ((@x7051 (mp ((_ quant-inst ?v0!19 ?v1!18) (or $x3578 (or $x6211 $x1888 $x7248))) @x6992 (or $x3578 $x6211 $x1888 $x7248))))
+(let ((@x8673 (unit-resolution (unit-resolution @x7051 @x4223 (hypothesis $x1889) (or $x6211 $x7248)) (unit-resolution @x7501 @x8658 @x7571 $x7499) $x6211)))
+(let (($x7222 (or $x7243 $x7246)))
+(let (($x6667 (fun_app$ ?x265 ?v1!18)))
+(let (($x6740 (= $x6667 $x7222)))
+(let (($x6746 (or $x4114 $x6740)))
+(let ((@x6743 (monotonicity (rewrite (= (ite $x7243 true $x7246) $x7222)) (= (= $x6667 (ite $x7243 true $x7246)) $x6740))))
+(let ((@x6845 (monotonicity @x6743 (= (or $x4114 (= $x6667 (ite $x7243 true $x7246))) $x6746))))
+(let ((@x4954 (trans @x6845 (rewrite (= $x6746 $x6746)) (= (or $x4114 (= $x6667 (ite $x7243 true $x7246))) $x6746))))
+(let ((@x6537 (mp ((_ quant-inst v_b_Visited_G_1$ v_b_v_G_1$ true ?v1!18) (or $x4114 (= $x6667 (ite $x7243 true $x7246)))) @x4954 $x6746)))
+(let ((@x8675 (mp (hypothesis $x1883) (symm (monotonicity @x5875 (= $x6667 $x1883)) (= $x1883 $x6667)) $x6667)))
+(let ((@x8676 (unit-resolution (def-axiom (or (not $x6740) (not $x6667) $x7222)) @x8675 (unit-resolution @x6537 @x3473 $x6740) $x7222)))
+(let ((@x4955 (def-axiom (or (not $x7222) $x7243 $x7246))))
+(let ((@x7000 (unit-resolution (hypothesis (not $x7003)) (monotonicity (monotonicity (hypothesis $x7243) (= ?x1884 ?x7110)) $x7003) false)))
+(let ((@x7002 (lemma @x7000 (or (not $x7243) $x7003))))
+(let ((@x7011 ((_ th-lemma arith triangle-eq) (or (not $x7003) $x7556))))
+(let ((@x8679 (unit-resolution @x7011 (unit-resolution @x7002 (unit-resolution @x4955 @x8676 @x8673 $x7243) $x7003) $x7556)))
+(let (($x7102 (<= (+ b_Infinity$ ?x7100) 0)))
+(let ((?x7171 (+ ?x257 ?x1894 ?x7111)))
+(let (($x7252 (>= ?x7171 0)))
+(let (($x7576 (not $x7252)))
+(let (($x7366 (<= (+ ?x257 ?x6721) 0)))
+(let (($x8449 (or $x3665 $x7246 $x7366)))
+(let (($x7357 (>= (+ ?x6619 ?x1173) 0)))
+(let (($x7358 (or $x7246 $x7357)))
+(let (($x8450 (or $x3665 $x7358)))
+(let ((@x8441 (monotonicity (rewrite (= (+ ?x6619 ?x1173) (+ ?x1173 ?x6619))) (= $x7357 (>= (+ ?x1173 ?x6619) 0)))))
+(let ((@x8445 (trans @x8441 (rewrite (= (>= (+ ?x1173 ?x6619) 0) $x7366)) (= $x7357 $x7366))))
+(let ((@x8454 (monotonicity (monotonicity @x8445 (= $x7358 (or $x7246 $x7366))) (= $x8450 (or $x3665 (or $x7246 $x7366))))))
+(let ((@x8458 (trans @x8454 (rewrite (= (or $x3665 (or $x7246 $x7366)) $x8449)) (= $x8450 $x8449))))
+(let ((@x8681 (unit-resolution (mp ((_ quant-inst ?v1!18) $x8450) @x8458 $x8449) (unit-resolution (def-axiom (or $x3809 $x3660)) @x6181 $x3660) @x8673 $x7366)))
+(let ((@x8685 (unit-resolution ((_ th-lemma arith assign-bounds -1 1 -1 1) (or $x7576 $x1896 (not $x7353) (not $x7366) (not $x7556))) @x8681 @x8679 @x7571 @x8658 $x7576)))
+(let ((@x8686 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x7171 0)) $x7252)) @x8685 (not (= ?x7171 0)))))
+(let (($x7117 (>= (+ ?x257 (* (- 1) (fun_app$c v_b_SP_G_1$ ?v0!19)) ?x7111) 0)))
+(let (($x7161 (not $x7117)))
+(let ((@x8688 ((_ th-lemma arith assign-bounds -1 -1 1 -1 1) (or $x7161 (not $x7076) $x1896 (not $x7353) (not $x7366) (not $x7556)))))
+(let (($x7174 (= ?x7171 0)))
+(let (($x7184 (or $x7102 $x7117 $x7174)))
+(let (($x7186 (or $x3675 $x7102 $x7117 $x7174)))
+(let (($x7104 (<= (+ (fun_app$c v_b_SP_G_1$ ?v0!19) ?x1173 ?x7100) 0)))
+(let (($x7165 (or $x7102 $x7104 (= (+ ?x257 ?x7111 ?x1894) 0))))
+(let (($x7187 (or $x3675 $x7165)))
+(let ((@x7183 (monotonicity (rewrite (= (+ ?x257 ?x7111 ?x1894) ?x7171)) (= (= (+ ?x257 ?x7111 ?x1894) 0) $x7174))))
+(let ((@x7119 (rewrite (= (<= (+ ?x1173 (fun_app$c v_b_SP_G_1$ ?v0!19) ?x7100) 0) $x7117))))
+(let (($x7112 (= (+ (fun_app$c v_b_SP_G_1$ ?v0!19) ?x1173 ?x7100) (+ ?x1173 (fun_app$c v_b_SP_G_1$ ?v0!19) ?x7100))))
+(let ((@x7115 (monotonicity (rewrite $x7112) (= $x7104 (<= (+ ?x1173 (fun_app$c v_b_SP_G_1$ ?v0!19) ?x7100) 0)))))
+(let ((@x7205 (monotonicity (monotonicity (trans @x7115 @x7119 (= $x7104 $x7117)) @x7183 (= $x7165 $x7184)) (= $x7187 (or $x3675 $x7184)))))
+(let ((@x7250 (mp ((_ quant-inst ?v0!19) $x7187) (trans @x7205 (rewrite (= (or $x3675 $x7184) $x7186)) (= $x7187 $x7186)) $x7186)))
+(let ((@x8690 (unit-resolution (unit-resolution @x7250 @x6588 $x7184) (unit-resolution @x8688 @x8681 @x8679 @x7571 @x8658 @x7496 $x7161) @x8686 $x7102)))
+(let ((@x8693 (lemma ((_ th-lemma arith farkas -1 1 1) @x8690 @x8679 (hypothesis $x1889) false) (or $x7618 $x1888 $x1896 $x2791))))
+(let ((@x7245 (mp ((_ quant-inst ?v1!18) (or $x3700 (or $x2791 $x6615))) (rewrite (= (or $x3700 (or $x2791 $x6615)) (or $x3700 $x2791 $x6615))) (or $x3700 $x2791 $x6615))))
+(let ((@x8285 (unit-resolution @x7245 @x7616 @x7607 (unit-resolution @x8693 @x7592 @x7571 @x7607 $x7618) false)))
+(unit-resolution (lemma @x8285 (or $x2806 $x1896)) @x8434 (unit-resolution @x8433 (lemma @x8013 $x3737) $x2811) false))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))
+
--- a/src/HOL/SMT_Examples/Boogie_Max.certs2	Tue Jun 03 16:22:01 2014 +0200
+++ b/src/HOL/SMT_Examples/Boogie_Max.certs2	Tue Jun 03 16:27:31 2014 +0200
@@ -1,844 +1,780 @@
-336198ca2566b9b7e0ce4a688dd7f9094f37a0b9 843 0
-unsat
-((set-logic AUFLIA)
-(declare-fun ?v0!5 () Int)
-(declare-fun ?v0!4 () Int)
-(declare-fun ?v0!3 () Int)
-(declare-fun ?v0!2 () Int)
-(declare-fun k!10 () Bool)
-(declare-fun k!00 () Bool)
-(proof
-(let (($x109 (= v_b_max_G_3$ v_b_max_G_2$)))
-(let ((?x135 (v_b_array$ v_b_k_G_1$)))
-(let (($x136 (= ?x135 v_b_max_G_3$)))
-(let (($x2120 (forall ((?v0 Int) )(!(let (($x1020 (<= (+ (v_b_array$ ?v0) (* (- 1) v_b_max_G_3$)) 0)))
-(let (($x1005 (>= (+ ?v0 (* (- 1) v_b_p_G_1$)) 0)))
-(let (($x838 (>= ?v0 0)))
-(let (($x1399 (not $x838)))
-(or $x1399 $x1005 $x1020))))) :pattern ( (v_b_array$ ?v0) )))
-))
-(let (($x2128 (or (not $x2120) $x136)))
-(let (($x2131 (not $x2128)))
-(let (($x1312 (>= (+ v_b_max_G_3$ (* (- 1) (v_b_array$ ?v0!5))) 0)))
-(let (($x1290 (<= (+ v_b_p_G_1$ (* (- 1) ?v0!5)) 0)))
-(let (($x1173 (>= ?v0!5 0)))
-(let (($x1540 (not $x1173)))
-(let (($x1555 (or $x1540 $x1290 $x1312)))
-(let (($x1560 (not $x1555)))
-(let (($x2134 (or $x1560 $x2131)))
-(let (($x2137 (not $x2134)))
-(let (($x996 (>= v_b_p_G_1$ 2)))
-(let (($x1606 (not $x996)))
-(let (($x991 (= (+ v_b_p_G_0$ (* (- 1) v_b_p_G_1$)) (- 1))))
-(let (($x1605 (not $x991)))
-(let (($x989 (>= v_b_k_G_1$ 0)))
-(let (($x1604 (not $x989)))
-(let (($x1603 (not $x109)))
-(let (($x107 (= v_b_k_G_1$ v_b_p_G_0$)))
-(let (($x1602 (not $x107)))
-(let ((?x101 (v_b_array$ v_b_p_G_0$)))
-(let (($x104 (= v_b_max_G_2$ ?x101)))
-(let (($x1601 (not $x104)))
-(let (($x980 (>= (+ v_b_max_G_1$ (* (- 1) ?x101)) 0)))
-(let (($x885 (>= v_b_p_G_0$ 1)))
-(let (($x1529 (not $x885)))
-(let (($x882 (>= v_b_k_G_0$ 0)))
-(let (($x1528 (not $x882)))
-(let (($x2140 (or $x1528 $x1529 $x980 $x1601 $x1602 $x1603 $x1604 $x1605 $x1606 $x2137)))
-(let (($x2143 (not $x2140)))
-(let (($x985 (not $x980)))
-(let (($x2146 (or $x1528 $x1529 $x985 (not (= v_b_k_G_1$ v_b_k_G_0$)) (not (= v_b_max_G_3$ v_b_max_G_1$)) $x1604 $x1605 $x1606 $x2137)))
-(let ((?x1179 (v_b_array$ ?v0!5)))
-(let (($x1799 (= ?x101 ?x1179)))
-(let (($x1803 (not $x1799)))
-(let (($x1703 (>= (+ ?x101 (* (- 1) ?x1179)) 0)))
-(let (($x1693 (not $x1703)))
-(let (($x2149 (not $x2146)))
-(let ((@x2389 (hypothesis $x2149)))
-(let (($x2024 (<= (+ v_b_max_G_1$ (* (- 1) v_b_max_G_3$)) 0)))
-(let (($x2022 (= v_b_max_G_1$ v_b_max_G_3$)))
-(let ((@x2401 (symm (commutativity (= $x2022 (= v_b_max_G_3$ v_b_max_G_1$))) (= (= v_b_max_G_3$ v_b_max_G_1$) $x2022))))
-(let (($x145 (= v_b_max_G_3$ v_b_max_G_1$)))
-(let ((@x2406 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x2022) $x2024)) (mp (unit-resolution (def-axiom (or $x2146 $x145)) @x2389 $x145) @x2401 $x2022) $x2024)))
-(let (($x1678 (not $x1312)))
-(let ((?x62 (v_b_array$ v_b_k_G_0$)))
-(let (($x63 (= ?x62 v_b_max_G_1$)))
-(let (($x2152 (or $x2143 $x2149)))
-(let (($x2155 (not $x2152)))
-(let (($x919 (<= (+ v_b_length$ (* (- 1) v_b_p_G_0$)) 0)))
-(let (($x2158 (or $x1528 $x1529 $x919 $x2155)))
-(let (($x2161 (not $x2158)))
-(let (($x1253 (>= (+ v_b_max_G_4$ (* (- 1) (v_b_array$ ?v0!4))) 0)))
-(let (($x1142 (<= (+ v_b_length$ (* (- 1) ?v0!4)) 0)))
-(let (($x1139 (>= ?v0!4 0)))
-(let (($x1489 (not $x1139)))
-(let (($x1131 (= (v_b_array$ ?v0!3) v_b_max_G_4$)))
-(let (($x1126 (<= (+ v_b_length$ (* (- 1) ?v0!3)) 0)))
-(let (($x1484 (or (not (>= ?v0!3 0)) $x1126 $x1131)))
-(let (($x1516 (or (not $x1484) $x1489 $x1142 $x1253)))
-(let (($x1517 (not $x1516)))
-(let (($x2103 (forall ((?v0 Int) )(!(let ((?x46 (v_b_array$ ?v0)))
-(let (($x86 (= ?x46 v_b_max_G_4$)))
-(let (($x930 (<= (+ v_b_length$ (* (- 1) ?v0)) 0)))
-(let (($x838 (>= ?v0 0)))
-(let (($x1399 (not $x838)))
-(let (($x1458 (or $x1399 $x930 $x86)))
-(not $x1458))))))) :pattern ( (v_b_array$ ?v0) )))
-))
-(let (($x2108 (or $x2103 $x1517)))
-(let (($x2111 (not $x2108)))
-(let (($x73 (= v_b_max_G_4$ v_b_max_G_1$)))
-(let (($x1531 (not $x73)))
-(let (($x971 (not $x919)))
-(let (($x2114 (or $x1528 $x1529 $x971 (not k!00) $x1531 (not k!10) $x2111)))
-(let (($x2117 (not $x2114)))
-(let (($x2164 (or $x2117 $x2161)))
-(let (($x2167 (not $x2164)))
-(let (($x2095 (forall ((?v0 Int) )(!(let (($x903 (<= (+ (v_b_array$ ?v0) (* (- 1) v_b_max_G_1$)) 0)))
-(let (($x888 (>= (+ ?v0 (* (- 1) v_b_p_G_0$)) 0)))
-(let (($x838 (>= ?v0 0)))
-(let (($x1399 (not $x838)))
-(or $x1399 $x888 $x903))))) :pattern ( (v_b_array$ ?v0) )))
-))
-(let (($x2100 (not $x2095)))
-(let (($x2170 (or $x1528 $x1529 $x2100 (not $x63) $x2167)))
-(let (($x2173 (not $x2170)))
-(let ((?x30 (v_b_array$ 0)))
-(let (($x50 (= ?x30 v_b_max_G_0$)))
-(let (($x1095 (not $x50)))
-(let (($x2176 (or $x1095 $x2173)))
-(let (($x2179 (not $x2176)))
-(let (($x2087 (forall ((?v0 Int) )(!(let (($x851 (>= (+ v_b_max_G_0$ (* (- 1) (v_b_array$ ?v0))) 0)))
-(let (($x841 (>= ?v0 1)))
-(let (($x838 (>= ?v0 0)))
-(let (($x1399 (not $x838)))
-(or $x1399 $x841 $x851))))) :pattern ( (v_b_array$ ?v0) )))
-))
-(let (($x2182 (or (not $x2087) $x2179)))
-(let (($x2185 (not $x2182)))
-(let (($x1083 (>= (+ v_b_max_G_0$ (* (- 1) (v_b_array$ ?v0!2))) 0)))
-(let (($x831 (>= ?v0!2 1)))
-(let (($x1391 (or (not (>= ?v0!2 0)) $x831 $x1083)))
-(let (($x1079 (not $x831)))
-(let (($x1396 (not $x1391)))
-(let ((@x1966 (hypothesis $x1396)))
-(let (($x1078 (>= ?v0!2 0)))
-(let ((@x1951 ((_ th-lemma arith eq-propagate 0 0) (unit-resolution (def-axiom (or $x1391 $x1078)) @x1966 $x1078) (unit-resolution (def-axiom (or $x1391 $x1079)) @x1966 $x1079) (= ?v0!2 0))))
-(let ((@x1955 (symm (monotonicity @x1951 (= (v_b_array$ ?v0!2) ?x30)) (= ?x30 (v_b_array$ ?v0!2)))))
-(let (($x31 (= v_b_max_G_0$ ?x30)))
-(let (($x201 (and (not (<= v_b_length$ 0)) $x31)))
-(let (($x572 (forall ((?v0 Int) )(let ((?x46 (v_b_array$ ?v0)))
-(let (($x132 (<= ?x46 v_b_max_G_3$)))
-(or (not (and (<= 0 ?v0) (not (<= v_b_p_G_1$ ?v0)))) $x132))))
-))
-(let (($x595 (or (not $x572) $x136)))
-(let (($x600 (and $x572 $x595)))
-(let (($x116 (<= 2 v_b_p_G_1$)))
-(let (($x456 (= v_b_p_G_1$ (+ 1 v_b_p_G_0$))))
-(let (($x110 (<= 0 v_b_k_G_1$)))
-(let (($x144 (= v_b_k_G_1$ v_b_k_G_0$)))
-(let (($x143 (<= ?x101 v_b_max_G_1$)))
-(let (($x54 (<= 1 v_b_p_G_0$)))
-(let (($x52 (<= 0 v_b_k_G_0$)))
-(let (($x654 (and $x52 $x54 $x143 $x144 $x145 $x110 $x456 $x116)))
-(let (($x669 (not $x654)))
-(let (($x670 (or $x669 $x600)))
-(let (($x441 (not $x143)))
-(let (($x544 (and $x52 $x54 $x441 $x104 $x107 $x109 $x110 $x456 $x116)))
-(let (($x606 (not $x544)))
-(let (($x607 (or $x606 $x600)))
-(let (($x675 (and $x607 $x670)))
-(let (($x69 (<= v_b_length$ v_b_p_G_0$)))
-(let (($x415 (not $x69)))
-(let (($x429 (and $x52 $x54 $x415)))
-(let (($x681 (not $x429)))
-(let (($x682 (or $x681 $x675)))
-(let (($x377 (forall ((?v0 Int) )(let ((?x46 (v_b_array$ ?v0)))
-(let (($x89 (<= ?x46 v_b_max_G_4$)))
-(let (($x351 (not (<= v_b_length$ ?v0))))
-(let (($x43 (<= 0 ?v0)))
-(let (($x354 (and $x43 $x351)))
-(let (($x360 (not $x354)))
-(or $x360 $x89))))))))
-))
-(let (($x366 (exists ((?v0 Int) )(let ((?x46 (v_b_array$ ?v0)))
-(let (($x86 (= ?x46 v_b_max_G_4$)))
-(let (($x351 (not (<= v_b_length$ ?v0))))
-(let (($x43 (<= 0 ?v0)))
-(let (($x354 (and $x43 $x351)))
-(let (($x360 (not $x354)))
-(or $x360 $x86))))))))
-))
-(let (($x398 (or (not $x366) $x377)))
-(let (($x403 (and $x366 $x398)))
-(let (($x75 (= v_b_p_G_2$ v_b_p_G_0$)))
-(let (($x71 (= v_b_k_G_2$ v_b_k_G_0$)))
-(let (($x338 (and $x52 $x54 $x69 $x71 $x73 $x75)))
-(let (($x409 (not $x338)))
-(let (($x410 (or $x409 $x403)))
-(let (($x687 (and $x410 $x682)))
-(let (($x259 (forall ((?v0 Int) )(let ((?x46 (v_b_array$ ?v0)))
-(let (($x59 (<= ?x46 v_b_max_G_1$)))
-(or (not (and (<= 0 ?v0) (not (<= v_b_p_G_0$ ?v0)))) $x59))))
-))
-(let (($x294 (and $x50 $x52 $x54 $x259 $x63)))
-(let (($x694 (or (not $x294) $x687)))
-(let (($x699 (and $x50 $x694)))
-(let (($x234 (forall ((?v0 Int) )(let ((?x46 (v_b_array$ ?v0)))
-(let (($x47 (<= ?x46 v_b_max_G_0$)))
-(or (not (and (<= 0 ?v0) (not (<= 1 ?v0)))) $x47))))
-))
-(let (($x705 (not $x234)))
-(let (($x706 (or $x705 $x699)))
-(let (($x711 (and $x234 $x706)))
-(let (($x718 (or (not $x201) $x711)))
-(let (($x138 (=> (and $x136 false) true)))
-(let (($x139 (and $x136 $x138)))
-(let (($x134 (forall ((?v0 Int) )(let ((?x46 (v_b_array$ ?v0)))
-(let (($x132 (<= ?x46 v_b_max_G_3$)))
-(=> (and (<= 0 ?v0) (< ?v0 v_b_p_G_1$)) $x132))))
-))
-(let (($x140 (=> $x134 $x139)))
-(let (($x141 (and $x134 $x140)))
-(let (($x117 (and $x110 $x116)))
-(let (($x118 (and $x117 true)))
-(let (($x119 (and (= v_b_p_G_1$ (+ v_b_p_G_0$ 1)) $x118)))
-(let (($x111 (and $x110 $x54)))
-(let (($x120 (and $x111 $x119)))
-(let (($x121 (and true $x120)))
-(let (($x146 (and $x145 $x121)))
-(let (($x147 (and $x144 $x146)))
-(let (($x148 (and true $x147)))
-(let (($x55 (and $x52 $x54)))
-(let (($x149 (and $x55 $x148)))
-(let (($x150 (and $x143 $x149)))
-(let (($x151 (and $x55 $x150)))
-(let (($x152 (and true $x151)))
-(let (($x153 (=> $x152 $x141)))
-(let (($x122 (and $x109 $x121)))
-(let (($x123 (and $x107 $x122)))
-(let (($x124 (and true $x123)))
-(let (($x105 (and $x54 $x54)))
-(let (($x125 (and $x105 $x124)))
-(let (($x126 (and $x104 $x125)))
-(let (($x127 (and (< v_b_max_G_1$ ?x101) $x126)))
-(let (($x128 (and $x55 $x127)))
-(let (($x129 (and true $x128)))
-(let (($x142 (=> $x129 $x141)))
-(let (($x98 (and (< v_b_p_G_0$ v_b_length$) $x55)))
-(let (($x99 (and $x55 $x98)))
-(let (($x100 (and true $x99)))
-(let (($x155 (=> $x100 (and $x142 $x153))))
-(let (($x91 (forall ((?v0 Int) )(let ((?x46 (v_b_array$ ?v0)))
-(let (($x89 (<= ?x46 v_b_max_G_4$)))
-(let (($x43 (<= 0 ?v0)))
-(let (($x85 (and $x43 (< ?v0 v_b_length$))))
-(=> $x85 $x89))))))
-))
-(let (($x92 (=> $x91 true)))
-(let (($x93 (and $x91 $x92)))
-(let (($x88 (exists ((?v0 Int) )(let ((?x46 (v_b_array$ ?v0)))
-(let (($x86 (= ?x46 v_b_max_G_4$)))
-(let (($x43 (<= 0 ?v0)))
-(let (($x85 (and $x43 (< ?v0 v_b_length$))))
-(=> $x85 $x86))))))
-))
-(let (($x94 (=> $x88 $x93)))
-(let (($x78 (and $x71 (and $x73 (and $x75 true)))))
-(let (($x79 (and true $x78)))
-(let (($x80 (and $x55 $x79)))
-(let (($x81 (and $x69 $x80)))
-(let (($x82 (and $x55 $x81)))
-(let (($x83 (and true $x82)))
-(let (($x96 (=> $x83 (and $x88 $x94))))
-(let (($x64 (and $x63 $x55)))
-(let (($x61 (forall ((?v0 Int) )(let ((?x46 (v_b_array$ ?v0)))
-(let (($x59 (<= ?x46 v_b_max_G_1$)))
-(=> (and (<= 0 ?v0) (< ?v0 v_b_p_G_0$)) $x59))))
-))
-(let (($x65 (and $x61 $x64)))
-(let (($x66 (and $x55 $x65)))
-(let (($x67 (and true $x66)))
-(let (($x68 (and $x50 $x67)))
-(let (($x157 (=> $x68 (and $x96 $x155))))
-(let (($x49 (forall ((?v0 Int) )(let ((?x46 (v_b_array$ ?v0)))
-(let (($x47 (<= ?x46 v_b_max_G_0$)))
-(=> (and (<= 0 ?v0) (< ?v0 1)) $x47))))
-))
-(let (($x159 (=> $x49 (and $x50 $x157))))
-(let (($x34 (<= 1 1)))
-(let (($x35 (and $x34 $x34)))
-(let (($x32 (<= 0 0)))
-(let (($x36 (and $x32 $x35)))
-(let (($x37 (and $x32 $x36)))
-(let (($x38 (and $x31 $x37)))
-(let (($x39 (and true $x38)))
-(let (($x41 (and true (and (< 0 v_b_length$) $x39))))
-(let (($x161 (=> $x41 (and $x49 $x159))))
-(let (($x162 (not $x161)))
-(let ((@x579 (monotonicity (rewrite (= (and $x136 false) false)) (= $x138 (=> false true)))))
-(let ((@x583 (trans @x579 (rewrite (= (=> false true) true)) (= $x138 true))))
-(let ((@x590 (trans (monotonicity @x583 (= $x139 (and $x136 true))) (rewrite (= (and $x136 true) $x136)) (= $x139 $x136))))
-(let ((?x46 (v_b_array$ ?0)))
-(let (($x132 (<= ?x46 v_b_max_G_3$)))
-(let (($x567 (or (not (and (<= 0 ?0) (not (<= v_b_p_G_1$ ?0)))) $x132)))
-(let (($x133 (=> (and (<= 0 ?0) (< ?0 v_b_p_G_1$)) $x132)))
-(let (($x568 (= (=> (and (<= 0 ?0) (not (<= v_b_p_G_1$ ?0))) $x132) $x567)))
-(let (($x564 (= $x133 (=> (and (<= 0 ?0) (not (<= v_b_p_G_1$ ?0))) $x132))))
-(let (($x557 (not (<= v_b_p_G_1$ ?0))))
-(let (($x43 (<= 0 ?0)))
-(let (($x560 (and $x43 $x557)))
-(let ((@x212 (rewrite (= $x43 $x43))))
-(let ((@x562 (monotonicity @x212 (rewrite (= (< ?0 v_b_p_G_1$) $x557)) (= (and $x43 (< ?0 v_b_p_G_1$)) $x560))))
-(let ((@x574 (quant-intro (trans (monotonicity @x562 $x564) (rewrite $x568) (= $x133 $x567)) (= $x134 $x572))))
-(let ((@x599 (trans (monotonicity @x574 @x590 (= $x140 (=> $x572 $x136))) (rewrite (= (=> $x572 $x136) $x595)) (= $x140 $x595))))
-(let ((@x656 (rewrite (= (and $x55 (and $x143 $x52 $x54 $x144 $x145 $x110 $x456 $x116)) $x654))))
-(let (($x646 (and $x143 $x52 $x54 $x144 $x145 $x110 $x456 $x116)))
-(let ((@x648 (rewrite (= (and $x143 (and $x52 $x54 $x144 $x145 $x110 $x456 $x116)) $x646))))
-(let (($x638 (and $x52 $x54 $x144 $x145 $x110 $x456 $x116)))
-(let (($x623 (and $x144 $x145 $x110 $x54 $x456 $x116)))
-(let (($x615 (and $x145 $x110 $x54 $x456 $x116)))
-(let (($x482 (and $x110 $x54 $x456 $x116)))
-(let ((@x463 (rewrite (= $x116 $x116))))
-(let ((@x450 (rewrite (= $x110 $x110))))
-(let ((@x467 (monotonicity (monotonicity @x450 @x463 (= $x117 $x117)) (= $x118 $x118))))
-(let ((@x460 (rewrite (= $x456 $x456))))
-(let ((@x458 (monotonicity (rewrite (= (+ v_b_p_G_0$ 1) (+ 1 v_b_p_G_0$))) (= (= v_b_p_G_1$ (+ v_b_p_G_0$ 1)) $x456))))
-(let ((@x473 (monotonicity (trans @x458 @x460 (= (= v_b_p_G_1$ (+ v_b_p_G_0$ 1)) $x456)) (trans @x467 (rewrite (= $x118 $x117)) (= $x118 $x117)) (= $x119 (and $x456 $x117)))))
-(let ((@x478 (trans @x473 (rewrite (= (and $x456 $x117) (and $x456 $x110 $x116))) (= $x119 (and $x456 $x110 $x116)))))
-(let ((@x481 (monotonicity (monotonicity @x450 (rewrite (= $x54 $x54)) (= $x111 $x111)) @x478 (= $x120 (and $x111 (and $x456 $x110 $x116))))))
-(let ((@x486 (trans @x481 (rewrite (= (and $x111 (and $x456 $x110 $x116)) $x482)) (= $x120 $x482))))
-(let ((@x493 (trans (monotonicity @x486 (= $x121 (and true $x482))) (rewrite (= (and true $x482) $x482)) (= $x121 $x482))))
-(let ((@x619 (trans (monotonicity @x493 (= $x146 (and $x145 $x482))) (rewrite (= (and $x145 $x482) $x615)) (= $x146 $x615))))
-(let ((@x627 (trans (monotonicity @x619 (= $x147 (and $x144 $x615))) (rewrite (= (and $x144 $x615) $x623)) (= $x147 $x623))))
-(let ((@x634 (trans (monotonicity @x627 (= $x148 (and true $x623))) (rewrite (= (and true $x623) $x623)) (= $x148 $x623))))
-(let ((@x240 (rewrite (= $x54 $x54))))
-(let ((@x238 (rewrite (= $x52 $x52))))
-(let ((@x242 (monotonicity @x238 @x240 (= $x55 $x55))))
-(let ((@x642 (trans (monotonicity @x242 @x634 (= $x149 (and $x55 $x623))) (rewrite (= (and $x55 $x623) $x638)) (= $x149 $x638))))
-(let ((@x650 (trans (monotonicity @x642 (= $x150 (and $x143 $x638))) @x648 (= $x150 $x646))))
-(let ((@x658 (trans (monotonicity @x242 @x650 (= $x151 (and $x55 $x646))) @x656 (= $x151 $x654))))
-(let ((@x665 (trans (monotonicity @x658 (= $x152 (and true $x654))) (rewrite (= (and true $x654) $x654)) (= $x152 $x654))))
-(let ((@x668 (monotonicity @x665 (monotonicity @x574 @x599 (= $x141 $x600)) (= $x153 (=> $x654 $x600)))))
-(let ((@x546 (rewrite (= (and $x55 (and $x441 $x104 $x54 $x107 $x109 $x110 $x456 $x116)) $x544))))
-(let (($x536 (and $x441 $x104 $x54 $x107 $x109 $x110 $x456 $x116)))
-(let ((@x538 (rewrite (= (and $x441 (and $x104 $x54 $x107 $x109 $x110 $x456 $x116)) $x536))))
-(let (($x528 (and $x104 $x54 $x107 $x109 $x110 $x456 $x116)))
-(let (($x520 (and $x54 $x107 $x109 $x110 $x456 $x116)))
-(let (($x505 (and $x107 $x109 $x110 $x54 $x456 $x116)))
-(let ((@x501 (trans (monotonicity @x493 (= $x122 (and $x109 $x482))) (rewrite (= (and $x109 $x482) (and $x109 $x110 $x54 $x456 $x116))) (= $x122 (and $x109 $x110 $x54 $x456 $x116)))))
-(let ((@x504 (monotonicity @x501 (= $x123 (and $x107 (and $x109 $x110 $x54 $x456 $x116))))))
-(let ((@x509 (trans @x504 (rewrite (= (and $x107 (and $x109 $x110 $x54 $x456 $x116)) $x505)) (= $x123 $x505))))
-(let ((@x516 (trans (monotonicity @x509 (= $x124 (and true $x505))) (rewrite (= (and true $x505) $x505)) (= $x124 $x505))))
-(let ((@x448 (trans (monotonicity @x240 @x240 (= $x105 $x105)) (rewrite (= $x105 $x54)) (= $x105 $x54))))
-(let ((@x524 (trans (monotonicity @x448 @x516 (= $x125 (and $x54 $x505))) (rewrite (= (and $x54 $x505) $x520)) (= $x125 $x520))))
-(let ((@x532 (trans (monotonicity @x524 (= $x126 (and $x104 $x520))) (rewrite (= (and $x104 $x520) $x528)) (= $x126 $x528))))
-(let ((@x535 (monotonicity (rewrite (= (< v_b_max_G_1$ ?x101) $x441)) @x532 (= $x127 (and $x441 $x528)))))
-(let ((@x543 (monotonicity @x242 (trans @x535 @x538 (= $x127 $x536)) (= $x128 (and $x55 $x536)))))
-(let ((@x551 (monotonicity (trans @x543 @x546 (= $x128 $x544)) (= $x129 (and true $x544)))))
-(let ((@x605 (monotonicity (trans @x551 (rewrite (= (and true $x544) $x544)) (= $x129 $x544)) (monotonicity @x574 @x599 (= $x141 $x600)) (= $x142 (=> $x544 $x600)))))
-(let ((@x677 (monotonicity (trans @x605 (rewrite (= (=> $x544 $x600) $x607)) (= $x142 $x607)) (trans @x668 (rewrite (= (=> $x654 $x600) $x670)) (= $x153 $x670)) (= (and $x142 $x153) $x675))))
-(let ((@x420 (monotonicity (rewrite (= (< v_b_p_G_0$ v_b_length$) $x415)) @x242 (= $x98 (and $x415 $x55)))))
-(let ((@x425 (trans @x420 (rewrite (= (and $x415 $x55) (and $x415 $x52 $x54))) (= $x98 (and $x415 $x52 $x54)))))
-(let ((@x433 (trans (monotonicity @x242 @x425 (= $x99 (and $x55 (and $x415 $x52 $x54)))) (rewrite (= (and $x55 (and $x415 $x52 $x54)) $x429)) (= $x99 $x429))))
-(let ((@x440 (trans (monotonicity @x433 (= $x100 (and true $x429))) (rewrite (= (and true $x429) $x429)) (= $x100 $x429))))
-(let ((@x686 (trans (monotonicity @x440 @x677 (= $x155 (=> $x429 $x675))) (rewrite (= (=> $x429 $x675) $x682)) (= $x155 $x682))))
-(let (($x89 (<= ?x46 v_b_max_G_4$)))
-(let (($x351 (not (<= v_b_length$ ?0))))
-(let (($x354 (and $x43 $x351)))
-(let (($x360 (not $x354)))
-(let (($x372 (or $x360 $x89)))
-(let (($x85 (and $x43 (< ?0 v_b_length$))))
-(let (($x90 (=> $x85 $x89)))
-(let ((@x356 (monotonicity @x212 (rewrite (= (< ?0 v_b_length$) $x351)) (= $x85 $x354))))
-(let ((@x376 (trans (monotonicity @x356 (= $x90 (=> $x354 $x89))) (rewrite (= (=> $x354 $x89) $x372)) (= $x90 $x372))))
-(let ((@x382 (monotonicity (quant-intro @x376 (= $x91 $x377)) (= $x92 (=> $x377 true)))))
-(let ((@x386 (trans @x382 (rewrite (= (=> $x377 true) true)) (= $x92 true))))
-(let ((@x389 (monotonicity (quant-intro @x376 (= $x91 $x377)) @x386 (= $x93 (and $x377 true)))))
-(let (($x86 (= ?x46 v_b_max_G_4$)))
-(let (($x361 (or $x360 $x86)))
-(let (($x87 (=> $x85 $x86)))
-(let ((@x365 (trans (monotonicity @x356 (= $x87 (=> $x354 $x86))) (rewrite (= (=> $x354 $x86) $x361)) (= $x87 $x361))))
-(let ((@x396 (monotonicity (quant-intro @x365 (= $x88 $x366)) (trans @x389 (rewrite (= (and $x377 true) $x377)) (= $x93 $x377)) (= $x94 (=> $x366 $x377)))))
-(let ((@x405 (monotonicity (quant-intro @x365 (= $x88 $x366)) (trans @x396 (rewrite (= (=> $x366 $x377) $x398)) (= $x94 $x398)) (= (and $x88 $x94) $x403))))
-(let (($x330 (and $x69 $x52 $x54 $x71 $x73 $x75)))
-(let (($x322 (and $x52 $x54 $x71 $x73 $x75)))
-(let ((@x316 (rewrite (= (and true (and $x71 $x73 $x75)) (and $x71 $x73 $x75)))))
-(let ((@x303 (monotonicity (rewrite (= (and $x75 true) $x75)) (= (and $x73 (and $x75 true)) (and $x73 $x75)))))
-(let ((@x311 (trans (monotonicity @x303 (= $x78 (and $x71 (and $x73 $x75)))) (rewrite (= (and $x71 (and $x73 $x75)) (and $x71 $x73 $x75))) (= $x78 (and $x71 $x73 $x75)))))
-(let ((@x318 (trans (monotonicity @x311 (= $x79 (and true (and $x71 $x73 $x75)))) @x316 (= $x79 (and $x71 $x73 $x75)))))
-(let ((@x326 (trans (monotonicity @x242 @x318 (= $x80 (and $x55 (and $x71 $x73 $x75)))) (rewrite (= (and $x55 (and $x71 $x73 $x75)) $x322)) (= $x80 $x322))))
-(let ((@x334 (trans (monotonicity @x326 (= $x81 (and $x69 $x322))) (rewrite (= (and $x69 $x322) $x330)) (= $x81 $x330))))
-(let ((@x342 (trans (monotonicity @x242 @x334 (= $x82 (and $x55 $x330))) (rewrite (= (and $x55 $x330) $x338)) (= $x82 $x338))))
-(let ((@x349 (trans (monotonicity @x342 (= $x83 (and true $x338))) (rewrite (= (and true $x338) $x338)) (= $x83 $x338))))
-(let ((@x414 (trans (monotonicity @x349 @x405 (= $x96 (=> $x338 $x403))) (rewrite (= (=> $x338 $x403) $x410)) (= $x96 $x410))))
-(let (($x279 (and $x52 $x54 $x259 $x63)))
-(let ((@x273 (rewrite (= (and $x259 (and $x63 $x52 $x54)) (and $x259 $x63 $x52 $x54)))))
-(let ((@x267 (trans (monotonicity @x242 (= $x64 $x64)) (rewrite (= $x64 (and $x63 $x52 $x54))) (= $x64 (and $x63 $x52 $x54)))))
-(let (($x59 (<= ?x46 v_b_max_G_1$)))
-(let (($x254 (or (not (and $x43 (not (<= v_b_p_G_0$ ?0)))) $x59)))
-(let (($x60 (=> (and $x43 (< ?0 v_b_p_G_0$)) $x59)))
-(let ((@x256 (rewrite (= (=> (and $x43 (not (<= v_b_p_G_0$ ?0))) $x59) $x254))))
-(let (($x244 (not (<= v_b_p_G_0$ ?0))))
-(let (($x247 (and $x43 $x244)))
-(let ((@x249 (monotonicity @x212 (rewrite (= (< ?0 v_b_p_G_0$) $x244)) (= (and $x43 (< ?0 v_b_p_G_0$)) $x247))))
-(let ((@x258 (trans (monotonicity @x249 (= $x60 (=> $x247 $x59))) @x256 (= $x60 $x254))))
-(let ((@x270 (monotonicity (quant-intro @x258 (= $x61 $x259)) @x267 (= $x65 (and $x259 (and $x63 $x52 $x54))))))
-(let ((@x278 (monotonicity @x242 (trans @x270 @x273 (= $x65 (and $x259 $x63 $x52 $x54))) (= $x66 (and $x55 (and $x259 $x63 $x52 $x54))))))
-(let ((@x283 (trans @x278 (rewrite (= (and $x55 (and $x259 $x63 $x52 $x54)) $x279)) (= $x66 $x279))))
-(let ((@x290 (trans (monotonicity @x283 (= $x67 (and true $x279))) (rewrite (= (and true $x279) $x279)) (= $x67 $x279))))
-(let ((@x298 (trans (monotonicity @x290 (= $x68 (and $x50 $x279))) (rewrite (= (and $x50 $x279) $x294)) (= $x68 $x294))))
-(let ((@x692 (monotonicity @x298 (monotonicity @x414 @x686 (= (and $x96 $x155) $x687)) (= $x157 (=> $x294 $x687)))))
-(let ((@x701 (monotonicity (trans @x692 (rewrite (= (=> $x294 $x687) $x694)) (= $x157 $x694)) (= (and $x50 $x157) $x699))))
-(let (($x47 (<= ?x46 v_b_max_G_0$)))
-(let (($x229 (or (not (and $x43 (not (<= 1 ?0)))) $x47)))
-(let (($x48 (=> (and $x43 (< ?0 1)) $x47)))
-(let ((@x220 (monotonicity (rewrite (= (<= 1 ?0) (<= 1 ?0))) (= (not (<= 1 ?0)) (not (<= 1 ?0))))))
-(let ((@x221 (trans (rewrite (= (< ?0 1) (not (<= 1 ?0)))) @x220 (= (< ?0 1) (not (<= 1 ?0))))))
-(let ((@x224 (monotonicity @x212 @x221 (= (and $x43 (< ?0 1)) (and $x43 (not (<= 1 ?0)))))))
-(let ((@x227 (monotonicity @x224 (= $x48 (=> (and $x43 (not (<= 1 ?0))) $x47)))))
-(let ((@x233 (trans @x227 (rewrite (= (=> (and $x43 (not (<= 1 ?0))) $x47) $x229)) (= $x48 $x229))))
-(let ((@x704 (monotonicity (quant-intro @x233 (= $x49 $x234)) @x701 (= $x159 (=> $x234 $x699)))))
-(let ((@x713 (monotonicity (quant-intro @x233 (= $x49 $x234)) (trans @x704 (rewrite (= (=> $x234 $x699) $x706)) (= $x159 $x706)) (= (and $x49 $x159) $x711))))
-(let ((@x176 (rewrite (= (and true true) true))))
-(let ((@x174 (monotonicity (rewrite (= $x34 true)) (rewrite (= $x34 true)) (= $x35 (and true true)))))
-(let ((@x180 (monotonicity (rewrite (= $x32 true)) (trans @x174 @x176 (= $x35 true)) (= $x36 (and true true)))))
-(let ((@x184 (monotonicity (rewrite (= $x32 true)) (trans @x180 @x176 (= $x36 true)) (= $x37 (and true true)))))
-(let ((@x189 (monotonicity (trans @x184 @x176 (= $x37 true)) (= $x38 (and $x31 true)))))
-(let ((@x196 (monotonicity (trans @x189 (rewrite (= (and $x31 true) $x31)) (= $x38 $x31)) (= $x39 (and true $x31)))))
-(let ((@x203 (monotonicity (rewrite (= (< 0 v_b_length$) (not (<= v_b_length$ 0)))) (trans @x196 (rewrite (= (and true $x31) $x31)) (= $x39 $x31)) (= (and (< 0 v_b_length$) $x39) $x201))))
-(let ((@x210 (trans (monotonicity @x203 (= $x41 (and true $x201))) (rewrite (= (and true $x201) $x201)) (= $x41 $x201))))
-(let ((@x722 (trans (monotonicity @x210 @x713 (= $x161 (=> $x201 $x711))) (rewrite (= (=> $x201 $x711) $x718)) (= $x161 $x718))))
-(let ((@x726 (mp (asserted $x162) (monotonicity @x722 (= $x162 (not $x718))) (not $x718))))
-(let ((@x737 (mp (and-elim (not-or-elim @x726 $x201) $x31) (rewrite* (= $x31 $x31)) $x31)))
-(let ((@x1930 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= v_b_max_G_0$ (v_b_array$ ?v0!2))) $x1083)) (unit-resolution (def-axiom (or $x1391 (not $x1083))) @x1966 (not $x1083)) (trans @x737 @x1955 (= v_b_max_G_0$ (v_b_array$ ?v0!2))) false)))
-(let (($x1582 (forall ((?v0 Int) )(let (($x1020 (<= (+ (v_b_array$ ?v0) (* (- 1) v_b_max_G_3$)) 0)))
-(let (($x1005 (>= (+ ?v0 (* (- 1) v_b_p_G_1$)) 0)))
-(let (($x838 (>= ?v0 0)))
-(let (($x1399 (not $x838)))
-(or $x1399 $x1005 $x1020))))))
-))
-(let (($x1590 (not (or (not $x1582) $x136))))
-(let (($x1595 (or $x1560 $x1590)))
-(let (($x1607 (not $x1595)))
-(let (($x1620 (not (or $x1528 $x1529 $x985 (not $x144) (not $x145) $x1604 $x1605 $x1606 $x1607))))
-(let (($x1609 (not (or $x1528 $x1529 $x980 $x1601 $x1602 $x1603 $x1604 $x1605 $x1606 $x1607))))
-(let (($x1625 (or $x1609 $x1620)))
-(let (($x1633 (not (or $x1528 $x1529 $x919 (not $x1625)))))
-(let (($x1466 (forall ((?v0 Int) )(let ((?x46 (v_b_array$ ?v0)))
-(let (($x86 (= ?x46 v_b_max_G_4$)))
-(let (($x930 (<= (+ v_b_length$ (* (- 1) ?v0)) 0)))
-(let (($x838 (>= ?v0 0)))
-(let (($x1399 (not $x838)))
-(let (($x1458 (or $x1399 $x930 $x86)))
-(not $x1458))))))))
-))
-(let (($x1522 (or $x1466 $x1517)))
-(let (($x1535 (not (or $x1528 $x1529 $x971 (not k!00) $x1531 (not k!10) (not $x1522)))))
-(let (($x1638 (or $x1535 $x1633)))
-(let (($x1441 (forall ((?v0 Int) )(let (($x903 (<= (+ (v_b_array$ ?v0) (* (- 1) v_b_max_G_1$)) 0)))
-(let (($x888 (>= (+ ?v0 (* (- 1) v_b_p_G_0$)) 0)))
-(let (($x838 (>= ?v0 0)))
-(let (($x1399 (not $x838)))
-(or $x1399 $x888 $x903))))))
-))
-(let (($x1648 (not (or $x1528 $x1529 (not $x1441) (not $x63) (not $x1638)))))
-(let (($x1653 (or $x1095 $x1648)))
-(let (($x1419 (forall ((?v0 Int) )(let (($x851 (>= (+ v_b_max_G_0$ (* (- 1) (v_b_array$ ?v0))) 0)))
-(let (($x841 (>= ?v0 1)))
-(let (($x838 (>= ?v0 0)))
-(let (($x1399 (not $x838)))
-(or $x1399 $x841 $x851))))))
-))
-(let (($x1662 (not (or (not $x1419) (not $x1653)))))
-(let (($x1667 (or $x1396 $x1662)))
-(let (($x2147 (= (or $x1528 $x1529 $x985 (not $x144) (not $x145) $x1604 $x1605 $x1606 $x1607) $x2146)))
-(let (($x1020 (<= (+ ?x46 (* (- 1) v_b_max_G_3$)) 0)))
-(let (($x1005 (>= (+ ?0 (* (- 1) v_b_p_G_1$)) 0)))
-(let (($x838 (>= ?0 0)))
-(let (($x1399 (not $x838)))
-(let (($x1577 (or $x1399 $x1005 $x1020)))
-(let ((@x2127 (monotonicity (quant-intro (refl (= $x1577 $x1577)) (= $x1582 $x2120)) (= (not $x1582) (not $x2120)))))
-(let ((@x2133 (monotonicity (monotonicity @x2127 (= (or (not $x1582) $x136) $x2128)) (= $x1590 $x2131))))
-(let ((@x2148 (monotonicity (monotonicity (monotonicity @x2133 (= $x1595 $x2134)) (= $x1607 $x2137)) $x2147)))
-(let ((@x2142 (monotonicity (monotonicity (monotonicity @x2133 (= $x1595 $x2134)) (= $x1607 $x2137)) (= (or $x1528 $x1529 $x980 $x1601 $x1602 $x1603 $x1604 $x1605 $x1606 $x1607) $x2140))))
-(let ((@x2154 (monotonicity (monotonicity @x2142 (= $x1609 $x2143)) (monotonicity @x2148 (= $x1620 $x2149)) (= $x1625 $x2152))))
-(let ((@x2160 (monotonicity (monotonicity @x2154 (= (not $x1625) $x2155)) (= (or $x1528 $x1529 $x919 (not $x1625)) $x2158))))
-(let (($x2115 (= (or $x1528 $x1529 $x971 (not k!00) $x1531 (not k!10) (not $x1522)) $x2114)))
-(let (($x930 (<= (+ v_b_length$ (* (- 1) ?0)) 0)))
-(let (($x1458 (or $x1399 $x930 $x86)))
-(let (($x1463 (not $x1458)))
-(let ((@x2110 (monotonicity (quant-intro (refl (= $x1463 $x1463)) (= $x1466 $x2103)) (= $x1522 $x2108))))
-(let ((@x2119 (monotonicity (monotonicity (monotonicity @x2110 (= (not $x1522) $x2111)) $x2115) (= $x1535 $x2117))))
-(let ((@x2166 (monotonicity @x2119 (monotonicity @x2160 (= $x1633 $x2161)) (= $x1638 $x2164))))
-(let (($x903 (<= (+ ?x46 (* (- 1) v_b_max_G_1$)) 0)))
-(let (($x888 (>= (+ ?0 (* (- 1) v_b_p_G_0$)) 0)))
-(let (($x1436 (or $x1399 $x888 $x903)))
-(let ((@x2102 (monotonicity (quant-intro (refl (= $x1436 $x1436)) (= $x1441 $x2095)) (= (not $x1441) $x2100))))
-(let ((@x2172 (monotonicity @x2102 (monotonicity @x2166 (= (not $x1638) $x2167)) (= (or $x1528 $x1529 (not $x1441) (not $x63) (not $x1638)) $x2170))))
-(let ((@x2181 (monotonicity (monotonicity (monotonicity @x2172 (= $x1648 $x2173)) (= $x1653 $x2176)) (= (not $x1653) $x2179))))
-(let (($x851 (>= (+ v_b_max_G_0$ (* (- 1) ?x46)) 0)))
-(let (($x841 (>= ?0 1)))
-(let (($x1414 (or $x1399 $x841 $x851)))
-(let ((@x2094 (monotonicity (quant-intro (refl (= $x1414 $x1414)) (= $x1419 $x2087)) (= (not $x1419) (not $x2087)))))
-(let ((@x2187 (monotonicity (monotonicity @x2094 @x2181 (= (or (not $x1419) (not $x1653)) $x2182)) (= $x1662 $x2185))))
-(let (($x1193 (not $x136)))
-(let (($x1026 (forall ((?v0 Int) )(let (($x1020 (<= (+ (v_b_array$ ?v0) (* (- 1) v_b_max_G_3$)) 0)))
-(let (($x838 (>= ?v0 0)))
-(let (($x1012 (and $x838 (not (>= (+ ?v0 (* (- 1) v_b_p_G_1$)) 0)))))
-(let (($x1015 (not $x1012)))
-(or $x1015 $x1020))))))
-))
-(let (($x1196 (and $x1026 $x1193)))
-(let (($x1295 (not $x1290)))
-(let (($x1298 (and $x1173 $x1295)))
-(let (($x1301 (not $x1298)))
-(let (($x1317 (or $x1301 $x1312)))
-(let (($x1320 (not $x1317)))
-(let (($x1323 (or $x1320 $x1196)))
-(let (($x1339 (and $x882 $x885 $x980 $x144 $x145 $x989 $x991 $x996 $x1323)))
-(let (($x1329 (and $x882 $x885 $x985 $x104 $x107 $x109 $x989 $x991 $x996 $x1323)))
-(let (($x1344 (or $x1329 $x1339)))
-(let (($x1350 (and $x882 $x885 $x971 $x1344)))
-(let (($x1145 (not (and $x1139 (not $x1142)))))
-(let (($x1258 (or $x1145 $x1253)))
-(let (($x1261 (not $x1258)))
-(let (($x1129 (not (and (>= ?v0!3 0) (not $x1126)))))
-(let (($x1132 (or $x1129 $x1131)))
-(let (($x1264 (and $x1132 $x1261)))
-(let (($x1119 (forall ((?v0 Int) )(let ((?x46 (v_b_array$ ?v0)))
-(let (($x86 (= ?x46 v_b_max_G_4$)))
-(let (($x838 (>= ?v0 0)))
-(let (($x936 (and $x838 (not (<= (+ v_b_length$ (* (- 1) ?v0)) 0)))))
-(let (($x939 (not $x936)))
-(let (($x942 (or $x939 $x86)))
-(not $x942))))))))
-))
-(let (($x1267 (or $x1119 $x1264)))
-(let (($x1273 (and $x882 $x885 $x919 k!00 $x73 k!10 $x1267)))
-(let (($x1355 (or $x1273 $x1350)))
-(let (($x909 (forall ((?v0 Int) )(let (($x903 (<= (+ (v_b_array$ ?v0) (* (- 1) v_b_max_G_1$)) 0)))
-(let (($x838 (>= ?v0 0)))
-(let (($x895 (and $x838 (not (>= (+ ?v0 (* (- 1) v_b_p_G_0$)) 0)))))
-(let (($x898 (not $x895)))
-(or $x898 $x903))))))
-))
-(let (($x1361 (and $x882 $x885 $x909 $x63 $x1355)))
-(let (($x1366 (or $x1095 $x1361)))
-(let (($x862 (forall ((?v0 Int) )(let (($x851 (>= (+ v_b_max_G_0$ (* (- 1) (v_b_array$ ?v0))) 0)))
-(let (($x838 (>= ?v0 0)))
-(let (($x849 (and $x838 (not (>= ?v0 1)))))
-(let (($x854 (not $x849)))
-(or $x854 $x851))))))
-))
-(let (($x1369 (and $x862 $x1366)))
-(let (($x1077 (not (and $x1078 $x1079))))
-(let (($x1084 (or $x1077 $x1083)))
-(let (($x1085 (not $x1084)))
-(let (($x1372 (or $x1085 $x1369)))
-(let ((@x1622 (rewrite (= (and $x882 $x885 $x980 $x144 $x145 $x989 $x991 $x996 $x1595) $x1620))))
-(let (($x1012 (and $x838 (not $x1005))))
-(let (($x1015 (not $x1012)))
-(let (($x1023 (or $x1015 $x1020)))
-(let ((@x1569 (monotonicity (rewrite (= $x1012 (not (or $x1399 $x1005)))) (= $x1015 (not (not (or $x1399 $x1005)))))))
-(let ((@x1573 (trans @x1569 (rewrite (= (not (not (or $x1399 $x1005))) (or $x1399 $x1005))) (= $x1015 (or $x1399 $x1005)))))
-(let ((@x1581 (trans (monotonicity @x1573 (= $x1023 (or (or $x1399 $x1005) $x1020))) (rewrite (= (or (or $x1399 $x1005) $x1020) $x1577)) (= $x1023 $x1577))))
-(let ((@x1587 (monotonicity (quant-intro @x1581 (= $x1026 $x1582)) (= $x1196 (and $x1582 $x1193)))))
-(let ((@x1547 (monotonicity (rewrite (= $x1298 (not (or $x1540 $x1290)))) (= $x1301 (not (not (or $x1540 $x1290)))))))
-(let ((@x1551 (trans @x1547 (rewrite (= (not (not (or $x1540 $x1290))) (or $x1540 $x1290))) (= $x1301 (or $x1540 $x1290)))))
-(let ((@x1559 (trans (monotonicity @x1551 (= $x1317 (or (or $x1540 $x1290) $x1312))) (rewrite (= (or (or $x1540 $x1290) $x1312) $x1555)) (= $x1317 $x1555))))
-(let ((@x1597 (monotonicity (monotonicity @x1559 (= $x1320 $x1560)) (trans @x1587 (rewrite (= (and $x1582 $x1193) $x1590)) (= $x1196 $x1590)) (= $x1323 $x1595))))
-(let ((@x1616 (monotonicity @x1597 (= $x1339 (and $x882 $x885 $x980 $x144 $x145 $x989 $x991 $x996 $x1595)))))
-(let ((@x1611 (rewrite (= (and $x882 $x885 $x985 $x104 $x107 $x109 $x989 $x991 $x996 $x1595) $x1609))))
-(let ((@x1600 (monotonicity @x1597 (= $x1329 (and $x882 $x885 $x985 $x104 $x107 $x109 $x989 $x991 $x996 $x1595)))))
-(let ((@x1627 (monotonicity (trans @x1600 @x1611 (= $x1329 $x1609)) (trans @x1616 @x1622 (= $x1339 $x1620)) (= $x1344 $x1625))))
-(let ((@x1637 (trans (monotonicity @x1627 (= $x1350 (and $x882 $x885 $x971 $x1625))) (rewrite (= (and $x882 $x885 $x971 $x1625) $x1633)) (= $x1350 $x1633))))
-(let ((@x1537 (rewrite (= (and $x882 $x885 $x919 k!00 $x73 k!10 $x1522) $x1535))))
-(let ((@x1496 (monotonicity (rewrite (= (and $x1139 (not $x1142)) (not (or $x1489 $x1142)))) (= $x1145 (not (not (or $x1489 $x1142)))))))
-(let ((@x1500 (trans @x1496 (rewrite (= (not (not (or $x1489 $x1142))) (or $x1489 $x1142))) (= $x1145 (or $x1489 $x1142)))))
-(let ((@x1508 (trans (monotonicity @x1500 (= $x1258 (or (or $x1489 $x1142) $x1253))) (rewrite (= (or (or $x1489 $x1142) $x1253) (or $x1489 $x1142 $x1253))) (= $x1258 (or $x1489 $x1142 $x1253)))))
-(let (($x1470 (or (not (>= ?v0!3 0)) $x1126)))
-(let ((@x1476 (monotonicity (rewrite (= (and (>= ?v0!3 0) (not $x1126)) (not $x1470))) (= $x1129 (not (not $x1470))))))
-(let ((@x1483 (monotonicity (trans @x1476 (rewrite (= (not (not $x1470)) $x1470)) (= $x1129 $x1470)) (= $x1132 (or $x1470 $x1131)))))
-(let ((@x1514 (monotonicity (trans @x1483 (rewrite (= (or $x1470 $x1131) $x1484)) (= $x1132 $x1484)) (monotonicity @x1508 (= $x1261 (not (or $x1489 $x1142 $x1253)))) (= $x1264 (and $x1484 (not (or $x1489 $x1142 $x1253)))))))
-(let ((@x1521 (trans @x1514 (rewrite (= (and $x1484 (not (or $x1489 $x1142 $x1253))) $x1517)) (= $x1264 $x1517))))
-(let (($x936 (and $x838 (not $x930))))
-(let (($x939 (not $x936)))
-(let (($x942 (or $x939 $x86)))
-(let ((@x1450 (monotonicity (rewrite (= $x936 (not (or $x1399 $x930)))) (= $x939 (not (not (or $x1399 $x930)))))))
-(let ((@x1454 (trans @x1450 (rewrite (= (not (not (or $x1399 $x930))) (or $x1399 $x930))) (= $x939 (or $x1399 $x930)))))
-(let ((@x1462 (trans (monotonicity @x1454 (= $x942 (or (or $x1399 $x930) $x86))) (rewrite (= (or (or $x1399 $x930) $x86) $x1458)) (= $x942 $x1458))))
-(let ((@x1468 (quant-intro (monotonicity @x1462 (= (not $x942) $x1463)) (= $x1119 $x1466))))
-(let ((@x1527 (monotonicity (monotonicity @x1468 @x1521 (= $x1267 $x1522)) (= $x1273 (and $x882 $x885 $x919 k!00 $x73 k!10 $x1522)))))
-(let (($x895 (and $x838 (not $x888))))
-(let (($x898 (not $x895)))
-(let (($x906 (or $x898 $x903)))
-(let ((@x1428 (monotonicity (rewrite (= $x895 (not (or $x1399 $x888)))) (= $x898 (not (not (or $x1399 $x888)))))))
-(let ((@x1432 (trans @x1428 (rewrite (= (not (not (or $x1399 $x888))) (or $x1399 $x888))) (= $x898 (or $x1399 $x888)))))
-(let ((@x1440 (trans (monotonicity @x1432 (= $x906 (or (or $x1399 $x888) $x903))) (rewrite (= (or (or $x1399 $x888) $x903) $x1436)) (= $x906 $x1436))))
-(let ((@x1643 (monotonicity (quant-intro @x1440 (= $x909 $x1441)) (monotonicity (trans @x1527 @x1537 (= $x1273 $x1535)) @x1637 (= $x1355 $x1638)) (= $x1361 (and $x882 $x885 $x1441 $x63 $x1638)))))
-(let ((@x1652 (trans @x1643 (rewrite (= (and $x882 $x885 $x1441 $x63 $x1638) $x1648)) (= $x1361 $x1648))))
-(let (($x849 (and $x838 (not $x841))))
-(let (($x854 (not $x849)))
-(let (($x859 (or $x854 $x851)))
-(let ((@x1406 (monotonicity (rewrite (= $x849 (not (or $x1399 $x841)))) (= $x854 (not (not (or $x1399 $x841)))))))
-(let ((@x1410 (trans @x1406 (rewrite (= (not (not (or $x1399 $x841))) (or $x1399 $x841))) (= $x854 (or $x1399 $x841)))))
-(let ((@x1418 (trans (monotonicity @x1410 (= $x859 (or (or $x1399 $x841) $x851))) (rewrite (= (or (or $x1399 $x841) $x851) $x1414)) (= $x859 $x1414))))
-(let ((@x1658 (monotonicity (quant-intro @x1418 (= $x862 $x1419)) (monotonicity @x1652 (= $x1366 $x1653)) (= $x1369 (and $x1419 $x1653)))))
-(let ((@x1385 (rewrite (= (not (not (or (not $x1078) $x831))) (or (not $x1078) $x831)))))
-(let ((@x1383 (monotonicity (rewrite (= (and $x1078 $x1079) (not (or (not $x1078) $x831)))) (= $x1077 (not (not (or (not $x1078) $x831)))))))
-(let ((@x1390 (monotonicity (trans @x1383 @x1385 (= $x1077 (or (not $x1078) $x831))) (= $x1084 (or (or (not $x1078) $x831) $x1083)))))
-(let ((@x1395 (trans @x1390 (rewrite (= (or (or (not $x1078) $x831) $x1083) $x1391)) (= $x1084 $x1391))))
-(let ((@x1669 (monotonicity (monotonicity @x1395 (= $x1085 $x1396)) (trans @x1658 (rewrite (= (and $x1419 $x1653) $x1662)) (= $x1369 $x1662)) (= $x1372 $x1667))))
-(let (($x1181 (<= (+ ?x1179 (* (- 1) v_b_max_G_3$)) 0)))
-(let (($x1182 (or (not (and $x1173 (not (>= (+ ?v0!5 (* (- 1) v_b_p_G_1$)) 0)))) $x1181)))
-(let (($x1183 (not $x1182)))
-(let (($x1200 (or $x1183 $x1196)))
-(let (($x1041 (and $x882 $x885 $x980 $x144 $x145 $x989 $x991 $x996)))
-(let (($x1044 (not $x1041)))
-(let (($x1208 (not $x1044)))
-(let (($x1211 (and $x1208 $x1200)))
-(let (($x999 (and $x882 $x885 $x985 $x104 $x107 $x109 $x989 $x991 $x996)))
-(let (($x1002 (not $x999)))
-(let (($x1169 (not $x1002)))
-(let (($x1204 (and $x1169 $x1200)))
-(let (($x1215 (or $x1204 $x1211)))
-(let (($x974 (and $x882 $x885 $x971)))
-(let (($x977 (not $x974)))
-(let (($x1166 (not $x977)))
-(let (($x1219 (and $x1166 $x1215)))
-(let (($x1150 (not (or $x1145 (<= (+ (v_b_array$ ?v0!4) (* (- 1) v_b_max_G_4$)) 0)))))
-(let (($x1154 (and $x1132 $x1150)))
-(let (($x1158 (or $x1119 $x1154)))
-(let (($x922 (and $x882 $x885 $x919 k!00 $x73 k!10)))
-(let (($x925 (not $x922)))
-(let (($x1113 (not $x925)))
-(let (($x1162 (and $x1113 $x1158)))
-(let (($x1223 (or $x1162 $x1219)))
-(let (($x912 (and $x882 $x885 $x909 $x63)))
-(let (($x1227 (and $x912 $x1223)))
-(let (($x1231 (or $x1095 $x1227)))
-(let (($x1235 (and $x862 $x1231)))
-(let (($x1239 (or $x1085 $x1235)))
-(let (($x1305 (= (+ ?x1179 (* (- 1) v_b_max_G_3$)) (+ (* (- 1) v_b_max_G_3$) ?x1179))))
-(let ((@x1309 (monotonicity (rewrite $x1305) (= $x1181 (<= (+ (* (- 1) v_b_max_G_3$) ?x1179) 0)))))
-(let ((@x1316 (trans @x1309 (rewrite (= (<= (+ (* (- 1) v_b_max_G_3$) ?x1179) 0) $x1312)) (= $x1181 $x1312))))
-(let (($x1302 (= (not (and $x1173 (not (>= (+ ?v0!5 (* (- 1) v_b_p_G_1$)) 0)))) $x1301)))
-(let (($x1299 (= (and $x1173 (not (>= (+ ?v0!5 (* (- 1) v_b_p_G_1$)) 0))) $x1298)))
-(let (($x1175 (>= (+ ?v0!5 (* (- 1) v_b_p_G_1$)) 0)))
-(let (($x1283 (= (+ ?v0!5 (* (- 1) v_b_p_G_1$)) (+ (* (- 1) v_b_p_G_1$) ?v0!5))))
-(let ((@x1287 (monotonicity (rewrite $x1283) (= $x1175 (>= (+ (* (- 1) v_b_p_G_1$) ?v0!5) 0)))))
-(let ((@x1294 (trans @x1287 (rewrite (= (>= (+ (* (- 1) v_b_p_G_1$) ?v0!5) 0) $x1290)) (= $x1175 $x1290))))
-(let ((@x1303 (monotonicity (monotonicity (monotonicity @x1294 (= (not $x1175) $x1295)) $x1299) $x1302)))
-(let ((@x1322 (monotonicity (monotonicity @x1303 @x1316 (= $x1182 $x1317)) (= $x1183 $x1320))))
-(let ((@x1338 (monotonicity (rewrite (= $x1208 $x1041)) (monotonicity @x1322 (= $x1200 $x1323)) (= $x1211 (and $x1041 $x1323)))))
-(let ((@x1328 (monotonicity (rewrite (= $x1169 $x999)) (monotonicity @x1322 (= $x1200 $x1323)) (= $x1204 (and $x999 $x1323)))))
-(let ((@x1346 (monotonicity (trans @x1328 (rewrite (= (and $x999 $x1323) $x1329)) (= $x1204 $x1329)) (trans @x1338 (rewrite (= (and $x1041 $x1323) $x1339)) (= $x1211 $x1339)) (= $x1215 $x1344))))
-(let ((@x1349 (monotonicity (rewrite (= $x1166 $x974)) @x1346 (= $x1219 (and $x974 $x1344)))))
-(let (($x1259 (= (or $x1145 (<= (+ (v_b_array$ ?v0!4) (* (- 1) v_b_max_G_4$)) 0)) $x1258)))
-(let (($x1148 (<= (+ (v_b_array$ ?v0!4) (* (- 1) v_b_max_G_4$)) 0)))
-(let (($x1254 (= (<= (+ (* (- 1) v_b_max_G_4$) (v_b_array$ ?v0!4)) 0) $x1253)))
-(let (($x1249 (= $x1148 (<= (+ (* (- 1) v_b_max_G_4$) (v_b_array$ ?v0!4)) 0))))
-(let (($x1246 (= (+ (v_b_array$ ?v0!4) (* (- 1) v_b_max_G_4$)) (+ (* (- 1) v_b_max_G_4$) (v_b_array$ ?v0!4)))))
-(let ((@x1257 (trans (monotonicity (rewrite $x1246) $x1249) (rewrite $x1254) (= $x1148 $x1253))))
-(let ((@x1266 (monotonicity (monotonicity (monotonicity @x1257 $x1259) (= $x1150 $x1261)) (= $x1154 $x1264))))
-(let ((@x1272 (monotonicity (rewrite (= $x1113 $x922)) (monotonicity @x1266 (= $x1158 $x1267)) (= $x1162 (and $x922 $x1267)))))
-(let ((@x1357 (monotonicity (trans @x1272 (rewrite (= (and $x922 $x1267) $x1273)) (= $x1162 $x1273)) (trans @x1349 (rewrite (= (and $x974 $x1344) $x1350)) (= $x1219 $x1350)) (= $x1223 $x1355))))
-(let ((@x1365 (trans (monotonicity @x1357 (= $x1227 (and $x912 $x1355))) (rewrite (= (and $x912 $x1355) $x1361)) (= $x1227 $x1361))))
-(let ((@x1374 (monotonicity (monotonicity (monotonicity @x1365 (= $x1231 $x1366)) (= $x1235 $x1369)) (= $x1239 $x1372))))
-(let (($x1029 (not $x1026)))
-(let (($x1032 (or $x1029 $x136)))
-(let (($x1035 (and $x1026 $x1032)))
-(let (($x1047 (or $x1044 $x1035)))
-(let (($x1038 (or $x1002 $x1035)))
-(let (($x1050 (and $x1038 $x1047)))
-(let (($x1053 (or $x977 $x1050)))
-(let (($x959 (forall ((?v0 Int) )(let (($x838 (>= ?v0 0)))
-(let (($x936 (and $x838 (not (<= (+ v_b_length$ (* (- 1) ?v0)) 0)))))
-(let (($x939 (not $x936)))
-(or $x939 (<= (+ (v_b_array$ ?v0) (* (- 1) v_b_max_G_4$)) 0))))))
-))
-(let (($x945 (exists ((?v0 Int) )(let ((?x46 (v_b_array$ ?v0)))
-(let (($x86 (= ?x46 v_b_max_G_4$)))
-(let (($x838 (>= ?v0 0)))
-(let (($x936 (and $x838 (not (<= (+ v_b_length$ (* (- 1) ?v0)) 0)))))
-(let (($x939 (not $x936)))
-(or $x939 $x86)))))))
-))
-(let (($x948 (not $x945)))
-(let (($x962 (or $x948 $x959)))
-(let (($x965 (and $x945 $x962)))
-(let (($x968 (or $x925 $x965)))
-(let (($x1056 (and $x968 $x1053)))
-(let (($x915 (not $x912)))
-(let (($x1059 (or $x915 $x1056)))
-(let (($x1062 (and $x50 $x1059)))
-(let (($x878 (not $x862)))
-(let (($x1065 (or $x878 $x1062)))
-(let (($x1071 (not (and $x862 $x1065))))
-(let ((@x1192 (nnf-neg (nnf-pos (refl (~ $x1023 $x1023)) (~ $x1026 $x1026)) (~ (not $x1029) $x1026))))
-(let ((@x1203 (nnf-neg (sk (~ $x1029 $x1183)) (nnf-neg @x1192 (refl (~ $x1193 $x1193)) (~ (not $x1032) $x1196)) (~ (not $x1035) $x1200))))
-(let ((@x1218 (nnf-neg (nnf-neg (refl (~ $x1169 $x1169)) @x1203 (~ (not $x1038) $x1204)) (nnf-neg (refl (~ $x1208 $x1208)) @x1203 (~ (not $x1047) $x1211)) (~ (not $x1050) $x1215))))
-(let ((@x1157 (nnf-neg (nnf-neg (sk (~ $x945 $x1132)) (~ (not $x948) $x1132)) (sk (~ (not $x959) $x1150)) (~ (not $x962) $x1154))))
-(let ((@x1161 (nnf-neg (nnf-neg (refl (~ (not $x942) (not $x942))) (~ $x948 $x1119)) @x1157 (~ (not $x965) $x1158))))
-(let ((@x1226 (nnf-neg (nnf-neg (refl (~ $x1113 $x1113)) @x1161 (~ (not $x968) $x1162)) (nnf-neg (refl (~ $x1166 $x1166)) @x1218 (~ (not $x1053) $x1219)) (~ (not $x1056) $x1223))))
-(let ((@x1109 (monotonicity (refl (~ $x882 $x882)) (refl (~ $x885 $x885)) (nnf-pos (refl (~ $x906 $x906)) (~ $x909 $x909)) (refl (~ $x63 $x63)) (~ $x912 $x912))))
-(let ((@x1230 (nnf-neg (nnf-neg @x1109 (~ (not $x915) $x912)) @x1226 (~ (not $x1059) $x1227))))
-(let ((@x1094 (nnf-neg (nnf-pos (refl (~ $x859 $x859)) (~ $x862 $x862)) (~ (not $x878) $x862))))
-(let ((@x1238 (nnf-neg @x1094 (nnf-neg (refl (~ $x1095 $x1095)) @x1230 (~ (not $x1062) $x1231)) (~ (not $x1065) $x1235))))
-(let (($x749 (and $x52 $x54 $x69 k!00 $x73 k!10)))
-(let (($x752 (not $x749)))
-(let (($x785 (or $x752 $x403)))
-(let (($x788 (and $x785 $x682)))
-(let (($x738 (not $x279)))
-(let (($x816 (or $x738 $x788)))
-(let (($x819 (and $x50 $x816)))
-(let (($x822 (or $x705 $x819)))
-(let (($x825 (and $x234 $x822)))
-(let (($x828 (not $x825)))
-(let ((@x1011 (monotonicity (rewrite (= (<= v_b_p_G_1$ ?0) $x1005)) (= $x557 (not $x1005)))))
-(let ((@x837 (rewrite (= $x43 $x838))))
-(let ((@x1017 (monotonicity (monotonicity @x837 @x1011 (= $x560 $x1012)) (= (not $x560) $x1015))))
-(let ((@x1028 (quant-intro (monotonicity @x1017 (rewrite (= $x132 $x1020)) (= $x567 $x1023)) (= $x572 $x1026))))
-(let ((@x1034 (monotonicity (monotonicity @x1028 (= (not $x572) $x1029)) (= $x595 $x1032))))
-(let ((@x886 (rewrite (= $x54 $x885))))
-(let ((@x883 (rewrite (= $x52 $x882))))
-(let ((@x1043 (monotonicity @x883 @x886 (rewrite (= $x143 $x980)) (rewrite (= $x110 $x989)) (rewrite (= $x456 $x991)) (rewrite (= $x116 $x996)) (= $x654 $x1041))))
-(let ((@x1049 (monotonicity (monotonicity @x1043 (= $x669 $x1044)) (monotonicity @x1028 @x1034 (= $x600 $x1035)) (= $x670 $x1047))))
-(let ((@x1001 (monotonicity @x883 @x886 (monotonicity (rewrite (= $x143 $x980)) (= $x441 $x985)) (rewrite (= $x110 $x989)) (rewrite (= $x456 $x991)) (rewrite (= $x116 $x996)) (= $x544 $x999))))
-(let ((@x1040 (monotonicity (monotonicity @x1001 (= $x606 $x1002)) (monotonicity @x1028 @x1034 (= $x600 $x1035)) (= $x607 $x1038))))
-(let ((@x976 (monotonicity @x883 @x886 (monotonicity (rewrite (= $x69 $x919)) (= $x415 $x971)) (= $x429 $x974))))
-(let ((@x1055 (monotonicity (monotonicity @x976 (= $x681 $x977)) (monotonicity @x1040 @x1049 (= $x675 $x1050)) (= $x682 $x1053))))
-(let ((@x935 (monotonicity (rewrite (= (<= v_b_length$ ?0) $x930)) (= $x351 (not $x930)))))
-(let ((@x941 (monotonicity (monotonicity @x837 @x935 (= $x354 $x936)) (= $x360 $x939))))
-(let ((@x958 (monotonicity @x941 (rewrite (= $x89 (<= (+ ?x46 (* (- 1) v_b_max_G_4$)) 0))) (= $x372 (or $x939 (<= (+ ?x46 (* (- 1) v_b_max_G_4$)) 0))))))
-(let ((@x950 (monotonicity (quant-intro (monotonicity @x941 (= $x361 $x942)) (= $x366 $x945)) (= (not $x366) $x948))))
-(let ((@x967 (monotonicity (quant-intro (monotonicity @x941 (= $x361 $x942)) (= $x366 $x945)) (monotonicity @x950 (quant-intro @x958 (= $x377 $x959)) (= $x398 $x962)) (= $x403 $x965))))
-(let ((@x927 (monotonicity (monotonicity @x883 @x886 (rewrite (= $x69 $x919)) (= $x749 $x922)) (= $x752 $x925))))
-(let ((@x1058 (monotonicity (monotonicity @x927 @x967 (= $x785 $x968)) @x1055 (= $x788 $x1056))))
-(let ((@x894 (monotonicity (rewrite (= (<= v_b_p_G_0$ ?0) $x888)) (= $x244 (not $x888)))))
-(let ((@x900 (monotonicity (monotonicity @x837 @x894 (= $x247 $x895)) (= (not $x247) $x898))))
-(let ((@x911 (quant-intro (monotonicity @x900 (rewrite (= $x59 $x903)) (= $x254 $x906)) (= $x259 $x909))))
-(let ((@x917 (monotonicity (monotonicity @x883 @x886 @x911 (= $x279 $x912)) (= $x738 $x915))))
-(let ((@x1064 (monotonicity (monotonicity @x917 @x1058 (= $x816 $x1059)) (= $x819 $x1062))))
-(let ((@x848 (monotonicity (rewrite (= (<= 1 ?0) $x841)) (= (not (<= 1 ?0)) (not $x841)))))
-(let ((@x834 (monotonicity (monotonicity @x837 @x848 (= (and $x43 (not (<= 1 ?0))) $x849)) (= (not (and $x43 (not (<= 1 ?0)))) $x854))))
-(let ((@x877 (quant-intro (monotonicity @x834 (rewrite (= $x47 $x851)) (= $x229 $x859)) (= $x234 $x862))))
-(let ((@x1067 (monotonicity (monotonicity @x877 (= $x705 $x878)) @x1064 (= $x822 $x1065))))
-(let ((@x1073 (monotonicity (monotonicity @x877 @x1067 (= $x825 (and $x862 $x1065))) (= $x828 $x1071))))
-(let ((@x796 (monotonicity (monotonicity @x238 @x240 @x450 @x460 @x463 (= $x654 $x654)) (= $x669 $x669))))
-(let ((@x784 (monotonicity (monotonicity @x238 @x240 @x450 @x460 @x463 (= $x544 $x544)) (= $x606 $x606))))
-(let ((@x800 (monotonicity (monotonicity @x784 (= $x607 $x607)) (monotonicity @x796 (= $x670 $x670)) (= $x675 $x675))))
-(let ((@x780 (monotonicity (monotonicity @x238 @x240 (= $x429 $x429)) (= $x681 $x681))))
-(let ((@x846 (monotonicity (monotonicity @x238 @x240 (= $x749 $x749)) (= $x752 $x752))))
-(let ((@x864 (monotonicity (monotonicity @x846 (= $x785 $x785)) (monotonicity @x780 @x800 (= $x682 $x682)) (= $x788 $x788))))
-(let ((@x762 (monotonicity (monotonicity @x238 @x240 (= $x279 $x279)) (= $x738 $x738))))
-(let ((@x868 (monotonicity (monotonicity @x762 @x864 (= $x816 $x816)) (= $x819 $x819))))
-(let ((@x874 (monotonicity (monotonicity (monotonicity @x868 (= $x822 $x822)) (= $x825 $x825)) (= $x828 $x828))))
-(let ((@x751 (monotonicity (apply-def (intro-def (= $x71 k!00)) (~ $x71 k!00)) (apply-def (intro-def (= $x75 k!10)) (~ $x75 k!10)) (= $x338 $x749))))
-(let ((@x790 (monotonicity (monotonicity (monotonicity @x751 (= $x409 $x752)) (= $x410 $x785)) (= $x687 $x788))))
-(let ((@x821 (monotonicity (monotonicity @x790 (= (or $x738 $x687) $x816)) (= (and $x50 (or $x738 $x687)) $x819))))
-(let ((@x827 (monotonicity (monotonicity @x821 (= (or $x705 (and $x50 (or $x738 $x687))) $x822)) (= (and $x234 (or $x705 (and $x50 (or $x738 $x687)))) $x825))))
-(let ((@x830 (monotonicity @x827 (= (not (and $x234 (or $x705 (and $x50 (or $x738 $x687))))) $x828))))
-(let (($x739 (or $x738 $x687)))
-(let (($x740 (and $x50 $x739)))
-(let (($x741 (or $x705 $x740)))
-(let (($x742 (and $x234 $x741)))
-(let (($x743 (not $x742)))
-(let ((@x766 (monotonicity (monotonicity @x238 @x240 (= $x338 $x338)) (= $x409 $x409))))
-(let ((@x804 (monotonicity (monotonicity @x766 (= $x410 $x410)) (monotonicity @x780 @x800 (= $x682 $x682)) (= $x687 $x687))))
-(let ((@x808 (monotonicity (monotonicity @x762 @x804 (= $x739 $x739)) (= $x740 $x740))))
-(let ((@x814 (monotonicity (monotonicity (monotonicity @x808 (= $x741 $x741)) (= $x742 $x742)) (= $x743 $x743))))
-(let ((@x746 (mp (not-or-elim @x726 (not $x711)) (rewrite* (= (not $x711) $x743)) $x743)))
-(let ((@x1242 (mp~ (mp (mp (mp (mp @x746 @x814 $x743) @x830 $x828) @x874 $x828) @x1073 $x1071) (nnf-neg (sk (~ $x878 $x1085)) @x1238 (~ $x1071 $x1239)) $x1239)))
-(let ((@x2191 (mp (mp (mp @x1242 @x1374 $x1372) @x1669 $x1667) (monotonicity @x2187 (= $x1667 (or $x1396 $x2185))) (or $x1396 $x2185))))
-(let ((@x2302 (unit-resolution (def-axiom (or $x2182 $x2176)) (unit-resolution @x2191 (lemma @x1930 $x1391) $x2185) $x2176)))
-(let ((@x2309 (unit-resolution (def-axiom (or $x2179 $x1095 $x2173)) (mp @x737 (symm (commutativity (= $x50 $x31)) (= $x31 $x50)) $x50) (or $x2179 $x2173))))
-(let ((@x2310 (unit-resolution @x2309 @x2302 $x2173)))
-(let ((@x2410 (monotonicity (unit-resolution (def-axiom (or $x2146 $x144)) @x2389 $x144) (= ?x135 ?x62))))
-(let ((@x2413 (trans @x2410 (unit-resolution (def-axiom (or $x2170 $x63)) @x2310 $x63) (= ?x135 v_b_max_G_1$))))
-(let ((@x2414 (trans @x2413 (symm (unit-resolution (def-axiom (or $x2146 $x145)) @x2389 $x145) $x2022) $x136)))
-(let ((@x2416 (unit-resolution (def-axiom (or $x2137 $x1560 $x2131)) (unit-resolution (def-axiom (or $x2128 $x1193)) @x2414 $x2128) (unit-resolution (def-axiom (or $x2146 $x2134)) @x2389 $x2134) $x1560)))
-(let ((@x2421 (unit-resolution ((_ th-lemma arith assign-bounds 1 -1 -1) (or $x1693 $x985 $x1312 (not $x2024))) (unit-resolution (def-axiom (or $x1555 $x1678)) @x2416 $x1678) @x2406 (unit-resolution (def-axiom (or $x2146 $x980)) @x2389 $x980) $x1693)))
-(let (($x1798 (= v_b_p_G_0$ ?v0!5)))
-(let (($x1800 (>= (+ v_b_p_G_0$ (* (- 1) ?v0!5)) 0)))
-(let (($x1764 (>= (+ v_b_p_G_0$ (* (- 1) v_b_p_G_1$)) (- 1))))
-(let ((@x2426 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x1605 $x1764)) (unit-resolution (def-axiom (or $x2146 $x991)) @x2389 $x991) $x1764)))
-(let ((@x2430 (unit-resolution ((_ th-lemma arith assign-bounds -1 -1) (or $x1800 $x1290 (not $x1764))) (unit-resolution (def-axiom (or $x1555 $x1295)) @x2416 $x1295) @x2426 $x1800)))
-(let (($x1751 (<= (+ v_b_p_G_0$ (* (- 1) ?v0!5)) 0)))
-(let (($x1728 (>= (+ v_b_max_G_1$ (* (- 1) ?x1179)) 0)))
-(let (($x2195 (not $x1728)))
-(let ((@x2433 (unit-resolution ((_ th-lemma arith assign-bounds -1 -1) (or $x2195 $x1312 (not $x2024))) @x2406 (unit-resolution (def-axiom (or $x1555 $x1678)) @x2416 $x1678) $x2195)))
-(let ((@x2333 (unit-resolution (def-axiom (or $x2170 $x2095)) @x2310 $x2095)))
-(let (($x1716 (or $x2100 $x1540 $x1751 $x1728)))
-(let (($x1775 (<= (+ ?x1179 (* (- 1) v_b_max_G_1$)) 0)))
-(let (($x1789 (>= (+ ?v0!5 (* (- 1) v_b_p_G_0$)) 0)))
-(let (($x1717 (or $x2100 (or $x1540 $x1789 $x1775))))
-(let (($x1739 (= (+ ?x1179 (* (- 1) v_b_max_G_1$)) (+ (* (- 1) v_b_max_G_1$) ?x1179))))
-(let ((@x1726 (monotonicity (rewrite $x1739) (= $x1775 (<= (+ (* (- 1) v_b_max_G_1$) ?x1179) 0)))))
-(let ((@x1732 (trans @x1726 (rewrite (= (<= (+ (* (- 1) v_b_max_G_1$) ?x1179) 0) $x1728)) (= $x1775 $x1728))))
-(let (($x1743 (= (+ ?v0!5 (* (- 1) v_b_p_G_0$)) (+ (* (- 1) v_b_p_G_0$) ?v0!5))))
-(let ((@x1749 (monotonicity (rewrite $x1743) (= $x1789 (>= (+ (* (- 1) v_b_p_G_0$) ?v0!5) 0)))))
-(let ((@x1755 (trans @x1749 (rewrite (= (>= (+ (* (- 1) v_b_p_G_0$) ?v0!5) 0) $x1751)) (= $x1789 $x1751))))
-(let ((@x1715 (monotonicity @x1755 @x1732 (= (or $x1540 $x1789 $x1775) (or $x1540 $x1751 $x1728)))))
-(let ((@x1690 (trans (monotonicity @x1715 (= $x1717 (or $x2100 (or $x1540 $x1751 $x1728)))) (rewrite (= (or $x2100 (or $x1540 $x1751 $x1728)) $x1716)) (= $x1717 $x1716))))
-(let ((@x2435 (unit-resolution (mp ((_ quant-inst ?v0!5) $x1717) @x1690 $x1716) @x2333 (unit-resolution (def-axiom (or $x1555 $x1173)) @x2416 $x1173) @x2433 $x1751)))
-(let ((@x2436 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x1798 (not $x1751) (not $x1800))) @x2435 @x2430 $x1798)))
-(let ((@x1807 (monotonicity (symm (hypothesis $x1798) (= ?v0!5 v_b_p_G_0$)) (= ?x1179 ?x101))))
-(let ((@x1796 (lemma (unit-resolution (hypothesis $x1803) (symm @x1807 $x1799) false) (or (not $x1798) $x1799))))
-(let ((@x2437 (unit-resolution @x1796 @x2436 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x1803 $x1703)) @x2421 $x1803) false)))
-(let (($x2228 (= v_b_max_G_1$ v_b_max_G_4$)))
-(let ((@x2349 (symm (unit-resolution (def-axiom (or $x2114 $x73)) (hypothesis $x2117) $x73) $x2228)))
-(let ((@x2352 ((_ th-lemma arith triangle-eq) (or (not $x2228) (<= (+ v_b_max_G_1$ (* (- 1) v_b_max_G_4$)) 0)))))
-(let ((@x2353 (unit-resolution @x2352 @x2349 (<= (+ v_b_max_G_1$ (* (- 1) v_b_max_G_4$)) 0))))
-(let (($x2265 (>= (+ v_b_max_G_1$ (* (- 1) (v_b_array$ ?v0!4))) 0)))
-(let (($x1143 (not $x1142)))
-(let (($x2077 (not $x2103)))
-(let (($x2282 (= ?x62 v_b_max_G_4$)))
-(let (($x2283 (or $x1528 (<= (+ v_b_length$ (* (- 1) v_b_k_G_0$)) 0) $x2282)))
-(let ((@x2313 (trans (unit-resolution (def-axiom (or $x2170 $x63)) @x2310 $x63) (symm (hypothesis $x73) $x2228) $x2282)))
-(let ((@x2316 (unit-resolution ((_ quant-inst v_b_k_G_0$) (or $x2077 (not $x2283))) (hypothesis $x2103) (unit-resolution (def-axiom (or $x2283 (not $x2282))) @x2313 $x2283) false)))
-(let ((@x2355 (unit-resolution (lemma @x2316 (or $x2077 $x1531)) (unit-resolution (def-axiom (or $x2114 $x73)) (hypothesis $x2117) $x73) $x2077)))
-(let ((@x2356 (unit-resolution (def-axiom (or $x2111 $x2103 $x1517)) @x2355 (unit-resolution (def-axiom (or $x2114 $x2108)) (hypothesis $x2117) $x2108) $x1517)))
-(let ((@x2343 ((_ th-lemma arith farkas -1 -1 1) (hypothesis (<= (+ v_b_p_G_0$ (* (- 1) ?v0!4)) 0)) (hypothesis $x919) (hypothesis $x1143) false)))
-(let ((@x2346 (lemma @x2343 (or (not (<= (+ v_b_p_G_0$ (* (- 1) ?v0!4)) 0)) $x971 $x1142))))
-(let ((@x2359 (unit-resolution @x2346 (unit-resolution (def-axiom (or $x2114 $x919)) (hypothesis $x2117) $x919) (unit-resolution (def-axiom (or $x1516 $x1143)) @x2356 $x1143) (not (<= (+ v_b_p_G_0$ (* (- 1) ?v0!4)) 0)))))
-(let (($x2272 (<= (+ v_b_p_G_0$ (* (- 1) ?v0!4)) 0)))
-(let (($x2296 (or $x2100 $x1489 $x2272 $x2265)))
-(let (($x2249 (<= (+ (v_b_array$ ?v0!4) (* (- 1) v_b_max_G_1$)) 0)))
-(let (($x2241 (>= (+ ?v0!4 (* (- 1) v_b_p_G_0$)) 0)))
-(let (($x2300 (or $x2100 (or $x1489 $x2241 $x2249))))
-(let (($x2266 (= (<= (+ (* (- 1) v_b_max_G_1$) (v_b_array$ ?v0!4)) 0) $x2265)))
-(let (($x2260 (= $x2249 (<= (+ (* (- 1) v_b_max_G_1$) (v_b_array$ ?v0!4)) 0))))
-(let (($x2278 (= (+ (v_b_array$ ?v0!4) (* (- 1) v_b_max_G_1$)) (+ (* (- 1) v_b_max_G_1$) (v_b_array$ ?v0!4)))))
-(let ((@x2292 (trans (monotonicity (rewrite $x2278) $x2260) (rewrite $x2266) (= $x2249 $x2265))))
-(let (($x2253 (= (+ ?v0!4 (* (- 1) v_b_p_G_0$)) (+ (* (- 1) v_b_p_G_0$) ?v0!4))))
-(let ((@x2258 (monotonicity (rewrite $x2253) (= $x2241 (>= (+ (* (- 1) v_b_p_G_0$) ?v0!4) 0)))))
-(let ((@x2276 (trans @x2258 (rewrite (= (>= (+ (* (- 1) v_b_p_G_0$) ?v0!4) 0) $x2272)) (= $x2241 $x2272))))
-(let ((@x2295 (monotonicity @x2276 @x2292 (= (or $x1489 $x2241 $x2249) (or $x1489 $x2272 $x2265)))))
-(let ((@x2319 (trans (monotonicity @x2295 (= $x2300 (or $x2100 (or $x1489 $x2272 $x2265)))) (rewrite (= (or $x2100 (or $x1489 $x2272 $x2265)) $x2296)) (= $x2300 $x2296))))
-(let ((@x2362 (unit-resolution (mp ((_ quant-inst ?v0!4) $x2300) @x2319 $x2296) @x2333 (unit-resolution (def-axiom (or $x1516 $x1139)) @x2356 $x1139) (or $x2272 $x2265))))
-(let ((@x2365 ((_ th-lemma arith farkas 1 -1 1) (unit-resolution (def-axiom (or $x1516 (not $x1253))) @x2356 (not $x1253)) (unit-resolution @x2362 @x2359 $x2265) @x2353 false)))
-(let ((@x2373 (unit-resolution (def-axiom (or $x2167 $x2117 $x2161)) (lemma @x2365 $x2114) (unit-resolution (def-axiom (or $x2170 $x2164)) @x2310 $x2164) $x2161)))
-(let ((@x2243 (unit-resolution (def-axiom (or $x2155 $x2143 $x2149)) (unit-resolution (def-axiom (or $x2158 $x2152)) @x2373 $x2152) $x2152)))
-(let ((@x2244 (unit-resolution @x2243 (lemma @x2437 $x2146) $x2143)))
-(let ((@x1791 (trans (monotonicity (hypothesis $x107) (= ?x135 ?x101)) (symm (hypothesis $x104) (= ?x101 v_b_max_G_2$)) (= ?x135 v_b_max_G_2$))))
-(let ((@x1769 (trans @x1791 (symm (hypothesis $x109) (= v_b_max_G_2$ v_b_max_G_3$)) $x136)))
-(let ((@x1771 (lemma (unit-resolution (hypothesis $x1193) @x1769 false) (or $x136 $x1603 $x1601 $x1602))))
-(let ((@x2380 (unit-resolution @x1771 (unit-resolution (def-axiom (or $x2140 $x109)) @x2244 $x109) (unit-resolution (def-axiom (or $x2140 $x104)) @x2244 $x104) (unit-resolution (def-axiom (or $x2140 $x107)) @x2244 $x107) $x136)))
-(let ((@x2368 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x1605 $x1764)) (unit-resolution (def-axiom (or $x2140 $x991)) @x2244 $x991) $x1764)))
-(let ((@x1699 (unit-resolution (def-axiom (or $x2137 $x1560 $x2131)) (unit-resolution (def-axiom (or $x2128 $x1193)) (hypothesis $x136) $x2128) (hypothesis $x2134) $x1560)))
-(let (($x2205 (not $x1800)))
-(let (($x1838 (<= (+ ?x101 (* (- 1) v_b_max_G_3$)) 0)))
-(let ((@x1685 (trans (symm (hypothesis $x104) (= ?x101 v_b_max_G_2$)) (symm (hypothesis $x109) (= v_b_max_G_2$ v_b_max_G_3$)) (= ?x101 v_b_max_G_3$))))
-(let ((@x1675 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x101 v_b_max_G_3$)) $x1838)) @x1685 $x1838)))
-(let ((@x1696 (lemma ((_ th-lemma arith farkas -1 -1 1) (hypothesis $x1678) (hypothesis $x1838) (hypothesis $x1703) false) (or $x1693 $x1312 (not $x1838)))))
-(let ((@x1677 (unit-resolution @x1696 (unit-resolution (def-axiom (or $x1555 $x1678)) @x1699 $x1678) @x1675 $x1693)))
-(let ((@x2193 (unit-resolution @x1796 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x1803 $x1703)) @x1677 $x1803) (not $x1798))))
-(let ((@x2198 (unit-resolution ((_ th-lemma arith assign-bounds 1 1 1) (or $x2195 $x1312 (not $x1838) $x980)) (unit-resolution (def-axiom (or $x1555 $x1678)) @x1699 $x1678) @x1675 (hypothesis $x985) $x2195)))
-(let ((@x2202 (unit-resolution (mp ((_ quant-inst ?v0!5) $x1717) @x1690 $x1716) (hypothesis $x2095) (unit-resolution (def-axiom (or $x1555 $x1173)) @x1699 $x1173) (or $x1751 $x1728))))
-(let ((@x2209 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x1798 (not $x1751) $x2205)) (unit-resolution @x2202 @x2198 $x1751) (or $x1798 $x2205))))
-(let ((@x2211 ((_ th-lemma arith farkas -1 1 1) (unit-resolution @x2209 @x2193 $x2205) (hypothesis $x1764) (unit-resolution (def-axiom (or $x1555 $x1295)) @x1699 $x1295) false)))
-(let ((@x2370 (unit-resolution (lemma @x2211 (or $x1193 (not $x1764) $x2100 $x980 $x2137 $x1601 $x1603)) @x2333 (or $x1193 (not $x1764) $x980 $x2137 $x1601 $x1603))))
-(unit-resolution @x2370 @x2368 @x2380 (unit-resolution (def-axiom (or $x2140 $x985)) @x2244 $x985) (unit-resolution (def-axiom (or $x2140 $x2134)) @x2244 $x2134) (unit-resolution (def-axiom (or $x2140 $x104)) @x2244 $x104) (unit-resolution (def-axiom (or $x2140 $x109)) @x2244 $x109) false)))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))
-
+3587bd3f21d47d812a1b3b30d0e7ce50216a24d3 779 0
+unsat
+((set-logic AUFLIA)
+(declare-fun ?v0!3 () Int)
+(declare-fun ?v0!2 () Int)
+(declare-fun ?v0!1 () Int)
+(declare-fun ?v0!0 () Int)
+(proof
+(let (($x109 (= v_b_max_G_3$ v_b_max_G_2$)))
+(let ((?x135 (v_b_array$ v_b_k_G_1$)))
+(let (($x136 (= ?x135 v_b_max_G_3$)))
+(let (($x1878 (forall ((?v0 Int) )(!(let (($x746 (<= (+ (v_b_array$ ?v0) (* (- 1) v_b_max_G_3$)) 0)))
+(let (($x733 (>= (+ ?v0 (* (- 1) v_b_p_G_1$)) 0)))
+(let (($x521 (>= ?v0 0)))
+(let (($x1157 (not $x521)))
+(or $x1157 $x733 $x746))))) :pattern ( (v_b_array$ ?v0) )))
+))
+(let (($x1883 (not $x1878)))
+(let (($x1886 (or $x1883 $x136)))
+(let (($x1889 (not $x1886)))
+(let (($x1070 (>= (+ v_b_max_G_3$ (* (- 1) (v_b_array$ ?v0!3))) 0)))
+(let (($x1048 (<= (+ v_b_p_G_1$ (* (- 1) ?v0!3)) 0)))
+(let (($x931 (>= ?v0!3 0)))
+(let (($x1298 (not $x931)))
+(let (($x1313 (or $x1298 $x1048 $x1070)))
+(let (($x1318 (not $x1313)))
+(let (($x1892 (or $x1318 $x1889)))
+(let (($x1895 (not $x1892)))
+(let (($x682 (>= v_b_p_G_1$ 2)))
+(let (($x1364 (not $x682)))
+(let (($x679 (>= v_b_k_G_1$ 0)))
+(let (($x1363 (not $x679)))
+(let ((?x685 (* (- 1) v_b_p_G_1$)))
+(let ((?x686 (+ v_b_p_G_0$ ?x685)))
+(let (($x684 (= ?x686 (- 1))))
+(let (($x1362 (not $x684)))
+(let (($x573 (>= v_b_p_G_0$ 1)))
+(let (($x1287 (not $x573)))
+(let (($x1361 (not $x109)))
+(let (($x107 (= v_b_k_G_1$ v_b_p_G_0$)))
+(let (($x1360 (not $x107)))
+(let ((?x101 (v_b_array$ v_b_p_G_0$)))
+(let (($x104 (= v_b_max_G_2$ ?x101)))
+(let (($x1359 (not $x104)))
+(let (($x689 (>= (+ v_b_max_G_1$ (* (- 1) ?x101)) 0)))
+(let (($x571 (>= v_b_k_G_0$ 0)))
+(let (($x1286 (not $x571)))
+(let (($x1898 (or $x1286 $x689 $x1359 $x1360 $x1361 $x1287 $x1362 $x1363 $x1364 $x1895)))
+(let (($x1901 (not $x1898)))
+(let (($x145 (= v_b_max_G_3$ v_b_max_G_1$)))
+(let (($x1376 (not $x145)))
+(let (($x144 (= v_b_k_G_1$ v_b_k_G_0$)))
+(let (($x1375 (not $x144)))
+(let (($x692 (not $x689)))
+(let (($x1904 (or $x692 $x1286 $x1375 $x1376 $x1287 $x1362 $x1363 $x1364 $x1895)))
+(let ((?x937 (v_b_array$ ?v0!3)))
+(let (($x1559 (= ?x101 ?x937)))
+(let (($x1563 (not $x1559)))
+(let ((?x1068 (* (- 1) ?x937)))
+(let ((?x1461 (+ ?x101 ?x1068)))
+(let (($x1445 (>= ?x1461 0)))
+(let (($x1453 (not $x1445)))
+(let (($x1907 (not $x1904)))
+(let ((@x2149 (hypothesis $x1907)))
+(let ((?x744 (* (- 1) v_b_max_G_3$)))
+(let ((?x1781 (+ v_b_max_G_1$ ?x744)))
+(let (($x1782 (<= ?x1781 0)))
+(let (($x1780 (= v_b_max_G_1$ v_b_max_G_3$)))
+(let ((@x2162 (mp (unit-resolution (def-axiom (or $x1904 $x145)) @x2149 $x145) (symm (commutativity (= $x1780 $x145)) (= $x145 $x1780)) $x1780)))
+(let (($x1436 (not $x1070)))
+(let ((?x62 (v_b_array$ v_b_k_G_0$)))
+(let (($x63 (= ?x62 v_b_max_G_1$)))
+(let (($x1910 (or $x1901 $x1907)))
+(let (($x1913 (not $x1910)))
+(let ((?x549 (* (- 1) v_b_p_G_0$)))
+(let ((?x599 (+ v_b_length$ ?x549)))
+(let (($x600 (<= ?x599 0)))
+(let (($x1916 (or $x600 $x1286 $x1287 $x1913)))
+(let (($x1919 (not $x1916)))
+(let (($x1011 (>= (+ v_b_max_G_4$ (* (- 1) (v_b_array$ ?v0!2))) 0)))
+(let (($x900 (<= (+ v_b_length$ (* (- 1) ?v0!2)) 0)))
+(let (($x897 (>= ?v0!2 0)))
+(let (($x1247 (not $x897)))
+(let (($x889 (= (v_b_array$ ?v0!1) v_b_max_G_4$)))
+(let (($x884 (<= (+ v_b_length$ (* (- 1) ?v0!1)) 0)))
+(let (($x881 (>= ?v0!1 0)))
+(let (($x1227 (not $x881)))
+(let (($x1242 (or $x1227 $x884 $x889)))
+(let (($x1273 (not $x1242)))
+(let (($x1274 (or $x1273 $x1247 $x900 $x1011)))
+(let (($x1275 (not $x1274)))
+(let (($x1861 (forall ((?v0 Int) )(!(let ((?x46 (v_b_array$ ?v0)))
+(let (($x86 (= ?x46 v_b_max_G_4$)))
+(let (($x622 (<= (+ v_b_length$ (* (- 1) ?v0)) 0)))
+(let (($x521 (>= ?v0 0)))
+(let (($x1157 (not $x521)))
+(let (($x1216 (or $x1157 $x622 $x86)))
+(not $x1216))))))) :pattern ( (v_b_array$ ?v0) )))
+))
+(let (($x1866 (or $x1861 $x1275)))
+(let (($x1869 (not $x1866)))
+(let (($x75 (= v_b_p_G_2$ v_b_p_G_0$)))
+(let (($x1290 (not $x75)))
+(let (($x73 (= v_b_max_G_4$ v_b_max_G_1$)))
+(let (($x1289 (not $x73)))
+(let (($x71 (= v_b_k_G_2$ v_b_k_G_0$)))
+(let (($x1288 (not $x71)))
+(let (($x661 (not $x600)))
+(let (($x1872 (or $x661 $x1286 $x1287 $x1288 $x1289 $x1290 $x1869)))
+(let (($x1875 (not $x1872)))
+(let (($x1922 (or $x1875 $x1919)))
+(let (($x1925 (not $x1922)))
+(let (($x1403 (not $x63)))
+(let (($x1853 (forall ((?v0 Int) )(!(let (($x561 (<= (+ (v_b_array$ ?v0) (* (- 1) v_b_max_G_1$)) 0)))
+(let (($x548 (>= (+ ?v0 (* (- 1) v_b_p_G_0$)) 0)))
+(let (($x521 (>= ?v0 0)))
+(let (($x1157 (not $x521)))
+(or $x1157 $x548 $x561))))) :pattern ( (v_b_array$ ?v0) )))
+))
+(let (($x1858 (not $x1853)))
+(let ((?x30 (v_b_array$ 0)))
+(let (($x50 (= ?x30 v_b_max_G_0$)))
+(let (($x851 (not $x50)))
+(let (($x1928 (or $x851 $x1858 $x1403 $x1286 $x1287 $x1925)))
+(let (($x1931 (not $x1928)))
+(let (($x1934 (or $x851 $x1931)))
+(let (($x1937 (not $x1934)))
+(let (($x1845 (forall ((?v0 Int) )(!(let (($x534 (>= (+ v_b_max_G_0$ (* (- 1) (v_b_array$ ?v0))) 0)))
+(let (($x524 (>= ?v0 1)))
+(let (($x521 (>= ?v0 0)))
+(let (($x1157 (not $x521)))
+(or $x1157 $x524 $x534))))) :pattern ( (v_b_array$ ?v0) )))
+))
+(let (($x1850 (not $x1845)))
+(let (($x1940 (or $x1850 $x1937)))
+(let (($x1943 (not $x1940)))
+(let (($x839 (>= (+ v_b_max_G_0$ (* (- 1) (v_b_array$ ?v0!0))) 0)))
+(let (($x832 (>= ?v0!0 1)))
+(let (($x835 (>= ?v0!0 0)))
+(let (($x1134 (not $x835)))
+(let (($x1149 (or $x1134 $x832 $x839)))
+(let (($x833 (not $x832)))
+(let (($x1154 (not $x1149)))
+(let ((@x1726 (hypothesis $x1154)))
+(let ((@x1711 ((_ th-lemma arith eq-propagate 0 0) (unit-resolution (def-axiom (or $x1149 $x835)) @x1726 $x835) (unit-resolution (def-axiom (or $x1149 $x833)) @x1726 $x833) (= ?v0!0 0))))
+(let ((@x1715 (symm (monotonicity @x1711 (= (v_b_array$ ?v0!0) ?x30)) (= ?x30 (v_b_array$ ?v0!0)))))
+(let (($x31 (= v_b_max_G_0$ ?x30)))
+(let (($x495 (<= v_b_length$ 0)))
+(let (($x496 (not $x495)))
+(let (($x511 (and $x496 $x31)))
+(let (($x752 (forall ((?v0 Int) )(let (($x746 (<= (+ (v_b_array$ ?v0) (* (- 1) v_b_max_G_3$)) 0)))
+(let (($x521 (>= ?v0 0)))
+(let (($x738 (and $x521 (not (>= (+ ?v0 (* (- 1) v_b_p_G_1$)) 0)))))
+(let (($x741 (not $x738)))
+(or $x741 $x746))))))
+))
+(let (($x755 (not $x752)))
+(let (($x758 (or $x755 $x136)))
+(let (($x761 (and $x752 $x758)))
+(let (($x784 (and $x689 $x571 $x144 $x145 $x573 $x684 $x679 $x682)))
+(let (($x789 (not $x784)))
+(let (($x792 (or $x789 $x761)))
+(let (($x725 (and $x571 $x692 $x104 $x107 $x109 $x573 $x684 $x679 $x682)))
+(let (($x730 (not $x725)))
+(let (($x764 (or $x730 $x761)))
+(let (($x795 (and $x764 $x792)))
+(let (($x670 (and $x661 $x571 $x573)))
+(let (($x675 (not $x670)))
+(let (($x798 (or $x675 $x795)))
+(let (($x649 (forall ((?v0 Int) )(let (($x521 (>= ?v0 0)))
+(let (($x626 (and $x521 (not (<= (+ v_b_length$ (* (- 1) ?v0)) 0)))))
+(let (($x629 (not $x626)))
+(or $x629 (<= (+ (v_b_array$ ?v0) (* (- 1) v_b_max_G_4$)) 0))))))
+))
+(let (($x635 (exists ((?v0 Int) )(let ((?x46 (v_b_array$ ?v0)))
+(let (($x86 (= ?x46 v_b_max_G_4$)))
+(let (($x521 (>= ?v0 0)))
+(let (($x626 (and $x521 (not (<= (+ v_b_length$ (* (- 1) ?v0)) 0)))))
+(let (($x629 (not $x626)))
+(or $x629 $x86)))))))
+))
+(let (($x638 (not $x635)))
+(let (($x652 (or $x638 $x649)))
+(let (($x655 (and $x635 $x652)))
+(let (($x612 (and $x600 $x571 $x573 $x71 $x73 $x75)))
+(let (($x617 (not $x612)))
+(let (($x658 (or $x617 $x655)))
+(let (($x801 (and $x658 $x798)))
+(let (($x567 (forall ((?v0 Int) )(let (($x561 (<= (+ (v_b_array$ ?v0) (* (- 1) v_b_max_G_1$)) 0)))
+(let (($x521 (>= ?v0 0)))
+(let (($x553 (and $x521 (not (>= (+ ?v0 (* (- 1) v_b_p_G_0$)) 0)))))
+(let (($x556 (not $x553)))
+(or $x556 $x561))))))
+))
+(let (($x591 (and $x50 $x567 $x63 $x571 $x573)))
+(let (($x596 (not $x591)))
+(let (($x804 (or $x596 $x801)))
+(let (($x807 (and $x50 $x804)))
+(let (($x541 (forall ((?v0 Int) )(let (($x534 (>= (+ v_b_max_G_0$ (* (- 1) (v_b_array$ ?v0))) 0)))
+(let (($x521 (>= ?v0 0)))
+(let (($x526 (and $x521 (not (>= ?v0 1)))))
+(let (($x529 (not $x526)))
+(or $x529 $x534))))))
+))
+(let (($x544 (not $x541)))
+(let (($x810 (or $x544 $x807)))
+(let (($x813 (and $x541 $x810)))
+(let (($x819 (not (or (not $x511) $x813))))
+(let (($x138 (=> (and $x136 false) true)))
+(let (($x139 (and $x136 $x138)))
+(let (($x134 (forall ((?v0 Int) )(let ((?x46 (v_b_array$ ?v0)))
+(let (($x132 (<= ?x46 v_b_max_G_3$)))
+(let (($x43 (<= 0 ?v0)))
+(let (($x131 (and $x43 (< ?v0 v_b_p_G_1$))))
+(=> $x131 $x132))))))
+))
+(let (($x140 (=> $x134 $x139)))
+(let (($x141 (and $x134 $x140)))
+(let (($x119 (and (= v_b_p_G_1$ (+ v_b_p_G_0$ 1)) (and (and (<= 0 v_b_k_G_1$) (<= 2 v_b_p_G_1$)) true))))
+(let (($x54 (<= 1 v_b_p_G_0$)))
+(let (($x110 (<= 0 v_b_k_G_1$)))
+(let (($x111 (and $x110 $x54)))
+(let (($x121 (and true (and $x111 $x119))))
+(let (($x148 (and true (and $x144 (and $x145 $x121)))))
+(let (($x55 (and (<= 0 v_b_k_G_0$) $x54)))
+(let (($x143 (<= ?x101 v_b_max_G_1$)))
+(let (($x152 (and true (and $x55 (and $x143 (and $x55 $x148))))))
+(let (($x153 (=> $x152 $x141)))
+(let (($x126 (and $x104 (and (and $x54 $x54) (and true (and $x107 (and $x109 $x121)))))))
+(let (($x102 (< v_b_max_G_1$ ?x101)))
+(let (($x129 (and true (and $x55 (and $x102 $x126)))))
+(let (($x142 (=> $x129 $x141)))
+(let (($x155 (=> (and true (and $x55 (and (< v_b_p_G_0$ v_b_length$) $x55))) (and $x142 $x153))))
+(let (($x91 (forall ((?v0 Int) )(let ((?x46 (v_b_array$ ?v0)))
+(let (($x89 (<= ?x46 v_b_max_G_4$)))
+(let (($x43 (<= 0 ?v0)))
+(let (($x85 (and $x43 (< ?v0 v_b_length$))))
+(=> $x85 $x89))))))
+))
+(let (($x92 (=> $x91 true)))
+(let (($x93 (and $x91 $x92)))
+(let (($x88 (exists ((?v0 Int) )(let ((?x46 (v_b_array$ ?v0)))
+(let (($x86 (= ?x46 v_b_max_G_4$)))
+(let (($x43 (<= 0 ?v0)))
+(let (($x85 (and $x43 (< ?v0 v_b_length$))))
+(=> $x85 $x86))))))
+))
+(let (($x94 (=> $x88 $x93)))
+(let (($x69 (<= v_b_length$ v_b_p_G_0$)))
+(let (($x81 (and $x69 (and $x55 (and true (and $x71 (and $x73 (and $x75 true))))))))
+(let (($x83 (and true (and $x55 $x81))))
+(let (($x96 (=> $x83 (and $x88 $x94))))
+(let (($x64 (and $x63 $x55)))
+(let (($x61 (forall ((?v0 Int) )(let ((?x46 (v_b_array$ ?v0)))
+(let (($x59 (<= ?x46 v_b_max_G_1$)))
+(let (($x43 (<= 0 ?v0)))
+(let (($x57 (and $x43 (< ?v0 v_b_p_G_0$))))
+(=> $x57 $x59))))))
+))
+(let (($x67 (and true (and $x55 (and $x61 $x64)))))
+(let (($x157 (=> (and $x50 $x67) (and $x96 $x155))))
+(let (($x49 (forall ((?v0 Int) )(let ((?x46 (v_b_array$ ?v0)))
+(let (($x47 (<= ?x46 v_b_max_G_0$)))
+(let (($x43 (<= 0 ?v0)))
+(let (($x45 (and $x43 (< ?v0 1))))
+(=> $x45 $x47))))))
+))
+(let (($x159 (=> $x49 (and $x50 $x157))))
+(let (($x32 (<= 0 0)))
+(let (($x38 (and $x31 (and $x32 (and $x32 (and (<= 1 1) (<= 1 1)))))))
+(let (($x39 (and true $x38)))
+(let (($x28 (< 0 v_b_length$)))
+(let (($x41 (and true (and $x28 $x39))))
+(let (($x161 (=> $x41 (and $x49 $x159))))
+(let (($x162 (not $x161)))
+(let (($x362 (forall ((?v0 Int) )(let ((?x46 (v_b_array$ ?v0)))
+(let (($x132 (<= ?x46 v_b_max_G_3$)))
+(or (not (and (<= 0 ?v0) (< ?v0 v_b_p_G_1$))) $x132))))
+))
+(let (($x385 (or (not $x362) $x136)))
+(let (($x390 (and $x362 $x385)))
+(let (($x117 (and $x110 (<= 2 v_b_p_G_1$))))
+(let (($x308 (= v_b_p_G_1$ (+ 1 v_b_p_G_0$))))
+(let (($x313 (and $x308 $x117)))
+(let (($x316 (and $x111 $x313)))
+(let (($x402 (and $x145 $x316)))
+(let (($x405 (and $x144 $x402)))
+(let (($x415 (and $x55 $x405)))
+(let (($x418 (and $x143 $x415)))
+(let (($x421 (and $x55 $x418)))
+(let (($x435 (or (not $x421) $x390)))
+(let (($x326 (and $x109 $x316)))
+(let (($x329 (and $x107 $x326)))
+(let (($x339 (and $x54 $x329)))
+(let (($x342 (and $x104 $x339)))
+(let (($x345 (and $x102 $x342)))
+(let (($x348 (and $x55 $x345)))
+(let (($x397 (or (not $x348) $x390)))
+(let (($x440 (and $x397 $x435)))
+(let (($x447 (or (not (and $x55 (and (< v_b_p_G_0$ v_b_length$) $x55))) $x440)))
+(let (($x263 (forall ((?v0 Int) )(let ((?x46 (v_b_array$ ?v0)))
+(let (($x89 (<= ?x46 v_b_max_G_4$)))
+(let (($x43 (<= 0 ?v0)))
+(let (($x85 (and $x43 (< ?v0 v_b_length$))))
+(let (($x253 (not $x85)))
+(or $x253 $x89)))))))
+))
+(let (($x257 (exists ((?v0 Int) )(let ((?x46 (v_b_array$ ?v0)))
+(let (($x86 (= ?x46 v_b_max_G_4$)))
+(let (($x43 (<= 0 ?v0)))
+(let (($x85 (and $x43 (< ?v0 v_b_length$))))
+(let (($x253 (not $x85)))
+(or $x253 $x86)))))))
+))
+(let (($x284 (or (not $x257) $x263)))
+(let (($x289 (and $x257 $x284)))
+(let (($x296 (or (not (and $x55 (and $x69 (and $x55 (and $x71 (and $x73 $x75)))))) $x289)))
+(let (($x452 (and $x296 $x447)))
+(let (($x203 (forall ((?v0 Int) )(let ((?x46 (v_b_array$ ?v0)))
+(let (($x59 (<= ?x46 v_b_max_G_1$)))
+(or (not (and (<= 0 ?v0) (< ?v0 v_b_p_G_0$))) $x59))))
+))
+(let (($x206 (and $x203 $x64)))
+(let (($x209 (and $x55 $x206)))
+(let (($x219 (and $x50 $x209)))
+(let (($x459 (or (not $x219) $x452)))
+(let (($x464 (and $x50 $x459)))
+(let (($x196 (forall ((?v0 Int) )(let ((?x46 (v_b_array$ ?v0)))
+(let (($x47 (<= ?x46 v_b_max_G_0$)))
+(or (not (and (<= 0 ?v0) (< ?v0 1))) $x47))))
+))
+(let (($x471 (or (not $x196) $x464)))
+(let (($x476 (and $x196 $x471)))
+(let (($x483 (or (not (and $x28 (and $x31 (and $x32 (and $x32 (<= 1 1)))))) $x476)))
+(let (($x746 (<= (+ (v_b_array$ ?0) ?x744) 0)))
+(let (($x521 (>= ?0 0)))
+(let (($x738 (and $x521 (not (>= (+ ?0 ?x685) 0)))))
+(let (($x741 (not $x738)))
+(let (($x749 (or $x741 $x746)))
+(let ((?x46 (v_b_array$ ?0)))
+(let (($x132 (<= ?x46 v_b_max_G_3$)))
+(let (($x359 (or (not (and (<= 0 ?0) (< ?0 v_b_p_G_1$))) $x132)))
+(let ((@x520 (rewrite (= (<= 0 ?0) $x521))))
+(let ((@x740 (monotonicity @x520 (rewrite (= (< ?0 v_b_p_G_1$) (not (>= (+ ?0 ?x685) 0)))) (= (and (<= 0 ?0) (< ?0 v_b_p_G_1$)) $x738))))
+(let ((@x743 (monotonicity @x740 (= (not (and (<= 0 ?0) (< ?0 v_b_p_G_1$))) $x741))))
+(let ((@x754 (quant-intro (monotonicity @x743 (rewrite (= $x132 $x746)) (= $x359 $x749)) (= $x362 $x752))))
+(let ((@x760 (monotonicity (monotonicity @x754 (= (not $x362) $x755)) (= $x385 $x758))))
+(let (($x772 (and $x144 (and $x145 (and (and $x679 $x573) (and $x684 (and $x679 $x682)))))))
+(let (($x576 (and $x571 $x573)))
+(let (($x770 (= $x402 (and $x145 (and (and $x679 $x573) (and $x684 (and $x679 $x682)))))))
+(let ((@x697 (monotonicity (rewrite (= $x110 $x679)) (rewrite (= (<= 2 v_b_p_G_1$) $x682)) (= $x117 (and $x679 $x682)))))
+(let ((@x700 (monotonicity (rewrite (= $x308 $x684)) @x697 (= $x313 (and $x684 (and $x679 $x682))))))
+(let ((@x575 (rewrite (= $x54 $x573))))
+(let ((@x703 (monotonicity (rewrite (= $x110 $x679)) @x575 (= $x111 (and $x679 $x573)))))
+(let ((@x706 (monotonicity @x703 @x700 (= $x316 (and (and $x679 $x573) (and $x684 (and $x679 $x682)))))))
+(let ((@x578 (monotonicity (rewrite (= (<= 0 v_b_k_G_0$) $x571)) @x575 (= $x55 $x576))))
+(let ((@x777 (monotonicity @x578 (monotonicity (monotonicity @x706 $x770) (= $x405 $x772)) (= $x415 (and $x576 $x772)))))
+(let ((@x780 (monotonicity (rewrite (= $x143 $x689)) @x777 (= $x418 (and $x689 (and $x576 $x772))))))
+(let ((@x783 (monotonicity @x578 @x780 (= $x421 (and $x576 (and $x689 (and $x576 $x772)))))))
+(let ((@x788 (trans @x783 (rewrite (= (and $x576 (and $x689 (and $x576 $x772))) $x784)) (= $x421 $x784))))
+(let ((@x794 (monotonicity (monotonicity @x788 (= (not $x421) $x789)) (monotonicity @x754 @x760 (= $x390 $x761)) (= $x435 $x792))))
+(let (($x710 (and $x107 (and $x109 (and (and $x679 $x573) (and $x684 (and $x679 $x682)))))))
+(let ((@x727 (rewrite (= (and $x576 (and $x692 (and $x104 (and $x573 $x710)))) $x725))))
+(let (($x708 (= $x326 (and $x109 (and (and $x679 $x573) (and $x684 (and $x679 $x682)))))))
+(let ((@x715 (monotonicity @x575 (monotonicity (monotonicity @x706 $x708) (= $x329 $x710)) (= $x339 (and $x573 $x710)))))
+(let ((@x721 (monotonicity (rewrite (= $x102 $x692)) (monotonicity @x715 (= $x342 (and $x104 (and $x573 $x710)))) (= $x345 (and $x692 (and $x104 (and $x573 $x710)))))))
+(let ((@x724 (monotonicity @x578 @x721 (= $x348 (and $x576 (and $x692 (and $x104 (and $x573 $x710))))))))
+(let ((@x732 (monotonicity (trans @x724 @x727 (= $x348 $x725)) (= (not $x348) $x730))))
+(let ((@x766 (monotonicity @x732 (monotonicity @x754 @x760 (= $x390 $x761)) (= $x397 $x764))))
+(let (($x99 (and $x55 (and (< v_b_p_G_0$ v_b_length$) $x55))))
+(let ((@x666 (monotonicity (rewrite (= (< v_b_p_G_0$ v_b_length$) $x661)) @x578 (= (and (< v_b_p_G_0$ v_b_length$) $x55) (and $x661 $x576)))))
+(let ((@x674 (trans (monotonicity @x578 @x666 (= $x99 (and $x576 (and $x661 $x576)))) (rewrite (= (and $x576 (and $x661 $x576)) $x670)) (= $x99 $x670))))
+(let ((@x800 (monotonicity (monotonicity @x674 (= (not $x99) $x675)) (monotonicity @x766 @x794 (= $x440 $x795)) (= $x447 $x798))))
+(let (($x626 (and $x521 (not (<= (+ v_b_length$ (* (- 1) ?0)) 0)))))
+(let (($x629 (not $x626)))
+(let (($x89 (<= ?x46 v_b_max_G_4$)))
+(let (($x43 (<= 0 ?0)))
+(let (($x85 (and $x43 (< ?0 v_b_length$))))
+(let (($x253 (not $x85)))
+(let (($x260 (or $x253 $x89)))
+(let (($x624 (= (< ?0 v_b_length$) (not (<= (+ v_b_length$ (* (- 1) ?0)) 0)))))
+(let ((@x631 (monotonicity (monotonicity @x520 (rewrite $x624) (= $x85 $x626)) (= $x253 $x629))))
+(let ((@x648 (monotonicity @x631 (rewrite (= $x89 (<= (+ ?x46 (* (- 1) v_b_max_G_4$)) 0))) (= $x260 (or $x629 (<= (+ ?x46 (* (- 1) v_b_max_G_4$)) 0))))))
+(let (($x86 (= ?x46 v_b_max_G_4$)))
+(let (($x632 (or $x629 $x86)))
+(let (($x254 (or $x253 $x86)))
+(let ((@x640 (monotonicity (quant-intro (monotonicity @x631 (= $x254 $x632)) (= $x257 $x635)) (= (not $x257) $x638))))
+(let ((@x657 (monotonicity (quant-intro (monotonicity @x631 (= $x254 $x632)) (= $x257 $x635)) (monotonicity @x640 (quant-intro @x648 (= $x263 $x649)) (= $x284 $x652)) (= $x289 $x655))))
+(let (($x618 (= (not (and $x55 (and $x69 (and $x55 (and $x71 (and $x73 $x75)))))) $x617)))
+(let (($x227 (and $x71 (and $x73 $x75))))
+(let (($x237 (and $x55 $x227)))
+(let (($x240 (and $x69 $x237)))
+(let (($x243 (and $x55 $x240)))
+(let ((@x608 (monotonicity (rewrite (= $x69 $x600)) (monotonicity @x578 (= $x237 (and $x576 $x227))) (= $x240 (and $x600 (and $x576 $x227))))))
+(let ((@x611 (monotonicity @x578 @x608 (= $x243 (and $x576 (and $x600 (and $x576 $x227)))))))
+(let ((@x616 (trans @x611 (rewrite (= (and $x576 (and $x600 (and $x576 $x227))) $x612)) (= $x243 $x612))))
+(let ((@x803 (monotonicity (monotonicity (monotonicity @x616 $x618) @x657 (= $x296 $x658)) @x800 (= $x452 $x801))))
+(let ((@x593 (rewrite (= (and $x50 (and $x576 (and $x567 (and $x63 $x576)))) $x591))))
+(let (($x561 (<= (+ ?x46 (* (- 1) v_b_max_G_1$)) 0)))
+(let (($x553 (and $x521 (not (>= (+ ?0 ?x549) 0)))))
+(let (($x556 (not $x553)))
+(let (($x564 (or $x556 $x561)))
+(let (($x59 (<= ?x46 v_b_max_G_1$)))
+(let (($x200 (or (not (and $x43 (< ?0 v_b_p_G_0$))) $x59)))
+(let ((@x555 (monotonicity @x520 (rewrite (= (< ?0 v_b_p_G_0$) (not (>= (+ ?0 ?x549) 0)))) (= (and $x43 (< ?0 v_b_p_G_0$)) $x553))))
+(let ((@x566 (monotonicity (monotonicity @x555 (= (not (and $x43 (< ?0 v_b_p_G_0$))) $x556)) (rewrite (= $x59 $x561)) (= $x200 $x564))))
+(let ((@x584 (monotonicity (quant-intro @x566 (= $x203 $x567)) (monotonicity @x578 (= $x64 (and $x63 $x576))) (= $x206 (and $x567 (and $x63 $x576))))))
+(let ((@x587 (monotonicity @x578 @x584 (= $x209 (and $x576 (and $x567 (and $x63 $x576)))))))
+(let ((@x590 (monotonicity @x587 (= $x219 (and $x50 (and $x576 (and $x567 (and $x63 $x576))))))))
+(let ((@x598 (monotonicity (trans @x590 @x593 (= $x219 $x591)) (= (not $x219) $x596))))
+(let ((@x809 (monotonicity (monotonicity @x598 @x803 (= $x459 $x804)) (= $x464 $x807))))
+(let (($x534 (>= (+ v_b_max_G_0$ (* (- 1) ?x46)) 0)))
+(let (($x526 (and $x521 (not (>= ?0 1)))))
+(let (($x529 (not $x526)))
+(let (($x538 (or $x529 $x534)))
+(let (($x47 (<= ?x46 v_b_max_G_0$)))
+(let (($x193 (or (not (and $x43 (< ?0 1))) $x47)))
+(let ((@x528 (monotonicity @x520 (rewrite (= (< ?0 1) (not (>= ?0 1)))) (= (and $x43 (< ?0 1)) $x526))))
+(let ((@x540 (monotonicity (monotonicity @x528 (= (not (and $x43 (< ?0 1))) $x529)) (rewrite (= $x47 $x534)) (= $x193 $x538))))
+(let ((@x546 (monotonicity (quant-intro @x540 (= $x196 $x541)) (= (not $x196) $x544))))
+(let ((@x815 (monotonicity (quant-intro @x540 (= $x196 $x541)) (monotonicity @x546 @x809 (= $x471 $x810)) (= $x476 $x813))))
+(let (($x517 (= (not (and $x28 (and $x31 (and $x32 (and $x32 (<= 1 1)))))) (not $x511))))
+(let (($x34 (<= 1 1)))
+(let (($x166 (and $x32 $x34)))
+(let (($x169 (and $x32 $x166)))
+(let (($x172 (and $x31 $x169)))
+(let (($x182 (and $x28 $x172)))
+(let ((@x513 (rewrite (= (and $x496 (and $x31 (and true (and true true)))) $x511))))
+(let ((@x501 (monotonicity (rewrite (= $x32 true)) (rewrite (= $x34 true)) (= $x166 (and true true)))))
+(let ((@x504 (monotonicity (rewrite (= $x32 true)) @x501 (= $x169 (and true (and true true))))))
+(let ((@x507 (monotonicity @x504 (= $x172 (and $x31 (and true (and true true)))))))
+(let ((@x510 (monotonicity (rewrite (= $x28 $x496)) @x507 (= $x182 (and $x496 (and $x31 (and true (and true true))))))))
+(let ((@x818 (monotonicity (monotonicity (trans @x510 @x513 (= $x182 $x511)) $x517) @x815 (= $x483 (or (not $x511) $x813)))))
+(let ((@x369 (monotonicity (rewrite (= (and $x136 false) false)) (= $x138 (=> false true)))))
+(let ((@x373 (trans @x369 (rewrite (= (=> false true) true)) (= $x138 true))))
+(let ((@x380 (trans (monotonicity @x373 (= $x139 (and $x136 true))) (rewrite (= (and $x136 true) $x136)) (= $x139 $x136))))
+(let ((@x364 (quant-intro (rewrite (= (=> (and $x43 (< ?0 v_b_p_G_1$)) $x132) $x359)) (= $x134 $x362))))
+(let ((@x389 (trans (monotonicity @x364 @x380 (= $x140 (=> $x362 $x136))) (rewrite (= (=> $x362 $x136) $x385)) (= $x140 $x385))))
+(let ((@x310 (monotonicity (rewrite (= (+ v_b_p_G_0$ 1) (+ 1 v_b_p_G_0$))) (= (= v_b_p_G_1$ (+ v_b_p_G_0$ 1)) $x308))))
+(let ((@x315 (monotonicity @x310 (rewrite (= (and $x117 true) $x117)) (= $x119 $x313))))
+(let ((@x321 (monotonicity (monotonicity @x315 (= (and $x111 $x119) $x316)) (= $x121 (and true $x316)))))
+(let ((@x404 (monotonicity (trans @x321 (rewrite (= (and true $x316) $x316)) (= $x121 $x316)) (= (and $x145 $x121) $x402))))
+(let ((@x410 (monotonicity (monotonicity @x404 (= (and $x144 (and $x145 $x121)) $x405)) (= $x148 (and true $x405)))))
+(let ((@x417 (monotonicity (trans @x410 (rewrite (= (and true $x405) $x405)) (= $x148 $x405)) (= (and $x55 $x148) $x415))))
+(let ((@x423 (monotonicity (monotonicity @x417 (= (and $x143 (and $x55 $x148)) $x418)) (= (and $x55 (and $x143 (and $x55 $x148))) $x421))))
+(let ((@x430 (trans (monotonicity @x423 (= $x152 (and true $x421))) (rewrite (= (and true $x421) $x421)) (= $x152 $x421))))
+(let ((@x433 (monotonicity @x430 (monotonicity @x364 @x389 (= $x141 $x390)) (= $x153 (=> $x421 $x390)))))
+(let (($x340 (= (and (and $x54 $x54) (and true (and $x107 (and $x109 $x121)))) $x339)))
+(let ((@x328 (monotonicity (trans @x321 (rewrite (= (and true $x316) $x316)) (= $x121 $x316)) (= (and $x109 $x121) $x326))))
+(let ((@x334 (monotonicity (monotonicity @x328 (= (and $x107 (and $x109 $x121)) $x329)) (= (and true (and $x107 (and $x109 $x121))) (and true $x329)))))
+(let ((@x338 (trans @x334 (rewrite (= (and true $x329) $x329)) (= (and true (and $x107 (and $x109 $x121))) $x329))))
+(let ((@x344 (monotonicity (monotonicity (rewrite (= (and $x54 $x54) $x54)) @x338 $x340) (= $x126 $x342))))
+(let ((@x350 (monotonicity (monotonicity @x344 (= (and $x102 $x126) $x345)) (= (and $x55 (and $x102 $x126)) $x348))))
+(let ((@x357 (trans (monotonicity @x350 (= $x129 (and true $x348))) (rewrite (= (and true $x348) $x348)) (= $x129 $x348))))
+(let ((@x395 (monotonicity @x357 (monotonicity @x364 @x389 (= $x141 $x390)) (= $x142 (=> $x348 $x390)))))
+(let ((@x442 (monotonicity (trans @x395 (rewrite (= (=> $x348 $x390) $x397)) (= $x142 $x397)) (trans @x433 (rewrite (= (=> $x421 $x390) $x435)) (= $x153 $x435)) (= (and $x142 $x153) $x440))))
+(let ((@x445 (monotonicity (rewrite (= (and true $x99) $x99)) @x442 (= $x155 (=> $x99 $x440)))))
+(let ((@x268 (monotonicity (quant-intro (rewrite (= (=> $x85 $x89) $x260)) (= $x91 $x263)) (= $x92 (=> $x263 true)))))
+(let ((@x272 (trans @x268 (rewrite (= (=> $x263 true) true)) (= $x92 true))))
+(let ((@x275 (monotonicity (quant-intro (rewrite (= (=> $x85 $x89) $x260)) (= $x91 $x263)) @x272 (= $x93 (and $x263 true)))))
+(let ((@x282 (monotonicity (quant-intro (rewrite (= (=> $x85 $x86) $x254)) (= $x88 $x257)) (trans @x275 (rewrite (= (and $x263 true) $x263)) (= $x93 $x263)) (= $x94 (=> $x257 $x263)))))
+(let ((@x291 (monotonicity (quant-intro (rewrite (= (=> $x85 $x86) $x254)) (= $x88 $x257)) (trans @x282 (rewrite (= (=> $x257 $x263) $x284)) (= $x94 $x284)) (= (and $x88 $x94) $x289))))
+(let (($x238 (= (and $x55 (and true (and $x71 (and $x73 (and $x75 true))))) $x237)))
+(let (($x79 (and true (and $x71 (and $x73 (and $x75 true))))))
+(let ((@x226 (monotonicity (rewrite (= (and $x75 true) $x75)) (= (and $x73 (and $x75 true)) (and $x73 $x75)))))
+(let ((@x229 (monotonicity @x226 (= (and $x71 (and $x73 (and $x75 true))) $x227))))
+(let ((@x236 (trans (monotonicity @x229 (= $x79 (and true $x227))) (rewrite (= (and true $x227) $x227)) (= $x79 $x227))))
+(let ((@x245 (monotonicity (monotonicity (monotonicity @x236 $x238) (= $x81 $x240)) (= (and $x55 $x81) $x243))))
+(let ((@x252 (trans (monotonicity @x245 (= $x83 (and true $x243))) (rewrite (= (and true $x243) $x243)) (= $x83 $x243))))
+(let ((@x300 (trans (monotonicity @x252 @x291 (= $x96 (=> $x243 $x289))) (rewrite (= (=> $x243 $x289) $x296)) (= $x96 $x296))))
+(let ((@x454 (monotonicity @x300 (trans @x445 (rewrite (= (=> $x99 $x440) $x447)) (= $x155 $x447)) (= (and $x96 $x155) $x452))))
+(let ((@x205 (quant-intro (rewrite (= (=> (and $x43 (< ?0 v_b_p_G_0$)) $x59) $x200)) (= $x61 $x203))))
+(let ((@x211 (monotonicity (monotonicity @x205 (= (and $x61 $x64) $x206)) (= (and $x55 (and $x61 $x64)) $x209))))
+(let ((@x218 (trans (monotonicity @x211 (= $x67 (and true $x209))) (rewrite (= (and true $x209) $x209)) (= $x67 $x209))))
+(let ((@x457 (monotonicity (monotonicity @x218 (= (and $x50 $x67) $x219)) @x454 (= $x157 (=> $x219 $x452)))))
+(let ((@x466 (monotonicity (trans @x457 (rewrite (= (=> $x219 $x452) $x459)) (= $x157 $x459)) (= (and $x50 $x157) $x464))))
+(let ((@x198 (quant-intro (rewrite (= (=> (and $x43 (< ?0 1)) $x47) $x193)) (= $x49 $x196))))
+(let ((@x475 (trans (monotonicity @x198 @x466 (= $x159 (=> $x196 $x464))) (rewrite (= (=> $x196 $x464) $x471)) (= $x159 $x471))))
+(let ((@x168 (monotonicity (rewrite (= (and $x34 $x34) $x34)) (= (and $x32 (and $x34 $x34)) $x166))))
+(let ((@x174 (monotonicity (monotonicity @x168 (= (and $x32 (and $x32 (and $x34 $x34))) $x169)) (= $x38 $x172))))
+(let ((@x181 (trans (monotonicity @x174 (= $x39 (and true $x172))) (rewrite (= (and true $x172) $x172)) (= $x39 $x172))))
+(let ((@x187 (monotonicity (monotonicity @x181 (= (and $x28 $x39) $x182)) (= $x41 (and true $x182)))))
+(let ((@x481 (monotonicity (trans @x187 (rewrite (= (and true $x182) $x182)) (= $x41 $x182)) (monotonicity @x198 @x475 (= (and $x49 $x159) $x476)) (= $x161 (=> $x182 $x476)))))
+(let ((@x490 (monotonicity (trans @x481 (rewrite (= (=> $x182 $x476) $x483)) (= $x161 $x483)) (= $x162 (not $x483)))))
+(let ((@x823 (trans @x490 (monotonicity @x818 (= (not $x483) $x819)) (= $x162 $x819))))
+(let ((@x827 (and-elim (not-or-elim (mp (asserted $x162) @x823 $x819) $x511) $x31)))
+(let ((@x1690 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= v_b_max_G_0$ (v_b_array$ ?v0!0))) $x839)) (unit-resolution (def-axiom (or $x1149 (not $x839))) @x1726 (not $x839)) (trans @x827 @x1715 (= v_b_max_G_0$ (v_b_array$ ?v0!0))) false)))
+(let (($x1946 (or $x1154 $x1943)))
+(let (($x1340 (forall ((?v0 Int) )(let (($x746 (<= (+ (v_b_array$ ?v0) (* (- 1) v_b_max_G_3$)) 0)))
+(let (($x733 (>= (+ ?v0 (* (- 1) v_b_p_G_1$)) 0)))
+(let (($x521 (>= ?v0 0)))
+(let (($x1157 (not $x521)))
+(or $x1157 $x733 $x746))))))
+))
+(let (($x1348 (not (or (not $x1340) $x136))))
+(let (($x1353 (or $x1318 $x1348)))
+(let (($x1365 (not $x1353)))
+(let (($x1378 (not (or $x692 $x1286 $x1375 $x1376 $x1287 $x1362 $x1363 $x1364 $x1365))))
+(let (($x1367 (not (or $x1286 $x689 $x1359 $x1360 $x1361 $x1287 $x1362 $x1363 $x1364 $x1365))))
+(let (($x1383 (or $x1367 $x1378)))
+(let (($x1391 (not (or $x600 $x1286 $x1287 (not $x1383)))))
+(let (($x1224 (forall ((?v0 Int) )(let ((?x46 (v_b_array$ ?v0)))
+(let (($x86 (= ?x46 v_b_max_G_4$)))
+(let (($x622 (<= (+ v_b_length$ (* (- 1) ?v0)) 0)))
+(let (($x521 (>= ?v0 0)))
+(let (($x1157 (not $x521)))
+(let (($x1216 (or $x1157 $x622 $x86)))
+(not $x1216))))))))
+))
+(let (($x1280 (or $x1224 $x1275)))
+(let (($x1293 (not (or $x661 $x1286 $x1287 $x1288 $x1289 $x1290 (not $x1280)))))
+(let (($x1396 (or $x1293 $x1391)))
+(let (($x1199 (forall ((?v0 Int) )(let (($x561 (<= (+ (v_b_array$ ?v0) (* (- 1) v_b_max_G_1$)) 0)))
+(let (($x548 (>= (+ ?v0 (* (- 1) v_b_p_G_0$)) 0)))
+(let (($x521 (>= ?v0 0)))
+(let (($x1157 (not $x521)))
+(or $x1157 $x548 $x561))))))
+))
+(let (($x1406 (not (or $x851 (not $x1199) $x1403 $x1286 $x1287 (not $x1396)))))
+(let (($x1411 (or $x851 $x1406)))
+(let (($x1177 (forall ((?v0 Int) )(let (($x534 (>= (+ v_b_max_G_0$ (* (- 1) (v_b_array$ ?v0))) 0)))
+(let (($x524 (>= ?v0 1)))
+(let (($x521 (>= ?v0 0)))
+(let (($x1157 (not $x521)))
+(or $x1157 $x524 $x534))))))
+))
+(let (($x1420 (not (or (not $x1177) (not $x1411)))))
+(let (($x1425 (or $x1154 $x1420)))
+(let (($x733 (>= (+ ?0 ?x685) 0)))
+(let (($x1157 (not $x521)))
+(let (($x1335 (or $x1157 $x733 $x746)))
+(let ((@x1885 (monotonicity (quant-intro (refl (= $x1335 $x1335)) (= $x1340 $x1878)) (= (not $x1340) $x1883))))
+(let ((@x1891 (monotonicity (monotonicity @x1885 (= (or (not $x1340) $x136) $x1886)) (= $x1348 $x1889))))
+(let ((@x1906 (monotonicity (monotonicity (monotonicity @x1891 (= $x1353 $x1892)) (= $x1365 $x1895)) (= (or $x692 $x1286 $x1375 $x1376 $x1287 $x1362 $x1363 $x1364 $x1365) $x1904))))
+(let ((@x1900 (monotonicity (monotonicity (monotonicity @x1891 (= $x1353 $x1892)) (= $x1365 $x1895)) (= (or $x1286 $x689 $x1359 $x1360 $x1361 $x1287 $x1362 $x1363 $x1364 $x1365) $x1898))))
+(let ((@x1912 (monotonicity (monotonicity @x1900 (= $x1367 $x1901)) (monotonicity @x1906 (= $x1378 $x1907)) (= $x1383 $x1910))))
+(let ((@x1918 (monotonicity (monotonicity @x1912 (= (not $x1383) $x1913)) (= (or $x600 $x1286 $x1287 (not $x1383)) $x1916))))
+(let (($x622 (<= (+ v_b_length$ (* (- 1) ?0)) 0)))
+(let (($x1216 (or $x1157 $x622 $x86)))
+(let (($x1221 (not $x1216)))
+(let ((@x1868 (monotonicity (quant-intro (refl (= $x1221 $x1221)) (= $x1224 $x1861)) (= $x1280 $x1866))))
+(let ((@x1874 (monotonicity (monotonicity @x1868 (= (not $x1280) $x1869)) (= (or $x661 $x1286 $x1287 $x1288 $x1289 $x1290 (not $x1280)) $x1872))))
+(let ((@x1924 (monotonicity (monotonicity @x1874 (= $x1293 $x1875)) (monotonicity @x1918 (= $x1391 $x1919)) (= $x1396 $x1922))))
+(let (($x548 (>= (+ ?0 ?x549) 0)))
+(let (($x1194 (or $x1157 $x548 $x561)))
+(let ((@x1860 (monotonicity (quant-intro (refl (= $x1194 $x1194)) (= $x1199 $x1853)) (= (not $x1199) $x1858))))
+(let ((@x1930 (monotonicity @x1860 (monotonicity @x1924 (= (not $x1396) $x1925)) (= (or $x851 (not $x1199) $x1403 $x1286 $x1287 (not $x1396)) $x1928))))
+(let ((@x1939 (monotonicity (monotonicity (monotonicity @x1930 (= $x1406 $x1931)) (= $x1411 $x1934)) (= (not $x1411) $x1937))))
+(let ((@x1847 (refl (= (or $x1157 (>= ?0 1) $x534) (or $x1157 (>= ?0 1) $x534)))))
+(let ((@x1852 (monotonicity (quant-intro @x1847 (= $x1177 $x1845)) (= (not $x1177) $x1850))))
+(let ((@x1945 (monotonicity (monotonicity @x1852 @x1939 (= (or (not $x1177) (not $x1411)) $x1940)) (= $x1420 $x1943))))
+(let (($x951 (not $x136)))
+(let (($x954 (and $x752 $x951)))
+(let (($x1053 (not $x1048)))
+(let (($x1056 (and $x931 $x1053)))
+(let (($x1059 (not $x1056)))
+(let (($x1075 (or $x1059 $x1070)))
+(let (($x1078 (not $x1075)))
+(let (($x1081 (or $x1078 $x954)))
+(let (($x1097 (and $x689 $x571 $x144 $x145 $x573 $x684 $x679 $x682 $x1081)))
+(let (($x1087 (and $x571 $x692 $x104 $x107 $x109 $x573 $x684 $x679 $x682 $x1081)))
+(let (($x1102 (or $x1087 $x1097)))
+(let (($x1108 (and $x661 $x571 $x573 $x1102)))
+(let (($x903 (not (and $x897 (not $x900)))))
+(let (($x1016 (or $x903 $x1011)))
+(let (($x1019 (not $x1016)))
+(let (($x887 (not (and $x881 (not $x884)))))
+(let (($x890 (or $x887 $x889)))
+(let (($x1022 (and $x890 $x1019)))
+(let (($x877 (forall ((?v0 Int) )(let ((?x46 (v_b_array$ ?v0)))
+(let (($x86 (= ?x46 v_b_max_G_4$)))
+(let (($x521 (>= ?v0 0)))
+(let (($x626 (and $x521 (not (<= (+ v_b_length$ (* (- 1) ?v0)) 0)))))
+(let (($x629 (not $x626)))
+(let (($x632 (or $x629 $x86)))
+(not $x632))))))))
+))
+(let (($x1025 (or $x877 $x1022)))
+(let (($x1031 (and $x600 $x571 $x573 $x71 $x73 $x75 $x1025)))
+(let (($x1113 (or $x1031 $x1108)))
+(let (($x1119 (and $x50 $x567 $x63 $x571 $x573 $x1113)))
+(let (($x1124 (or $x851 $x1119)))
+(let (($x1127 (and $x541 $x1124)))
+(let (($x831 (not (and $x835 $x833))))
+(let (($x840 (or $x831 $x839)))
+(let (($x841 (not $x840)))
+(let (($x1130 (or $x841 $x1127)))
+(let ((@x1380 (rewrite (= (and $x689 $x571 $x144 $x145 $x573 $x684 $x679 $x682 $x1353) $x1378))))
+(let ((@x1327 (monotonicity (rewrite (= $x738 (not (or $x1157 $x733)))) (= $x741 (not (not (or $x1157 $x733)))))))
+(let ((@x1331 (trans @x1327 (rewrite (= (not (not (or $x1157 $x733))) (or $x1157 $x733))) (= $x741 (or $x1157 $x733)))))
+(let ((@x1339 (trans (monotonicity @x1331 (= $x749 (or (or $x1157 $x733) $x746))) (rewrite (= (or (or $x1157 $x733) $x746) $x1335)) (= $x749 $x1335))))
+(let ((@x1345 (monotonicity (quant-intro @x1339 (= $x752 $x1340)) (= $x954 (and $x1340 $x951)))))
+(let ((@x1305 (monotonicity (rewrite (= $x1056 (not (or $x1298 $x1048)))) (= $x1059 (not (not (or $x1298 $x1048)))))))
+(let ((@x1309 (trans @x1305 (rewrite (= (not (not (or $x1298 $x1048))) (or $x1298 $x1048))) (= $x1059 (or $x1298 $x1048)))))
+(let ((@x1317 (trans (monotonicity @x1309 (= $x1075 (or (or $x1298 $x1048) $x1070))) (rewrite (= (or (or $x1298 $x1048) $x1070) $x1313)) (= $x1075 $x1313))))
+(let ((@x1355 (monotonicity (monotonicity @x1317 (= $x1078 $x1318)) (trans @x1345 (rewrite (= (and $x1340 $x951) $x1348)) (= $x954 $x1348)) (= $x1081 $x1353))))
+(let ((@x1374 (monotonicity @x1355 (= $x1097 (and $x689 $x571 $x144 $x145 $x573 $x684 $x679 $x682 $x1353)))))
+(let ((@x1369 (rewrite (= (and $x571 $x692 $x104 $x107 $x109 $x573 $x684 $x679 $x682 $x1353) $x1367))))
+(let ((@x1358 (monotonicity @x1355 (= $x1087 (and $x571 $x692 $x104 $x107 $x109 $x573 $x684 $x679 $x682 $x1353)))))
+(let ((@x1385 (monotonicity (trans @x1358 @x1369 (= $x1087 $x1367)) (trans @x1374 @x1380 (= $x1097 $x1378)) (= $x1102 $x1383))))
+(let ((@x1395 (trans (monotonicity @x1385 (= $x1108 (and $x661 $x571 $x573 $x1383))) (rewrite (= (and $x661 $x571 $x573 $x1383) $x1391)) (= $x1108 $x1391))))
+(let ((@x1254 (monotonicity (rewrite (= (and $x897 (not $x900)) (not (or $x1247 $x900)))) (= $x903 (not (not (or $x1247 $x900)))))))
+(let ((@x1258 (trans @x1254 (rewrite (= (not (not (or $x1247 $x900))) (or $x1247 $x900))) (= $x903 (or $x1247 $x900)))))
+(let ((@x1266 (trans (monotonicity @x1258 (= $x1016 (or (or $x1247 $x900) $x1011))) (rewrite (= (or (or $x1247 $x900) $x1011) (or $x1247 $x900 $x1011))) (= $x1016 (or $x1247 $x900 $x1011)))))
+(let ((@x1234 (monotonicity (rewrite (= (and $x881 (not $x884)) (not (or $x1227 $x884)))) (= $x887 (not (not (or $x1227 $x884)))))))
+(let ((@x1238 (trans @x1234 (rewrite (= (not (not (or $x1227 $x884))) (or $x1227 $x884))) (= $x887 (or $x1227 $x884)))))
+(let ((@x1246 (trans (monotonicity @x1238 (= $x890 (or (or $x1227 $x884) $x889))) (rewrite (= (or (or $x1227 $x884) $x889) $x1242)) (= $x890 $x1242))))
+(let ((@x1272 (monotonicity @x1246 (monotonicity @x1266 (= $x1019 (not (or $x1247 $x900 $x1011)))) (= $x1022 (and $x1242 (not (or $x1247 $x900 $x1011)))))))
+(let ((@x1279 (trans @x1272 (rewrite (= (and $x1242 (not (or $x1247 $x900 $x1011))) $x1275)) (= $x1022 $x1275))))
+(let ((@x1208 (monotonicity (rewrite (= $x626 (not (or $x1157 $x622)))) (= $x629 (not (not (or $x1157 $x622)))))))
+(let ((@x1212 (trans @x1208 (rewrite (= (not (not (or $x1157 $x622))) (or $x1157 $x622))) (= $x629 (or $x1157 $x622)))))
+(let ((@x1220 (trans (monotonicity @x1212 (= $x632 (or (or $x1157 $x622) $x86))) (rewrite (= (or (or $x1157 $x622) $x86) $x1216)) (= $x632 $x1216))))
+(let ((@x1226 (quant-intro (monotonicity @x1220 (= (not $x632) $x1221)) (= $x877 $x1224))))
+(let ((@x1285 (monotonicity (monotonicity @x1226 @x1279 (= $x1025 $x1280)) (= $x1031 (and $x600 $x571 $x573 $x71 $x73 $x75 $x1280)))))
+(let ((@x1297 (trans @x1285 (rewrite (= (and $x600 $x571 $x573 $x71 $x73 $x75 $x1280) $x1293)) (= $x1031 $x1293))))
+(let ((@x1186 (monotonicity (rewrite (= $x553 (not (or $x1157 $x548)))) (= $x556 (not (not (or $x1157 $x548)))))))
+(let ((@x1190 (trans @x1186 (rewrite (= (not (not (or $x1157 $x548))) (or $x1157 $x548))) (= $x556 (or $x1157 $x548)))))
+(let ((@x1198 (trans (monotonicity @x1190 (= $x564 (or (or $x1157 $x548) $x561))) (rewrite (= (or (or $x1157 $x548) $x561) $x1194)) (= $x564 $x1194))))
+(let ((@x1401 (monotonicity (quant-intro @x1198 (= $x567 $x1199)) (monotonicity @x1297 @x1395 (= $x1113 $x1396)) (= $x1119 (and $x50 $x1199 $x63 $x571 $x573 $x1396)))))
+(let ((@x1410 (trans @x1401 (rewrite (= (and $x50 $x1199 $x63 $x571 $x573 $x1396) $x1406)) (= $x1119 $x1406))))
+(let (($x524 (>= ?0 1)))
+(let (($x1172 (or $x1157 $x524 $x534)))
+(let ((@x1164 (monotonicity (rewrite (= $x526 (not (or $x1157 $x524)))) (= $x529 (not (not (or $x1157 $x524)))))))
+(let ((@x1168 (trans @x1164 (rewrite (= (not (not (or $x1157 $x524))) (or $x1157 $x524))) (= $x529 (or $x1157 $x524)))))
+(let ((@x1176 (trans (monotonicity @x1168 (= $x538 (or (or $x1157 $x524) $x534))) (rewrite (= (or (or $x1157 $x524) $x534) $x1172)) (= $x538 $x1172))))
+(let ((@x1416 (monotonicity (quant-intro @x1176 (= $x541 $x1177)) (monotonicity @x1410 (= $x1124 $x1411)) (= $x1127 (and $x1177 $x1411)))))
+(let ((@x1141 (monotonicity (rewrite (= (and $x835 $x833) (not (or $x1134 $x832)))) (= $x831 (not (not (or $x1134 $x832)))))))
+(let ((@x1145 (trans @x1141 (rewrite (= (not (not (or $x1134 $x832))) (or $x1134 $x832))) (= $x831 (or $x1134 $x832)))))
+(let ((@x1153 (trans (monotonicity @x1145 (= $x840 (or (or $x1134 $x832) $x839))) (rewrite (= (or (or $x1134 $x832) $x839) $x1149)) (= $x840 $x1149))))
+(let ((@x1427 (monotonicity (monotonicity @x1153 (= $x841 $x1154)) (trans @x1416 (rewrite (= (and $x1177 $x1411) $x1420)) (= $x1127 $x1420)) (= $x1130 $x1425))))
+(let (($x939 (<= (+ ?x937 ?x744) 0)))
+(let (($x941 (not (or (not (and $x931 (not (>= (+ ?v0!3 ?x685) 0)))) $x939))))
+(let (($x958 (or $x941 $x954)))
+(let (($x966 (not $x789)))
+(let (($x969 (and $x966 $x958)))
+(let (($x927 (not $x730)))
+(let (($x962 (and $x927 $x958)))
+(let (($x973 (or $x962 $x969)))
+(let (($x924 (not $x675)))
+(let (($x977 (and $x924 $x973)))
+(let (($x908 (not (or $x903 (<= (+ (v_b_array$ ?v0!2) (* (- 1) v_b_max_G_4$)) 0)))))
+(let (($x912 (and $x890 $x908)))
+(let (($x916 (or $x877 $x912)))
+(let (($x871 (not $x617)))
+(let (($x920 (and $x871 $x916)))
+(let (($x981 (or $x920 $x977)))
+(let (($x985 (and $x591 $x981)))
+(let (($x989 (or $x851 $x985)))
+(let (($x993 (and $x541 $x989)))
+(let (($x997 (or $x841 $x993)))
+(let (($x1076 (= (or (not (and $x931 (not (>= (+ ?v0!3 ?x685) 0)))) $x939) $x1075)))
+(let ((@x1067 (monotonicity (rewrite (= (+ ?x937 ?x744) (+ ?x744 ?x937))) (= $x939 (<= (+ ?x744 ?x937) 0)))))
+(let ((@x1074 (trans @x1067 (rewrite (= (<= (+ ?x744 ?x937) 0) $x1070)) (= $x939 $x1070))))
+(let ((@x1045 (monotonicity (rewrite (= (+ ?v0!3 ?x685) (+ ?x685 ?v0!3))) (= (>= (+ ?v0!3 ?x685) 0) (>= (+ ?x685 ?v0!3) 0)))))
+(let ((@x1052 (trans @x1045 (rewrite (= (>= (+ ?x685 ?v0!3) 0) $x1048)) (= (>= (+ ?v0!3 ?x685) 0) $x1048))))
+(let ((@x1058 (monotonicity (monotonicity @x1052 (= (not (>= (+ ?v0!3 ?x685) 0)) $x1053)) (= (and $x931 (not (>= (+ ?v0!3 ?x685) 0))) $x1056))))
+(let ((@x1061 (monotonicity @x1058 (= (not (and $x931 (not (>= (+ ?v0!3 ?x685) 0)))) $x1059))))
+(let ((@x1083 (monotonicity (monotonicity (monotonicity @x1061 @x1074 $x1076) (= $x941 $x1078)) (= $x958 $x1081))))
+(let ((@x1096 (monotonicity (rewrite (= $x966 $x784)) @x1083 (= $x969 (and $x784 $x1081)))))
+(let ((@x1086 (monotonicity (rewrite (= $x927 $x725)) @x1083 (= $x962 (and $x725 $x1081)))))
+(let ((@x1104 (monotonicity (trans @x1086 (rewrite (= (and $x725 $x1081) $x1087)) (= $x962 $x1087)) (trans @x1096 (rewrite (= (and $x784 $x1081) $x1097)) (= $x969 $x1097)) (= $x973 $x1102))))
+(let ((@x1107 (monotonicity (rewrite (= $x924 $x670)) @x1104 (= $x977 (and $x670 $x1102)))))
+(let (($x1017 (= (or $x903 (<= (+ (v_b_array$ ?v0!2) (* (- 1) v_b_max_G_4$)) 0)) $x1016)))
+(let (($x906 (<= (+ (v_b_array$ ?v0!2) (* (- 1) v_b_max_G_4$)) 0)))
+(let (($x1012 (= (<= (+ (* (- 1) v_b_max_G_4$) (v_b_array$ ?v0!2)) 0) $x1011)))
+(let (($x1007 (= $x906 (<= (+ (* (- 1) v_b_max_G_4$) (v_b_array$ ?v0!2)) 0))))
+(let (($x1004 (= (+ (v_b_array$ ?v0!2) (* (- 1) v_b_max_G_4$)) (+ (* (- 1) v_b_max_G_4$) (v_b_array$ ?v0!2)))))
+(let ((@x1015 (trans (monotonicity (rewrite $x1004) $x1007) (rewrite $x1012) (= $x906 $x1011))))
+(let ((@x1024 (monotonicity (monotonicity (monotonicity @x1015 $x1017) (= $x908 $x1019)) (= $x912 $x1022))))
+(let ((@x1030 (monotonicity (rewrite (= $x871 $x612)) (monotonicity @x1024 (= $x916 $x1025)) (= $x920 (and $x612 $x1025)))))
+(let ((@x1115 (monotonicity (trans @x1030 (rewrite (= (and $x612 $x1025) $x1031)) (= $x920 $x1031)) (trans @x1107 (rewrite (= (and $x670 $x1102) $x1108)) (= $x977 $x1108)) (= $x981 $x1113))))
+(let ((@x1123 (trans (monotonicity @x1115 (= $x985 (and $x591 $x1113))) (rewrite (= (and $x591 $x1113) $x1119)) (= $x985 $x1119))))
+(let ((@x1132 (monotonicity (monotonicity (monotonicity @x1123 (= $x989 $x1124)) (= $x993 $x1127)) (= $x997 $x1130))))
+(let ((@x950 (nnf-neg (nnf-pos (refl (~ $x749 $x749)) (~ $x752 $x752)) (~ (not $x755) $x752))))
+(let ((@x961 (nnf-neg (sk (~ $x755 $x941)) (nnf-neg @x950 (refl (~ $x951 $x951)) (~ (not $x758) $x954)) (~ (not $x761) $x958))))
+(let ((@x976 (nnf-neg (nnf-neg (refl (~ $x927 $x927)) @x961 (~ (not $x764) $x962)) (nnf-neg (refl (~ $x966 $x966)) @x961 (~ (not $x792) $x969)) (~ (not $x795) $x973))))
+(let ((@x915 (nnf-neg (nnf-neg (sk (~ $x635 $x890)) (~ (not $x638) $x890)) (sk (~ (not $x649) $x908)) (~ (not $x652) $x912))))
+(let ((@x919 (nnf-neg (nnf-neg (refl (~ (not $x632) (not $x632))) (~ $x638 $x877)) @x915 (~ (not $x655) $x916))))
+(let ((@x984 (nnf-neg (nnf-neg (refl (~ $x871 $x871)) @x919 (~ (not $x658) $x920)) (nnf-neg (refl (~ $x924 $x924)) @x976 (~ (not $x798) $x977)) (~ (not $x801) $x981))))
+(let ((@x867 (monotonicity (refl (~ $x50 $x50)) (nnf-pos (refl (~ $x564 $x564)) (~ $x567 $x567)) (refl (~ $x63 $x63)) (refl (~ $x571 $x571)) (refl (~ $x573 $x573)) (~ $x591 $x591))))
+(let ((@x988 (nnf-neg (nnf-neg @x867 (~ (not $x596) $x591)) @x984 (~ (not $x804) $x985))))
+(let ((@x850 (nnf-neg (nnf-pos (refl (~ $x538 $x538)) (~ $x541 $x541)) (~ (not $x544) $x541))))
+(let ((@x996 (nnf-neg @x850 (nnf-neg (refl (~ $x851 $x851)) @x988 (~ (not $x807) $x989)) (~ (not $x810) $x993))))
+(let ((@x1000 (mp~ (not-or-elim (mp (asserted $x162) @x823 $x819) (not $x813)) (nnf-neg (sk (~ $x544 $x841)) @x996 (~ (not $x813) $x997)) $x997)))
+(let ((@x1949 (mp (mp (mp @x1000 @x1132 $x1130) @x1427 $x1425) (monotonicity @x1945 (= $x1425 $x1946)) $x1946)))
+(let ((@x2062 (unit-resolution (def-axiom (or $x1940 $x1934)) (unit-resolution @x1949 (lemma @x1690 $x1149) $x1943) $x1934)))
+(let ((@x2069 (unit-resolution (def-axiom (or $x1937 $x851 $x1931)) (mp @x827 (symm (commutativity (= $x50 $x31)) (= $x31 $x50)) $x50) (or $x1937 $x1931))))
+(let ((@x2070 (unit-resolution @x2069 @x2062 $x1931)))
+(let ((@x2170 (monotonicity (unit-resolution (def-axiom (or $x1904 $x144)) @x2149 $x144) (= ?x135 ?x62))))
+(let ((@x2173 (trans @x2170 (unit-resolution (def-axiom (or $x1928 $x63)) @x2070 $x63) (= ?x135 v_b_max_G_1$))))
+(let ((@x2174 (trans @x2173 (symm (unit-resolution (def-axiom (or $x1904 $x145)) @x2149 $x145) $x1780) $x136)))
+(let ((@x1523 (def-axiom (or $x1886 $x951))))
+(let ((@x1808 (def-axiom (or $x1895 $x1318 $x1889))))
+(let ((@x2176 (unit-resolution @x1808 (unit-resolution @x1523 @x2174 $x1886) (unit-resolution (def-axiom (or $x1904 $x1892)) @x2149 $x1892) $x1318)))
+(let ((@x1812 (def-axiom (or $x1313 $x1436))))
+(let ((@x2181 (unit-resolution ((_ th-lemma arith assign-bounds 1 -1 -1) (or $x1453 $x692 $x1070 (not $x1782))) (unit-resolution @x1812 @x2176 $x1436) (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x1780) $x1782)) @x2162 $x1782) (unit-resolution (def-axiom (or $x1904 $x689)) @x2149 $x689) $x1453)))
+(let ((@x1565 ((_ th-lemma arith triangle-eq) (or $x1563 $x1445))))
+(let (($x1558 (= v_b_p_G_0$ ?v0!3)))
+(let ((?x1046 (* (- 1) ?v0!3)))
+(let ((?x1510 (+ v_b_p_G_0$ ?x1046)))
+(let (($x1560 (>= ?x1510 0)))
+(let (($x1522 (>= ?x686 (- 1))))
+(let ((@x2186 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x1362 $x1522)) (unit-resolution (def-axiom (or $x1904 $x684)) @x2149 $x684) $x1522)))
+(let ((@x2190 (unit-resolution ((_ th-lemma arith assign-bounds -1 -1) (or $x1560 $x1048 (not $x1522))) (unit-resolution (def-axiom (or $x1313 $x1053)) @x2176 $x1053) @x2186 $x1560)))
+(let (($x1511 (<= ?x1510 0)))
+(let (($x1488 (>= (+ v_b_max_G_1$ ?x1068) 0)))
+(let (($x1955 (not $x1488)))
+(let ((@x2193 (unit-resolution ((_ th-lemma arith assign-bounds -1 -1) (or $x1955 $x1070 (not $x1782))) (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x1780) $x1782)) @x2162 $x1782) (unit-resolution @x1812 @x2176 $x1436) $x1955)))
+(let ((@x2093 (unit-resolution (def-axiom (or $x1928 $x1853)) @x2070 $x1853)))
+(let (($x1476 (or $x1858 $x1298 $x1511 $x1488)))
+(let (($x1535 (<= (+ ?x937 (* (- 1) v_b_max_G_1$)) 0)))
+(let (($x1549 (>= (+ ?v0!3 ?x549) 0)))
+(let (($x1501 (or $x1298 $x1549 $x1535)))
+(let (($x1464 (or $x1858 $x1501)))
+(let (($x1478 (= (+ ?x937 (* (- 1) v_b_max_G_1$)) (+ (* (- 1) v_b_max_G_1$) ?x937))))
+(let ((@x1486 (monotonicity (rewrite $x1478) (= $x1535 (<= (+ (* (- 1) v_b_max_G_1$) ?x937) 0)))))
+(let ((@x1472 (trans @x1486 (rewrite (= (<= (+ (* (- 1) v_b_max_G_1$) ?x937) 0) $x1488)) (= $x1535 $x1488))))
+(let ((@x1509 (monotonicity (rewrite (= (+ ?v0!3 ?x549) (+ ?x549 ?v0!3))) (= $x1549 (>= (+ ?x549 ?v0!3) 0)))))
+(let ((@x1497 (trans @x1509 (rewrite (= (>= (+ ?x549 ?v0!3) 0) $x1511)) (= $x1549 $x1511))))
+(let ((@x1470 (monotonicity (monotonicity @x1497 @x1472 (= $x1501 (or $x1298 $x1511 $x1488))) (= $x1464 (or $x1858 (or $x1298 $x1511 $x1488))))))
+(let ((@x1450 (trans @x1470 (rewrite (= (or $x1858 (or $x1298 $x1511 $x1488)) $x1476)) (= $x1464 $x1476))))
+(let ((@x2195 (unit-resolution (mp ((_ quant-inst ?v0!3) $x1464) @x1450 $x1476) @x2093 (unit-resolution (def-axiom (or $x1313 $x931)) @x2176 $x931) @x2193 $x1511)))
+(let ((@x2196 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x1558 (not $x1511) (not $x1560))) @x2195 @x2190 $x1558)))
+(let ((@x1551 (monotonicity (symm (hypothesis $x1558) (= ?v0!3 v_b_p_G_0$)) (= ?x937 ?x101))))
+(let ((@x1540 (lemma (unit-resolution (hypothesis $x1563) (symm @x1551 $x1559) false) (or (not $x1558) $x1559))))
+(let ((@x2198 (lemma (unit-resolution @x1540 @x2196 (unit-resolution @x1565 @x2181 $x1563) false) $x1904)))
+(let (($x1990 (<= (+ v_b_max_G_1$ (* (- 1) v_b_max_G_4$)) 0)))
+(let (($x1988 (= v_b_max_G_1$ v_b_max_G_4$)))
+(let ((@x2109 (symm (unit-resolution (def-axiom (or $x1872 $x73)) (hypothesis $x1875) $x73) $x1988)))
+(let (($x2025 (>= (+ v_b_max_G_1$ (* (- 1) (v_b_array$ ?v0!2))) 0)))
+(let (($x901 (not $x900)))
+(let (($x1835 (not $x1861)))
+(let (($x2042 (= ?x62 v_b_max_G_4$)))
+(let (($x2043 (or $x1286 (<= (+ v_b_length$ (* (- 1) v_b_k_G_0$)) 0) $x2042)))
+(let ((@x2073 (trans (unit-resolution (def-axiom (or $x1928 $x63)) @x2070 $x63) (symm (hypothesis $x73) $x1988) $x2042)))
+(let ((@x2076 (unit-resolution ((_ quant-inst v_b_k_G_0$) (or $x1835 (not $x2043))) (hypothesis $x1861) (unit-resolution (def-axiom (or $x2043 (not $x2042))) @x2073 $x2043) false)))
+(let ((@x2115 (unit-resolution (lemma @x2076 (or $x1835 $x1289)) (unit-resolution (def-axiom (or $x1872 $x73)) (hypothesis $x1875) $x73) $x1835)))
+(let ((@x2116 (unit-resolution (def-axiom (or $x1869 $x1861 $x1275)) @x2115 (unit-resolution (def-axiom (or $x1872 $x1866)) (hypothesis $x1875) $x1866) $x1275)))
+(let ((@x2103 ((_ th-lemma arith farkas -1 -1 1) (hypothesis (<= (+ v_b_p_G_0$ (* (- 1) ?v0!2)) 0)) (hypothesis $x600) (hypothesis $x901) false)))
+(let ((@x2106 (lemma @x2103 (or (not (<= (+ v_b_p_G_0$ (* (- 1) ?v0!2)) 0)) $x661 $x900))))
+(let ((@x2119 (unit-resolution @x2106 (unit-resolution (def-axiom (or $x1872 $x600)) (hypothesis $x1875) $x600) (unit-resolution (def-axiom (or $x1274 $x901)) @x2116 $x901) (not (<= (+ v_b_p_G_0$ (* (- 1) ?v0!2)) 0)))))
+(let (($x2032 (<= (+ v_b_p_G_0$ (* (- 1) ?v0!2)) 0)))
+(let (($x2056 (or $x1858 $x1247 $x2032 $x2025)))
+(let (($x2009 (<= (+ (v_b_array$ ?v0!2) (* (- 1) v_b_max_G_1$)) 0)))
+(let (($x2001 (>= (+ ?v0!2 ?x549) 0)))
+(let (($x2010 (or $x1247 $x2001 $x2009)))
+(let (($x2060 (or $x1858 $x2010)))
+(let (($x2026 (= (<= (+ (* (- 1) v_b_max_G_1$) (v_b_array$ ?v0!2)) 0) $x2025)))
+(let (($x2020 (= $x2009 (<= (+ (* (- 1) v_b_max_G_1$) (v_b_array$ ?v0!2)) 0))))
+(let (($x2038 (= (+ (v_b_array$ ?v0!2) (* (- 1) v_b_max_G_1$)) (+ (* (- 1) v_b_max_G_1$) (v_b_array$ ?v0!2)))))
+(let ((@x2052 (trans (monotonicity (rewrite $x2038) $x2020) (rewrite $x2026) (= $x2009 $x2025))))
+(let ((@x2018 (monotonicity (rewrite (= (+ ?v0!2 ?x549) (+ ?x549 ?v0!2))) (= $x2001 (>= (+ ?x549 ?v0!2) 0)))))
+(let ((@x2036 (trans @x2018 (rewrite (= (>= (+ ?x549 ?v0!2) 0) $x2032)) (= $x2001 $x2032))))
+(let ((@x2031 (monotonicity (monotonicity @x2036 @x2052 (= $x2010 (or $x1247 $x2032 $x2025))) (= $x2060 (or $x1858 (or $x1247 $x2032 $x2025))))))
+(let ((@x2079 (trans @x2031 (rewrite (= (or $x1858 (or $x1247 $x2032 $x2025)) $x2056)) (= $x2060 $x2056))))
+(let ((@x2122 (unit-resolution (mp ((_ quant-inst ?v0!2) $x2060) @x2079 $x2056) @x2093 (unit-resolution (def-axiom (or $x1274 $x897)) @x2116 $x897) (or $x2032 $x2025))))
+(let ((@x2125 ((_ th-lemma arith farkas 1 -1 1) (unit-resolution (def-axiom (or $x1274 (not $x1011))) @x2116 (not $x1011)) (unit-resolution @x2122 @x2119 $x2025) (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x1988) $x1990)) @x2109 $x1990) false)))
+(let ((@x2133 (unit-resolution (def-axiom (or $x1925 $x1875 $x1919)) (lemma @x2125 $x1872) (unit-resolution (def-axiom (or $x1928 $x1922)) @x2070 $x1922) $x1919)))
+(let ((@x2003 (unit-resolution (def-axiom (or $x1913 $x1901 $x1907)) (unit-resolution (def-axiom (or $x1916 $x1910)) @x2133 $x1910) $x1910)))
+(let ((@x2004 (unit-resolution @x2003 @x2198 $x1901)))
+(let ((@x1528 (trans (monotonicity (hypothesis $x107) (= ?x135 ?x101)) (symm (hypothesis $x104) (= ?x101 v_b_max_G_2$)) (= ?x135 v_b_max_G_2$))))
+(let ((@x1529 (trans @x1528 (symm (hypothesis $x109) (= v_b_max_G_2$ v_b_max_G_3$)) $x136)))
+(let ((@x1532 (lemma (unit-resolution (hypothesis $x951) @x1529 false) (or $x136 $x1361 $x1359 $x1360))))
+(let ((@x2140 (unit-resolution @x1532 (unit-resolution (def-axiom (or $x1898 $x109)) @x2004 $x109) (unit-resolution (def-axiom (or $x1898 $x104)) @x2004 $x104) (unit-resolution (def-axiom (or $x1898 $x107)) @x2004 $x107) $x136)))
+(let ((@x2128 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x1362 $x1522)) (unit-resolution (def-axiom (or $x1898 $x684)) @x2004 $x684) $x1522)))
+(let ((@x1460 (unit-resolution @x1808 (unit-resolution @x1523 (hypothesis $x136) $x1886) (hypothesis $x1892) $x1318)))
+(let ((@x1539 (def-axiom (or $x1313 $x1053))))
+(let (($x1965 (not $x1560)))
+(let (($x1597 (<= (+ ?x101 ?x744) 0)))
+(let ((@x1431 (trans (symm (hypothesis $x104) (= ?x101 v_b_max_G_2$)) (symm (hypothesis $x109) (= v_b_max_G_2$ v_b_max_G_3$)) (= ?x101 v_b_max_G_3$))))
+(let ((@x1435 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x101 v_b_max_G_3$)) $x1597)) @x1431 $x1597)))
+(let ((@x1437 (lemma ((_ th-lemma arith farkas -1 -1 1) (hypothesis $x1436) (hypothesis $x1597) (hypothesis $x1445) false) (or $x1453 $x1070 (not $x1597)))))
+(let ((@x1952 (unit-resolution @x1565 (unit-resolution @x1437 (unit-resolution @x1812 @x1460 $x1436) @x1435 $x1453) $x1563)))
+(let ((@x1958 (unit-resolution ((_ th-lemma arith assign-bounds 1 1 1) (or $x1955 $x1070 (not $x1597) $x689)) (unit-resolution @x1812 @x1460 $x1436) @x1435 (hypothesis $x692) $x1955)))
+(let ((@x1962 (unit-resolution (mp ((_ quant-inst ?v0!3) $x1464) @x1450 $x1476) (hypothesis $x1853) (unit-resolution (def-axiom (or $x1313 $x931)) @x1460 $x931) (or $x1511 $x1488))))
+(let ((@x1969 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x1558 (not $x1511) $x1965)) (unit-resolution @x1962 @x1958 $x1511) (or $x1558 $x1965))))
+(let ((@x1971 ((_ th-lemma arith farkas -1 1 1) (unit-resolution @x1969 (unit-resolution @x1540 @x1952 (not $x1558)) $x1965) (hypothesis $x1522) (unit-resolution @x1539 @x1460 $x1053) false)))
+(let ((@x2130 (unit-resolution (lemma @x1971 (or $x951 (not $x1522) $x1858 $x689 $x1895 $x1359 $x1361)) @x2093 (or $x951 (not $x1522) $x689 $x1895 $x1359 $x1361))))
+(unit-resolution @x2130 @x2128 @x2140 (unit-resolution (def-axiom (or $x1898 $x692)) @x2004 $x692) (unit-resolution (def-axiom (or $x1898 $x1892)) @x2004 $x1892) (unit-resolution (def-axiom (or $x1898 $x104)) @x2004 $x104) (unit-resolution (def-axiom (or $x1898 $x109)) @x2004 $x109) false)))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))
+
--- a/src/HOL/SMT_Examples/SMT_Examples.certs2	Tue Jun 03 16:22:01 2014 +0200
+++ b/src/HOL/SMT_Examples/SMT_Examples.certs2	Tue Jun 03 16:27:31 2014 +0200
@@ -1,4 +1,19 @@
-6ef15d5757e12551f288742c4dce61fbb4a48e2d 9 0
+3e49cb365d2f84977be8ddb3771bcc354b18e2da 6 0
+unsat
+((set-logic AUFLIA)
+(proof
+(let ((@x30 (rewrite (= (not true) false))))
+(mp (asserted (not true)) @x30 false))))
+
+eda548b925b5843c60e62dbbde93cd51aec726cd 7 0
+unsat
+((set-logic AUFLIA)
+(proof
+(let ((@x36 (monotonicity (rewrite (= (or p$ (not p$)) true)) (= (not (or p$ (not p$))) (not true)))))
+(let ((@x40 (trans @x36 (rewrite (= (not true) false)) (= (not (or p$ (not p$))) false))))
+(mp (asserted (not (or p$ (not p$)))) @x40 false)))))
+
+853f72b15f802590d68a8ff710d53b08079e9f25 9 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -8,22 +23,33 @@
 (let ((@x47 (trans @x43 (rewrite (= (not true) false)) (= (not (= (and p$ true) p$)) false))))
 (mp (asserted (not (= (and p$ true) p$))) @x47 false)))))))
 
-d23c7684cffd678dfbdd7b614197ecef170e9b21 6 0
+bc944fad642a1e33cb760904138c7fbd5c55fe99 13 0
 unsat
 ((set-logic AUFLIA)
 (proof
-(let ((@x30 (rewrite (= (not true) false))))
-(mp (asserted (not true)) @x30 false))))
+(let (($x33 (not (=> (and (or p$ q$) (not p$)) q$))))
+(let (($x37 (= (=> (and (or p$ q$) (not p$)) q$) (or (not (and (or p$ q$) (not p$))) q$))))
+(let ((@x41 (monotonicity (rewrite $x37) (= $x33 (not (or (not (and (or p$ q$) (not p$))) q$))))))
+(let ((@x44 (mp (asserted $x33) @x41 (not (or (not (and (or p$ q$) (not p$))) q$)))))
+(let ((@x45 (and-elim (not-or-elim @x44 (and (or p$ q$) (not p$))) (not p$))))
+(let ((@x54 (monotonicity (iff-false @x45 (= p$ false)) (iff-false (not-or-elim @x44 (not q$)) (= q$ false)) (= (or p$ q$) (or false false)))))
+(let ((@x58 (trans @x54 (rewrite (= (or false false) false)) (= (or p$ q$) false))))
+(let (($x29 (or p$ q$)))
+(mp (and-elim (not-or-elim @x44 (and $x29 (not p$))) $x29) @x58 false)))))))))))
 
-85938d4e39bdd250fc7d6d1310c58a831798d91d 7 0
+0254fd7dc9fb99b1e3c68f22cbe647c82b00ce69 11 0
 unsat
 ((set-logic AUFLIA)
 (proof
-(let ((@x36 (monotonicity (rewrite (= (or p$ (not p$)) true)) (= (not (or p$ (not p$))) (not true)))))
-(let ((@x40 (trans @x36 (rewrite (= (not true) false)) (= (not (or p$ (not p$))) false))))
-(mp (asserted (not (or p$ (not p$)))) @x40 false)))))
+(let (($x32 (and c$ d$)))
+(let (($x29 (and a$ b$)))
+(let (($x33 (or $x29 $x32)))
+(let (($x34 (=> $x33 $x33)))
+(let (($x35 (not $x34)))
+(let ((@x45 (trans (monotonicity (rewrite (= $x34 true)) (= $x35 (not true))) (rewrite (= (not true) false)) (= $x35 false))))
+(mp (asserted $x35) @x45 false)))))))))
 
-11b5ff41fb5050714ac35f86f3cf14c21ab6bd0f 23 0
+e6c423a181ed233be5f1dc2cac4fddfbc7fcf552 23 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -47,33 +73,7 @@
 (let ((@x58 (monotonicity (trans @x49 (rewrite (= (=> $x31 $x44) $x51)) (= $x37 $x51)) (= $x38 $x56))))
 (mp (asserted $x38) (trans @x58 @x67 (= $x38 false)) false)))))))))))))))))))))
 
-09401881a11dd403572091d4efe07f044e1df713 13 0
-unsat
-((set-logic AUFLIA)
-(proof
-(let (($x33 (not (=> (and (or p$ q$) (not p$)) q$))))
-(let (($x37 (= (=> (and (or p$ q$) (not p$)) q$) (or (not (and (or p$ q$) (not p$))) q$))))
-(let ((@x41 (monotonicity (rewrite $x37) (= $x33 (not (or (not (and (or p$ q$) (not p$))) q$))))))
-(let ((@x44 (mp (asserted $x33) @x41 (not (or (not (and (or p$ q$) (not p$))) q$)))))
-(let ((@x45 (and-elim (not-or-elim @x44 (and (or p$ q$) (not p$))) (not p$))))
-(let ((@x54 (monotonicity (iff-false @x45 (= p$ false)) (iff-false (not-or-elim @x44 (not q$)) (= q$ false)) (= (or p$ q$) (or false false)))))
-(let ((@x58 (trans @x54 (rewrite (= (or false false) false)) (= (or p$ q$) false))))
-(let (($x29 (or p$ q$)))
-(mp (and-elim (not-or-elim @x44 (and $x29 (not p$))) $x29) @x58 false)))))))))))
-
-a4d516e1422eb475560be574681f28b06985be50 11 0
-unsat
-((set-logic AUFLIA)
-(proof
-(let (($x32 (and c$ d$)))
-(let (($x29 (and a$ b$)))
-(let (($x33 (or $x29 $x32)))
-(let (($x34 (=> $x33 $x33)))
-(let (($x35 (not $x34)))
-(let ((@x45 (trans (monotonicity (rewrite (= $x34 true)) (= $x35 (not true))) (rewrite (= (not true) false)) (= $x35 false))))
-(mp (asserted $x35) @x45 false)))))))))
-
-f900e7bf7b793a5fde805469aaa724607533e84e 24 0
+cc37a013f00f1a8a65604ca2822223c8c303278e 24 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -98,7 +98,7 @@
 (let ((@x82 (trans (monotonicity @x75 (= $x37 (not true))) (rewrite (= (not true) false)) (= $x37 false))))
 (mp (asserted $x37) @x82 false))))))))))))))))))))))
 
-c6e2ff75bf3674f3670b76a57974bcdbe3b2e34a 39 0
+40b39e2d1a04236093e96081605bcd51392df4b4 39 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -138,7 +138,7 @@
 (let ((@x40 (mp (asserted (or a$ (or b$ (or c$ d$)))) (rewrite (= (or a$ (or b$ (or c$ d$))) $x37)) $x37)))
 (mp @x40 @x202 false)))))))))))))))))))))))))))))))))))))
 
-37c8cbfd0b65b6e0dbafd0d63335000db1e88a45 27 0
+685995a75ef22cfac4fa1571ee30f23149426b18 27 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -166,46 +166,7 @@
 (let ((@x61 ((_ quant-inst a$ b$) $x149)))
 (unit-resolution @x61 @x485 @x57 false)))))))))))))))))))
 
-c107a75e14d611a8e5d82479c10abfc46dd5c755 38 0
-unsat
-((set-logic AUFLIA)
-(declare-fun ?v0!0 () Int)
-(declare-fun ?v1!1 () Int)
-(proof
-(let (($x48 (p$ ?v0!0)))
-(let (($x50 (not $x48)))
-(let (($x64 (not (or $x48 (p$ ?v1!1)))))
-(let ((@x77 (monotonicity (rewrite (= (not $x50) $x48)) (= (and (not $x50) $x64) (and $x48 $x64)))))
-(let (($x57 (not $x50)))
-(let (($x67 (and $x57 $x64)))
-(let (($x41 (forall ((?v0 Int) )(let (($x32 (forall ((?v1 Int) )(let (($x28 (p$ ?v1)))
-(or (p$ ?v0) $x28)))
-))
-(or (not (p$ ?v0)) $x32)))
-))
-(let (($x44 (not $x41)))
-(let (($x52 (forall ((?v1 Int) )(let (($x28 (p$ ?v1)))
-(let (($x48 (p$ ?v0!0)))
-(or $x48 $x28))))
-))
-(let ((@x69 (nnf-neg (refl (~ $x57 $x57)) (sk (~ (not $x52) $x64)) (~ (not (or $x50 $x52)) $x67))))
-(let (($x34 (forall ((?v0 Int) )(let (($x32 (forall ((?v1 Int) )(let (($x28 (p$ ?v1)))
-(or (p$ ?v0) $x28)))
-))
-(let (($x28 (p$ ?v0)))
-(=> $x28 $x32))))
-))
-(let (($x35 (not $x34)))
-(let (($x32 (forall ((?v1 Int) )(let (($x28 (p$ ?v1)))
-(or (p$ ?0) $x28)))
-))
-(let ((@x43 (quant-intro (rewrite (= (=> (p$ ?0) $x32) (or (not (p$ ?0)) $x32))) (= $x34 $x41))))
-(let ((@x72 (mp~ (mp (asserted $x35) (monotonicity @x43 (= $x35 $x44)) $x44) (trans (sk (~ $x44 (not (or $x50 $x52)))) @x69 (~ $x44 $x67)) $x67)))
-(let ((@x81 (not-or-elim (and-elim (mp @x72 @x77 (and $x48 $x64)) $x64) $x50)))
-(let ((@x79 (and-elim (mp @x72 @x77 (and $x48 $x64)) $x48)))
-(unit-resolution @x79 @x81 false))))))))))))))))))))
-
-ea70394857a4c8c662289548e2d7f9f3803b42bb 637 0
+f4fa77f2d3aebec03f0078d83a92f590ad57699e 637 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -843,7 +804,46 @@
 (let ((@x1722 (unit-resolution @x1662 (unit-resolution @x472 @x1718 $x467) (unit-resolution @x565 @x1715 $x482) $x355)))
 (unit-resolution @x1647 @x1722 (unit-resolution @x472 @x1718 $x467) (unit-resolution @x565 @x1715 $x482) (unit-resolution @x480 @x1718 $x397) false)))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))
 
-eeecd6c9779ef5d70c86f61cca0282e6f6b227b5 53 0
+f21bf7f9491a17ae420581bdb52bbd1d9857412e 38 0
+unsat
+((set-logic AUFLIA)
+(declare-fun ?v0!0 () Int)
+(declare-fun ?v1!1 () Int)
+(proof
+(let (($x48 (p$ ?v0!0)))
+(let (($x50 (not $x48)))
+(let (($x63 (not (or $x48 (p$ ?v1!1)))))
+(let ((@x77 (monotonicity (rewrite (= (not $x50) $x48)) (= (and (not $x50) $x63) (and $x48 $x63)))))
+(let (($x57 (not $x50)))
+(let (($x67 (and $x57 $x63)))
+(let (($x41 (forall ((?v0 Int) )(let (($x32 (forall ((?v1 Int) )(let (($x28 (p$ ?v1)))
+(or (p$ ?v0) $x28)))
+))
+(or (not (p$ ?v0)) $x32)))
+))
+(let (($x44 (not $x41)))
+(let (($x52 (forall ((?v1 Int) )(let (($x28 (p$ ?v1)))
+(let (($x48 (p$ ?v0!0)))
+(or $x48 $x28))))
+))
+(let ((@x69 (nnf-neg (refl (~ $x57 $x57)) (sk (~ (not $x52) $x63)) (~ (not (or $x50 $x52)) $x67))))
+(let (($x34 (forall ((?v0 Int) )(let (($x32 (forall ((?v1 Int) )(let (($x28 (p$ ?v1)))
+(or (p$ ?v0) $x28)))
+))
+(let (($x28 (p$ ?v0)))
+(=> $x28 $x32))))
+))
+(let (($x35 (not $x34)))
+(let (($x32 (forall ((?v1 Int) )(let (($x28 (p$ ?v1)))
+(or (p$ ?0) $x28)))
+))
+(let ((@x43 (quant-intro (rewrite (= (=> (p$ ?0) $x32) (or (not (p$ ?0)) $x32))) (= $x34 $x41))))
+(let ((@x72 (mp~ (mp (asserted $x35) (monotonicity @x43 (= $x35 $x44)) $x44) (trans (sk (~ $x44 (not (or $x50 $x52)))) @x69 (~ $x44 $x67)) $x67)))
+(let ((@x81 (not-or-elim (and-elim (mp @x72 @x77 (and $x48 $x63)) $x63) $x50)))
+(let ((@x79 (and-elim (mp @x72 @x77 (and $x48 $x63)) $x48)))
+(unit-resolution @x79 @x81 false))))))))))))))))))))
+
+9c45fe28ef4034444b16a63b5d3ef9ee357f8069 53 0
 unsat
 ((set-logic AUFLIA)
 (declare-fun ?v0!0 () A$)
@@ -870,34 +870,34 @@
 (let ((@x503 ((_ quant-inst x$ c$) $x170)))
 (let (($x73 (p$ x$ ?v0!0)))
 (let (($x179 (= $x73 x$)))
-(let (($x84 (or $x73 $x44)))
+(let (($x85 (or $x73 $x44)))
 (let (($x81 (not $x44)))
 (let (($x69 (forall ((?v0 A$) )(let (($x40 (p$ x$ ?v0)))
 (not $x40)))
 ))
-(let (($x85 (or $x69 $x81)))
+(let (($x84 (or $x69 $x81)))
 (let (($x42 (exists ((?v0 A$) )(p$ x$ ?v0))
 ))
 (let (($x54 (not $x42)))
 (let (($x55 (= $x54 $x44)))
 (let ((@x71 (nnf-neg (refl (~ (not (p$ x$ ?0)) (not (p$ x$ ?0)))) (~ $x54 $x69))))
-(let ((@x88 (nnf-pos @x71 (nnf-neg (sk (~ $x42 $x73)) (~ (not $x54) $x73)) (refl (~ $x44 $x44)) (refl (~ $x81 $x81)) (~ $x55 (and $x84 $x85)))))
+(let ((@x88 (nnf-pos @x71 (nnf-neg (sk (~ $x42 $x73)) (~ (not $x54) $x73)) (refl (~ $x44 $x44)) (refl (~ $x81 $x81)) (~ $x55 (and $x85 $x84)))))
 (let ((@x53 (monotonicity (rewrite (= (= $x42 $x44) (= $x42 $x44))) (= (not (= $x42 $x44)) (not (= $x42 $x44))))))
 (let ((@x59 (trans @x53 (rewrite (= (not (= $x42 $x44)) $x55)) (= (not (= $x42 $x44)) $x55))))
-(let ((@x89 (mp~ (mp (asserted (not (= $x42 $x44))) @x59 $x55) @x88 (and $x84 $x85))))
-(let ((@x92 (and-elim @x89 $x84)))
+(let ((@x89 (mp~ (mp (asserted (not (= $x42 $x44))) @x59 $x55) @x88 (and $x85 $x84))))
+(let ((@x92 (and-elim @x89 $x85)))
 (let ((@x484 (unit-resolution (def-axiom (or (not $x179) (not $x73) x$)) (unit-resolution @x92 (hypothesis $x81) $x73) (or (not $x179) x$))))
 (let ((@x145 (unit-resolution @x484 (unit-resolution ((_ quant-inst x$ ?v0!0) (or (not $x510) $x179)) @x515 $x179) x$)))
 (let ((@x147 (unit-resolution (def-axiom (or (not $x91) $x44 (not x$))) (hypothesis $x81) (or (not $x91) (not x$)))))
 (let ((@x485 (lemma (unit-resolution @x147 @x145 (unit-resolution @x503 @x515 $x91) false) $x44)))
 (let (($x522 (or $x517 $x81)))
 (let ((@x521 (quant-intro (refl (= (not (p$ x$ ?0)) (not (p$ x$ ?0)))) (= $x69 $x517))))
-(let ((@x525 (mp (and-elim @x89 $x85) (monotonicity @x521 (= $x85 $x522)) $x522)))
+(let ((@x525 (mp (and-elim @x89 $x84) (monotonicity @x521 (= $x84 $x522)) $x522)))
 (let (($x160 (or (not $x517) $x81)))
 (let ((@x161 ((_ quant-inst c$) $x160)))
 (unit-resolution @x161 @x485 (unit-resolution @x525 @x485 $x517) false)))))))))))))))))))))))))))))))))))))))
 
-48e1796773de6c2c0546e34aa9ce5aa2097adf0a 53 0
+add25b227a3fe99971fe1b09f27504b2c1357233 53 0
 unsat
 ((set-logic AUFLIA)
 (declare-fun ?v0!3 () A$)
@@ -924,34 +924,34 @@
 (let ((@x221 ((_ quant-inst x$ c$) $x220)))
 (let (($x124 (p$ x$ ?v0!3)))
 (let (($x141 (= $x124 x$)))
-(let (($x135 (or $x124 $x55)))
+(let (($x136 (or $x124 $x55)))
 (let (($x132 (not $x55)))
 (let (($x120 (forall ((?v0 A$) )(let (($x52 (p$ x$ ?v0)))
 (not $x52)))
 ))
-(let (($x136 (or $x120 $x132)))
+(let (($x135 (or $x120 $x132)))
 (let (($x54 (exists ((?v0 A$) )(p$ x$ ?v0))
 ))
 (let (($x65 (not $x54)))
 (let (($x66 (= $x65 $x55)))
 (let ((@x122 (nnf-neg (refl (~ (not (p$ x$ ?0)) (not (p$ x$ ?0)))) (~ $x65 $x120))))
-(let ((@x139 (nnf-pos @x122 (nnf-neg (sk (~ $x54 $x124)) (~ (not $x65) $x124)) (refl (~ $x55 $x55)) (refl (~ $x132 $x132)) (~ $x66 (and $x135 $x136)))))
+(let ((@x139 (nnf-pos @x122 (nnf-neg (sk (~ $x54 $x124)) (~ (not $x65) $x124)) (refl (~ $x55 $x55)) (refl (~ $x132 $x132)) (~ $x66 (and $x136 $x135)))))
 (let ((@x64 (monotonicity (rewrite (= (= $x54 $x55) (= $x54 $x55))) (= (not (= $x54 $x55)) (not (= $x54 $x55))))))
 (let ((@x70 (trans @x64 (rewrite (= (not (= $x54 $x55)) $x66)) (= (not (= $x54 $x55)) $x66))))
-(let ((@x140 (mp~ (mp (asserted (not (= $x54 $x55))) @x70 $x66) @x139 (and $x135 $x136))))
-(let ((@x143 (and-elim @x140 $x135)))
+(let ((@x140 (mp~ (mp (asserted (not (= $x54 $x55))) @x70 $x66) @x139 (and $x136 $x135))))
+(let ((@x143 (and-elim @x140 $x136)))
 (let ((@x193 (unit-resolution (def-axiom (or (not $x141) (not $x124) x$)) (unit-resolution @x143 (hypothesis $x132) $x124) (or (not $x141) x$))))
 (let ((@x535 (unit-resolution @x193 (unit-resolution ((_ quant-inst x$ ?v0!3) (or (not $x561) $x141)) @x566 $x141) x$)))
 (let ((@x197 (unit-resolution (def-axiom (or (not $x230) $x55 (not x$))) (hypothesis $x132) (or (not $x230) (not x$)))))
 (let ((@x199 (lemma (unit-resolution @x197 @x535 (unit-resolution @x221 @x566 $x230) false) $x55)))
 (let (($x589 (or $x584 $x132)))
 (let ((@x588 (quant-intro (refl (= (not (p$ x$ ?0)) (not (p$ x$ ?0)))) (= $x120 $x584))))
-(let ((@x592 (mp (and-elim @x140 $x136) (monotonicity @x588 (= $x136 $x589)) $x589)))
+(let ((@x592 (mp (and-elim @x140 $x135) (monotonicity @x588 (= $x135 $x589)) $x589)))
 (let (($x549 (or (not $x584) $x132)))
 (let ((@x211 ((_ quant-inst c$) $x549)))
 (unit-resolution @x211 @x199 (unit-resolution @x592 @x199 $x584) false)))))))))))))))))))))))))))))))))))))))
 
-2df8e4308f7ae8ea39388023f7bd76c530ffef8c 26 0
+6e1ff5fbd8bb1e07db66392756af68190f5710fc 26 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -978,7 +978,7 @@
 (let ((@x70 ((_ quant-inst x$) $x156)))
 (unit-resolution @x70 @x491 @x49 false)))))))))))))))))))
 
-80de60849dcf0651c1aedd7f781a8e7ca39f83d7 7 0
+4d06340faf678d780abe1b549d370cfbc6a06283 7 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -986,7 +986,7 @@
 (let ((@x39 (trans @x35 (rewrite (= (not true) false)) (= (not (= 3 3)) false))))
 (mp (asserted (not (= 3 3))) @x39 false)))))
 
-e65839fa5c1f3589cfc5db6ea43029f8639a17fe 7 0
+c50285acac95353711e1b3c14e259c11a865a457 7 0
 unsat
 ((set-logic AUFLIRA)
 (proof
@@ -994,7 +994,7 @@
 (let ((@x39 (trans @x35 (rewrite (= (not true) false)) (= (not (= 3.0 3.0)) false))))
 (mp (asserted (not (= 3.0 3.0))) @x39 false)))))
 
-e571eb0660d494fd6aa308bebdd9b517a21af759 9 0
+9ea7ebd4a1255b1c69f10ddd25579a26623a9829 9 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -1004,7 +1004,7 @@
 (let ((@x48 (trans @x44 (rewrite (= (not true) false)) (= (not (= (+ 3 1) 4)) false))))
 (mp (asserted (not (= (+ 3 1) 4))) @x48 false)))))))
 
-c7eed2f76baba4a0c01a800ee2da514b0162cac7 16 0
+acf4f35bbccceadec51bcf1732fa619318da6e6a 16 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -1021,7 +1021,7 @@
 (let ((@x63 (trans (monotonicity @x56 (= $x35 (not true))) (rewrite (= (not true) false)) (= $x35 false))))
 (mp (asserted $x35) @x63 false))))))))))))))
 
-38b869bfd4118f2fcf9bed900c8fd8af524dcd76 11 0
+f7062dfbd56ef142487caec036d85622d510acc0 11 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -1033,7 +1033,7 @@
 (let ((@x59 (trans @x55 (rewrite (= (not true) false)) (= (not (< 5 (ite (<= 3 8) 8 3))) false))))
 (mp (asserted (not (< 5 (ite (<= 3 8) 8 3)))) @x59 false)))))))))
 
-eb4f0cbaa80520a62b72d8aba335f8d20fb56cb8 88 0
+5869334c390e42307ff6dacd4cb34b2fbcd91f23 88 0
 unsat
 ((set-logic AUFLIRA)
 (proof
@@ -1122,7 +1122,7 @@
 (let ((@x234 (unit-resolution @x136 (unit-resolution @x138 (lemma @x231 (not $x134)) $x83) $x133)))
 ((_ th-lemma arith farkas -2 1 -1 -1 1) (unit-resolution @x138 (lemma @x231 (not $x134)) $x83) @x221 @x126 @x226 (unit-resolution @x173 @x234 $x149) false))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))
 
-b033145c396900caefe8b7b0bb0eb6f18ba1b976 16 0
+23e93683167899d4e5714fd0dd3ef72db374d210 16 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -1139,7 +1139,7 @@
 (let ((@x46 (monotonicity @x43 (= $x34 (not (= (p$ $x29) ?x32))))))
 (mp (asserted $x34) (trans @x46 @x63 (= $x34 false)) false))))))))))))))
 
-8b9e890789d51395030c5121155b5df222b5edc3 16 0
+0dacec367e5e4a73f1a722bdecfc5909ba863310 16 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -1156,7 +1156,7 @@
 (let ((@x70 (trans @x48 @x68 (= (not (or (<= 4 (+ x$ 3)) $x33)) false))))
 (mp (asserted (not (or (<= 4 (+ x$ 3)) $x33))) @x70 false))))))))))))))
 
-154bdf1c6ef792cc3795d45472fcc25a640e2843 18 0
+c1f070b03c72df3665299559abe6324267b678f4 18 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -1175,7 +1175,7 @@
 (let ((@x83 (mp (asserted $x58) (trans (monotonicity @x66 (= $x58 $x67)) @x80 (= $x58 $x70)) $x70)))
 (mp @x83 @x90 false))))))))))))))))
 
-a3d554bfa10b48cb1a494a10bb1e501be6292b39 11 0
+8d9f7ab3847c14170f0ea8f147f2c27593d2f794 11 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -1187,7 +1187,7 @@
 (let ((@x57 (trans @x53 (rewrite (= (not true) false)) (= (not (not (= (+ 2 2) 5))) false))))
 (mp (asserted (not (not (= (+ 2 2) 5)))) @x57 false)))))))))
 
-574989c0cc54480cb40b21b6e42362819c4a33e8 22 0
+da06c9772c963270cacb44bca84fb24a6715b6b0 22 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -1210,7 +1210,7 @@
 (let ((@x78 (trans (monotonicity @x71 (= $x40 (not true))) (rewrite (= (not true) false)) (= $x40 false))))
 (mp (asserted $x40) @x78 false))))))))))))))))))))
 
-e52dc26c77bd7d10a72f38a2499294aa0ff205b3 19 0
+2b2e1c484321a806c0b36f3310c53635c9c2585c 19 0
 unsat
 ((set-logic AUFLIRA)
 (proof
@@ -1230,7 +1230,7 @@
 (let ((@x67 (mp (asserted (not (< a$ 0.0))) @x66 $x58)))
 ((_ th-lemma arith farkas 7 3/2 1) @x67 @x52 @x40 false)))))))))))))))))
 
-c39f49e54187d0a817f3e4a791616e6b5ccf322c 159 0
+6aeae777626a0656caf5988c97b33e73009f1993 159 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -1390,28 +1390,7 @@
 (let ((@x433 (mp (not-or-elim @x205 (not $x57)) @x432 $x422)))
 (unit-resolution @x433 @x488 (mp @x478 @x480 $x44) false)))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))
 
-08815a713893cf2f2359b61906c2360b4a2a841e 20 0
-unsat
-((set-logic AUFLIRA)
-(proof
-(let ((?x30 (* 2.0 x$)))
-(let ((?x32 (+ ?x30 1.0)))
-(let ((?x28 (+ x$ x$)))
-(let (($x33 (< ?x28 ?x32)))
-(let (($x34 (or false $x33)))
-(let (($x35 (or $x33 $x34)))
-(let (($x36 (not $x35)))
-(let ((@x67 (monotonicity (rewrite (= (< ?x30 (+ 1.0 ?x30)) true)) (= (not (< ?x30 (+ 1.0 ?x30))) (not true)))))
-(let ((@x71 (trans @x67 (rewrite (= (not true) false)) (= (not (< ?x30 (+ 1.0 ?x30))) false))))
-(let ((?x40 (+ 1.0 ?x30)))
-(let (($x43 (< ?x30 ?x40)))
-(let ((@x45 (monotonicity (rewrite (= ?x28 ?x30)) (rewrite (= ?x32 ?x40)) (= $x33 $x43))))
-(let ((@x52 (trans (monotonicity @x45 (= $x34 (or false $x43))) (rewrite (= (or false $x43) $x43)) (= $x34 $x43))))
-(let ((@x59 (trans (monotonicity @x45 @x52 (= $x35 (or $x43 $x43))) (rewrite (= (or $x43 $x43) $x43)) (= $x35 $x43))))
-(let ((@x62 (monotonicity @x59 (= $x36 (not $x43)))))
-(mp (asserted $x36) (trans @x62 @x71 (= $x36 false)) false))))))))))))))))))
-
-65e2c3423bd20786a741d330830050f8c51df180 933 0
+bc03e4aa9e0481125feaa6ba37a3c4bea0d39acd 933 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -2345,120 +2324,28 @@
 (let ((@x2059 (unit-resolution @x1592 (unit-resolution @x1271 (unit-resolution @x591 @x2050 $x588) $x672) @x2026 @x2058 (unit-resolution @x693 (unit-resolution @x599 @x2014 $x596) $x678) (unit-resolution @x725 (unit-resolution @x591 @x2050 $x588) $x681) $x653)))
 (unit-resolution @x1307 @x2059 @x2055 @x1942 false)))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))
 
-4a8a0bf3d43500148c2184dcd30bf04139ef48a8 112 0
+cb06f8242245a2a9fa59299555f1031ed2fbcc42 20 0
 unsat
-((set-logic <null>)
+((set-logic AUFLIRA)
 (proof
-(let ((?x224 (mod x$ 2)))
-(let (($x318 (>= ?x224 2)))
-(let (($x319 (not $x318)))
-(let ((?x258 (* (- 1) ?x224)))
-(let ((?x29 (mod$ x$ 2)))
-(let ((?x259 (+ ?x29 ?x258)))
-(let (($x275 (<= ?x259 0)))
-(let (($x260 (= ?x259 0)))
-(let (($x201 (forall ((?v0 Int) (?v1 Int) )(!(let ((?x132 (mod ?v0 ?v1)))
-(let ((?x89 (* (- 1) ?v1)))
-(let ((?x86 (* (- 1) ?v0)))
-(let ((?x140 (mod ?x86 ?x89)))
-(let ((?x146 (* (- 1) ?x140)))
-(let (($x107 (<= ?v1 0)))
-(let ((?x166 (ite $x107 ?x146 ?x132)))
-(let (($x74 (= ?v1 0)))
-(let ((?x171 (ite $x74 ?v0 ?x166)))
-(let ((?x131 (mod$ ?v0 ?v1)))
-(= ?x131 ?x171))))))))))) :pattern ( (mod$ ?v0 ?v1) )))
-))
-(let (($x177 (forall ((?v0 Int) (?v1 Int) )(let ((?x132 (mod ?v0 ?v1)))
-(let ((?x89 (* (- 1) ?v1)))
-(let ((?x86 (* (- 1) ?v0)))
-(let ((?x140 (mod ?x86 ?x89)))
-(let ((?x146 (* (- 1) ?x140)))
-(let (($x107 (<= ?v1 0)))
-(let ((?x166 (ite $x107 ?x146 ?x132)))
-(let (($x74 (= ?v1 0)))
-(let ((?x171 (ite $x74 ?v0 ?x166)))
-(let ((?x131 (mod$ ?v0 ?v1)))
-(= ?x131 ?x171))))))))))))
-))
-(let ((?x132 (mod ?1 ?0)))
-(let ((?x89 (* (- 1) ?0)))
-(let ((?x86 (* (- 1) ?1)))
-(let ((?x140 (mod ?x86 ?x89)))
-(let ((?x146 (* (- 1) ?x140)))
-(let (($x107 (<= ?0 0)))
-(let ((?x166 (ite $x107 ?x146 ?x132)))
-(let (($x74 (= ?0 0)))
-(let ((?x171 (ite $x74 ?1 ?x166)))
-(let ((?x131 (mod$ ?1 ?0)))
-(let (($x174 (= ?x131 ?x171)))
-(let (($x138 (forall ((?v0 Int) (?v1 Int) )(let (($x74 (= ?v1 0)))
-(let ((?x136 (ite $x74 ?v0 (ite (< 0 ?v1) (mod ?v0 ?v1) (- (mod (- ?v0) (- ?v1)))))))
-(let ((?x131 (mod$ ?v0 ?v1)))
-(= ?x131 ?x136)))))
-))
-(let (($x160 (forall ((?v0 Int) (?v1 Int) )(let ((?x89 (* (- 1) ?v1)))
-(let ((?x86 (* (- 1) ?v0)))
-(let ((?x140 (mod ?x86 ?x89)))
-(let ((?x146 (* (- 1) ?x140)))
-(let ((?x132 (mod ?v0 ?v1)))
-(let (($x75 (< 0 ?v1)))
-(let ((?x151 (ite $x75 ?x132 ?x146)))
-(let (($x74 (= ?v1 0)))
-(let ((?x154 (ite $x74 ?v0 ?x151)))
-(let ((?x131 (mod$ ?v0 ?v1)))
-(= ?x131 ?x154))))))))))))
-))
-(let ((@x165 (monotonicity (rewrite (= (< 0 ?0) (not $x107))) (= (ite (< 0 ?0) ?x132 ?x146) (ite (not $x107) ?x132 ?x146)))))
-(let ((@x170 (trans @x165 (rewrite (= (ite (not $x107) ?x132 ?x146) ?x166)) (= (ite (< 0 ?0) ?x132 ?x146) ?x166))))
-(let ((@x173 (monotonicity @x170 (= (ite $x74 ?1 (ite (< 0 ?0) ?x132 ?x146)) ?x171))))
-(let ((@x176 (monotonicity @x173 (= (= ?x131 (ite $x74 ?1 (ite (< 0 ?0) ?x132 ?x146))) $x174))))
-(let (($x75 (< 0 ?0)))
-(let ((?x151 (ite $x75 ?x132 ?x146)))
-(let ((?x154 (ite $x74 ?1 ?x151)))
-(let (($x157 (= ?x131 ?x154)))
-(let (($x158 (= (= ?x131 (ite $x74 ?1 (ite $x75 ?x132 (- (mod (- ?1) (- ?0)))))) $x157)))
-(let ((@x142 (monotonicity (rewrite (= (- ?1) ?x86)) (rewrite (= (- ?0) ?x89)) (= (mod (- ?1) (- ?0)) ?x140))))
-(let ((@x150 (trans (monotonicity @x142 (= (- (mod (- ?1) (- ?0))) (- ?x140))) (rewrite (= (- ?x140) ?x146)) (= (- (mod (- ?1) (- ?0))) ?x146))))
-(let ((@x153 (monotonicity @x150 (= (ite $x75 ?x132 (- (mod (- ?1) (- ?0)))) ?x151))))
-(let ((@x156 (monotonicity @x153 (= (ite $x74 ?1 (ite $x75 ?x132 (- (mod (- ?1) (- ?0))))) ?x154))))
-(let ((@x181 (trans (quant-intro (monotonicity @x156 $x158) (= $x138 $x160)) (quant-intro @x176 (= $x160 $x177)) (= $x138 $x177))))
-(let ((@x192 (mp~ (mp (asserted $x138) @x181 $x177) (nnf-pos (refl (~ $x174 $x174)) (~ $x177 $x177)) $x177)))
-(let ((@x206 (mp @x192 (quant-intro (refl (= $x174 $x174)) (= $x177 $x201)) $x201)))
-(let (($x266 (or (not $x201) $x260)))
-(let ((?x221 (* (- 1) 2)))
-(let ((?x220 (* (- 1) x$)))
-(let ((?x222 (mod ?x220 ?x221)))
-(let ((?x223 (* (- 1) ?x222)))
-(let (($x219 (<= 2 0)))
-(let ((?x225 (ite $x219 ?x223 ?x224)))
-(let (($x218 (= 2 0)))
-(let ((?x226 (ite $x218 x$ ?x225)))
-(let (($x227 (= ?x29 ?x226)))
-(let ((@x240 (monotonicity (monotonicity (rewrite (= ?x221 (- 2))) (= ?x222 (mod ?x220 (- 2)))) (= ?x223 (* (- 1) (mod ?x220 (- 2)))))))
-(let ((@x243 (monotonicity (rewrite (= $x219 false)) @x240 (= ?x225 (ite false (* (- 1) (mod ?x220 (- 2))) ?x224)))))
-(let ((@x247 (trans @x243 (rewrite (= (ite false (* (- 1) (mod ?x220 (- 2))) ?x224) ?x224)) (= ?x225 ?x224))))
-(let ((@x250 (monotonicity (rewrite (= $x218 false)) @x247 (= ?x226 (ite false x$ ?x224)))))
-(let ((@x257 (monotonicity (trans @x250 (rewrite (= (ite false x$ ?x224) ?x224)) (= ?x226 ?x224)) (= $x227 (= ?x29 ?x224)))))
-(let ((@x270 (monotonicity (trans @x257 (rewrite (= (= ?x29 ?x224) $x260)) (= $x227 $x260)) (= (or (not $x201) $x227) $x266))))
-(let ((@x273 (trans @x270 (rewrite (= $x266 $x266)) (= (or (not $x201) $x227) $x266))))
-(let ((@x274 (mp ((_ quant-inst x$ 2) (or (not $x201) $x227)) @x273 $x266)))
-(let ((@x336 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x260) $x275)) (unit-resolution @x274 @x206 $x260) $x275)))
-(let (($x63 (>= ?x29 2)))
-(let ((?x37 (* 2 ?x29)))
-(let (($x56 (>= ?x37 3)))
-(let (($x46 (< (+ x$ ?x37) (+ 3 x$))))
-(let (($x49 (not $x46)))
-(let ((@x58 (monotonicity (rewrite (= $x46 (not $x56))) (= $x49 (not (not $x56))))))
-(let ((@x67 (trans (trans @x58 (rewrite (= (not (not $x56)) $x56)) (= $x49 $x56)) (rewrite (= $x56 $x63)) (= $x49 $x63))))
-(let ((@x42 (monotonicity (rewrite (= (+ ?x29 ?x29) ?x37)) (= (+ x$ (+ ?x29 ?x29)) (+ x$ ?x37)))))
-(let ((@x48 (monotonicity @x42 (rewrite (= (+ x$ 3) (+ 3 x$))) (= (< (+ x$ (+ ?x29 ?x29)) (+ x$ 3)) $x46))))
-(let ((@x51 (monotonicity @x48 (= (not (< (+ x$ (+ ?x29 ?x29)) (+ x$ 3))) $x49))))
-(let ((@x69 (trans @x51 @x67 (= (not (< (+ x$ (+ ?x29 ?x29)) (+ x$ 3))) $x63))))
-(let ((@x70 (mp (asserted (not (< (+ x$ (+ ?x29 ?x29)) (+ x$ 3)))) @x69 $x63)))
-((_ th-lemma arith farkas -1 1 1) @x70 @x336 (unit-resolution ((_ th-lemma arith) (or false $x319)) (true-axiom true) $x319) false)))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))
+(let ((?x30 (* 2.0 x$)))
+(let ((?x32 (+ ?x30 1.0)))
+(let ((?x28 (+ x$ x$)))
+(let (($x33 (< ?x28 ?x32)))
+(let (($x34 (or false $x33)))
+(let (($x35 (or $x33 $x34)))
+(let (($x36 (not $x35)))
+(let ((@x67 (monotonicity (rewrite (= (< ?x30 (+ 1.0 ?x30)) true)) (= (not (< ?x30 (+ 1.0 ?x30))) (not true)))))
+(let ((@x71 (trans @x67 (rewrite (= (not true) false)) (= (not (< ?x30 (+ 1.0 ?x30))) false))))
+(let ((?x40 (+ 1.0 ?x30)))
+(let (($x43 (< ?x30 ?x40)))
+(let ((@x45 (monotonicity (rewrite (= ?x28 ?x30)) (rewrite (= ?x32 ?x40)) (= $x33 $x43))))
+(let ((@x52 (trans (monotonicity @x45 (= $x34 (or false $x43))) (rewrite (= (or false $x43) $x43)) (= $x34 $x43))))
+(let ((@x59 (trans (monotonicity @x45 @x52 (= $x35 (or $x43 $x43))) (rewrite (= (or $x43 $x43) $x43)) (= $x35 $x43))))
+(let ((@x62 (monotonicity @x59 (= $x36 (not $x43)))))
+(mp (asserted $x36) (trans @x62 @x71 (= $x36 false)) false))))))))))))))))))
 
-79755c254382365be942468233fcaccea51e52f9 113 0
+3b9ce43e2740f87b7b76af427475ff5d8f44cbe5 113 0
 unsat
 ((set-logic <null>)
 (proof
@@ -2572,7 +2459,120 @@
 (let ((@x74 (mp (asserted $x36) @x73 $x67)))
 ((_ th-lemma arith farkas -1 1 1) @x74 (unit-resolution ((_ th-lemma arith) (or false $x305)) (true-axiom true) $x305) @x337 false))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))
 
-fddd35182d98a66f939d6ead708e259190268f17 32 0
+65dbdf3c35230cd95a2270964f818bd947c20f0c 112 0
+unsat
+((set-logic <null>)
+(proof
+(let ((?x224 (mod x$ 2)))
+(let (($x318 (>= ?x224 2)))
+(let (($x319 (not $x318)))
+(let ((?x258 (* (- 1) ?x224)))
+(let ((?x29 (mod$ x$ 2)))
+(let ((?x259 (+ ?x29 ?x258)))
+(let (($x275 (<= ?x259 0)))
+(let (($x260 (= ?x259 0)))
+(let (($x201 (forall ((?v0 Int) (?v1 Int) )(!(let ((?x132 (mod ?v0 ?v1)))
+(let ((?x89 (* (- 1) ?v1)))
+(let ((?x86 (* (- 1) ?v0)))
+(let ((?x140 (mod ?x86 ?x89)))
+(let ((?x146 (* (- 1) ?x140)))
+(let (($x107 (<= ?v1 0)))
+(let ((?x166 (ite $x107 ?x146 ?x132)))
+(let (($x74 (= ?v1 0)))
+(let ((?x171 (ite $x74 ?v0 ?x166)))
+(let ((?x131 (mod$ ?v0 ?v1)))
+(= ?x131 ?x171))))))))))) :pattern ( (mod$ ?v0 ?v1) )))
+))
+(let (($x177 (forall ((?v0 Int) (?v1 Int) )(let ((?x132 (mod ?v0 ?v1)))
+(let ((?x89 (* (- 1) ?v1)))
+(let ((?x86 (* (- 1) ?v0)))
+(let ((?x140 (mod ?x86 ?x89)))
+(let ((?x146 (* (- 1) ?x140)))
+(let (($x107 (<= ?v1 0)))
+(let ((?x166 (ite $x107 ?x146 ?x132)))
+(let (($x74 (= ?v1 0)))
+(let ((?x171 (ite $x74 ?v0 ?x166)))
+(let ((?x131 (mod$ ?v0 ?v1)))
+(= ?x131 ?x171))))))))))))
+))
+(let ((?x132 (mod ?1 ?0)))
+(let ((?x89 (* (- 1) ?0)))
+(let ((?x86 (* (- 1) ?1)))
+(let ((?x140 (mod ?x86 ?x89)))
+(let ((?x146 (* (- 1) ?x140)))
+(let (($x107 (<= ?0 0)))
+(let ((?x166 (ite $x107 ?x146 ?x132)))
+(let (($x74 (= ?0 0)))
+(let ((?x171 (ite $x74 ?1 ?x166)))
+(let ((?x131 (mod$ ?1 ?0)))
+(let (($x174 (= ?x131 ?x171)))
+(let (($x138 (forall ((?v0 Int) (?v1 Int) )(let (($x74 (= ?v1 0)))
+(let ((?x136 (ite $x74 ?v0 (ite (< 0 ?v1) (mod ?v0 ?v1) (- (mod (- ?v0) (- ?v1)))))))
+(let ((?x131 (mod$ ?v0 ?v1)))
+(= ?x131 ?x136)))))
+))
+(let (($x160 (forall ((?v0 Int) (?v1 Int) )(let ((?x89 (* (- 1) ?v1)))
+(let ((?x86 (* (- 1) ?v0)))
+(let ((?x140 (mod ?x86 ?x89)))
+(let ((?x146 (* (- 1) ?x140)))
+(let ((?x132 (mod ?v0 ?v1)))
+(let (($x75 (< 0 ?v1)))
+(let ((?x151 (ite $x75 ?x132 ?x146)))
+(let (($x74 (= ?v1 0)))
+(let ((?x154 (ite $x74 ?v0 ?x151)))
+(let ((?x131 (mod$ ?v0 ?v1)))
+(= ?x131 ?x154))))))))))))
+))
+(let ((@x165 (monotonicity (rewrite (= (< 0 ?0) (not $x107))) (= (ite (< 0 ?0) ?x132 ?x146) (ite (not $x107) ?x132 ?x146)))))
+(let ((@x170 (trans @x165 (rewrite (= (ite (not $x107) ?x132 ?x146) ?x166)) (= (ite (< 0 ?0) ?x132 ?x146) ?x166))))
+(let ((@x173 (monotonicity @x170 (= (ite $x74 ?1 (ite (< 0 ?0) ?x132 ?x146)) ?x171))))
+(let ((@x176 (monotonicity @x173 (= (= ?x131 (ite $x74 ?1 (ite (< 0 ?0) ?x132 ?x146))) $x174))))
+(let (($x75 (< 0 ?0)))
+(let ((?x151 (ite $x75 ?x132 ?x146)))
+(let ((?x154 (ite $x74 ?1 ?x151)))
+(let (($x157 (= ?x131 ?x154)))
+(let (($x158 (= (= ?x131 (ite $x74 ?1 (ite $x75 ?x132 (- (mod (- ?1) (- ?0)))))) $x157)))
+(let ((@x142 (monotonicity (rewrite (= (- ?1) ?x86)) (rewrite (= (- ?0) ?x89)) (= (mod (- ?1) (- ?0)) ?x140))))
+(let ((@x150 (trans (monotonicity @x142 (= (- (mod (- ?1) (- ?0))) (- ?x140))) (rewrite (= (- ?x140) ?x146)) (= (- (mod (- ?1) (- ?0))) ?x146))))
+(let ((@x153 (monotonicity @x150 (= (ite $x75 ?x132 (- (mod (- ?1) (- ?0)))) ?x151))))
+(let ((@x156 (monotonicity @x153 (= (ite $x74 ?1 (ite $x75 ?x132 (- (mod (- ?1) (- ?0))))) ?x154))))
+(let ((@x181 (trans (quant-intro (monotonicity @x156 $x158) (= $x138 $x160)) (quant-intro @x176 (= $x160 $x177)) (= $x138 $x177))))
+(let ((@x192 (mp~ (mp (asserted $x138) @x181 $x177) (nnf-pos (refl (~ $x174 $x174)) (~ $x177 $x177)) $x177)))
+(let ((@x206 (mp @x192 (quant-intro (refl (= $x174 $x174)) (= $x177 $x201)) $x201)))
+(let (($x266 (or (not $x201) $x260)))
+(let ((?x221 (* (- 1) 2)))
+(let ((?x220 (* (- 1) x$)))
+(let ((?x222 (mod ?x220 ?x221)))
+(let ((?x223 (* (- 1) ?x222)))
+(let (($x219 (<= 2 0)))
+(let ((?x225 (ite $x219 ?x223 ?x224)))
+(let (($x218 (= 2 0)))
+(let ((?x226 (ite $x218 x$ ?x225)))
+(let (($x227 (= ?x29 ?x226)))
+(let ((@x240 (monotonicity (monotonicity (rewrite (= ?x221 (- 2))) (= ?x222 (mod ?x220 (- 2)))) (= ?x223 (* (- 1) (mod ?x220 (- 2)))))))
+(let ((@x243 (monotonicity (rewrite (= $x219 false)) @x240 (= ?x225 (ite false (* (- 1) (mod ?x220 (- 2))) ?x224)))))
+(let ((@x247 (trans @x243 (rewrite (= (ite false (* (- 1) (mod ?x220 (- 2))) ?x224) ?x224)) (= ?x225 ?x224))))
+(let ((@x250 (monotonicity (rewrite (= $x218 false)) @x247 (= ?x226 (ite false x$ ?x224)))))
+(let ((@x257 (monotonicity (trans @x250 (rewrite (= (ite false x$ ?x224) ?x224)) (= ?x226 ?x224)) (= $x227 (= ?x29 ?x224)))))
+(let ((@x270 (monotonicity (trans @x257 (rewrite (= (= ?x29 ?x224) $x260)) (= $x227 $x260)) (= (or (not $x201) $x227) $x266))))
+(let ((@x273 (trans @x270 (rewrite (= $x266 $x266)) (= (or (not $x201) $x227) $x266))))
+(let ((@x274 (mp ((_ quant-inst x$ 2) (or (not $x201) $x227)) @x273 $x266)))
+(let ((@x336 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x260) $x275)) (unit-resolution @x274 @x206 $x260) $x275)))
+(let (($x63 (>= ?x29 2)))
+(let ((?x37 (* 2 ?x29)))
+(let (($x56 (>= ?x37 3)))
+(let (($x46 (< (+ x$ ?x37) (+ 3 x$))))
+(let (($x49 (not $x46)))
+(let ((@x58 (monotonicity (rewrite (= $x46 (not $x56))) (= $x49 (not (not $x56))))))
+(let ((@x67 (trans (trans @x58 (rewrite (= (not (not $x56)) $x56)) (= $x49 $x56)) (rewrite (= $x56 $x63)) (= $x49 $x63))))
+(let ((@x42 (monotonicity (rewrite (= (+ ?x29 ?x29) ?x37)) (= (+ x$ (+ ?x29 ?x29)) (+ x$ ?x37)))))
+(let ((@x48 (monotonicity @x42 (rewrite (= (+ x$ 3) (+ 3 x$))) (= (< (+ x$ (+ ?x29 ?x29)) (+ x$ 3)) $x46))))
+(let ((@x51 (monotonicity @x48 (= (not (< (+ x$ (+ ?x29 ?x29)) (+ x$ 3))) $x49))))
+(let ((@x69 (trans @x51 @x67 (= (not (< (+ x$ (+ ?x29 ?x29)) (+ x$ 3))) $x63))))
+(let ((@x70 (mp (asserted (not (< (+ x$ (+ ?x29 ?x29)) (+ x$ 3)))) @x69 $x63)))
+((_ th-lemma arith farkas -1 1 1) @x70 @x336 (unit-resolution ((_ th-lemma arith) (or false $x319)) (true-axiom true) $x319) false)))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))
+
+5821addf2e306ce7cacfa0f38fedab2f627b2a07 32 0
 unsat
 ((set-logic <null>)
 (proof
@@ -2605,7 +2605,7 @@
 (let ((@x117 (unit-resolution ((_ th-lemma arith assign-bounds 1) (or $x102 (not $x100))) (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x95) $x100)) @x98 $x100) $x102)))
 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x28 (not $x101) (not $x102))) @x117 @x110 @x30 false))))))))))))))))))))))))))))))
 
-6137ebc1a4dee6ad5f0013ba64ccdfe87c956a4c 236 0
+ab2477be99ba02ce738f9e8292c948cefb65d1f0 236 0
 unsat
 ((set-logic <null>)
 (proof
@@ -2821,9 +2821,9 @@
 (let (($x404 (>= ?x398 0)))
 (let ((@x552 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x396) $x404)) (unit-resolution ((_ th-lemma arith) (or false $x396)) @x26 $x396) $x404)))
 (let (($x380 (>= ?x364 0)))
-(let ((@x274 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x365) $x380)) (unit-resolution @x378 @x196 $x365) $x380)))
+(let ((@x273 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x365) $x380)) (unit-resolution @x378 @x196 $x365) $x380)))
 (let (($x436 (>= ?x35 3)))
-(let ((@x545 ((_ th-lemma arith farkas -1/2 -1/2 -1/2 -1/2 -1/2 -1/2 -1/2 -1/2 1) (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x37) $x436)) @x38 $x436) @x274 @x552 @x549 @x537 @x531 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x32) $x434)) @x33 $x434) @x566 @x565 false)))
+(let ((@x545 ((_ th-lemma arith farkas -1/2 -1/2 -1/2 -1/2 -1/2 -1/2 -1/2 -1/2 1) (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x37) $x436)) @x38 $x436) @x273 @x552 @x549 @x537 @x531 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x32) $x434)) @x33 $x434) @x566 @x565 false)))
 (let (($x171 (or $x169 (not $x43))))
 (let ((@x177 (monotonicity (rewrite (= (and $x41 $x43) (not $x171))) (= (not (and $x41 $x43)) (not (not $x171))))))
 (let ((@x181 (trans @x177 (rewrite (= (not (not $x171)) $x171)) (= (not (and $x41 $x43)) $x171))))
@@ -2840,9 +2840,22 @@
 (let (($x427 (>= ?x421 0)))
 (let ((@x584 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x419) $x427)) (unit-resolution ((_ th-lemma arith) (or false $x419)) @x26 $x419) $x427)))
 (let (($x542 (>= ?x519 0)))
-((_ th-lemma arith farkas -1/2 -1/2 -1/2 -1/2 -1/2 1) (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x37) $x436)) @x38 $x436) @x552 (unit-resolution ((_ th-lemma arith) (or false $x542)) @x26 $x542) @x584 @x274 (lemma @x742 (not $x706)) false)))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))
+((_ th-lemma arith farkas -1/2 -1/2 -1/2 -1/2 -1/2 1) (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x37) $x436)) @x38 $x436) @x552 (unit-resolution ((_ th-lemma arith) (or false $x542)) @x26 $x542) @x584 @x273 (lemma @x742 (not $x706)) false)))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))
 
-53b87189d4fa854317dcd8674e77536e36b623a9 12 0
+a9300dbe9262a69a3cfdc9c56fd42d7c0342cf18 12 0
+unsat
+((set-logic AUFLIA)
+(proof
+(let (($x28 (exists ((?v0 Int) )false)
+))
+(let (($x27 (not $x28)))
+(let (($x29 (not $x27)))
+(let ((@x35 (monotonicity (elim-unused (= $x28 false)) (= $x27 (not false)))))
+(let ((@x42 (monotonicity (trans @x35 (rewrite (= (not false) true)) (= $x27 true)) (= $x29 (not true)))))
+(let ((@x46 (trans @x42 (rewrite (= (not true) false)) (= $x29 false))))
+(mp (asserted $x29) @x46 false)))))))))
+
+89d6b345b16adb1e835f69f2b12bdfbb65f85d6f 12 0
 unsat
 ((set-logic AUFLIRA)
 (proof
@@ -2855,20 +2868,7 @@
 (let ((@x46 (trans @x42 (rewrite (= (not true) false)) (= $x29 false))))
 (mp (asserted $x29) @x46 false)))))))))
 
-c290998049722e9064991552da49de93b1870890 12 0
-unsat
-((set-logic AUFLIA)
-(proof
-(let (($x28 (exists ((?v0 Int) )false)
-))
-(let (($x27 (not $x28)))
-(let (($x29 (not $x27)))
-(let ((@x35 (monotonicity (elim-unused (= $x28 false)) (= $x27 (not false)))))
-(let ((@x42 (monotonicity (trans @x35 (rewrite (= (not false) true)) (= $x27 true)) (= $x29 (not true)))))
-(let ((@x46 (trans @x42 (rewrite (= (not true) false)) (= $x29 false))))
-(mp (asserted $x29) @x46 false)))))))))
-
-006eb5bfd7c221833bed8cb6329632aaa194fbfb 22 0
+c0b457d231443ee740b4ce5f216d64438244549d 22 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -2891,7 +2891,7 @@
 (let ((@x49 (mp~ (mp (asserted $x30) (monotonicity @x40 (= $x30 $x41)) $x41) @x48 $x46)))
 (mp (mp @x49 @x54 $x52) (rewrite (= $x52 false)) false)))))))))))))
 
-4b537bd0ac915a6248e7ab628729c96862196610 22 0
+f5a6840d663a7151c77679eb31df85fbe38d8fde 22 0
 unsat
 ((set-logic AUFLIRA)
 (proof
@@ -2914,7 +2914,7 @@
 (let ((@x48 (mp~ (mp (asserted $x29) (monotonicity @x39 (= $x29 $x40)) $x40) @x47 $x45)))
 (mp (mp @x48 @x53 $x51) (rewrite (= $x51 false)) false)))))))))))))
 
-a4d78976c78e2e93de6480dddf342fdcc4b645d0 31 0
+1697215d42414548a1a7c4f39d164dce39494e28 31 0
 unsat
 ((set-logic AUFLIA)
 (declare-fun ?v0!0 () Int)
@@ -2946,7 +2946,7 @@
 (let ((@x74 (mp (mp~ (mp (asserted $x32) @x51 $x49) @x67 $x63) (quant-intro (rewrite (= $x60 $x54)) (= $x63 $x71)) $x71)))
 (mp @x74 (rewrite (= $x71 false)) false))))))))))))))))))
 
-0599cab93c20e7ec32e4ccd96b617b98c9583ac6 22 0
+89a6480b8f6ca7084b8763d66b725709c1e2b14b 22 0
 unsat
 ((set-logic AUFLIA)
 (declare-fun ?v1!0 () Int)
@@ -2969,7 +2969,7 @@
 (let ((@x70 (trans (symm (and-elim @x65 (= ?v0!1 0)) (= 0 ?v0!1)) @x68 (= 0 ?v1!0))))
 (mp (trans @x70 @x67 (= 0 1)) (rewrite (= (= 0 1) false)) false))))))))))))))))
 
-d8593d44297c3187a702aba2fd49f4ad76117020 55 0
+0b631409631fd9a48d7e052718176c2734d9970a 55 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -3025,7 +3025,7 @@
 (let ((@x50 (monotonicity @x47 (= $x36 $x48))))
 (mp (asserted $x36) (trans @x50 @x101 (= $x36 false)) false)))))))))))))))))))))))))))
 
-75068fac55f5cd4cceebee82c7f07a7dd4bf9104 42 0
+a02fbab78826794399de97e7fb644c926c1c3876 42 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -3068,7 +3068,7 @@
 (let ((@x60 (monotonicity (quant-intro @x54 (= $x37 $x55)) (= $x38 $x58))))
 (mp (asserted $x38) (trans @x60 @x97 (= $x38 false)) false))))))))))))))))))))))))))
 
-a2f9a6aa539c30e09dd3b64e591e790324d7c645 32 0
+bac06e4ce21a6a92b3a2ccdc8f904797ab357514 32 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -3101,7 +3101,7 @@
 (let ((@x53 (monotonicity @x50 (= $x37 $x51))))
 (mp (asserted $x37) (trans @x53 @x76 (= $x37 false)) false)))))))))))))))))))
 
-94385afe5a4674c0cf5e8e53c895cbd5392d7e69 43 0
+ae1c03bd9e800e427a6747d8b2266cc9c537b295 43 0
 unsat
 ((set-logic AUFLIA)
 (declare-fun ?v0!1 () Int)
@@ -3145,7 +3145,7 @@
 (let ((@x103 (not-or-elim @x102 $x81)))
 (unit-resolution (unit-resolution ((_ th-lemma arith triangle-eq) (or $x87 $x84 $x93)) @x103 (or $x87 $x93)) @x106 @x105 false)))))))))))))))))))))))))))))))))
 
-e71a92d0ec57041b4a90cd14085e39ffbc344b71 46 0
+db63155888d6756cde4a625ef2b3d96c4b5dda9e 46 0
 unsat
 ((set-logic AUFLIA)
 (declare-fun ?v0!0 () Int)
@@ -3192,7 +3192,7 @@
 (let ((@x114 (unit-resolution (def-axiom (or $x88 (not $x83) $x84)) @x92 (or (not $x83) $x84))))
 (unit-resolution @x114 (unit-resolution ((_ th-lemma arith farkas 1 1) (or $x85 (not $x83))) @x109 $x85) @x109 false)))))))))))))))))))))))))))))))))
 
-cec63c4e61277cab3f34c858a58786d0b6b7272b 31 0
+a8dac4a7ecab6f2724d194d43b8ea416f1162aeb 31 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -3224,47 +3224,7 @@
 (let ((@x66 (mp~ (mp (asserted $x33) @x60 $x56) (nnf-pos (refl (~ $x53 $x53)) (~ $x56 $x56)) $x56)))
 (unit-resolution @x66 @x464 false)))))))))))))))))))))))))
 
-3ad025eb052c9510c89e0ee0394bb351383dc7cd 39 0
-unsat
-((set-logic AUFLIA)
-(proof
-(let (($x38 (exists ((?v0 Int) (?v1 Int) (?v2 Int) )(let ((?x33 (- 6)))
-(let ((?x34 (* ?x33 ?v1)))
-(let ((?x31 (* 4 ?v0)))
-(let ((?x35 (+ ?x31 ?x34)))
-(= ?x35 1))))))
-))
-(let (($x29 (not $x38)))
-(let (($x39 (not $x29)))
-(let (($x61 (exists ((?v0 Int) (?v1 Int) )(let ((?x58 (* (- 6) ?v1)))
-(let ((?x57 (* 4 ?v0)))
-(let ((?x59 (+ ?x57 ?x58)))
-(= ?x59 1)))))
-))
-(let (($x77 (exists ((?v0 Int) (?v1 Int) )false)
-))
-(let ((@x81 (quant-intro (rewrite (= (= (+ (* 4 ?1) (* (- 6) ?0)) 1) false)) (= $x61 $x77))))
-(let ((@x85 (trans @x81 (elim-unused (= $x77 false)) (= $x61 false))))
-(let (($x53 (exists ((?v0 Int) (?v1 Int) (?v2 Int) )(let ((?x44 (* (- 6) ?v1)))
-(let ((?x31 (* 4 ?v0)))
-(let ((?x47 (+ ?x31 ?x44)))
-(= ?x47 1)))))
-))
-(let ((?x44 (* (- 6) ?1)))
-(let ((?x31 (* 4 ?2)))
-(let ((?x47 (+ ?x31 ?x44)))
-(let (($x50 (= ?x47 1)))
-(let ((?x33 (- 6)))
-(let ((?x34 (* ?x33 ?1)))
-(let ((?x35 (+ ?x31 ?x34)))
-(let (($x37 (= ?x35 1)))
-(let ((@x49 (monotonicity (monotonicity (rewrite (= ?x33 (- 6))) (= ?x34 ?x44)) (= ?x35 ?x47))))
-(let ((@x65 (trans (quant-intro (monotonicity @x49 (= $x37 $x50)) (= $x38 $x53)) (elim-unused (= $x53 $x61)) (= $x38 $x61))))
-(let ((@x71 (monotonicity (monotonicity @x65 (= $x29 (not $x61))) (= $x39 (not (not $x61))))))
-(let ((@x75 (trans @x71 (rewrite (= (not (not $x61)) $x61)) (= $x39 $x61))))
-(mp (asserted $x39) (trans @x75 @x85 (= $x39 false)) false)))))))))))))))))))))))
-
-742605321b1c1bf714414e704f5fbaa4881d29be 62 0
+e2aa0dee3f7e85b2864ff5156cfcfdfb81794763 62 0
 unsat
 ((set-logic AUFLIA)
 (declare-fun ?v0!1 () Int)
@@ -3327,7 +3287,47 @@
 (let ((@x515 (unit-resolution (def-axiom (or z3name!0 $x220)) (unit-resolution @x131 @x238 $x88) $x220)))
 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x220) (>= ?x96 3))) @x515 @x245 false))))))))))))))))))))))))))))))))))))))))))))))))))))))
 
-b419771c87952c92c2e97909ff791914992c4c92 52 0
+b8b49f331abce2ef652c812e5388c9b1eb2103d4 39 0
+unsat
+((set-logic AUFLIA)
+(proof
+(let (($x38 (exists ((?v0 Int) (?v1 Int) (?v2 Int) )(let ((?x33 (- 6)))
+(let ((?x34 (* ?x33 ?v1)))
+(let ((?x31 (* 4 ?v0)))
+(let ((?x35 (+ ?x31 ?x34)))
+(= ?x35 1))))))
+))
+(let (($x29 (not $x38)))
+(let (($x39 (not $x29)))
+(let (($x61 (exists ((?v0 Int) (?v1 Int) )(let ((?x58 (* (- 6) ?v1)))
+(let ((?x57 (* 4 ?v0)))
+(let ((?x59 (+ ?x57 ?x58)))
+(= ?x59 1)))))
+))
+(let (($x77 (exists ((?v0 Int) (?v1 Int) )false)
+))
+(let ((@x81 (quant-intro (rewrite (= (= (+ (* 4 ?1) (* (- 6) ?0)) 1) false)) (= $x61 $x77))))
+(let ((@x85 (trans @x81 (elim-unused (= $x77 false)) (= $x61 false))))
+(let (($x53 (exists ((?v0 Int) (?v1 Int) (?v2 Int) )(let ((?x44 (* (- 6) ?v1)))
+(let ((?x31 (* 4 ?v0)))
+(let ((?x47 (+ ?x31 ?x44)))
+(= ?x47 1)))))
+))
+(let ((?x44 (* (- 6) ?1)))
+(let ((?x31 (* 4 ?2)))
+(let ((?x47 (+ ?x31 ?x44)))
+(let (($x50 (= ?x47 1)))
+(let ((?x33 (- 6)))
+(let ((?x34 (* ?x33 ?1)))
+(let ((?x35 (+ ?x31 ?x34)))
+(let (($x37 (= ?x35 1)))
+(let ((@x49 (monotonicity (monotonicity (rewrite (= ?x33 (- 6))) (= ?x34 ?x44)) (= ?x35 ?x47))))
+(let ((@x65 (trans (quant-intro (monotonicity @x49 (= $x37 $x50)) (= $x38 $x53)) (elim-unused (= $x53 $x61)) (= $x38 $x61))))
+(let ((@x71 (monotonicity (monotonicity @x65 (= $x29 (not $x61))) (= $x39 (not (not $x61))))))
+(let ((@x75 (trans @x71 (rewrite (= (not (not $x61)) $x61)) (= $x39 $x61))))
+(mp (asserted $x39) (trans @x75 @x85 (= $x39 false)) false)))))))))))))))))))))))
+
+eb19c818b6d733ebf111be3722a0ce2595e03179 52 0
 unsat
 ((set-logic AUFLIA)
 (declare-fun ?v1!1 () Int)
@@ -3380,7 +3380,7 @@
 (let ((@x117 (and-elim (not-or-elim @x112 (and $x100 $x102)) $x102)))
 ((_ th-lemma arith farkas 1 1 1) @x117 @x116 @x118 false)))))))))))))))))))))))))))))))))))
 
-aca1057d33e2c20ed6a4e7340ea11d94647e9dc8 46 0
+094447109c844652a6f546ce3ffd0f6694fd8927 46 0
 unsat
 ((set-logic AUFLIRA)
 (declare-fun ?v1!1 () Int)
@@ -3427,7 +3427,7 @@
 (let ((@x115 (and-elim (not-or-elim @x111 (and $x100 (not (<= ?v2!0 0.0)))) $x100)))
 (unit-resolution (unit-resolution ((_ th-lemma arith farkas 1 1) (or $x106 $x99)) @x115 $x106) @x117 false)))))))))))))))))))))))))))))))
 
-271acbb7e8a77900a25a72e272c627346e8e5aad 110 0
+276d0c1b7b2ca7d8710b2346fa41fe39d8e39aa4 110 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -3538,7 +3538,7 @@
 (let ((@x125 (mp (mp @x110 (quant-intro @x115 (= $x107 $x116)) $x116) (quant-intro (rewrite (= $x113 $x104)) (= $x116 $x122)) $x122)))
 (mp (mp @x125 @x156 $x152) @x180 false))))))))))))))))))))))))))))))))))))))))))))))
 
-d435f7f9afa42bb528c08b9973fb84251457cc61 36 0
+4548ba5cb4f4d4ca35cf5ce5a77f8d0693dbfe20 36 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -3575,7 +3575,7 @@
 (let ((@x47 (monotonicity (quant-intro (rewrite (= (=> $x29 $x33) $x39)) (= $x35 $x42)) (= $x36 $x45))))
 (mp (asserted $x36) (trans @x47 @x84 (= $x36 false)) false))))))))))))))))))))))
 
-6da91cb6f227cacea1dfaf3034cb4a390ac0baa5 24 0
+a5a9936b807e06c40471a61664d8a592934c9cca 24 0
 unsat
 ((set-logic AUFLIA)
 (declare-fun ?v1!0 () Int)
@@ -3600,7 +3600,7 @@
 (let ((@x73 (not-or-elim @x70 $x62)))
 (unit-resolution (unit-resolution ((_ th-lemma arith farkas 1 1) (or $x65 (not $x62))) @x73 $x65) @x74 false))))))))))))))))))
 
-fe3b63dadb4f4e5b321fc5b7c5f730628f383434 26 0
+91259a177773bafc6d480a897160dabc2e374303 26 0
 unsat
 ((set-logic <null>)
 (proof
@@ -3627,7 +3627,7 @@
 (let ((@x73 (and-elim (not-or-elim (mp (asserted $x35) @x69 $x65) $x52) $x49)))
 ((_ th-lemma arith farkas 1 1 1) @x73 @x72 @x74 false))))))))))))))))))))))))
 
-24c8f0dd4aa6c97766e14b2f7117e047e77febf6 26 0
+4cf7e84f6612e6723de979a5590429ed0bdc2149 26 0
 unsat
 ((set-logic <null>)
 (proof
@@ -3654,7 +3654,7 @@
 (let ((@x92 (trans @x88 (rewrite (= (not true) false)) (= $x39 false))))
 (mp (asserted $x39) @x92 false))))))))))))))))))))))))
 
-e22e8faf67fe7e4aace8b3f6a8b1454fcc24ea86 23 0
+ef2a46fc25a1446e4cb5ba92171b8904421d3d93 23 0
 unsat
 ((set-logic <null>)
 (proof
@@ -3678,7 +3678,7 @@
 (let ((@x82 (trans (monotonicity @x75 (= $x39 (not true))) (rewrite (= (not true) false)) (= $x39 false))))
 (mp (asserted $x39) @x82 false)))))))))))))))))))))
 
-c0e8a04cf61a70a02319dafd0746e974e08efce6 51 0
+27ccfe7c1b0e81ae67ba7604acc7a5a88ebafbcc 51 0
 unsat
 ((set-logic <null>)
 (proof
@@ -3730,7 +3730,7 @@
 (let ((@x152 (trans (monotonicity @x145 (= $x52 (not true))) (rewrite (= (not true) false)) (= $x52 false))))
 (mp (asserted $x52) @x152 false)))))))))))))))))))))))))))))))))))))))))))))))))
 
-cbab19031067d3b53edcf7fe0ab1b4b285157eaf 126 0
+2084de0906ecde328438829773f63c6ae64addcf 126 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -3857,7 +3857,7 @@
 (let (($x486 (<= ?x212 1)))
 ((_ th-lemma arith gcd-test -1/2 -1/2 -1/2 -1/2) (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x485) $x487)) @x356 $x487) (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x485) $x486)) @x356 $x486) (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x531) $x514)) @x470 $x514) (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x531) $x513)) @x470 $x513) false))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))
 
-a26825fade3f4c15b8fd2d7864ae3dcd4a826d6d 22 0
+ebb67e656a1cacdf82196bc885af68a17da94cdf 22 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -3880,7 +3880,7 @@
 (let ((@x70 (not-or-elim (mp (asserted (not (=> $x30 $x34))) @x68 $x64) $x45)))
 (unit-resolution (unit-resolution ((_ th-lemma arith farkas 1 1) (or $x58 $x47)) @x70 $x58) @x71 false))))))))))))))))))))
 
-0e96d2bcbd5540b8d6a69936d530d9d9ced1c4be 147 0
+c28551c93998b294bbaffa72349cb5e28c52bc85 147 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -4028,7 +4028,7 @@
 (let ((@x72 (mp (asserted $x38) (trans (monotonicity @x55 (= $x38 $x56)) @x69 (= $x38 $x59)) $x59)))
 ((_ th-lemma arith farkas -1 -1 1) @x72 @x453 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x532) $x513)) @x459 $x513) false)))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))
 
-0ca03284fa57fab888696978d182e9520b70a64b 145 0
+d9bfa018c73582b83eab8ae6958210b79fde3ced 145 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -4174,7 +4174,7 @@
 (let ((@x538 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x612) $x595)) (unit-resolution (unit-resolution @x594 @x631 $x616) @x545 $x612) $x595)))
 ((_ th-lemma arith farkas 1 -1 -1 1) (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x559) $x557)) @x539 $x557) @x106 @x538 @x457 false)))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))
 
-ed992e8735f6c9b531d67fd3885b90b06272f149 78 0
+7206a08fff0e511601448c72b67eb8b3b6aa2599 78 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -4253,7 +4253,7 @@
 (let ((@x257 (unit-resolution ((_ th-lemma arith farkas 1 1) (or $x578 $x254)) (unit-resolution @x576 @x81 @x593 $x255) $x578)))
 ((_ th-lemma arith farkas 1 1 1) @x257 @x198 @x566 false)))))))))))))))))))))))))))))))))))))))))))))))))))))))
 
-859305ec6d928beaf23fc5a8882356fcb3b97d7d 312 0
+aa1937ae6bc1e22ce854bc70cf99a1e60ddb4dc9 312 0
 unsat
 ((set-logic AUFLIA)
 (declare-fun ?v1!0 (Nat$) Nat$)
@@ -4301,11 +4301,11 @@
 (let (($x342 (or $x369 $x700)))
 (let (($x684 (not $x342)))
 (let (($x738 (forall ((?v0 Nat$) )(!(let (($x219 (or (not (dvd$ (?v1!0 ?v0) ?v0)) (= (?v1!0 ?v0) (nat$ 1)) (= (?v1!0 ?v0) ?v0))))
-(let (($x221 (not $x219)))
+(let (($x220 (not $x219)))
 (let ((?x30 (of_nat$ ?v0)))
 (let (($x65 (<= ?x30 1)))
 (let (($x28 (prime_nat$ ?v0)))
-(let (($x245 (or $x28 $x65 $x221)))
+(let (($x245 (or $x28 $x65 $x220)))
 (let (($x710 (forall ((?v1 Nat$) )(!(let ((?x34 (nat$ 1)))
 (let (($x35 (= ?v1 ?x34)))
 (or (not (dvd$ ?v1 ?v0)) $x35 (= ?v1 ?v0)))) :pattern ( (dvd$ ?v1 ?v0) )))
@@ -4314,27 +4314,27 @@
 (not (or (not (or $x200 (not (or $x65 (not $x710))))) (not $x245))))))))))) :pattern ( (prime_nat$ ?v0) ) :pattern ( (of_nat$ ?v0) )))
 ))
 (let (($x290 (forall ((?v0 Nat$) )(let (($x219 (or (not (dvd$ (?v1!0 ?v0) ?v0)) (= (?v1!0 ?v0) (nat$ 1)) (= (?v1!0 ?v0) ?v0))))
-(let (($x221 (not $x219)))
+(let (($x220 (not $x219)))
 (let ((?x30 (of_nat$ ?v0)))
 (let (($x65 (<= ?x30 1)))
 (let (($x28 (prime_nat$ ?v0)))
-(let (($x245 (or $x28 $x65 $x221)))
+(let (($x245 (or $x28 $x65 $x220)))
 (let (($x72 (forall ((?v1 Nat$) )(let ((?x34 (nat$ 1)))
 (let (($x35 (= ?v1 ?x34)))
 (or (not (dvd$ ?v1 ?v0)) $x35 (= ?v1 ?v0)))))
 ))
-(let (($x220 (not $x72)))
-(let (($x273 (not (or $x65 $x220))))
+(let (($x221 (not $x72)))
+(let (($x273 (not (or $x65 $x221))))
 (let (($x200 (not $x28)))
 (let (($x276 (or $x200 $x273)))
 (not (or (not $x276) (not $x245)))))))))))))))
 ))
 (let (($x219 (or (not (dvd$ (?v1!0 ?0) ?0)) (= (?v1!0 ?0) ?x34) (= (?v1!0 ?0) ?0))))
-(let (($x221 (not $x219)))
+(let (($x220 (not $x219)))
 (let ((?x30 (of_nat$ ?0)))
 (let (($x65 (<= ?x30 1)))
 (let (($x28 (prime_nat$ ?0)))
-(let (($x245 (or $x28 $x65 $x221)))
+(let (($x245 (or $x28 $x65 $x220)))
 (let (($x710 (forall ((?v1 Nat$) )(!(let ((?x34 (nat$ 1)))
 (let (($x35 (= ?v1 ?x34)))
 (or (not (dvd$ ?v1 ?0)) $x35 (= ?v1 ?0)))) :pattern ( (dvd$ ?v1 ?0) )))
@@ -4344,24 +4344,24 @@
 (let (($x35 (= ?v1 ?x34)))
 (or (not (dvd$ ?v1 ?0)) $x35 (= ?v1 ?0)))))
 ))
-(let (($x220 (not $x72)))
-(let (($x273 (not (or $x65 $x220))))
+(let (($x221 (not $x72)))
+(let (($x273 (not (or $x65 $x221))))
 (let (($x276 (or $x200 $x273)))
 (let (($x285 (not (or (not $x276) (not $x245)))))
 (let (($x734 (= $x285 (not (or (not (or $x200 (not (or $x65 (not $x710))))) (not $x245))))))
 (let (($x731 (= (or (not $x276) (not $x245)) (or (not (or $x200 (not (or $x65 (not $x710))))) (not $x245)))))
 (let (($x35 (= ?0 ?x34)))
 (let (($x69 (or (not (dvd$ ?0 ?1)) $x35 (= ?0 ?1))))
-(let ((@x717 (monotonicity (quant-intro (refl (= $x69 $x69)) (= $x72 $x710)) (= $x220 (not $x710)))))
-(let ((@x723 (monotonicity (monotonicity @x717 (= (or $x65 $x220) (or $x65 (not $x710)))) (= $x273 (not (or $x65 (not $x710)))))))
+(let ((@x717 (monotonicity (quant-intro (refl (= $x69 $x69)) (= $x72 $x710)) (= $x221 (not $x710)))))
+(let ((@x723 (monotonicity (monotonicity @x717 (= (or $x65 $x221) (or $x65 (not $x710)))) (= $x273 (not (or $x65 (not $x710)))))))
 (let ((@x729 (monotonicity (monotonicity @x723 (= $x276 (or $x200 (not (or $x65 (not $x710)))))) (= (not $x276) (not (or $x200 (not (or $x65 (not $x710)))))))))
 (let ((@x740 (quant-intro (monotonicity (monotonicity @x729 $x731) $x734) (= $x290 $x738))))
 (let (($x253 (forall ((?v0 Nat$) )(let (($x219 (or (not (dvd$ (?v1!0 ?v0) ?v0)) (= (?v1!0 ?v0) (nat$ 1)) (= (?v1!0 ?v0) ?v0))))
-(let (($x221 (not $x219)))
+(let (($x220 (not $x219)))
 (let ((?x30 (of_nat$ ?v0)))
 (let (($x65 (<= ?x30 1)))
 (let (($x28 (prime_nat$ ?v0)))
-(let (($x245 (or $x28 $x65 $x221)))
+(let (($x245 (or $x28 $x65 $x220)))
 (let (($x72 (forall ((?v1 Nat$) )(let ((?x34 (nat$ 1)))
 (let (($x35 (= ?v1 ?x34)))
 (or (not (dvd$ ?v1 ?v0)) $x35 (= ?v1 ?v0)))))
@@ -4369,40 +4369,40 @@
 (let (($x66 (not $x65)))
 (let (($x75 (and $x66 $x72)))
 (let (($x200 (not $x28)))
-(let (($x228 (or $x200 $x75)))
-(and $x228 $x245)))))))))))))
+(let (($x229 (or $x200 $x75)))
+(and $x229 $x245)))))))))))))
 ))
 (let ((@x278 (monotonicity (rewrite (= (and (not $x65) $x72) $x273)) (= (or $x200 (and (not $x65) $x72)) $x276))))
 (let ((@x281 (monotonicity @x278 (= (and (or $x200 (and (not $x65) $x72)) $x245) (and $x276 $x245)))))
 (let ((@x289 (trans @x281 (rewrite (= (and $x276 $x245) $x285)) (= (and (or $x200 (and (not $x65) $x72)) $x245) $x285))))
 (let (($x233 (forall ((?v0 Nat$) )(let (($x219 (or (not (dvd$ (?v1!0 ?v0) ?v0)) (= (?v1!0 ?v0) (nat$ 1)) (= (?v1!0 ?v0) ?v0))))
-(let (($x221 (not $x219)))
+(let (($x220 (not $x219)))
 (let ((?x30 (of_nat$ ?v0)))
 (let (($x65 (<= ?x30 1)))
 (let (($x66 (not $x65)))
 (let (($x211 (not $x66)))
-(let (($x224 (or $x211 $x221)))
+(let (($x224 (or $x211 $x220)))
 (let (($x28 (prime_nat$ ?v0)))
-(let (($x229 (or $x28 $x224)))
+(let (($x228 (or $x28 $x224)))
 (let (($x72 (forall ((?v1 Nat$) )(let ((?x34 (nat$ 1)))
 (let (($x35 (= ?v1 ?x34)))
 (or (not (dvd$ ?v1 ?v0)) $x35 (= ?v1 ?v0)))))
 ))
 (let (($x75 (and $x66 $x72)))
 (let (($x200 (not $x28)))
-(let (($x228 (or $x200 $x75)))
-(and $x228 $x229)))))))))))))))
+(let (($x229 (or $x200 $x75)))
+(and $x229 $x228)))))))))))))))
 ))
 (let (($x66 (not $x65)))
 (let (($x75 (and $x66 $x72)))
-(let (($x228 (or $x200 $x75)))
-(let (($x250 (and $x228 $x245)))
+(let (($x229 (or $x200 $x75)))
+(let (($x250 (and $x229 $x245)))
 (let (($x211 (not $x66)))
-(let (($x224 (or $x211 $x221)))
-(let (($x229 (or $x28 $x224)))
-(let (($x230 (and $x228 $x229)))
-(let ((@x244 (monotonicity (monotonicity (rewrite (= $x211 $x65)) (= $x224 (or $x65 $x221))) (= $x229 (or $x28 (or $x65 $x221))))))
-(let ((@x249 (trans @x244 (rewrite (= (or $x28 (or $x65 $x221)) $x245)) (= $x229 $x245))))
+(let (($x224 (or $x211 $x220)))
+(let (($x228 (or $x28 $x224)))
+(let (($x230 (and $x229 $x228)))
+(let ((@x244 (monotonicity (monotonicity (rewrite (= $x211 $x65)) (= $x224 (or $x65 $x220))) (= $x228 (or $x28 (or $x65 $x220))))))
+(let ((@x249 (trans @x244 (rewrite (= (or $x28 (or $x65 $x220)) $x245)) (= $x228 $x245))))
 (let (($x81 (forall ((?v0 Nat$) )(let (($x72 (forall ((?v1 Nat$) )(let ((?x34 (nat$ 1)))
 (let (($x35 (= ?v1 ?x34)))
 (or (not (dvd$ ?v1 ?v0)) $x35 (= ?v1 ?v0)))))
@@ -4414,7 +4414,7 @@
 (let (($x28 (prime_nat$ ?v0)))
 (= $x28 $x75))))))))
 ))
-(let ((@x227 (nnf-neg (refl (~ $x211 $x211)) (sk (~ $x220 $x221)) (~ (not $x75) $x224))))
+(let ((@x227 (nnf-neg (refl (~ $x211 $x211)) (sk (~ $x221 $x220)) (~ (not $x75) $x224))))
 (let ((@x210 (monotonicity (refl (~ $x66 $x66)) (nnf-pos (refl (~ $x69 $x69)) (~ $x72 $x72)) (~ $x75 $x75))))
 (let ((@x232 (nnf-pos (refl (~ $x28 $x28)) (refl (~ $x200 $x200)) @x210 @x227 (~ (= $x28 $x75) $x230))))
 (let (($x42 (forall ((?v0 Nat$) )(let (($x39 (forall ((?v1 Nat$) )(let (($x33 (dvd$ ?v1 ?v0)))
@@ -4566,7 +4566,7 @@
 (let ((@x133 (not-or-elim (mp (asserted $x96) @x129 $x125) (not (>= ?x89 1)))))
 ((_ th-lemma arith farkas -4 1 1) @x133 (unit-resolution (def-axiom (or $x357 $x687)) @x572 $x687) (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x597) $x574)) @x532 $x574) false)))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))
 
-632a5cc60479c47e39f08b133241258ad5a60c0d 23 0
+fa52995d8e0d975d4935c3463171969be61873a0 23 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -4590,7 +4590,7 @@
 (let ((@x54 (not-or-elim (mp (asserted (not (=> $x39 $x40))) @x50 (not (or (not $x39) $x40))) (not $x40))))
 (unit-resolution @x54 @x150 false)))))))))))))))))))
 
-ef7d2926debcf081d5863191925f0342f600bafa 42 0
+0717916b99d003f0eebdfca4e5036aea3ba20b2e 42 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -4633,7 +4633,7 @@
 (let ((@x76 (not-or-elim (mp (asserted (not (=> $x57 $x60))) @x70 (not (or (not $x57) $x60))) (not $x60))))
 (unit-resolution @x76 (trans @x489 @x504 $x60) false))))))))))))))))))))))))))))))))))))
 
-a7b6c0ca99c35f7f160cb791dff0471341a655d2 60 0
+218e2ca9c8438c8bc69109bc405a4e8afb307ea3 60 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -4694,7 +4694,7 @@
 (let ((@x86 (not-or-elim (mp (asserted (not (=> $x58 $x70))) @x80 (not (or (not $x58) $x70))) (not $x70))))
 (unit-resolution @x86 @x470 false))))))))))))))))))))))))))))))))))))))))))))))))
 
-398e19463db97884db9b1a6cf323ad9e8d7ed595 24 0
+32036f8366ebb8f5f28e560f469c51fe27adf147 24 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -4719,7 +4719,7 @@
 (let ((@x80 (mp (not-or-elim @x70 (not $x44)) (rewrite (= (not $x44) $x77)) $x77)))
 (mp @x80 @x93 false))))))))))))))))))))))
 
-c7546359abeadcc57d79b687aff33f5d29209729 45 0
+09a1df859386cd5f0beadf3cfac6ffd9d984b2b0 45 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -4765,7 +4765,7 @@
 (let ((@x496 ((_ quant-inst x$) $x163)))
 (unit-resolution @x496 @x508 (unit-resolution @x84 (lemma @x495 $x47) $x73) false)))))))))))))))))))))))))))))))))
 
-0c570d8faa2ef80523f83dbdeb271e428451f2b8 14 0
+c18561c3bde17d16d60757484a2fa97d9fae4e9d 14 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -4780,7 +4780,7 @@
 (let ((@x53 (trans (monotonicity @x46 (= $x33 (not true))) (rewrite (= (not true) false)) (= $x33 false))))
 (mp (asserted $x33) @x53 false)))))))))))
 
-0acbd728d248ce2e753dfea749c0f4b89e597d4d 14 0
+f2a4bc3ff3a59823ea7b57650a442bcda5da2bcf 14 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -4795,7 +4795,7 @@
 (let ((@x53 (trans (monotonicity @x46 (= $x33 (not true))) (rewrite (= (not true) false)) (= $x33 false))))
 (mp (asserted $x33) @x53 false)))))))))))
 
-9adfad76d5881b3c86f178d354224ff6c8530870 46 0
+6c254d9b7c5214823eb3d2838ec7a0a8299d4e32 46 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -4842,7 +4842,7 @@
 (let ((@x478 (mp ((_ quant-inst 3 42) (or (not $x52) $x171)) (trans (monotonicity @x131 $x137) (rewrite (= $x134 $x134)) $x137) $x134)))
 (unit-resolution (unit-resolution @x478 @x78 $x168) (mp @x77 @x472 (not $x168)) false)))))))))))))))))))))))))))))))))))
 
-95598ecc48263b667471a0a5145776d543f7750b 189 0
+358e9258315cd854d736e1b5ba21615744cfd921 189 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -5032,7 +5032,7 @@
 (let ((@x79 (asserted $x78)))
 (unit-resolution @x79 (trans (unit-resolution @x367 @x603 $x266) @x279 $x77) false))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))
 
-f9d9f73f1f276df0f7f9790713a13204b3df5ba4 11 0
+a88907c053a7ee53678749394daefd6c9f4b68cb 11 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -5044,7 +5044,7 @@
 (let ((@x42 (trans (monotonicity (rewrite (= $x31 true)) (= $x32 (not true))) (rewrite (= (not true) false)) (= $x32 false))))
 (mp (asserted $x32) @x42 false))))))))
 
-d75b1250831c7be693f7d73dc2069f59a82284f3 190 0
+7ccde197585af1e99e41c45491749be9bfb7aea3 190 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -5235,7 +5235,7 @@
 (let ((@x90 (asserted $x89)))
 (unit-resolution @x90 @x323 false)))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))
 
-28f9e3a56fce77e7784b19fdbe43fc5b9f9bc5b0 336 0
+677dbfda71252b7d1a479255e9abc091ee9a806b 336 0
 unsat
 ((set-logic <null>)
 (proof
@@ -5544,7 +5544,7 @@
 (let (($x890 (<= ?x889 0)))
 (let ((@x1023 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x887) $x890)) (trans @x965 (symm (unit-resolution @x620 @x384 $x610) $x881) $x887) $x890)))
 (let (($x793 (>= ?x791 0)))
-(let ((@x521 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x364 $x793)) (unit-resolution (def-axiom (or $x365 $x120)) @x583 $x120) $x793)))
+(let ((@x522 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x364 $x793)) (unit-resolution (def-axiom (or $x365 $x120)) @x583 $x120) $x793)))
 (let ((@x1085 (unit-resolution ((_ th-lemma arith) (or false (not (>= ?x530 2)))) @x26 (not (>= ?x530 2)))))
 (let (($x665 (<= ?x649 0)))
 (let ((@x767 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x650) $x665)) (unit-resolution @x664 @x425 $x650) $x665)))
@@ -5558,7 +5558,7 @@
 (let ((@x1104 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x503) (>= ?x502 0))) @x907 (>= ?x502 0))))
 (let ((@x1107 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x539) (<= ?x542 0))) (unit-resolution ((_ th-lemma arith) (or false $x539)) @x26 $x539) (<= ?x542 0))))
 (let ((@x1108 ((_ th-lemma arith farkas 1 -2 -2 -1 -2 1 1 1 1 1 1) @x1107 @x1104 (hypothesis $x793) @x1100 (hypothesis $x1078) (hypothesis $x890) @x1095 @x1092 @x858 @x767 @x1085 false)))
-(let ((@x576 (unit-resolution (lemma @x1108 (or (not $x1078) (not $x793) (not $x890))) @x521 @x1023 (not $x1078))))
+(let ((@x576 (unit-resolution (lemma @x1108 (or (not $x1078) (not $x793) (not $x890))) @x522 @x1023 (not $x1078))))
 (let ((@x966 (unit-resolution @x576 ((_ th-lemma arith) @x962 @x775 @x934 @x924 @x921 @x604 $x1078) false)))
 (let ((@x967 (lemma @x966 $x365)))
 (let ((@x445 (unit-resolution (def-axiom (or $x98 $x366 (not $x372))) @x377 (or $x98 $x366))))
@@ -5572,7 +5572,7 @@
 (let ((@x569 (unit-resolution (unit-resolution (def-axiom (or $x366 $x363 $x364)) @x967 $x365) (lemma @x1060 $x120) $x363)))
 (unit-resolution @x569 @x1067 false)))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))
 
-d351417cb827933b8da0a8b279e29eee0719819b 64 0
+5c5741c570cfdb433453abf31d1834a33ff261a7 64 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -5637,7 +5637,7 @@
 (let ((@x570 (mp ((_ quant-inst (sup$ ?x108) (sup$ ?x111) (sup$ ?x108)) (or $x251 (or $x160 $x247 $x117))) (rewrite (= (or $x251 (or $x160 $x247 $x117)) $x252)) $x252)))
 (unit-resolution @x570 @x584 @x114 @x116 @x119 false)))))))))))))))))))))))))))))))))))))))
 
-5a12a7134fe0a0d7becdd33ab1e66b9929fb9200 25 0
+b9f96986f08dff1e22d14a54a59ba0d994d1a5a6 25 0
 unsat
 ((set-logic AUFLIA)
 (proof
@@ -5663,7 +5663,7 @@
 (let ((@x258 ((_ quant-inst 1) $x257)))
 (unit-resolution @x258 @x620 @x145 false))))))))))))))))))
 
-27dedd7bdd019ed24c64571c329ee3a3f8abfec6 170 0
+90515e71e62ef453a5373f0331cce954b2c8e0f5 170 0
 unsat
 ((set-logic AUFLIA)
 (proof
--- a/src/HOL/SMT_Examples/SMT_Tests.thy	Tue Jun 03 16:22:01 2014 +0200
+++ b/src/HOL/SMT_Examples/SMT_Tests.thy	Tue Jun 03 16:27:31 2014 +0200
@@ -174,13 +174,11 @@
 
 lemma
   "a \<noteq> b \<and> a \<noteq> c \<and> b \<noteq> c \<and> (\<forall>x y. f x = f y \<longrightarrow> y = x) \<longrightarrow> f a \<noteq> f b"
-  using [[smt2_oracle=true]] (* FIXME: disable refine_inj_axiom in Z3 *)
   by smt2
 
 lemma
   "(\<forall>x y z. f x y = f x z \<longrightarrow> y = z) \<and> b \<noteq> c \<longrightarrow> f a b \<noteq> f a c"
   "(\<forall>x y z. f x y = f z y \<longrightarrow> x = z) \<and> a \<noteq> d \<longrightarrow> f a b \<noteq> f d b"
-  using [[smt2_oracle=true]] (* FIXME: disable refine_inj_axiom in Z3 *)
   by smt2+
 
 
--- a/src/HOL/SMT_Examples/SMT_Word_Examples.certs2	Tue Jun 03 16:22:01 2014 +0200
+++ b/src/HOL/SMT_Examples/SMT_Word_Examples.certs2	Tue Jun 03 16:27:31 2014 +0200
@@ -1,4 +1,4 @@
-ce41fb71f7c517682982b0f93f9e2ff5851420aa 8 0
+05ec0bc653bb980e7b2d8a64fcdbd39bf25dcaaa 8 0
 unsat
 ((set-logic <null>)
 (proof
@@ -7,7 +7,7 @@
 (let ((@x49 (trans (monotonicity @x42 (= (not (= (_ bv11 4) (bvneg (_ bv5 4)))) (not true))) (rewrite (= (not true) false)) (= (not (= (_ bv11 4) (bvneg (_ bv5 4)))) false))))
 (mp (asserted (not (= (_ bv11 4) (bvneg (_ bv5 4))))) @x49 false))))))
 
-7325b3de463bba9b3acec049992ae8e3bd84095c 7 0
+14099c150931519c703d279e4d77ff1b1016c31f 7 0
 unsat
 ((set-logic <null>)
 (proof
@@ -15,7 +15,7 @@
 (let ((@x39 (trans @x35 (rewrite (= (not true) false)) (= (not (= (_ bv11 4) (_ bv11 4))) false))))
 (mp (asserted (not (= (_ bv11 4) (_ bv11 4)))) @x39 false)))))
 
-23777227062fe10ce464941fc1e922676db603bc 7 0
+20d47424a7a34697fefe151cead57274409d19a7 7 0
 unsat
 ((set-logic <null>)
 (proof
@@ -23,7 +23,7 @@
 (let ((@x42 (trans @x38 (rewrite (= (not true) false)) (= (not (bvult (_ bv23 8) (_ bv27 8))) false))))
 (mp (asserted (not (bvult (_ bv23 8) (_ bv27 8)))) @x42 false)))))
 
-3fd9c0547528aa1b8bae9f52b77a315328f9b96f 9 0
+269da6b4ec3bfbe1037aca5daa32b7203e019162 9 0
 unsat
 ((set-logic <null>)
 (proof
@@ -33,7 +33,7 @@
 (let ((@x49 (trans @x45 (rewrite (= (not true) false)) (= (not (= (bvadd (_ bv27 5) (_ bv11 5)) (_ bv6 5))) false))))
 (mp (asserted (not (= (bvadd (_ bv27 5) (_ bv11 5)) (_ bv6 5)))) @x49 false)))))))
 
-666c4335f919bac608558e6bff8d2961e7974e97 9 0
+88864598d6a389e7a3d6c3f263e996fc5bc02af5 9 0
 unsat
 ((set-logic <null>)
 (proof
@@ -43,7 +43,7 @@
 (let ((@x49 (trans @x45 (rewrite (= (not true) false)) (= (not (= (bvmul (_ bv7 8) (_ bv3 8)) (_ bv21 8))) false))))
 (mp (asserted (not (= (bvmul (_ bv7 8) (_ bv3 8)) (_ bv21 8)))) @x49 false)))))))
 
-d1056c70663a614cd643028a7f6a9eac0e9c530f 9 0
+3a89a668465c3bdfa370a8a35d4c00de6035c388 9 0
 unsat
 ((set-logic <null>)
 (proof
@@ -53,7 +53,7 @@
 (let ((@x54 (trans @x50 (rewrite (= (not true) false)) (= (not (= (bvsub (_ bv11 8) (_ bv27 8)) (bvneg (_ bv16 8)))) false))))
 (mp (asserted (not (= (bvsub (_ bv11 8) (_ bv27 8)) (bvneg (_ bv16 8))))) @x54 false)))))))
 
-19c0dbd45ab3fc5b4fd54e1a565097dafc4b15aa 7 0
+6ac5f1f2168c9cba8c066fe8fba0691fcd0720ea 7 0
 unsat
 ((set-logic <null>)
 (proof
@@ -61,7 +61,7 @@
 (let ((@x39 (trans @x35 (rewrite (= (not true) false)) (= (not (= (_ bv11 5) (_ bv11 5))) false))))
 (mp (asserted (not (= (_ bv11 5) (_ bv11 5)))) @x39 false)))))
 
-287abeacd5cb5140a799c8f4f18a80225d062f81 11 0
+d88c56050b5020110d7aaf8e2503429964eba6e2 11 0
 unsat
 ((set-logic <null>)
 (proof
@@ -73,7 +73,7 @@
 (let ((@x63 (trans @x59 (rewrite (= (not true) false)) (= (not (= (bvadd (bvneg (_ bv40 7)) (_ bv1 7)) (bvneg (_ bv39 7)))) false))))
 (mp (asserted (not (= (bvadd (bvneg (_ bv40 7)) (_ bv1 7)) (bvneg (_ bv39 7))))) @x63 false)))))))))
 
-040c6f02771b1c516b52571900cb6fa5a5aabb39 19 0
+126c54378729ffdb76513e44c4a24ad9bb5ec0e5 19 0
 unsat
 ((set-logic <null>)
 (proof
@@ -93,7 +93,7 @@
 (let ((@x67 (trans @x63 (rewrite (= (not true) false)) (= $x38 false))))
 (mp (asserted $x38) @x67 false)))))))))))))))))
 
-266542f0767de16755644d9ae6de01b4da6720d0 18 0
+646a5730339e2c255c7e97b65e0064519875fc50 18 0
 unsat
 ((set-logic <null>)
 (proof
@@ -112,7 +112,7 @@
 (let ((@x84 (trans (monotonicity @x77 (= (not (= (_ bv4 4) ?x31)) (not true))) (rewrite (= (not true) false)) (= (not (= (_ bv4 4) ?x31)) false))))
 (mp (not-or-elim (mp (asserted $x34) @x60 $x56) (not (= (_ bv4 4) ?x31))) @x84 false))))))))))))))))
 
-9137ccc15de2c1c931d3b46d1d69025a9741a669 9 0
+db6783d09d27b1dd27f02ac7997f554083229f0e 9 0
 unsat
 ((set-logic <null>)
 (proof
@@ -122,7 +122,7 @@
 (let ((@x48 (trans @x44 (rewrite (= (not true) false)) (= (not (= (bvand (_ bv6 32) (_ bv5 32)) (_ bv4 32))) false))))
 (mp (asserted (not (= (bvand (_ bv6 32) (_ bv5 32)) (_ bv4 32)))) @x48 false)))))))
 
-a0cc2e473d859a107afe1adc11b287b98facf0dc 9 0
+caaca28f45463c8ac3330a15d5fe0ce34815a957 9 0
 unsat
 ((set-logic <null>)
 (proof
@@ -132,7 +132,7 @@
 (let ((@x48 (trans @x44 (rewrite (= (not true) false)) (= (not (= (bvor (_ bv6 8) (_ bv3 8)) (_ bv7 8))) false))))
 (mp (asserted (not (= (bvor (_ bv6 8) (_ bv3 8)) (_ bv7 8)))) @x48 false)))))))
 
-e3aa830bf4137713f98d1be224746b07ab5dde9e 9 0
+4cc2ef20dffa648829a897e5149ef7ca7a3e8392 9 0
 unsat
 ((set-logic <null>)
 (proof
@@ -142,7 +142,7 @@
 (let ((@x48 (trans @x44 (rewrite (= (not true) false)) (= (not (= (bvxor (_ bv240 8) (_ bv255 8)) (_ bv15 8))) false))))
 (mp (asserted (not (= (bvxor (_ bv240 8) (_ bv255 8)) (_ bv15 8)))) @x48 false)))))))
 
-860de692ca30ccc8528c0b8bf8e0107a887f31ca 8 0
+f6a406ff8446b18273f2321a90f5cffe4a87ef36 8 0
 unsat
 ((set-logic <null>)
 (proof
@@ -151,17 +151,7 @@
 (let ((@x47 (trans (monotonicity @x40 (= (not (= (bvnot (_ bv240 16)) (_ bv65295 16))) (not true))) (rewrite (= (not true) false)) (= (not (= (bvnot (_ bv240 16)) (_ bv65295 16))) false))))
 (mp (asserted (not (= (bvnot (_ bv240 16)) (_ bv65295 16)))) @x47 false))))))
 
-b09831d957da6fd7dc01ad2903ee64ea6163dd71 9 0
-unsat
-((set-logic <null>)
-(proof
-(let ((@x37 (monotonicity (rewrite (= (concat (_ bv3 4) (_ bv15 6)) (_ bv207 10))) (= (= (concat (_ bv3 4) (_ bv15 6)) (_ bv207 10)) (= (_ bv207 10) (_ bv207 10))))))
-(let ((@x41 (trans @x37 (rewrite (= (= (_ bv207 10) (_ bv207 10)) true)) (= (= (concat (_ bv3 4) (_ bv15 6)) (_ bv207 10)) true))))
-(let ((@x44 (monotonicity @x41 (= (not (= (concat (_ bv3 4) (_ bv15 6)) (_ bv207 10))) (not true)))))
-(let ((@x48 (trans @x44 (rewrite (= (not true) false)) (= (not (= (concat (_ bv3 4) (_ bv15 6)) (_ bv207 10))) false))))
-(mp (asserted (not (= (concat (_ bv3 4) (_ bv15 6)) (_ bv207 10)))) @x48 false)))))))
-
-754c79ba46ed9ca6826e2bd89107d64a3bda946c 9 0
+73073d457e5938da82c066eeab49ee274aa8c29c 9 0
 unsat
 ((set-logic <null>)
 (proof
@@ -171,7 +161,17 @@
 (let ((@x48 (trans @x44 (rewrite (= (not true) false)) (= (not (= (concat (_ bv11 4) (_ bv27 8)) (_ bv2843 12))) false))))
 (mp (asserted (not (= (concat (_ bv11 4) (_ bv27 8)) (_ bv2843 12)))) @x48 false)))))))
 
-ec3f2df20c6525ebf42f7503f7272036edb7945b 8 0
+65593ed080180204ff70dd46bc3cfb6c61a3b194 9 0
+unsat
+((set-logic <null>)
+(proof
+(let ((@x37 (monotonicity (rewrite (= (concat (_ bv3 4) (_ bv15 6)) (_ bv207 10))) (= (= (concat (_ bv3 4) (_ bv15 6)) (_ bv207 10)) (= (_ bv207 10) (_ bv207 10))))))
+(let ((@x41 (trans @x37 (rewrite (= (= (_ bv207 10) (_ bv207 10)) true)) (= (= (concat (_ bv3 4) (_ bv15 6)) (_ bv207 10)) true))))
+(let ((@x44 (monotonicity @x41 (= (not (= (concat (_ bv3 4) (_ bv15 6)) (_ bv207 10))) (not true)))))
+(let ((@x48 (trans @x44 (rewrite (= (not true) false)) (= (not (= (concat (_ bv3 4) (_ bv15 6)) (_ bv207 10))) false))))
+(mp (asserted (not (= (concat (_ bv3 4) (_ bv15 6)) (_ bv207 10)))) @x48 false)))))))
+
+4f6b1e0ff79913f7a2c5808fd6ef26cc8f37792d 8 0
 unsat
 ((set-logic <null>)
 (proof
@@ -180,7 +180,7 @@
 (let ((@x47 (trans (monotonicity @x40 (= (not (= ((_ extract 2 1) (_ bv6 4)) (_ bv3 2))) (not true))) (rewrite (= (not true) false)) (= (not (= ((_ extract 2 1) (_ bv6 4)) (_ bv3 2))) false))))
 (mp (asserted (not (= ((_ extract 2 1) (_ bv6 4)) (_ bv3 2)))) @x47 false))))))
 
-7f259d911b25f4f07d4578393dfd19c111adf0a1 9 0
+d86ad7c38fa16f519de4ec003010d1a8f081565c 9 0
 unsat
 ((set-logic <null>)
 (proof
@@ -190,7 +190,7 @@
 (let ((@x47 (trans @x43 (rewrite (= (not true) false)) (= (not (= ((_ zero_extend 6) (_ bv10 4)) (_ bv10 10))) false))))
 (mp (asserted (not (= ((_ zero_extend 6) (_ bv10 4)) (_ bv10 10)))) @x47 false)))))))
 
-cdeeacf51114f18ccd2f08e989ac540e7f6e65fe 9 0
+81c41e9044102d7a30c0580e58f69b452ee38a4b 9 0
 unsat
 ((set-logic <null>)
 (proof
@@ -200,17 +200,7 @@
 (let ((@x47 (trans @x43 (rewrite (= (not true) false)) (= (not (= ((_ sign_extend 2) (_ bv10 4)) (_ bv58 6))) false))))
 (mp (asserted (not (= ((_ sign_extend 2) (_ bv10 4)) (_ bv58 6)))) @x47 false)))))))
 
-a47b7af2f61edceb589d429fdc3caf416bf4289a 9 0
-unsat
-((set-logic <null>)
-(proof
-(let ((@x37 (monotonicity (rewrite (= (bvlshr (_ bv25 8) (_ bv2 8)) (_ bv6 8))) (= (= (bvlshr (_ bv25 8) (_ bv2 8)) (_ bv6 8)) (= (_ bv6 8) (_ bv6 8))))))
-(let ((@x41 (trans @x37 (rewrite (= (= (_ bv6 8) (_ bv6 8)) true)) (= (= (bvlshr (_ bv25 8) (_ bv2 8)) (_ bv6 8)) true))))
-(let ((@x44 (monotonicity @x41 (= (not (= (bvlshr (_ bv25 8) (_ bv2 8)) (_ bv6 8))) (not true)))))
-(let ((@x48 (trans @x44 (rewrite (= (not true) false)) (= (not (= (bvlshr (_ bv25 8) (_ bv2 8)) (_ bv6 8))) false))))
-(mp (asserted (not (= (bvlshr (_ bv25 8) (_ bv2 8)) (_ bv6 8)))) @x48 false)))))))
-
-b6c9268772e2e87691aac0285f81ee86c12fcbec 9 0
+11e634df3fd58dbe8bf7158dad75f4ae2701eb4c 9 0
 unsat
 ((set-logic <null>)
 (proof
@@ -220,7 +210,17 @@
 (let ((@x48 (trans @x44 (rewrite (= (not true) false)) (= (not (= (bvshl (_ bv19 8) (_ bv2 8)) (_ bv76 8))) false))))
 (mp (asserted (not (= (bvshl (_ bv19 8) (_ bv2 8)) (_ bv76 8)))) @x48 false)))))))
 
-9ab700e0dd6f49a60b128de87d210acc7f635d17 9 0
+237a24b121caa9070d8b35520f80e0ccba0d2f4f 9 0
+unsat
+((set-logic <null>)
+(proof
+(let ((@x37 (monotonicity (rewrite (= (bvlshr (_ bv25 8) (_ bv2 8)) (_ bv6 8))) (= (= (bvlshr (_ bv25 8) (_ bv2 8)) (_ bv6 8)) (= (_ bv6 8) (_ bv6 8))))))
+(let ((@x41 (trans @x37 (rewrite (= (= (_ bv6 8) (_ bv6 8)) true)) (= (= (bvlshr (_ bv25 8) (_ bv2 8)) (_ bv6 8)) true))))
+(let ((@x44 (monotonicity @x41 (= (not (= (bvlshr (_ bv25 8) (_ bv2 8)) (_ bv6 8))) (not true)))))
+(let ((@x48 (trans @x44 (rewrite (= (not true) false)) (= (not (= (bvlshr (_ bv25 8) (_ bv2 8)) (_ bv6 8))) false))))
+(mp (asserted (not (= (bvlshr (_ bv25 8) (_ bv2 8)) (_ bv6 8)))) @x48 false)))))))
+
+24384117f1fb154bc6416e4dd7ebc58ae0ca58d0 9 0
 unsat
 ((set-logic <null>)
 (proof
@@ -230,7 +230,7 @@
 (let ((@x48 (trans @x44 (rewrite (= (not true) false)) (= (not (= (bvashr (_ bv19 8) (_ bv2 8)) (_ bv4 8))) false))))
 (mp (asserted (not (= (bvashr (_ bv19 8) (_ bv2 8)) (_ bv4 8)))) @x48 false)))))))
 
-a99b8e8be40d80553ba4b11a508f78f6f4c87603 9 0
+5b9579066b20879b403fc98591f59c3d91708905 9 0
 unsat
 ((set-logic <null>)
 (proof
@@ -240,7 +240,17 @@
 (let ((@x47 (trans @x43 (rewrite (= (not true) false)) (= (not (= ((_ rotate_right 2) (_ bv6 4)) (_ bv9 4))) false))))
 (mp (asserted (not (= ((_ rotate_right 2) (_ bv6 4)) (_ bv9 4)))) @x47 false)))))))
 
-94eb73825d5572a2deeedb3cd9d62b002e25b9c9 17 0
+e1c17c42e520700c8fd0a10aafa28bafb081d5a9 9 0
+unsat
+((set-logic <null>)
+(proof
+(let ((@x36 (monotonicity (rewrite (= ((_ rotate_left 1) (_ bv14 4)) (_ bv13 4))) (= (= ((_ rotate_left 1) (_ bv14 4)) (_ bv13 4)) (= (_ bv13 4) (_ bv13 4))))))
+(let ((@x40 (trans @x36 (rewrite (= (= (_ bv13 4) (_ bv13 4)) true)) (= (= ((_ rotate_left 1) (_ bv14 4)) (_ bv13 4)) true))))
+(let ((@x43 (monotonicity @x40 (= (not (= ((_ rotate_left 1) (_ bv14 4)) (_ bv13 4))) (not true)))))
+(let ((@x47 (trans @x43 (rewrite (= (not true) false)) (= (not (= ((_ rotate_left 1) (_ bv14 4)) (_ bv13 4))) false))))
+(mp (asserted (not (= ((_ rotate_left 1) (_ bv14 4)) (_ bv13 4)))) @x47 false)))))))
+
+724e976f30fe0ee5563da7659ab27d5a1ccc8ec7 17 0
 unsat
 ((set-logic <null>)
 (proof
@@ -258,47 +268,7 @@
 (let ((@x55 (unit-resolution ((_ th-lemma bv) $x53) @x26 @x26 @x26 @x26 @x26 @x26 @x26 @x26 @x26 @x26 @x26 @x26 @x26 @x26 @x26 @x26 $x52)))
 (unit-resolution @x55 @x63 false)))))))))))))))
 
-1f7f153791a05b2fcd257d295cb279a51cb236cc 9 0
-unsat
-((set-logic <null>)
-(proof
-(let ((@x36 (monotonicity (rewrite (= ((_ rotate_left 1) (_ bv14 4)) (_ bv13 4))) (= (= ((_ rotate_left 1) (_ bv14 4)) (_ bv13 4)) (= (_ bv13 4) (_ bv13 4))))))
-(let ((@x40 (trans @x36 (rewrite (= (= (_ bv13 4) (_ bv13 4)) true)) (= (= ((_ rotate_left 1) (_ bv14 4)) (_ bv13 4)) true))))
-(let ((@x43 (monotonicity @x40 (= (not (= ((_ rotate_left 1) (_ bv14 4)) (_ bv13 4))) (not true)))))
-(let ((@x47 (trans @x43 (rewrite (= (not true) false)) (= (not (= ((_ rotate_left 1) (_ bv14 4)) (_ bv13 4))) false))))
-(mp (asserted (not (= ((_ rotate_left 1) (_ bv14 4)) (_ bv13 4)))) @x47 false)))))))
-
-85eff1077503d712336bf007dbc3d299f880dd8c 29 0
-unsat
-((set-logic <null>)
-(proof
-(let ((?x28 (bv2int$ (_ bv0 2))))
-(let (($x183 (<= ?x28 0)))
-(let (($x184 (not $x183)))
-(let (($x175 (forall ((?v0 (_ BitVec 2)) )(!(let ((?x47 (bv2int$ ?v0)))
-(let (($x53 (<= ?x47 0)))
-(not $x53))) :pattern ( (bv2int$ ?v0) )))
-))
-(let (($x57 (forall ((?v0 (_ BitVec 2)) )(let ((?x47 (bv2int$ ?v0)))
-(let (($x53 (<= ?x47 0)))
-(not $x53))))
-))
-(let ((@x177 (refl (= (not (<= (bv2int$ ?0) 0)) (not (<= (bv2int$ ?0) 0))))))
-(let ((@x112 (refl (~ (not (<= (bv2int$ ?0) 0)) (not (<= (bv2int$ ?0) 0))))))
-(let (($x49 (forall ((?v0 (_ BitVec 2)) )(let ((?x47 (bv2int$ ?v0)))
-(< 0 ?x47)))
-))
-(let ((@x56 (rewrite (= (< 0 (bv2int$ ?0)) (not (<= (bv2int$ ?0) 0))))))
-(let ((@x115 (mp~ (mp (asserted $x49) (quant-intro @x56 (= $x49 $x57)) $x57) (nnf-pos @x112 (~ $x57 $x57)) $x57)))
-(let ((@x180 (mp @x115 (quant-intro @x177 (= $x57 $x175)) $x175)))
-(let (($x187 (not $x175)))
-(let (($x188 (or $x187 $x184)))
-(let ((@x189 ((_ quant-inst (_ bv0 2)) $x188)))
-(let (($x29 (= ?x28 0)))
-(let ((@x30 (asserted $x29)))
-(unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x29) $x183)) @x30 (unit-resolution @x189 @x180 $x184) false)))))))))))))))))))
-
-5257e6fa7cd9238326b5139a4fdf82173f5411bf 51 0
+c0a99051efa07ae43e711d87b3b223ac1405eccc 51 0
 unsat
 ((set-logic <null>)
 (proof
@@ -350,7 +320,37 @@
 (let ((@x314 (unit-resolution ((_ th-lemma bv) $x312) @x26 @x26 @x26 @x26 @x26 @x26 @x26 @x26 (unit-resolution (def-axiom (or $x95 (not $x74))) @x303 (not $x74)) (unit-resolution (def-axiom (or $x95 (not $x75))) @x303 (not $x75)) (unit-resolution (def-axiom (or $x95 (not $x76))) @x303 (not $x76)) (unit-resolution (def-axiom (or $x95 (not $x77))) @x303 (not $x77)) (unit-resolution (def-axiom (or $x95 (not $x78))) @x303 (not $x78)) (unit-resolution (def-axiom (or $x95 (not $x79))) @x303 (not $x79)) (unit-resolution (def-axiom (or $x95 (not $x80))) @x303 (not $x80)) (unit-resolution (def-axiom (or $x95 $x264)) @x303 $x264) $x300)))
 (unit-resolution @x314 @x322 false)))))))))))))))))))))))))))))))))))))))))))))))))
 
-24d6f4fed7bbcb314acc273e33b6c33e838be536 16 0
+601b503239ecedf3719684b019abb944c178da93 29 0
+unsat
+((set-logic <null>)
+(proof
+(let ((?x28 (bv2int$ (_ bv0 2))))
+(let (($x183 (<= ?x28 0)))
+(let (($x184 (not $x183)))
+(let (($x175 (forall ((?v0 (_ BitVec 2)) )(!(let ((?x47 (bv2int$ ?v0)))
+(let (($x53 (<= ?x47 0)))
+(not $x53))) :pattern ( (bv2int$ ?v0) )))
+))
+(let (($x57 (forall ((?v0 (_ BitVec 2)) )(let ((?x47 (bv2int$ ?v0)))
+(let (($x53 (<= ?x47 0)))
+(not $x53))))
+))
+(let ((@x177 (refl (= (not (<= (bv2int$ ?0) 0)) (not (<= (bv2int$ ?0) 0))))))
+(let ((@x112 (refl (~ (not (<= (bv2int$ ?0) 0)) (not (<= (bv2int$ ?0) 0))))))
+(let (($x49 (forall ((?v0 (_ BitVec 2)) )(let ((?x47 (bv2int$ ?v0)))
+(< 0 ?x47)))
+))
+(let ((@x56 (rewrite (= (< 0 (bv2int$ ?0)) (not (<= (bv2int$ ?0) 0))))))
+(let ((@x115 (mp~ (mp (asserted $x49) (quant-intro @x56 (= $x49 $x57)) $x57) (nnf-pos @x112 (~ $x57 $x57)) $x57)))
+(let ((@x180 (mp @x115 (quant-intro @x177 (= $x57 $x175)) $x175)))
+(let (($x187 (not $x175)))
+(let (($x188 (or $x187 $x184)))
+(let ((@x189 ((_ quant-inst (_ bv0 2)) $x188)))
+(let (($x29 (= ?x28 0)))
+(let ((@x30 (asserted $x29)))
+(unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x29) $x183)) @x30 (unit-resolution @x189 @x180 $x184) false)))))))))))))))))))
+
+a68762d8c188bac63c09eec7c0a6f37774c2ce8c 16 0
 unsat
 ((set-logic <null>)
 (proof
--- a/src/HOL/SMT_Examples/VCC_Max.certs2	Tue Jun 03 16:22:01 2014 +0200
+++ b/src/HOL/SMT_Examples/VCC_Max.certs2	Tue Jun 03 16:27:31 2014 +0200
@@ -1,2831 +1,2973 @@
-d89d419269a26cf0f9e2b838b7d86233eeb72c17 2830 0
-unsat
-((set-logic <null>)
-(declare-fun ?v0!14 () Int)
-(declare-fun ?v0!15 () Int)
-(declare-fun ?v0!13 () Int)
-(proof
-(let ((?x12534 (* (- 1) v_b_L_H_max_G_3$)))
-(let ((?x3680 (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$)))
-(let ((?x3922 (b_S_idx$ ?x3680 v_b_L_H_p_G_0$ b_T_T_u1$)))
-(let ((?x3929 (b_S_read_n_u1$ v_b_S_s$ ?x3922)))
-(let (($x24191 (<= (+ ?x3929 ?x12534) 0)))
-(let (($x3940 (= v_b_L_H_max_G_3$ v_b_L_H_max_G_2$)))
-(let ((?x3974 (b_S_idx$ ?x3680 v_b_SL_H_witness_G_1$ b_T_T_u1$)))
-(let ((?x3975 (b_S_read_n_u1$ v_b_S_s$ ?x3974)))
-(let (($x3976 (= ?x3975 v_b_L_H_max_G_3$)))
-(let (($x12550 (<= (+ v_b_P_H_len$ (* (- 1) v_b_SL_H_witness_G_1$)) 0)))
-(let (($x20130 (or $x12550 (not $x3976))))
-(let (($x20131 (not $x20130)))
-(let (($x21049 (forall ((?v0 Int) )(!(let ((?x12534 (* (- 1) v_b_L_H_max_G_3$)))
-(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x12536 (<= (+ ?x3765 ?x12534) 0)))
-(let (($x12521 (>= (+ ?v0 (* (- 1) v_b_L_H_p_G_1$)) 0)))
-(let (($x14211 (<= ?v0 4294967295)))
-(let (($x17271 (not $x14211)))
-(let (($x10138 (>= ?v0 0)))
-(let (($x10556 (not $x10138)))
-(or $x10556 $x17271 $x12521 $x12536))))))))) :pattern ( (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$) )))
-))
-(let (($x21057 (or (not $x21049) $x20131)))
-(let (($x21060 (not $x21057)))
-(let ((?x16374 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ ?x3680 ?v0!14 b_T_T_u1$))))
-(let ((?x16620 (* (- 1) ?x16374)))
-(let (($x16622 (>= (+ v_b_L_H_max_G_3$ ?x16620) 0)))
-(let (($x16600 (<= (+ v_b_L_H_p_G_1$ (* (- 1) ?v0!14)) 0)))
-(let (($x16367 (<= ?v0!14 4294967295)))
-(let (($x20084 (not $x16367)))
-(let (($x16366 (>= ?v0!14 0)))
-(let (($x20083 (not $x16366)))
-(let (($x20099 (or $x20083 $x20084 $x16600 $x16622)))
-(let (($x20104 (not $x20099)))
-(let (($x21063 (or $x20104 $x21060)))
-(let (($x21066 (not $x21063)))
-(let (($x12514 (>= (+ v_b_P_H_len$ (* (- 1) v_b_L_H_p_G_1$)) 0)))
-(let (($x12518 (not $x12514)))
-(let (($x21069 (or $x12518 $x21066)))
-(let (($x21072 (not $x21069)))
-(let (($x21075 (or $x12518 $x21072)))
-(let (($x21078 (not $x21075)))
-(let (($x12486 (>= v_b_SL_H_witness_G_1$ 0)))
-(let (($x20173 (not $x12486)))
-(let (($x3960 (b_S_local_n_value_n_is$ v_b_S_s$ b_H_tok_S_1_T_16_o_24$ b_H_loc_o_p$ v_b_L_H_p_G_1$ b_T_T_u4$)))
-(let (($x12500 (= (+ v_b_L_H_p_G_0$ (* (- 1) v_b_L_H_p_G_1$)) (- 1))))
-(let (($x20170 (not $x12500)))
-(let (($x13856 (<= v_b_L_H_p_G_0$ 4294967294)))
-(let (($x16354 (not $x13856)))
-(let (($x12494 (>= v_b_L_H_p_G_0$ (- 1))))
-(let (($x16351 (not $x12494)))
-(let (($x21081 (or $x16351 $x16354 $x20170 (not $x3960) (not (>= v_b_L_H_p_G_1$ 2)) $x20173 $x21078)))
-(let (($x21084 (not $x21081)))
-(let (($x21087 (or $x16351 $x16354 $x21084)))
-(let (($x21090 (not $x21087)))
-(let (($x12404 (>= v_b_L_H_p_G_0$ 1)))
-(let (($x20190 (not $x12404)))
-(let (($x3937 (b_S_local_n_value_n_is$ v_b_S_s$ b_H_tok_S_1_T_24_o_47$ b_H_loc_o_witness$ v_b_L_H_p_G_0$ b_T_T_u4$)))
-(let (($x3936 (b_S_local_n_value_n_is$ v_b_S_s$ b_H_tok_S_1_T_23_o_7$ b_H_loc_o_max$ v_b_L_H_max_G_2$ b_T_T_u1$)))
-(let (($x3926 (b_S_thread_n_local$ v_b_S_s$ ?x3922)))
-(let (($x16339 (not $x3926)))
-(let (($x3923 (b_S_is$ ?x3922 b_T_T_u1$)))
-(let (($x16330 (not $x3923)))
-(let (($x21093 (or $x16330 $x16339 (not (= v_b_L_H_max_G_2$ ?x3929)) (not $x3936) (not $x3937) $x20190 (not $x3940) (not (= v_b_SL_H_witness_G_1$ v_b_L_H_p_G_0$)) $x20173 $x21090)))
-(let (($x21096 (not $x21093)))
-(let ((?x24124 (b_S_ref$ ?x3922)))
-(let ((?x23972 (b_S_ptr$ b_T_T_u1$ ?x24124)))
-(let (($x24221 (or (= (b_S_owner$ v_b_S_s$ ?x23972) b_S_me$) (b_S_in_n_wrapped_n_domain$ v_b_S_s$ ?x23972))))
-(let (($x24198 (= (b_S_kind_n_of$ (b_S_typ$ ?x23972)) b_S_kind_n_primitive$)))
-(let ((?x3874 (b_S_typemap$ v_b_S_s$)))
-(let ((?x24200 (b_S_select_o_tm$ ?x3874 ?x23972)))
-(let ((?x24203 (b_S_ts_n_emb$ ?x24200)))
-(let (($x24212 (= (b_S_owner$ v_b_S_s$ ?x24203) b_S_me$)))
-(let (($x24214 (or $x24212 (b_S_in_n_wrapped_n_domain$ v_b_S_s$ ?x24203))))
-(let (($x24210 (= (b_S_kind_n_of$ (b_S_typ$ ?x24203)) b_S_kind_n_primitive$)))
-(let (($x24201 (b_S_ts_n_is_n_volatile$ ?x24200)))
-(let (($x24202 (not $x24201)))
-(let (($x24206 (or $x24202 (not (b_S_closed$ v_b_S_s$ ?x24203)))))
-(let (($x24207 (not $x24206)))
-(let (($x24199 (not $x24198)))
-(let (($x24217 (not (or $x24199 $x24207 $x24210 (not $x24214)))))
-(let (($x24226 (not (or $x24217 (not (or $x24198 (not $x24221)))))))
-(let (($x24194 (b_S_typed$ v_b_S_s$ ?x23972)))
-(let (($x24195 (not $x24194)))
-(let (($x24227 (or $x24195 $x24226)))
-(let (($x24228 (not $x24227)))
-(let (($x24193 (b_S_thread_n_local$ v_b_S_s$ ?x23972)))
-(let (($x24229 (= $x24193 $x24228)))
-(let (($x19790 (forall ((?v0 B_S_state$) (?v1 B_S_ptr$) )(!(let (($x3184 (b_S_in_n_wrapped_n_domain$ ?v0 ?v1)))
-(let ((?x1103 (b_S_owner$ ?v0 ?v1)))
-(let (($x1104 (= ?x1103 b_S_me$)))
-(let (($x1001 (= (b_S_kind_n_of$ (b_S_typ$ ?v1)) b_S_kind_n_primitive$)))
-(let ((?x1215 (b_S_typemap$ ?v0)))
-(let ((?x3166 (b_S_select_o_tm$ ?x1215 ?v1)))
-(let ((?x3169 (b_S_ts_n_emb$ ?x3166)))
-(let (($x3180 (or (= (b_S_owner$ ?v0 ?x3169) b_S_me$) (b_S_in_n_wrapped_n_domain$ ?v0 ?x3169))))
-(let (($x3172 (or (not (b_S_ts_n_is_n_volatile$ ?x3166)) (not (b_S_closed$ ?v0 ?x3169)))))
-(let (($x1024 (not $x1001)))
-(let (($x19765 (or $x1024 (not $x3172) (= (b_S_kind_n_of$ (b_S_typ$ ?x3169)) b_S_kind_n_primitive$) (not $x3180))))
-(let (($x19774 (or (not $x19765) (not (or $x1001 (not (or $x1104 $x3184)))))))
-(let (($x1106 (b_S_typed$ ?v0 ?v1)))
-(let (($x8534 (not $x1106)))
-(let (($x19782 (not (or $x8534 (not $x19774)))))
-(let (($x3165 (b_S_thread_n_local$ ?v0 ?v1)))
-(= $x3165 $x19782))))))))))))))))) :pattern ( (b_S_thread_n_local$ ?v0 ?v1) )))
-))
-(let (($x12140 (forall ((?v0 B_S_state$) (?v1 B_S_ptr$) )(!(let (($x3184 (b_S_in_n_wrapped_n_domain$ ?v0 ?v1)))
-(let ((?x1103 (b_S_owner$ ?v0 ?v1)))
-(let (($x1104 (= ?x1103 b_S_me$)))
-(let (($x1001 (= (b_S_kind_n_of$ (b_S_typ$ ?v1)) b_S_kind_n_primitive$)))
-(let (($x1024 (not $x1001)))
-(let (($x3186 (and $x1024 (or $x1104 $x3184))))
-(let ((?x1215 (b_S_typemap$ ?v0)))
-(let ((?x3166 (b_S_select_o_tm$ ?x1215 ?v1)))
-(let ((?x3169 (b_S_ts_n_emb$ ?x3166)))
-(let (($x3180 (or (= (b_S_owner$ ?v0 ?x3169) b_S_me$) (b_S_in_n_wrapped_n_domain$ ?v0 ?x3169))))
-(let (($x3176 (not (= (b_S_kind_n_of$ (b_S_typ$ ?x3169)) b_S_kind_n_primitive$))))
-(let (($x3172 (or (not (b_S_ts_n_is_n_volatile$ ?x3166)) (not (b_S_closed$ ?v0 ?x3169)))))
-(let (($x8324 (and $x1001 $x3172 $x3176 $x3180)))
-(let (($x8329 (or $x8324 $x3186)))
-(let (($x1106 (b_S_typed$ ?v0 ?v1)))
-(let (($x8332 (and $x1106 $x8329)))
-(let (($x3165 (b_S_thread_n_local$ ?v0 ?v1)))
-(= $x3165 $x8332)))))))))))))))))) :pattern ( (b_S_thread_n_local$ ?v0 ?v1) )))
-))
-(let (($x3184 (b_S_in_n_wrapped_n_domain$ ?1 ?0)))
-(let ((?x1103 (b_S_owner$ ?1 ?0)))
-(let (($x1104 (= ?x1103 b_S_me$)))
-(let (($x1001 (= (b_S_kind_n_of$ (b_S_typ$ ?0)) b_S_kind_n_primitive$)))
-(let ((?x1215 (b_S_typemap$ ?1)))
-(let ((?x3166 (b_S_select_o_tm$ ?x1215 ?0)))
-(let ((?x3169 (b_S_ts_n_emb$ ?x3166)))
-(let (($x3180 (or (= (b_S_owner$ ?1 ?x3169) b_S_me$) (b_S_in_n_wrapped_n_domain$ ?1 ?x3169))))
-(let (($x3172 (or (not (b_S_ts_n_is_n_volatile$ ?x3166)) (not (b_S_closed$ ?1 ?x3169)))))
-(let (($x1024 (not $x1001)))
-(let (($x19765 (or $x1024 (not $x3172) (= (b_S_kind_n_of$ (b_S_typ$ ?x3169)) b_S_kind_n_primitive$) (not $x3180))))
-(let (($x19774 (or (not $x19765) (not (or $x1001 (not (or $x1104 $x3184)))))))
-(let (($x1106 (b_S_typed$ ?1 ?0)))
-(let (($x8534 (not $x1106)))
-(let (($x19782 (not (or $x8534 (not $x19774)))))
-(let (($x3165 (b_S_thread_n_local$ ?1 ?0)))
-(let (($x3186 (and $x1024 (or $x1104 $x3184))))
-(let (($x3176 (not (= (b_S_kind_n_of$ (b_S_typ$ ?x3169)) b_S_kind_n_primitive$))))
-(let (($x8324 (and $x1001 $x3172 $x3176 $x3180)))
-(let (($x8329 (or $x8324 $x3186)))
-(let (($x8332 (and $x1106 $x8329)))
-(let (($x12136 (= $x3165 $x8332)))
-(let ((@x19776 (monotonicity (rewrite (= $x8324 (not $x19765))) (rewrite (= $x3186 (not (or $x1001 (not (or $x1104 $x3184)))))) (= $x8329 $x19774))))
-(let ((@x19786 (trans (monotonicity @x19776 (= $x8332 (and $x1106 $x19774))) (rewrite (= (and $x1106 $x19774) $x19782)) (= $x8332 $x19782))))
-(let ((@x19792 (quant-intro (monotonicity @x19786 (= $x12136 (= $x3165 $x19782))) (= $x12140 $x19790))))
-(let (($x8338 (forall ((?v0 B_S_state$) (?v1 B_S_ptr$) )(!(let (($x3184 (b_S_in_n_wrapped_n_domain$ ?v0 ?v1)))
-(let ((?x1103 (b_S_owner$ ?v0 ?v1)))
-(let (($x1104 (= ?x1103 b_S_me$)))
-(let (($x1001 (= (b_S_kind_n_of$ (b_S_typ$ ?v1)) b_S_kind_n_primitive$)))
-(let (($x1024 (not $x1001)))
-(let (($x3186 (and $x1024 (or $x1104 $x3184))))
-(let ((?x1215 (b_S_typemap$ ?v0)))
-(let ((?x3166 (b_S_select_o_tm$ ?x1215 ?v1)))
-(let ((?x3169 (b_S_ts_n_emb$ ?x3166)))
-(let (($x3180 (or (= (b_S_owner$ ?v0 ?x3169) b_S_me$) (b_S_in_n_wrapped_n_domain$ ?v0 ?x3169))))
-(let (($x3176 (not (= (b_S_kind_n_of$ (b_S_typ$ ?x3169)) b_S_kind_n_primitive$))))
-(let (($x3172 (or (not (b_S_ts_n_is_n_volatile$ ?x3166)) (not (b_S_closed$ ?v0 ?x3169)))))
-(let (($x8324 (and $x1001 $x3172 $x3176 $x3180)))
-(let (($x8329 (or $x8324 $x3186)))
-(let (($x1106 (b_S_typed$ ?v0 ?v1)))
-(let (($x8332 (and $x1106 $x8329)))
-(let (($x3165 (b_S_thread_n_local$ ?v0 ?v1)))
-(= $x3165 $x8332)))))))))))))))))) :pattern ( (b_S_thread_n_local$ ?v0 ?v1) )))
-))
-(let (($x3191 (forall ((?v0 B_S_state$) (?v1 B_S_ptr$) )(!(let (($x3184 (b_S_in_n_wrapped_n_domain$ ?v0 ?v1)))
-(let ((?x1103 (b_S_owner$ ?v0 ?v1)))
-(let (($x1104 (= ?x1103 b_S_me$)))
-(let (($x1001 (= (b_S_kind_n_of$ (b_S_typ$ ?v1)) b_S_kind_n_primitive$)))
-(let (($x1024 (not $x1001)))
-(let (($x3186 (and $x1024 (or $x1104 $x3184))))
-(let ((?x1215 (b_S_typemap$ ?v0)))
-(let ((?x3166 (b_S_select_o_tm$ ?x1215 ?v1)))
-(let ((?x3169 (b_S_ts_n_emb$ ?x3166)))
-(let (($x3180 (or (= (b_S_owner$ ?v0 ?x3169) b_S_me$) (b_S_in_n_wrapped_n_domain$ ?v0 ?x3169))))
-(let (($x3176 (not (= (b_S_kind_n_of$ (b_S_typ$ ?x3169)) b_S_kind_n_primitive$))))
-(let (($x3172 (or (not (b_S_ts_n_is_n_volatile$ ?x3166)) (not (b_S_closed$ ?v0 ?x3169)))))
-(let (($x3183 (and $x1001 (and $x3172 (and $x3176 $x3180)))))
-(let (($x1106 (b_S_typed$ ?v0 ?v1)))
-(let (($x3165 (b_S_thread_n_local$ ?v0 ?v1)))
-(= $x3165 (and $x1106 (or $x3183 $x3186)))))))))))))))))) :pattern ( (b_S_thread_n_local$ ?v0 ?v1) )))
-))
-(let (($x8335 (= $x3165 $x8332)))
-(let (($x8336 (= (= $x3165 (and $x1106 (or (and $x1001 (and $x3172 (and $x3176 $x3180))) $x3186))) $x8335)))
-(let (($x8333 (= (and $x1106 (or (and $x1001 (and $x3172 (and $x3176 $x3180))) $x3186)) $x8332)))
-(let (($x3183 (and $x1001 (and $x3172 (and $x3176 $x3180)))))
-(let ((@x8323 (monotonicity (rewrite (= (and $x3172 (and $x3176 $x3180)) (and $x3172 $x3176 $x3180))) (= $x3183 (and $x1001 (and $x3172 $x3176 $x3180))))))
-(let ((@x8328 (trans @x8323 (rewrite (= (and $x1001 (and $x3172 $x3176 $x3180)) $x8324)) (= $x3183 $x8324))))
-(let ((@x8337 (monotonicity (monotonicity (monotonicity @x8328 (= (or $x3183 $x3186) $x8329)) $x8333) $x8336)))
-(let ((@x12145 (mp (mp (asserted $x3191) (quant-intro @x8337 (= $x3191 $x8338)) $x8338) (quant-intro (rewrite (= $x8335 $x12136)) (= $x8338 $x12140)) $x12140)))
-(let ((@x19793 (mp (mp~ @x12145 (nnf-pos (refl (~ $x12136 $x12136)) (~ $x12140 $x12140)) $x12140) @x19792 $x19790)))
-(let (($x23973 (= ?x3922 ?x23972)))
-(let ((?x23986 (b_S_typ$ ?x3922)))
-(let (($x23984 (= ?x23986 b_T_T_u1$)))
-(let ((?x3652 (b_S_sizeof$ b_T_T_u1$)))
-(let ((?x24037 (* ?x3652 v_b_L_H_p_G_0$)))
-(let ((?x3739 (b_S_idx$ ?x3680 0 b_T_T_u1$)))
-(let ((?x23186 (b_S_ref$ ?x3739)))
-(let ((?x23206 (b_S_ptr$ b_T_T_u1$ ?x23186)))
-(let ((?x23612 (b_S_ref$ ?x23206)))
-(let ((?x24040 (+ ?x23612 ?x24037)))
-(let ((?x24043 (b_S_ptr$ b_T_T_u1$ ?x24040)))
-(let (($x20974 (forall ((?v0 B_S_ctype$) (?v1 Int) )(!(= (b_S_typ$ (b_S_ptr$ ?v0 ?v1)) ?v0) :pattern ( (b_S_ptr$ ?v0 ?v1) )))
-))
-(let (($x3462 (forall ((?v0 B_S_ctype$) (?v1 Int) )(= (b_S_typ$ (b_S_ptr$ ?v0 ?v1)) ?v0))
-))
-(let (($x3461 (= (b_S_typ$ (b_S_ptr$ ?1 ?0)) ?1)))
-(let ((@x16101 (mp~ (asserted $x3462) (nnf-pos (refl (~ $x3461 $x3461)) (~ $x3462 $x3462)) $x3462)))
-(let ((@x20979 (mp @x16101 (quant-intro (refl (= $x3461 $x3461)) (= $x3462 $x20974)) $x20974)))
-(let ((@x24995 (unit-resolution ((_ quant-inst b_T_T_u1$ (+ ?x23612 ?x24037)) (or (not $x20974) (= (b_S_typ$ ?x24043) b_T_T_u1$))) @x20979 (= (b_S_typ$ ?x24043) b_T_T_u1$))))
-(let ((?x23996 (b_S_idx$ ?x23206 v_b_L_H_p_G_0$ b_T_T_u1$)))
-(let (($x24957 (= ?x23996 ?x24043)))
-(let (($x24973 (or (not (b_S_extent_n_hint$ ?x23996 ?x23206)) (not $x24957))))
-(let (($x24976 (not $x24973)))
-(let (($x18898 (forall ((?v0 B_S_ptr$) (?v1 Int) (?v2 B_S_ctype$) )(!(let ((?x2466 (* ?v1 (b_S_sizeof$ ?v2))))
-(let ((?x2467 (+ (b_S_ref$ ?v0) ?x2466)))
-(let ((?x2468 (b_S_ptr$ ?v2 ?x2467)))
-(let ((?x2462 (b_S_idx$ ?v0 ?v1 ?v2)))
-(let (($x2469 (= ?x2462 ?x2468)))
-(not (or (not (b_S_extent_n_hint$ ?x2462 ?v0)) (not $x2469)))))))) :pattern ( (b_S_idx$ ?v0 ?v1 ?v2) )))
-))
-(let (($x2472 (forall ((?v0 B_S_ptr$) (?v1 Int) (?v2 B_S_ctype$) )(!(let ((?x2466 (* ?v1 (b_S_sizeof$ ?v2))))
-(let ((?x2467 (+ (b_S_ref$ ?v0) ?x2466)))
-(let ((?x2468 (b_S_ptr$ ?v2 ?x2467)))
-(let ((?x2462 (b_S_idx$ ?v0 ?v1 ?v2)))
-(let (($x2469 (= ?x2462 ?x2468)))
-(let (($x2463 (b_S_extent_n_hint$ ?x2462 ?v0)))
-(and $x2463 $x2469))))))) :pattern ( (b_S_idx$ ?v0 ?v1 ?v2) )))
-))
-(let ((?x2466 (* ?1 (b_S_sizeof$ ?0))))
-(let ((?x2467 (+ (b_S_ref$ ?2) ?x2466)))
-(let ((?x2468 (b_S_ptr$ ?0 ?x2467)))
-(let ((?x2462 (b_S_idx$ ?2 ?1 ?0)))
-(let (($x2469 (= ?x2462 ?x2468)))
-(let (($x2463 (b_S_extent_n_hint$ ?x2462 ?2)))
-(let (($x2470 (and $x2463 $x2469)))
-(let ((@x18900 (quant-intro (rewrite (= $x2470 (not (or (not $x2463) (not $x2469))))) (= $x2472 $x18898))))
-(let (($x7455 (forall ((?v0 B_S_ptr$) (?v1 Int) (?v2 B_S_ctype$) )(!(let ((?x7440 (* (b_S_sizeof$ ?v2) ?v1)))
-(let ((?x7443 (+ (b_S_ref$ ?v0) ?x7440)))
-(let ((?x7446 (b_S_ptr$ ?v2 ?x7443)))
-(let ((?x2462 (b_S_idx$ ?v0 ?v1 ?v2)))
-(let (($x7449 (= ?x2462 ?x7446)))
-(let (($x2463 (b_S_extent_n_hint$ ?x2462 ?v0)))
-(and $x2463 $x7449))))))) :pattern ( (b_S_idx$ ?v0 ?v1 ?v2) )))
-))
-(let ((?x7440 (* (b_S_sizeof$ ?0) ?1)))
-(let ((?x7443 (+ (b_S_ref$ ?2) ?x7440)))
-(let ((?x7446 (b_S_ptr$ ?0 ?x7443)))
-(let (($x7449 (= ?x2462 ?x7446)))
-(let (($x7452 (and $x2463 $x7449)))
-(let ((@x11827 (monotonicity (monotonicity (rewrite (= ?x7440 ?x2466)) (= ?x7443 ?x2467)) (= ?x7446 ?x2468))))
-(let ((@x11833 (quant-intro (monotonicity (monotonicity @x11827 (= $x7449 $x2469)) (= $x7452 $x2470)) (= $x7455 $x2472))))
-(let ((@x7448 (monotonicity (monotonicity (rewrite (= ?x2466 ?x7440)) (= ?x2467 ?x7443)) (= ?x2468 ?x7446))))
-(let ((@x7457 (quant-intro (monotonicity (monotonicity @x7448 (= $x2469 $x7449)) (= $x2470 $x7452)) (= $x2472 $x7455))))
-(let ((@x15301 (mp~ (mp (mp (asserted $x2472) @x7457 $x7455) @x11833 $x2472) (nnf-pos (refl (~ $x2470 $x2470)) (~ $x2472 $x2472)) $x2472)))
-(let ((@x18901 (mp @x15301 @x18900 $x18898)))
-(let (($x23217 (not $x18898)))
-(let (($x24981 (or $x23217 $x24976)))
-(let (($x24034 (not (= ?x23996 (b_S_ptr$ b_T_T_u1$ (+ ?x23612 (* v_b_L_H_p_G_0$ ?x3652)))))))
-(let (($x24986 (= (or $x23217 (not (or (not (b_S_extent_n_hint$ ?x23996 ?x23206)) $x24034))) $x24981)))
-(let (($x24958 (= (= ?x23996 (b_S_ptr$ b_T_T_u1$ (+ ?x23612 (* v_b_L_H_p_G_0$ ?x3652)))) $x24957)))
-(let ((@x24955 (monotonicity (rewrite (= (* v_b_L_H_p_G_0$ ?x3652) ?x24037)) (= (+ ?x23612 (* v_b_L_H_p_G_0$ ?x3652)) ?x24040))))
-(let ((@x24956 (monotonicity @x24955 (= (b_S_ptr$ b_T_T_u1$ (+ ?x23612 (* v_b_L_H_p_G_0$ ?x3652))) ?x24043))))
-(let ((@x24975 (monotonicity (monotonicity (monotonicity @x24956 $x24958) (= $x24034 (not $x24957))) (= (or (not (b_S_extent_n_hint$ ?x23996 ?x23206)) $x24034) $x24973))))
-(let ((@x24983 (monotonicity @x24975 (= (not (or (not (b_S_extent_n_hint$ ?x23996 ?x23206)) $x24034)) $x24976))))
-(let ((@x24985 ((_ quant-inst (b_S_ptr$ b_T_T_u1$ ?x23186) v_b_L_H_p_G_0$ b_T_T_u1$) (or $x23217 (not (or (not (b_S_extent_n_hint$ ?x23996 ?x23206)) $x24034))))))
-(let ((@x23295 (mp @x24985 (trans (monotonicity @x24983 $x24986) (rewrite (= $x24981 $x24981)) $x24986) $x24981)))
-(let ((@x25587 (unit-resolution (def-axiom (or $x24973 $x24957)) (unit-resolution @x23295 @x18901 $x24976) $x24957)))
-(let (($x23207 (= ?x3739 ?x23206)))
-(let (($x3740 (b_S_is$ ?x3739 b_T_T_u1$)))
-(let ((?x23215 (b_S_typ$ ?x3739)))
-(let (($x23216 (= ?x23215 b_T_T_u1$)))
-(let ((@x23266 (unit-resolution ((_ quant-inst b_T_T_u1$ v_b_P_H_arr$) (or (not $x20974) (= (b_S_typ$ ?x3680) b_T_T_u1$))) @x20979 (= (b_S_typ$ ?x3680) b_T_T_u1$))))
-(let (($x20968 (forall ((?v0 B_S_ctype$) (?v1 Int) )(!(= (b_S_ref$ (b_S_ptr$ ?v0 ?v1)) ?v1) :pattern ( (b_S_ptr$ ?v0 ?v1) )))
-))
-(let (($x3459 (forall ((?v0 B_S_ctype$) (?v1 Int) )(= (b_S_ref$ (b_S_ptr$ ?v0 ?v1)) ?v1))
-))
-(let (($x3458 (= (b_S_ref$ (b_S_ptr$ ?1 ?0)) ?0)))
-(let ((@x16096 (mp~ (asserted $x3459) (nnf-pos (refl (~ $x3458 $x3458)) (~ $x3459 $x3459)) $x3459)))
-(let ((@x20973 (mp @x16096 (quant-intro (refl (= $x3458 $x3458)) (= $x3459 $x20968)) $x20968)))
-(let ((@x23283 (unit-resolution ((_ quant-inst b_T_T_u1$ v_b_P_H_arr$) (or (not $x20968) (= (b_S_ref$ ?x3680) v_b_P_H_arr$))) @x20973 (= (b_S_ref$ ?x3680) v_b_P_H_arr$))))
-(let ((?x3681 (b_S_ref$ ?x3680)))
-(let ((?x23203 (b_S_ptr$ b_T_T_u1$ ?x3681)))
-(let (($x23188 (= ?x3739 ?x23203)))
-(let (($x23208 (or (not (b_S_extent_n_hint$ ?x3739 ?x3680)) (not $x23188))))
-(let (($x23213 (not $x23208)))
-(let (($x23220 (or $x23217 $x23213)))
-(let (($x23243 (or (not (b_S_extent_n_hint$ ?x3739 ?x3680)) (not (= ?x3739 (b_S_ptr$ b_T_T_u1$ (+ ?x3681 (* 0 ?x3652))))))))
-(let (($x23209 (= (not (= ?x3739 (b_S_ptr$ b_T_T_u1$ (+ ?x3681 (* 0 ?x3652))))) (not $x23188))))
-(let ((@x23198 (monotonicity (rewrite (= (* 0 ?x3652) 0)) (= (+ ?x3681 (* 0 ?x3652)) (+ ?x3681 0)))))
-(let ((@x23202 (trans @x23198 (rewrite (= (+ ?x3681 0) ?x3681)) (= (+ ?x3681 (* 0 ?x3652)) ?x3681))))
-(let ((@x23190 (monotonicity @x23202 (= (b_S_ptr$ b_T_T_u1$ (+ ?x3681 (* 0 ?x3652))) ?x23203))))
-(let ((@x23192 (monotonicity @x23190 (= (= ?x3739 (b_S_ptr$ b_T_T_u1$ (+ ?x3681 (* 0 ?x3652)))) $x23188))))
-(let ((@x23219 (monotonicity (monotonicity (monotonicity @x23192 $x23209) (= $x23243 $x23208)) (= (not $x23243) $x23213))))
-(let ((@x23232 (trans (monotonicity @x23219 (= (or $x23217 (not $x23243)) $x23220)) (rewrite (= $x23220 $x23220)) (= (or $x23217 (not $x23243)) $x23220))))
-(let ((@x23284 (unit-resolution (mp ((_ quant-inst (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) 0 b_T_T_u1$) (or $x23217 (not $x23243))) @x23232 $x23220) @x18901 $x23213)))
-(let ((@x23269 (unit-resolution (def-axiom (or $x23208 $x23188)) @x23284 $x23188)))
-(let ((@x23248 (monotonicity (trans @x23269 (monotonicity @x23283 (= ?x23203 ?x3680)) (= ?x3739 ?x3680)) (= ?x23215 (b_S_typ$ ?x3680)))))
-(let (($x23163 (not $x23216)))
-(let (($x23223 (= $x3740 $x23216)))
-(let (($x20961 (forall ((?v0 B_S_ptr$) (?v1 B_S_ctype$) )(!(let ((?x2296 (b_S_typ$ ?v0)))
-(let (($x2741 (= ?x2296 ?v1)))
-(let (($x3427 (b_S_is$ ?v0 ?v1)))
-(= $x3427 $x2741)))) :pattern ( (b_S_is$ ?v0 ?v1) )))
-))
-(let (($x12230 (forall ((?v0 B_S_ptr$) (?v1 B_S_ctype$) )(let ((?x2296 (b_S_typ$ ?v0)))
-(let (($x2741 (= ?x2296 ?v1)))
-(let (($x3427 (b_S_is$ ?v0 ?v1)))
-(= $x3427 $x2741)))))
-))
-(let ((?x2296 (b_S_typ$ ?1)))
-(let (($x2741 (= ?x2296 ?0)))
-(let (($x3427 (b_S_is$ ?1 ?0)))
-(let (($x12201 (= $x3427 $x2741)))
-(let (($x3434 (forall ((?v0 B_S_ptr$) (?v1 B_S_ctype$) )(let ((?x2296 (b_S_typ$ ?v0)))
-(let (($x2741 (= ?x2296 ?v1)))
-(let (($x3427 (b_S_is$ ?v0 ?v1)))
-(= $x3427 $x2741)))))
-))
-(let ((@x12235 (mp (asserted $x3434) (quant-intro (rewrite (= (= $x3427 $x2741) $x12201)) (= $x3434 $x12230)) $x12230)))
-(let ((@x20966 (mp (mp~ @x12235 (nnf-pos (refl (~ $x12201 $x12201)) (~ $x12230 $x12230)) $x12230) (quant-intro (refl (= $x12201 $x12201)) (= $x12230 $x20961)) $x20961)))
-(let ((@x23281 (unit-resolution (def-axiom (or (not $x23223) $x3740 $x23163)) (hypothesis (not $x3740)) (or (not $x23223) $x23163))))
-(let ((@x23282 (unit-resolution @x23281 (unit-resolution ((_ quant-inst (b_S_idx$ ?x3680 0 b_T_T_u1$) b_T_T_u1$) (or (not $x20961) $x23223)) @x20966 $x23223) $x23163)))
-(let ((@x23251 (lemma (unit-resolution @x23282 (trans @x23248 @x23266 $x23216) false) $x3740)))
-(let (($x8559 (forall ((?v0 B_S_ptr$) (?v1 B_S_ctype$) )(!(or (not (b_S_is$ ?v0 ?v1)) (= ?v0 (b_S_ptr$ ?v1 (b_S_ref$ ?v0)))) :pattern ( (b_S_is$ ?v0 ?v1) )))
-))
-(let (($x8556 (or (not $x3427) (= ?1 (b_S_ptr$ ?0 (b_S_ref$ ?1))))))
-(let (($x3432 (forall ((?v0 B_S_ptr$) (?v1 B_S_ctype$) )(!(let (($x3427 (b_S_is$ ?v0 ?v1)))
-(=> $x3427 (= ?v0 (b_S_ptr$ ?v1 (b_S_ref$ ?v0))))) :pattern ( (b_S_is$ ?v0 ?v1) )))
-))
-(let ((@x8558 (rewrite (= (=> $x3427 (= ?1 (b_S_ptr$ ?0 (b_S_ref$ ?1)))) $x8556))))
-(let ((@x16076 (mp~ (mp (asserted $x3432) (quant-intro @x8558 (= $x3432 $x8559)) $x8559) (nnf-pos (refl (~ $x8556 $x8556)) (~ $x8559 $x8559)) $x8559)))
-(let (($x23403 (= (or (not $x8559) (or (not $x3740) $x23207)) (or (not $x8559) (not $x3740) $x23207))))
-(let ((@x23405 (mp ((_ quant-inst (b_S_idx$ ?x3680 0 b_T_T_u1$) b_T_T_u1$) (or (not $x8559) (or (not $x3740) $x23207))) (rewrite $x23403) (or (not $x8559) (not $x3740) $x23207))))
-(let ((@x24358 (monotonicity (symm @x23283 (= v_b_P_H_arr$ ?x3681)) (= ?x3680 ?x23203))))
-(let ((@x24998 (trans (trans @x24358 (symm @x23269 (= ?x23203 ?x3739)) (= ?x3680 ?x3739)) (unit-resolution @x23405 @x16076 @x23251 $x23207) (= ?x3680 ?x23206))))
-(let ((@x25027 (monotonicity (trans (monotonicity @x24998 (= ?x3922 ?x23996)) @x25587 (= ?x3922 ?x24043)) (= ?x23986 (b_S_typ$ ?x24043)))))
-(let (($x25000 (not $x23984)))
-(let (($x23994 (= $x3923 $x23984)))
-(let ((@x24895 (unit-resolution (def-axiom (or (not $x23994) $x3923 $x25000)) (hypothesis $x16330) (or (not $x23994) $x25000))))
-(let ((@x24903 (unit-resolution @x24895 (unit-resolution ((_ quant-inst (b_S_idx$ ?x3680 v_b_L_H_p_G_0$ b_T_T_u1$) b_T_T_u1$) (or (not $x20961) $x23994)) @x20966 $x23994) $x25000)))
-(let ((@x25032 (lemma (unit-resolution @x24903 (trans @x25027 @x24995 $x23984) false) $x3923)))
-(let ((@x24892 (rewrite (= (or (not $x8559) (or $x16330 $x23973)) (or (not $x8559) $x16330 $x23973)))))
-(let ((@x24894 (mp ((_ quant-inst (b_S_idx$ ?x3680 v_b_L_H_p_G_0$ b_T_T_u1$) b_T_T_u1$) (or (not $x8559) (or $x16330 $x23973))) @x24892 (or (not $x8559) $x16330 $x23973))))
-(let ((@x24935 (unit-resolution @x24894 @x16076 (hypothesis $x3923) (hypothesis (not $x23973)) false)))
-(let ((@x25156 (unit-resolution (lemma @x24935 (or $x16330 $x23973)) @x25032 $x23973)))
-(let ((@x25212 (symm (monotonicity (symm @x25156 (= ?x23972 ?x3922)) (= $x24193 $x3926)) (= $x3926 $x24193))))
-(let ((@x25225 (mp (hypothesis $x16339) (monotonicity @x25212 (= $x16339 (not $x24193))) (not $x24193))))
-(let ((@x25226 (unit-resolution (def-axiom (or (not $x24229) $x24193 $x24227)) @x25225 (unit-resolution ((_ quant-inst v_b_S_s$ (b_S_ptr$ b_T_T_u1$ ?x24124)) (or (not $x19790) $x24229)) @x19793 $x24229) $x24227)))
-(let ((@x25350 (monotonicity (symm (hypothesis $x23973) (= ?x23972 ?x3922)) (= $x24194 (b_S_typed$ v_b_S_s$ ?x3922)))))
-(let (($x3924 (b_S_typed$ v_b_S_s$ ?x3922)))
-(let ((?x23936 (b_S_select_o_tm$ ?x3874 ?x3922)))
-(let (($x24081 (b_S_ts_n_is_n_volatile$ ?x23936)))
-(let (($x16333 (not $x3924)))
-(let (($x24082 (or $x16333 $x24081)))
-(let (($x24083 (not $x24082)))
-(let (($x12397 (>= v_b_L_H_p_G_0$ 0)))
-(let (($x21173 (forall ((?v0 Int) )(!(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x3840 (= ?x3765 v_b_S_result_G_0$)))
-(let (($x12631 (>= (+ ?v0 (* (- 1) v_b_P_H_len$)) 0)))
-(let (($x14211 (<= ?v0 4294967295)))
-(let (($x17271 (not $x14211)))
-(let (($x10138 (>= ?v0 0)))
-(let (($x10556 (not $x10138)))
-(or $x10556 $x17271 $x12631 (not $x3840))))))))) :pattern ( (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$) )))
-))
-(let (($x21178 (not $x21173)))
-(let (($x21165 (forall ((?v0 Int) )(!(let ((?x12644 (* (- 1) v_b_S_result_G_0$)))
-(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x12646 (<= (+ ?x3765 ?x12644) 0)))
-(let (($x12631 (>= (+ ?v0 (* (- 1) v_b_P_H_len$)) 0)))
-(let (($x14211 (<= ?v0 4294967295)))
-(let (($x17271 (not $x14211)))
-(let (($x10138 (>= ?v0 0)))
-(let (($x10556 (not $x10138)))
-(or $x10556 $x17271 $x12631 $x12646))))))))) :pattern ( (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$) )))
-))
-(let (($x21181 (or (not $x21165) $x21178)))
-(let (($x21184 (not $x21181)))
-(let ((?x16481 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ ?x3680 ?v0!15 b_T_T_u1$))))
-(let (($x16760 (>= (+ v_b_S_result_G_0$ (* (- 1) ?x16481)) 0)))
-(let (($x16738 (<= (+ v_b_P_H_len$ (* (- 1) ?v0!15)) 0)))
-(let (($x16474 (<= ?v0!15 4294967295)))
-(let (($x20278 (not $x16474)))
-(let (($x16473 (>= ?v0!15 0)))
-(let (($x20277 (not $x16473)))
-(let (($x20293 (or $x20277 $x20278 $x16738 $x16760)))
-(let (($x20298 (not $x20293)))
-(let (($x21187 (or $x20298 $x21184)))
-(let (($x21190 (not $x21187)))
-(let (($x3824 (= v_b_S_result_G_0$ v_b_L_H_max_G_1$)))
-(let (($x20358 (not $x3824)))
-(let (($x12389 (>= v_b_SL_H_witness_G_0$ 0)))
-(let (($x20219 (not $x12389)))
-(let (($x12453 (<= (+ v_b_P_H_len$ (* (- 1) v_b_L_H_p_G_0$)) 0)))
-(let (($x12456 (not $x12453)))
-(let (($x21193 (or $x12456 $x20190 $x20219 (not (= v_b_L_H_max_G_4$ v_b_L_H_max_G_1$)) (not (= v_b_L_H_p_G_2$ v_b_L_H_p_G_0$)) (not (= v_b_SL_H_witness_G_2$ v_b_SL_H_witness_G_0$)) $x20358 $x21190)))
-(let (($x21196 (not $x21193)))
-(let (($x3993 (= v_b_L_H_max_G_3$ v_b_L_H_max_G_1$)))
-(let (($x20230 (not $x3993)))
-(let (($x12471 (>= (+ v_b_L_H_max_G_1$ (* (- 1) ?x3929)) 0)))
-(let (($x12476 (not $x12471)))
-(let (($x21123 (or $x20190 $x20219 $x12476 $x20230 (not (= v_b_SL_H_witness_G_1$ v_b_SL_H_witness_G_0$)) $x20173 $x21090)))
-(let (($x21126 (not $x21123)))
-(let (($x21099 (or $x16330 $x16339 $x21096)))
-(let (($x21102 (not $x21099)))
-(let (($x21105 (or $x16330 $x16333 $x21102)))
-(let (($x21108 (not $x21105)))
-(let (($x21111 (or $x16330 $x16333 $x21108)))
-(let (($x21114 (not $x21111)))
-(let (($x21117 (or $x20190 $x20219 $x12471 $x21114)))
-(let (($x21120 (not $x21117)))
-(let (($x21129 (or $x21120 $x21126)))
-(let (($x21132 (not $x21129)))
-(let (($x21135 (or $x16330 $x16339 $x20190 $x20219 $x21132)))
-(let (($x21138 (not $x21135)))
-(let (($x21141 (or $x16330 $x16339 $x21138)))
-(let (($x21144 (not $x21141)))
-(let (($x21147 (or $x16330 $x16333 $x21144)))
-(let (($x21150 (not $x21147)))
-(let (($x21153 (or $x16330 $x16333 $x21150)))
-(let (($x21156 (not $x21153)))
-(let (($x21159 (or $x20190 $x20219 $x12453 $x21156)))
-(let (($x21162 (not $x21159)))
-(let (($x21199 (or $x21162 $x21196)))
-(let (($x21202 (not $x21199)))
-(let ((?x991 (b_S_ptr_n_to$ b_T_T_u1$)))
-(let (($x3898 (b_S_local_n_value_n_is_n_ptr$ v_b_S_s$ b_H_tok_S_1_T_16_o_3$ b_H_loc_o_arr$ ?x3680 ?x991)))
-(let (($x3897 (b_S_local_n_value_n_is$ v_b_S_s$ b_H_tok_S_1_T_16_o_3$ b_H_loc_o_arr$ (b_S_ptr_n_to_n_int$ ?x3680) ?x991)))
-(let (($x3896 (b_S_local_n_value_n_is$ v_b_S_s$ b_H_tok_S_1_T_16_o_3$ b_H_loc_o_len$ v_b_P_H_len$ b_T_T_u4$)))
-(let (($x3895 (b_S_local_n_value_n_is$ v_b_S_s$ b_H_tok_S_1_T_16_o_3$ b_H_loc_o_max$ v_b_L_H_max_G_1$ b_T_T_u1$)))
-(let (($x3894 (b_S_local_n_value_n_is$ v_b_S_s$ b_H_tok_S_1_T_16_o_3$ b_H_loc_o_witness$ v_b_SL_H_witness_G_0$ b_T_T_u4$)))
-(let (($x3893 (b_S_local_n_value_n_is$ v_b_S_s$ b_H_tok_S_1_T_16_o_3$ b_H_loc_o_p$ v_b_L_H_p_G_0$ b_T_T_u4$)))
-(let ((?x3793 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ ?x3680 v_b_SL_H_witness_G_0$ b_T_T_u1$))))
-(let (($x3794 (= ?x3793 v_b_L_H_max_G_1$)))
-(let (($x20379 (not $x3794)))
-(let (($x12435 (<= (+ v_b_P_H_len$ (* (- 1) v_b_SL_H_witness_G_0$)) 0)))
-(let (($x21041 (forall ((?v0 Int) )(!(let ((?x12384 (* (- 1) v_b_L_H_max_G_1$)))
-(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x12425 (<= (+ ?x3765 ?x12384) 0)))
-(let (($x12411 (>= (+ ?v0 (* (- 1) v_b_L_H_p_G_0$)) 0)))
-(let (($x14211 (<= ?v0 4294967295)))
-(let (($x17271 (not $x14211)))
-(let (($x10138 (>= ?v0 0)))
-(let (($x10556 (not $x10138)))
-(or $x10556 $x17271 $x12411 $x12425))))))))) :pattern ( (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$) )))
-))
-(let (($x21046 (not $x21041)))
-(let (($x20375 (not $x12397)))
-(let (($x12834 (<= v_b_SL_H_witness_G_0$ 4294967295)))
-(let (($x20374 (not $x12834)))
-(let ((?x3746 (b_S_read_n_u1$ v_b_S_s$ ?x3739)))
-(let (($x3769 (= ?x3746 v_b_L_H_max_G_0$)))
-(let (($x16288 (not $x3769)))
-(let (($x8666 (<= v_b_P_H_len$ 0)))
-(let (($x21205 (or $x8666 $x16288 (not (>= v_b_L_H_max_G_1$ 0)) (not (<= v_b_L_H_max_G_1$ 255)) $x20374 $x20375 (not (<= v_b_L_H_p_G_0$ 4294967295)) (not (>= (+ v_b_P_H_len$ (* (- 1) v_b_L_H_p_G_0$)) 0)) $x21046 $x12435 $x20379 $x20190 $x20219 (not (b_S_call_n_transition$ v_b_S_s$ v_b_S_s$)) (not (b_S_good_n_state_n_ext$ b_H_tok_S_1_T_16_o_3$ v_b_S_s$)) (not $x3893) (not $x3894) (not $x3895) (not $x3896) (not $x3897) (not $x3898) $x21202)))
-(let (($x21208 (not $x21205)))
-(let (($x21211 (or $x8666 $x16288 $x21208)))
-(let (($x21214 (not $x21211)))
-(let (($x21033 (forall ((?v0 Int) )(!(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x12367 (>= (+ v_b_L_H_max_G_0$ (* (- 1) ?x3765)) 0)))
-(let (($x12354 (>= ?v0 1)))
-(let (($x14211 (<= ?v0 4294967295)))
-(let (($x17271 (not $x14211)))
-(let (($x10138 (>= ?v0 0)))
-(let (($x10556 (not $x10138)))
-(or $x10556 $x17271 $x12354 $x12367)))))))) :pattern ( (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$) )))
-))
-(let (($x21217 (or (not $x21033) $x21214)))
-(let (($x21220 (not $x21217)))
-(let ((?x16270 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ ?x3680 ?v0!13 b_T_T_u1$))))
-(let (($x16273 (>= (+ v_b_L_H_max_G_0$ (* (- 1) ?x16270)) 0)))
-(let (($x16265 (>= ?v0!13 1)))
-(let (($x20031 (or (not (>= ?v0!13 0)) (not (<= ?v0!13 4294967295)) $x16265 $x16273)))
-(let (($x20036 (not $x20031)))
-(let (($x21223 (or $x20036 $x21220)))
-(let (($x21226 (not $x21223)))
-(let (($x12348 (>= v_b_P_H_len$ 1)))
-(let (($x12351 (not $x12348)))
-(let (($x21229 (or $x12351 $x21226)))
-(let (($x21232 (not $x21229)))
-(let (($x8667 (not $x8666)))
-(let (($x3720 (<= v_b_P_H_len$ b_S_max_o_u4$)))
-(let (($x3719 (<= 0 v_b_P_H_len$)))
-(let (($x8707 (forall ((?v0 B_S_ptr$) )(!(let (($x3715 (b_S_in_n_writes_n_at$ v_b_H_wrTime_S_1_T_6_o_1$ ?v0)))
-(not $x3715)) :pattern ( (b_S_in_n_writes_n_at$ v_b_H_wrTime_S_1_T_6_o_1$ ?v0) )))
-))
-(let ((?x3713 (b_S_current_n_timestamp$ v_b_S_s$)))
-(let (($x3714 (= v_b_H_wrTime_S_1_T_6_o_1$ ?x3713)))
-(let (($x3711 (b_S_local_n_value_n_is$ v_b_S_s$ b_H_tok_S_1_T_6_o_1$ b_H_loc_o_len$ v_b_P_H_len$ b_T_T_u4$)))
-(let (($x3709 (b_S_local_n_value_n_is_n_ptr$ v_b_S_s$ b_H_tok_S_1_T_6_o_1$ b_H_loc_o_arr$ ?x3680 ?x991)))
-(let (($x3708 (b_S_local_n_value_n_is$ v_b_S_s$ b_H_tok_S_1_T_6_o_1$ b_H_loc_o_arr$ (b_S_ptr_n_to_n_int$ ?x3680) ?x991)))
-(let (($x8701 (forall ((?v0 B_S_pure_n_function$) )(!(not (<= b_S_current_n_frame_n_level$ (b_S_frame_n_level$ ?v0))) :pattern ( (b_S_frame_n_level$ ?v0) )))
-))
-(let (($x3699 (b_S_full_n_stop$ v_b_S_s$)))
-(let (($x3698 (b_S_good_n_state_n_ext$ b_H_tok_S_1_T_6_o_1$ v_b_S_s$)))
-(let (($x3697 (b_S_function_n_entry$ v_b_S_s$)))
-(let ((?x3678 (b_S_array$ b_T_T_u1$ v_b_P_H_len$)))
-(let (($x3691 (b_S_is_n_non_n_primitive$ ?x3678)))
-(let (($x3690 (not (= (b_S_kind_n_of$ ?x3678) b_S_kind_n_primitive$))))
-(let ((?x3682 (b_S_ptr$ ?x3678 ?x3681)))
-(let (($x3687 (b_S_typed$ v_b_S_s$ ?x3682)))
-(let (($x3686 (b_S_is$ ?x3682 ?x3678)))
-(let ((?x3684 (b_S_owner$ v_b_S_s$ ?x3682)))
-(let (($x3685 (= ?x3684 b_S_me$)))
-(let (($x3683 (b_S_closed$ v_b_S_s$ ?x3682)))
-(let (($x8657 (<= 1099511627776 v_b_P_H_len$)))
-(let (($x8658 (not $x8657)))
-(let (($x3672 (<= v_b_SL_H_witness$ b_S_max_o_u4$)))
-(let (($x3671 (<= 0 v_b_SL_H_witness$)))
-(let (($x3668 (<= v_b_L_H_p$ b_S_max_o_u4$)))
-(let (($x3667 (<= 0 v_b_L_H_p$)))
-(let (($x3663 (<= 0 v_b_L_H_max$)))
-(let (($x8820 (and $x3663 (<= v_b_L_H_max$ b_S_max_o_u1$) $x3667 $x3668 $x3671 $x3672 $x8658 $x8667 $x3683 $x3685 $x3686 $x3687 $x3690 $x3691 $x3697 $x3698 $x3699 $x8701 $x3708 $x3709 $x3711 $x3714 $x8707 $x3719 $x3720)))
-(let (($x9207 (exists ((?v0 Int) )(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x3840 (= ?x3765 v_b_S_result_G_0$)))
-(let (($x9165 (not (<= v_b_P_H_len$ ?v0))))
-(let (($x1344 (<= ?v0 b_S_max_o_u4$)))
-(let (($x1212 (<= 0 ?v0)))
-(and $x1212 $x1344 $x9165 $x3840)))))))
-))
-(let (($x9185 (forall ((?v0 Int) )(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x3837 (<= ?x3765 v_b_S_result_G_0$)))
-(let (($x9165 (not (<= v_b_P_H_len$ ?v0))))
-(let (($x1344 (<= ?v0 b_S_max_o_u4$)))
-(let (($x1212 (<= 0 ?v0)))
-(let (($x9171 (and $x1212 $x1344 $x9165)))
-(or (not $x9171) $x3837))))))))
-))
-(let (($x9228 (or (not $x9185) $x9207)))
-(let (($x9233 (and $x9185 $x9228)))
-(let (($x3822 (= v_b_SL_H_witness_G_2$ v_b_SL_H_witness_G_0$)))
-(let (($x3820 (= v_b_L_H_p_G_2$ v_b_L_H_p_G_0$)))
-(let (($x3818 (= v_b_L_H_max_G_4$ v_b_L_H_max_G_1$)))
-(let (($x3776 (<= 0 v_b_SL_H_witness_G_0$)))
-(let (($x3783 (<= 1 v_b_L_H_p_G_0$)))
-(let (($x9159 (and b_S_position_n_marker$ $x3783 $x3776 $x3818 $x3820 $x3822 $x3824)))
-(let (($x9240 (or (not $x9159) $x9233)))
-(let (($x9245 (and b_S_position_n_marker$ $x9240)))
-(let (($x9963 (or (not (and $x3783 $x3776 (<= v_b_P_H_len$ v_b_L_H_p_G_0$))) $x9245)))
-(let (($x9687 (not (<= v_b_P_H_len$ v_b_SL_H_witness_G_1$))))
-(let (($x9690 (and $x9687 $x3976)))
-(let (($x9683 (forall ((?v0 Int) )(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x3970 (<= ?x3765 v_b_L_H_max_G_3$)))
-(let (($x9663 (not (<= v_b_L_H_p_G_1$ ?v0))))
-(let (($x1344 (<= ?v0 b_S_max_o_u4$)))
-(let (($x1212 (<= 0 ?v0)))
-(let (($x9669 (and $x1212 $x1344 $x9663)))
-(or (not $x9669) $x3970))))))))
-))
-(let (($x9718 (or (not $x9683) $x9690)))
-(let (($x9723 (and $x9683 $x9718)))
-(let (($x9730 (or (not (<= v_b_L_H_p_G_1$ v_b_P_H_len$)) $x9723)))
-(let (($x3967 (<= v_b_L_H_p_G_1$ v_b_P_H_len$)))
-(let (($x9735 (and $x3967 $x9730)))
-(let (($x3943 (<= 0 v_b_SL_H_witness_G_1$)))
-(let (($x3961 (<= 2 v_b_L_H_p_G_1$)))
-(let ((?x9600 (+ 1 v_b_L_H_p_G_0$)))
-(let (($x9623 (= v_b_L_H_p_G_1$ ?x9600)))
-(let (($x9615 (<= v_b_L_H_p_G_0$ (+ (- 1) b_S_max_o_u4$))))
-(let (($x9606 (<= (- 1) v_b_L_H_p_G_0$)))
-(let (($x9657 (and $x9606 $x9615 $x9623 $x3960 $x3961 $x3943)))
-(let (($x9742 (or (not $x9657) $x9735)))
-(let (($x9750 (and $x9606 $x9615 $x9742)))
-(let (($x3994 (= v_b_SL_H_witness_G_1$ v_b_SL_H_witness_G_0$)))
-(let (($x3992 (<= ?x3929 v_b_L_H_max_G_1$)))
-(let (($x9858 (and $x3783 $x3776 $x3992 $x3993 $x3994 $x3943)))
-(let (($x9874 (or (not $x9858) $x9750)))
-(let (($x3942 (= v_b_SL_H_witness_G_1$ v_b_L_H_p_G_0$)))
-(let (($x3935 (= v_b_L_H_max_G_2$ ?x3929)))
-(let (($x9595 (and $x3923 $x3926 $x3935 $x3936 $x3937 $x3783 $x3940 $x3942 $x3943)))
-(let (($x9759 (or (not $x9595) $x9750)))
-(let (($x9767 (and $x3923 $x3926 $x9759)))
-(let (($x3925 (and $x3923 $x3924)))
-(let (($x9775 (not $x3925)))
-(let (($x9776 (or $x9775 $x9767)))
-(let (($x9784 (and $x3923 $x3924 $x9776)))
-(let (($x9793 (or (not (and $x3783 $x3776 (not $x3992))) $x9784)))
-(let (($x9879 (and $x9793 $x9874)))
-(let (($x9886 (or (not (and $x3923 $x3926 $x3783 $x3776)) $x9879)))
-(let (($x9894 (and $x3923 $x3926 $x9886)))
-(let (($x9902 (or $x9775 $x9894)))
-(let (($x9910 (and $x3923 $x3924 $x9902)))
-(let (($x9919 (or (not (and $x3783 $x3776 (not (<= v_b_P_H_len$ v_b_L_H_p_G_0$)))) $x9910)))
-(let (($x9968 (and $x9919 $x9963)))
-(let (($x3806 (b_S_good_n_state_n_ext$ b_H_tok_S_1_T_16_o_3$ v_b_S_s$)))
-(let (($x3886 (b_S_call_n_transition$ v_b_S_s$ v_b_S_s$)))
-(let (($x9434 (and $x3783 $x3776 $x3886 $x3806 $x3699 $x3893 $x3894 $x3895 $x3896 $x3897 $x3898)))
-(let (($x9974 (not $x9434)))
-(let (($x8960 (not (<= v_b_P_H_len$ v_b_SL_H_witness_G_0$))))
-(let (($x8956 (forall ((?v0 Int) )(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x3788 (<= ?x3765 v_b_L_H_max_G_1$)))
-(let (($x8936 (not (<= v_b_L_H_p_G_0$ ?v0))))
-(let (($x1344 (<= ?v0 b_S_max_o_u4$)))
-(let (($x1212 (<= 0 ?v0)))
-(let (($x8942 (and $x1212 $x1344 $x8936)))
-(or (not $x8942) $x3788))))))))
-))
-(let (($x3785 (<= v_b_L_H_p_G_0$ v_b_P_H_len$)))
-(let (($x3781 (<= v_b_L_H_p_G_0$ b_S_max_o_u4$)))
-(let (($x3780 (<= 0 v_b_L_H_p_G_0$)))
-(let (($x3777 (<= v_b_SL_H_witness_G_0$ b_S_max_o_u4$)))
-(let (($x3773 (<= v_b_L_H_max_G_1$ b_S_max_o_u1$)))
-(let (($x3772 (<= 0 v_b_L_H_max_G_1$)))
-(let (($x9032 (and $x8667 $x3769 $x3772 $x3773 $x3776 $x3777 $x3780 $x3781 $x3783 $x3785 $x8956 $x8960 $x3794)))
-(let (($x9991 (or (not $x9032) $x9974 $x9968)))
-(let (($x9999 (and $x8667 $x3769 $x9991)))
-(let (($x8913 (forall ((?v0 Int) )(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x3766 (<= ?x3765 v_b_L_H_max_G_0$)))
-(let (($x8887 (<= 1 ?v0)))
-(let (($x8888 (not $x8887)))
-(let (($x1344 (<= ?v0 b_S_max_o_u4$)))
-(let (($x1212 (<= 0 ?v0)))
-(let (($x8899 (and $x1212 $x1344 $x8888)))
-(or (not $x8899) $x3766)))))))))
-))
-(let (($x10008 (or (not $x8913) $x9999)))
-(let (($x10013 (and $x8913 $x10008)))
-(let (($x10020 (or (not (<= 1 v_b_P_H_len$)) $x10013)))
-(let (($x3761 (<= 1 v_b_P_H_len$)))
-(let (($x10025 (and $x3761 $x10020)))
-(let (($x3750 (b_S_local_n_value_n_is$ v_b_S_s$ b_H_tok_S_1_T_16_o_8$ b_H_loc_o_p$ 1 b_T_T_u4$)))
-(let (($x3749 (b_S_local_n_value_n_is$ v_b_S_s$ b_H_tok_S_1_T_14_o_3$ b_H_loc_o_witness$ 0 b_T_T_u4$)))
-(let (($x3748 (b_S_local_n_value_n_is$ v_b_S_s$ b_H_tok_S_1_T_12_o_3$ b_H_loc_o_max$ v_b_L_H_max_G_0$ b_T_T_u1$)))
-(let (($x3747 (= v_b_L_H_max_G_0$ ?x3746)))
-(let (($x3743 (b_S_thread_n_local$ v_b_S_s$ ?x3739)))
-(let (($x8880 (and $x3740 $x3743 $x3747 $x3748 $x3749 $x3750)))
-(let (($x10031 (not $x8880)))
-(let (($x10032 (or $x10031 $x10025)))
-(let (($x10040 (and $x3740 $x3743 $x10032)))
-(let (($x3741 (b_S_typed$ v_b_S_s$ ?x3739)))
-(let (($x3742 (and $x3740 $x3741)))
-(let (($x10048 (not $x3742)))
-(let (($x10049 (or $x10048 $x10040)))
-(let (($x10057 (and $x3740 $x3741 $x10049)))
-(let (($x3738 (b_S_in_n_domain_n_lab$ v_b_S_s$ ?x3682 ?x3682 b_l_H_public$)))
-(let (($x10065 (not $x3738)))
-(let (($x10066 (or $x10065 $x10057)))
-(let (($x10071 (and $x3738 $x10066)))
-(let (($x10078 (or (not $x8820) $x10071)))
-(let (($x3844 (exists ((?v0 Int) )(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x3840 (= ?x3765 v_b_S_result_G_0$)))
-(let (($x3835 (< ?v0 v_b_P_H_len$)))
-(let (($x1344 (<= ?v0 b_S_max_o_u4$)))
-(let (($x3842 (and $x1344 (and $x3835 $x3840))))
-(let (($x1212 (<= 0 ?v0)))
-(and $x1212 $x3842))))))))
-))
-(let (($x3845 (=> $x3844 true)))
-(let (($x3846 (and $x3844 $x3845)))
-(let (($x3839 (forall ((?v0 Int) )(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x3837 (<= ?x3765 v_b_S_result_G_0$)))
-(let (($x3835 (< ?v0 v_b_P_H_len$)))
-(let (($x1344 (<= ?v0 b_S_max_o_u4$)))
-(let (($x1212 (<= 0 ?v0)))
-(let (($x1345 (and $x1212 $x1344)))
-(let (($x3836 (and $x1345 $x3835)))
-(=> $x3836 $x3837)))))))))
-))
-(let (($x3847 (=> $x3839 $x3846)))
-(let (($x3827 (and $x3820 (and $x3822 (and $x3824 true)))))
-(let (($x3828 (and $x3818 $x3827)))
-(let (($x3829 (and true $x3828)))
-(let (($x3784 (and $x3783 $x3776)))
-(let (($x3830 (and $x3784 $x3829)))
-(let (($x3831 (and $x3784 $x3830)))
-(let (($x3832 (and true $x3831)))
-(let (($x3833 (and $x3784 $x3832)))
-(let (($x3834 (and b_S_position_n_marker$ $x3833)))
-(let (($x3849 (=> $x3834 (and $x3839 $x3847))))
-(let (($x3850 (and b_S_position_n_marker$ $x3849)))
-(let (($x3808 (and true $x3784)))
-(let (($x3809 (and $x3784 $x3808)))
-(let (($x4013 (and $x3784 $x3809)))
-(let (($x4014 (and true $x4013)))
-(let (($x4015 (and $x3784 $x4014)))
-(let (($x4012 (<= v_b_P_H_len$ v_b_L_H_p_G_0$)))
-(let (($x4016 (and $x4012 $x4015)))
-(let (($x4017 (and $x3784 $x4016)))
-(let (($x4018 (and true $x4017)))
-(let (($x4019 (=> $x4018 $x3850)))
-(let (($x3977 (and (< v_b_SL_H_witness_G_1$ v_b_P_H_len$) $x3976)))
-(let (($x3978 (and $x3977 false)))
-(let (($x3979 (=> $x3978 true)))
-(let (($x3980 (and $x3977 $x3979)))
-(let (($x3972 (forall ((?v0 Int) )(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x3970 (<= ?x3765 v_b_L_H_max_G_3$)))
-(let (($x1344 (<= ?v0 b_S_max_o_u4$)))
-(let (($x1212 (<= 0 ?v0)))
-(let (($x1345 (and $x1212 $x1344)))
-(let (($x3969 (and $x1345 (< ?v0 v_b_L_H_p_G_1$))))
-(=> $x3969 $x3970))))))))
-))
-(let (($x3981 (=> $x3972 $x3980)))
-(let (($x3983 (=> $x3967 (and $x3972 $x3981))))
-(let (($x3962 (and $x3961 $x3943)))
-(let (($x3963 (and $x3962 true)))
-(let (($x3964 (and $x3960 $x3963)))
-(let (($x3965 (and (= v_b_L_H_p_G_1$ (+ v_b_L_H_p_G_0$ 1)) $x3964)))
-(let ((?x3954 (+ v_b_L_H_p_G_0$ 1)))
-(let (($x3956 (<= ?x3954 b_S_max_o_u4$)))
-(let (($x3955 (<= 0 ?x3954)))
-(let (($x3957 (and $x3955 $x3956)))
-(let (($x3966 (and $x3957 $x3965)))
-(let (($x3985 (=> $x3966 (and $x3967 $x3983))))
-(let (($x3986 (and $x3957 $x3985)))
-(let (($x3944 (and $x3783 $x3943)))
-(let (($x3945 (and true $x3944)))
-(let (($x3995 (and $x3994 $x3945)))
-(let (($x3996 (and $x3993 $x3995)))
-(let (($x3997 (and true $x3996)))
-(let (($x3998 (and $x3784 $x3997)))
-(let (($x3999 (and $x3784 $x3998)))
-(let (($x4000 (and true $x3999)))
-(let (($x4001 (and $x3784 $x4000)))
-(let (($x4002 (and $x3992 $x4001)))
-(let (($x4003 (and $x3784 $x4002)))
-(let (($x4004 (and true $x4003)))
-(let (($x4005 (=> $x4004 $x3986)))
-(let (($x3946 (and $x3942 $x3945)))
-(let (($x3947 (and $x3940 $x3946)))
-(let (($x3948 (and true $x3947)))
-(let (($x3938 (and $x3783 $x3783)))
-(let (($x3949 (and $x3938 $x3948)))
-(let (($x3950 (and $x3937 $x3949)))
-(let (($x3951 (and $x3936 $x3950)))
-(let (($x3952 (and $x3935 $x3951)))
-(let (($x3927 (and $x3923 $x3926)))
-(let (($x3953 (and $x3927 $x3952)))
-(let (($x3987 (=> $x3953 $x3986)))
-(let (($x3988 (and $x3927 $x3987)))
-(let (($x3989 (=> $x3925 $x3988)))
-(let (($x3990 (and $x3925 $x3989)))
-(let (($x3931 (and (< v_b_L_H_max_G_1$ ?x3929) $x3809)))
-(let (($x3932 (and $x3784 $x3931)))
-(let (($x3933 (and true $x3932)))
-(let (($x3991 (=> $x3933 $x3990)))
-(let (($x3928 (and $x3927 $x3784)))
-(let (($x4007 (=> $x3928 (and $x3991 $x4005))))
-(let (($x4008 (and $x3927 $x4007)))
-(let (($x4009 (=> $x3925 $x4008)))
-(let (($x4010 (and $x3925 $x4009)))
-(let (($x3919 (and (< v_b_L_H_p_G_0$ v_b_P_H_len$) $x3809)))
-(let (($x3920 (and $x3784 $x3919)))
-(let (($x3921 (and true $x3920)))
-(let (($x4011 (=> $x3921 $x4010)))
-(let (($x3902 (and (= ?x3874 ?x3874) (= (b_S_statusmap$ v_b_S_s$) (b_S_statusmap$ v_b_S_s$)))))
-(let (($x3903 (and $x3902 $x3784)))
-(let (($x3904 (and (and $x3897 $x3898) $x3903)))
-(let (($x3905 (and $x3896 $x3904)))
-(let (($x3906 (and $x3895 $x3905)))
-(let (($x3907 (and $x3894 $x3906)))
-(let (($x3908 (and $x3893 $x3907)))
-(let (($x3807 (and $x3806 $x3699)))
-(let (($x3909 (and $x3807 $x3908)))
-(let (($x3885 (forall ((?v0 B_S_ptr$) )(!(let ((?x3882 (b_S_timestamp$ v_b_S_s$ ?v0)))
-(<= ?x3882 ?x3882)) :pattern ( (b_S_timestamp$ v_b_S_s$ ?v0) )))
-))
-(let (($x3887 (and $x3885 $x3886)))
-(let (($x3888 (and (<= ?x3713 ?x3713) $x3887)))
-(let (($x3910 (and $x3888 $x3909)))
-(let (($x3880 (forall ((?v0 B_S_ptr$) )(!(let (($x3862 (b_S_thread_n_local$ v_b_S_s$ ?v0)))
-(let ((?x3874 (b_S_typemap$ v_b_S_s$)))
-(let ((?x3875 (b_S_select_o_tm$ ?x3874 ?v0)))
-(let (($x3877 (and (= ?x3875 ?x3875) $x3862)))
-(=> $x3862 $x3877))))) :pattern ( (b_S_select_o_tm$ (b_S_typemap$ v_b_S_s$) ?v0) )))
-))
-(let (($x3889 (and $x3880 $x3888)))
-(let (($x3873 (forall ((?v0 B_S_ptr$) )(!(let (($x3862 (b_S_thread_n_local$ v_b_S_s$ ?v0)))
-(let ((?x3858 (b_S_statusmap$ v_b_S_s$)))
-(let ((?x3859 (b_S_select_o_sm$ ?x3858 ?v0)))
-(let (($x3871 (and (= ?x3859 ?x3859) $x3862)))
-(=> $x3862 $x3871))))) :pattern ( (b_S_select_o_sm$ (b_S_statusmap$ v_b_S_s$) ?v0) )))
-))
-(let (($x3890 (and $x3873 $x3889)))
-(let (($x3869 (forall ((?v0 B_S_ptr$) )(!(let (($x3862 (b_S_thread_n_local$ v_b_S_s$ ?v0)))
-(let ((?x3864 (b_S_select_o_mem$ (b_S_memory$ v_b_S_s$) ?v0)))
-(let (($x3866 (and (= ?x3864 ?x3864) $x3862)))
-(=> $x3862 $x3866)))) :pattern ( (b_S_select_o_mem$ (b_S_memory$ v_b_S_s$) ?v0) )))
-))
-(let (($x3891 (and $x3869 $x3890)))
-(let (($x3861 (forall ((?v0 B_S_ptr$) )(!(let (($x3855 (= (b_S_kind_n_of$ (b_S_typ$ (b_S_owner$ v_b_S_s$ ?v0))) b_S_kind_n_thread$)))
-(=> (not $x3855) (not $x3855))) :pattern ( (b_S_select_o_sm$ (b_S_statusmap$ v_b_S_s$) ?v0) )))
-))
-(let (($x3892 (and $x3861 $x3891)))
-(let (($x3911 (and $x3892 $x3910)))
-(let (($x3912 (and $x3784 $x3911)))
-(let (($x3913 (and true $x3912)))
-(let (($x3914 (and $x3784 $x3913)))
-(let (($x3915 (and true $x3914)))
-(let (($x3916 (and $x3784 $x3915)))
-(let (($x3917 (and true $x3916)))
-(let (($x4021 (=> $x3917 (and $x4011 $x4019))))
-(let (($x3810 (and $x3807 $x3809)))
-(let (($x3811 (and $x3784 $x3810)))
-(let (($x3812 (and true $x3811)))
-(let (($x3813 (and $x3784 $x3812)))
-(let (($x3805 (not true)))
-(let (($x3814 (and $x3805 $x3813)))
-(let (($x3815 (and $x3784 $x3814)))
-(let (($x3816 (and true $x3815)))
-(let (($x3851 (=> $x3816 $x3850)))
-(let (($x4022 (and $x3851 $x4021)))
-(let (($x3796 (and (and (< v_b_SL_H_witness_G_0$ v_b_P_H_len$) $x3794) $x3784)))
-(let (($x3790 (forall ((?v0 Int) )(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x3788 (<= ?x3765 v_b_L_H_max_G_1$)))
-(let (($x1344 (<= ?v0 b_S_max_o_u4$)))
-(let (($x1212 (<= 0 ?v0)))
-(let (($x1345 (and $x1212 $x1344)))
-(let (($x3787 (and $x1345 (< ?v0 v_b_L_H_p_G_0$))))
-(=> $x3787 $x3788))))))))
-))
-(let (($x3797 (and $x3790 $x3796)))
-(let (($x3798 (and $x3785 $x3797)))
-(let (($x3799 (and $x3784 $x3798)))
-(let (($x3782 (and $x3780 $x3781)))
-(let (($x3800 (and $x3782 $x3799)))
-(let (($x3778 (and $x3776 $x3777)))
-(let (($x3801 (and $x3778 $x3800)))
-(let (($x3774 (and $x3772 $x3773)))
-(let (($x3802 (and $x3774 $x3801)))
-(let (($x3803 (and true $x3802)))
-(let (($x3676 (< 0 v_b_P_H_len$)))
-(let (($x3770 (and $x3676 $x3769)))
-(let (($x3804 (and $x3770 $x3803)))
-(let (($x4023 (=> $x3804 $x4022)))
-(let (($x4024 (and $x3770 $x4023)))
-(let (($x3768 (forall ((?v0 Int) )(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x3766 (<= ?x3765 v_b_L_H_max_G_0$)))
-(let (($x1344 (<= ?v0 b_S_max_o_u4$)))
-(let (($x1212 (<= 0 ?v0)))
-(let (($x1345 (and $x1212 $x1344)))
-(let (($x3763 (and $x1345 (< ?v0 1))))
-(=> $x3763 $x3766))))))))
-))
-(let (($x4025 (=> $x3768 $x4024)))
-(let (($x4027 (=> $x3761 (and $x3768 $x4025))))
-(let (($x3752 (<= 0 0)))
-(let (($x3753 (and $x3752 $x3752)))
-(let (($x3751 (<= 1 1)))
-(let (($x3754 (and $x3751 $x3753)))
-(let (($x3755 (and $x3751 $x3754)))
-(let (($x3756 (and $x3750 $x3755)))
-(let (($x3758 (and $x3748 (and $x3749 $x3756))))
-(let (($x3759 (and $x3747 $x3758)))
-(let (($x3744 (and $x3740 $x3743)))
-(let (($x3760 (and $x3744 $x3759)))
-(let (($x4029 (=> $x3760 (and $x3761 $x4027))))
-(let (($x4030 (and $x3744 $x4029)))
-(let (($x4031 (=> $x3742 $x4030)))
-(let (($x4032 (and $x3742 $x4031)))
-(let (($x4033 (=> $x3738 $x4032)))
-(let (($x3721 (and $x3719 $x3720)))
-(let (($x3718 (forall ((?v0 B_S_ptr$) )(!(let (($x3715 (b_S_in_n_writes_n_at$ v_b_H_wrTime_S_1_T_6_o_1$ ?v0)))
-(= $x3715 false)) :pattern ( (b_S_in_n_writes_n_at$ v_b_H_wrTime_S_1_T_6_o_1$ ?v0) )))
-))
-(let (($x3722 (and $x3718 $x3721)))
-(let (($x3723 (and $x3714 $x3722)))
-(let (($x3724 (and $x3711 $x3723)))
-(let (($x3725 (and (and $x3708 $x3709) $x3724)))
-(let (($x3706 (forall ((?v0 B_S_pure_n_function$) )(!(let ((?x3702 (b_S_frame_n_level$ ?v0)))
-(< ?x3702 b_S_current_n_frame_n_level$)) :pattern ( (b_S_frame_n_level$ ?v0) )))
-))
-(let (($x3726 (and $x3706 $x3725)))
-(let (($x3727 (and (and $x3698 $x3699) $x3726)))
-(let (($x3728 (and $x3697 $x3727)))
-(let (($x3729 (and true $x3728)))
-(let (($x3694 (and $x3686 (and $x3687 (and $x3690 $x3691)))))
-(let (($x3695 (and $x3685 $x3694)))
-(let (($x3696 (and $x3683 $x3695)))
-(let (($x3730 (and $x3696 $x3729)))
-(let (($x3731 (and $x3676 $x3730)))
-(let (($x3732 (and (< v_b_P_H_len$ 1099511627776) $x3731)))
-(let (($x3673 (and $x3671 $x3672)))
-(let (($x3733 (and $x3673 $x3732)))
-(let (($x3669 (and $x3667 $x3668)))
-(let (($x3734 (and $x3669 $x3733)))
-(let (($x3665 (and $x3663 (<= v_b_L_H_max$ b_S_max_o_u1$))))
-(let (($x3735 (and $x3665 $x3734)))
-(let (($x3736 (and true $x3735)))
-(let (($x4035 (=> $x3736 (and $x3738 $x4033))))
-(let (($x4036 (not $x4035)))
-(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ ?x3680 ?0 b_T_T_u1$))))
-(let (($x3840 (= ?x3765 v_b_S_result_G_0$)))
-(let (($x9165 (not (<= v_b_P_H_len$ ?0))))
-(let (($x1344 (<= ?0 b_S_max_o_u4$)))
-(let (($x1212 (<= 0 ?0)))
-(let (($x9202 (and $x1212 $x1344 $x9165 $x3840)))
-(let (($x3842 (and $x1344 (and (< ?0 v_b_P_H_len$) $x3840))))
-(let (($x3843 (and $x1212 $x3842)))
-(let ((@x9190 (monotonicity (rewrite (= (< ?0 v_b_P_H_len$) $x9165)) (= (and (< ?0 v_b_P_H_len$) $x3840) (and $x9165 $x3840)))))
-(let ((@x9198 (trans (monotonicity @x9190 (= $x3842 (and $x1344 (and $x9165 $x3840)))) (rewrite (= (and $x1344 (and $x9165 $x3840)) (and $x1344 $x9165 $x3840))) (= $x3842 (and $x1344 $x9165 $x3840)))))
-(let ((@x5396 (rewrite (= $x1212 $x1212))))
-(let ((@x9206 (trans (monotonicity @x5396 @x9198 (= $x3843 (and $x1212 (and $x1344 $x9165 $x3840)))) (rewrite (= (and $x1212 (and $x1344 $x9165 $x3840)) $x9202)) (= $x3843 $x9202))))
-(let ((@x9212 (monotonicity (quant-intro @x9206 (= $x3844 $x9207)) (= $x3845 (=> $x9207 true)))))
-(let ((@x9216 (trans @x9212 (rewrite (= (=> $x9207 true) true)) (= $x3845 true))))
-(let ((@x9219 (monotonicity (quant-intro @x9206 (= $x3844 $x9207)) @x9216 (= $x3846 (and $x9207 true)))))
-(let (($x3837 (<= ?x3765 v_b_S_result_G_0$)))
-(let (($x9180 (or (not (and $x1212 $x1344 $x9165)) $x3837)))
-(let (($x3835 (< ?0 v_b_P_H_len$)))
-(let (($x1345 (and $x1212 $x1344)))
-(let (($x3836 (and $x1345 $x3835)))
-(let (($x3838 (=> $x3836 $x3837)))
-(let ((@x5523 (monotonicity @x5396 (= $x1345 $x1345))))
-(let ((@x9170 (monotonicity @x5523 (rewrite (= $x3835 $x9165)) (= $x3836 (and $x1345 $x9165)))))
-(let ((@x9175 (trans @x9170 (rewrite (= (and $x1345 $x9165) (and $x1212 $x1344 $x9165))) (= $x3836 (and $x1212 $x1344 $x9165)))))
-(let ((@x9184 (trans (monotonicity @x9175 (= $x3838 (=> (and $x1212 $x1344 $x9165) $x3837))) (rewrite (= (=> (and $x1212 $x1344 $x9165) $x3837) $x9180)) (= $x3838 $x9180))))
-(let ((@x9226 (monotonicity (quant-intro @x9184 (= $x3839 $x9185)) (trans @x9219 (rewrite (= (and $x9207 true) $x9207)) (= $x3846 $x9207)) (= $x3847 (=> $x9185 $x9207)))))
-(let ((@x9235 (monotonicity (quant-intro @x9184 (= $x3839 $x9185)) (trans @x9226 (rewrite (= (=> $x9185 $x9207) $x9228)) (= $x3847 $x9228)) (= (and $x3839 $x3847) $x9233))))
-(let (($x9160 (= (and b_S_position_n_marker$ (and $x3783 $x3776 $x3818 $x3820 $x3822 $x3824)) $x9159)))
-(let (($x9157 (= $x3834 (and b_S_position_n_marker$ (and $x3783 $x3776 $x3818 $x3820 $x3822 $x3824)))))
-(let (($x9133 (and $x3783 $x3776 $x3818 $x3820 $x3822 $x3824)))
-(let (($x9138 (and $x3784 $x9133)))
-(let (($x9118 (and $x3818 $x3820 $x3822 $x3824)))
-(let ((@x9106 (monotonicity (rewrite (= (and $x3824 true) $x3824)) (= (and $x3822 (and $x3824 true)) (and $x3822 $x3824)))))
-(let ((@x9114 (trans (monotonicity @x9106 (= $x3827 (and $x3820 (and $x3822 $x3824)))) (rewrite (= (and $x3820 (and $x3822 $x3824)) (and $x3820 $x3822 $x3824))) (= $x3827 (and $x3820 $x3822 $x3824)))))
-(let ((@x9122 (trans (monotonicity @x9114 (= $x3828 (and $x3818 (and $x3820 $x3822 $x3824)))) (rewrite (= (and $x3818 (and $x3820 $x3822 $x3824)) $x9118)) (= $x3828 $x9118))))
-(let ((@x9129 (trans (monotonicity @x9122 (= $x3829 (and true $x9118))) (rewrite (= (and true $x9118) $x9118)) (= $x3829 $x9118))))
-(let ((@x8932 (rewrite (= $x3783 $x3783))))
-(let ((@x8934 (monotonicity @x8932 (rewrite (= $x3776 $x3776)) (= $x3784 $x3784))))
-(let ((@x9137 (trans (monotonicity @x8934 @x9129 (= $x3830 (and $x3784 $x9118))) (rewrite (= (and $x3784 $x9118) $x9133)) (= $x3830 $x9133))))
-(let ((@x9144 (trans (monotonicity @x8934 @x9137 (= $x3831 $x9138)) (rewrite (= $x9138 $x9133)) (= $x3831 $x9133))))
-(let ((@x9151 (trans (monotonicity @x9144 (= $x3832 (and true $x9133))) (rewrite (= (and true $x9133) $x9133)) (= $x3832 $x9133))))
-(let ((@x9155 (trans (monotonicity @x8934 @x9151 (= $x3833 $x9138)) (rewrite (= $x9138 $x9133)) (= $x3833 $x9133))))
-(let ((@x9238 (monotonicity (trans (monotonicity @x9155 $x9157) (rewrite $x9160) (= $x3834 $x9159)) @x9235 (= $x3849 (=> $x9159 $x9233)))))
-(let ((@x9247 (monotonicity (trans @x9238 (rewrite (= (=> $x9159 $x9233) $x9240)) (= $x3849 $x9240)) (= $x3850 $x9245))))
-(let ((@x9956 (rewrite (= (and true (and $x3783 $x3776 $x4012)) (and $x3783 $x3776 $x4012)))))
-(let ((@x9048 (rewrite (= (and $x3784 $x3784) $x3784))))
-(let ((@x9042 (rewrite (= $x3808 $x3784))))
-(let ((@x9046 (monotonicity @x8934 (trans (monotonicity @x8934 (= $x3808 $x3808)) @x9042 (= $x3808 $x3784)) (= $x3809 (and $x3784 $x3784)))))
-(let ((@x9050 (trans @x9046 @x9048 (= $x3809 $x3784))))
-(let ((@x9927 (trans (monotonicity @x8934 @x9050 (= $x4013 (and $x3784 $x3784))) @x9048 (= $x4013 $x3784))))
-(let ((@x9933 (monotonicity @x8934 (trans (monotonicity @x9927 (= $x4014 $x3808)) @x9042 (= $x4014 $x3784)) (= $x4015 (and $x3784 $x3784)))))
-(let ((@x9938 (monotonicity (trans @x9933 @x9048 (= $x4015 $x3784)) (= $x4016 (and $x4012 $x3784)))))
-(let ((@x9943 (trans @x9938 (rewrite (= (and $x4012 $x3784) (and $x4012 $x3783 $x3776))) (= $x4016 (and $x4012 $x3783 $x3776)))))
-(let ((@x9951 (trans (monotonicity @x8934 @x9943 (= $x4017 (and $x3784 (and $x4012 $x3783 $x3776)))) (rewrite (= (and $x3784 (and $x4012 $x3783 $x3776)) (and $x3783 $x3776 $x4012))) (= $x4017 (and $x3783 $x3776 $x4012)))))
-(let ((@x9958 (trans (monotonicity @x9951 (= $x4018 (and true (and $x3783 $x3776 $x4012)))) @x9956 (= $x4018 (and $x3783 $x3776 $x4012)))))
-(let ((@x9967 (trans (monotonicity @x9958 @x9247 (= $x4019 (=> (and $x3783 $x3776 $x4012) $x9245))) (rewrite (= (=> (and $x3783 $x3776 $x4012) $x9245) $x9963)) (= $x4019 $x9963))))
-(let ((@x9692 (monotonicity (rewrite (= (< v_b_SL_H_witness_G_1$ v_b_P_H_len$) $x9687)) (= $x3977 $x9690))))
-(let ((@x9699 (trans (monotonicity @x9692 (= $x3978 (and $x9690 false))) (rewrite (= (and $x9690 false) false)) (= $x3978 false))))
-(let ((@x9706 (trans (monotonicity @x9699 (= $x3979 (=> false true))) (rewrite (= (=> false true) true)) (= $x3979 true))))
-(let ((@x9713 (trans (monotonicity @x9692 @x9706 (= $x3980 (and $x9690 true))) (rewrite (= (and $x9690 true) $x9690)) (= $x3980 $x9690))))
-(let (($x3970 (<= ?x3765 v_b_L_H_max_G_3$)))
-(let (($x9678 (or (not (and $x1212 $x1344 (not (<= v_b_L_H_p_G_1$ ?0)))) $x3970)))
-(let (($x3969 (and $x1345 (< ?0 v_b_L_H_p_G_1$))))
-(let (($x3971 (=> $x3969 $x3970)))
-(let ((@x9680 (rewrite (= (=> (and $x1212 $x1344 (not (<= v_b_L_H_p_G_1$ ?0))) $x3970) $x9678))))
-(let (($x9663 (not (<= v_b_L_H_p_G_1$ ?0))))
-(let (($x9669 (and $x1212 $x1344 $x9663)))
-(let ((@x9668 (monotonicity @x5523 (rewrite (= (< ?0 v_b_L_H_p_G_1$) $x9663)) (= $x3969 (and $x1345 $x9663)))))
-(let ((@x9676 (monotonicity (trans @x9668 (rewrite (= (and $x1345 $x9663) $x9669)) (= $x3969 $x9669)) (= $x3971 (=> $x9669 $x3970)))))
-(let ((@x9716 (monotonicity (quant-intro (trans @x9676 @x9680 (= $x3971 $x9678)) (= $x3972 $x9683)) @x9713 (= $x3981 (=> $x9683 $x9690)))))
-(let ((@x9725 (monotonicity (quant-intro (trans @x9676 @x9680 (= $x3971 $x9678)) (= $x3972 $x9683)) (trans @x9716 (rewrite (= (=> $x9683 $x9690) $x9718)) (= $x3981 $x9718)) (= (and $x3972 $x3981) $x9723))))
-(let ((@x9734 (trans (monotonicity @x9725 (= $x3983 (=> $x3967 $x9723))) (rewrite (= (=> $x3967 $x9723) $x9730)) (= $x3983 $x9730))))
-(let ((@x9651 (rewrite (= (and $x9623 (and $x3960 $x3961 $x3943)) (and $x9623 $x3960 $x3961 $x3943)))))
-(let ((@x9632 (monotonicity (rewrite (= $x3961 $x3961)) (rewrite (= $x3943 $x3943)) (= $x3962 $x3962))))
-(let ((@x9637 (trans (monotonicity @x9632 (= $x3963 $x3963)) (rewrite (= $x3963 $x3962)) (= $x3963 $x3962))))
-(let ((@x9645 (trans (monotonicity @x9637 (= $x3964 (and $x3960 $x3962))) (rewrite (= (and $x3960 $x3962) (and $x3960 $x3961 $x3943))) (= $x3964 (and $x3960 $x3961 $x3943)))))
-(let ((@x9602 (rewrite (= ?x3954 ?x9600))))
-(let ((@x9628 (trans (monotonicity @x9602 (= (= v_b_L_H_p_G_1$ ?x3954) $x9623)) (rewrite (= $x9623 $x9623)) (= (= v_b_L_H_p_G_1$ ?x3954) $x9623))))
-(let ((@x9653 (trans (monotonicity @x9628 @x9645 (= $x3965 (and $x9623 (and $x3960 $x3961 $x3943)))) @x9651 (= $x3965 (and $x9623 $x3960 $x3961 $x3943)))))
-(let ((@x9619 (trans (monotonicity @x9602 (= $x3956 (<= ?x9600 b_S_max_o_u4$))) (rewrite (= (<= ?x9600 b_S_max_o_u4$) $x9615)) (= $x3956 $x9615))))
-(let ((@x9610 (trans (monotonicity @x9602 (= $x3955 (<= 0 ?x9600))) (rewrite (= (<= 0 ?x9600) $x9606)) (= $x3955 $x9606))))
-(let ((@x9656 (monotonicity (monotonicity @x9610 @x9619 (= $x3957 (and $x9606 $x9615))) @x9653 (= $x3966 (and (and $x9606 $x9615) (and $x9623 $x3960 $x3961 $x3943))))))
-(let ((@x9661 (trans @x9656 (rewrite (= (and (and $x9606 $x9615) (and $x9623 $x3960 $x3961 $x3943)) $x9657)) (= $x3966 $x9657))))
-(let ((@x9740 (monotonicity @x9661 (monotonicity @x9734 (= (and $x3967 $x3983) $x9735)) (= $x3985 (=> $x9657 $x9735)))))
-(let ((@x9749 (monotonicity (monotonicity @x9610 @x9619 (= $x3957 (and $x9606 $x9615))) (trans @x9740 (rewrite (= (=> $x9657 $x9735) $x9742)) (= $x3985 $x9742)) (= $x3986 (and (and $x9606 $x9615) $x9742)))))
-(let ((@x9754 (trans @x9749 (rewrite (= (and (and $x9606 $x9615) $x9742) $x9750)) (= $x3986 $x9750))))
-(let (($x9850 (and $x3992 $x3783 $x3776 $x3993 $x3994 $x3943)))
-(let (($x9824 (and $x3783 $x3776 $x3993 $x3994 $x3943)))
-(let (($x9829 (and $x3784 $x9824)))
-(let (($x9809 (and $x3993 $x3994 $x3783 $x3943)))
-(let ((@x9533 (monotonicity (monotonicity @x8932 (rewrite (= $x3943 $x3943)) (= $x3944 $x3944)) (= $x3945 $x3945))))
-(let ((@x9800 (monotonicity (trans @x9533 (rewrite (= $x3945 $x3944)) (= $x3945 $x3944)) (= $x3995 (and $x3994 $x3944)))))
-(let ((@x9805 (trans @x9800 (rewrite (= (and $x3994 $x3944) (and $x3994 $x3783 $x3943))) (= $x3995 (and $x3994 $x3783 $x3943)))))
-(let ((@x9813 (trans (monotonicity @x9805 (= $x3996 (and $x3993 (and $x3994 $x3783 $x3943)))) (rewrite (= (and $x3993 (and $x3994 $x3783 $x3943)) $x9809)) (= $x3996 $x9809))))
-(let ((@x9820 (trans (monotonicity @x9813 (= $x3997 (and true $x9809))) (rewrite (= (and true $x9809) $x9809)) (= $x3997 $x9809))))
-(let ((@x9828 (trans (monotonicity @x8934 @x9820 (= $x3998 (and $x3784 $x9809))) (rewrite (= (and $x3784 $x9809) $x9824)) (= $x3998 $x9824))))
-(let ((@x9835 (trans (monotonicity @x8934 @x9828 (= $x3999 $x9829)) (rewrite (= $x9829 $x9824)) (= $x3999 $x9824))))
-(let ((@x9842 (trans (monotonicity @x9835 (= $x4000 (and true $x9824))) (rewrite (= (and true $x9824) $x9824)) (= $x4000 $x9824))))
-(let ((@x9846 (trans (monotonicity @x8934 @x9842 (= $x4001 $x9829)) (rewrite (= $x9829 $x9824)) (= $x4001 $x9824))))
-(let ((@x9854 (trans (monotonicity @x9846 (= $x4002 (and $x3992 $x9824))) (rewrite (= (and $x3992 $x9824) $x9850)) (= $x4002 $x9850))))
-(let ((@x9862 (trans (monotonicity @x8934 @x9854 (= $x4003 (and $x3784 $x9850))) (rewrite (= (and $x3784 $x9850) $x9858)) (= $x4003 $x9858))))
-(let ((@x9869 (trans (monotonicity @x9862 (= $x4004 (and true $x9858))) (rewrite (= (and true $x9858) $x9858)) (= $x4004 $x9858))))
-(let ((@x9878 (trans (monotonicity @x9869 @x9754 (= $x4005 (=> $x9858 $x9750))) (rewrite (= (=> $x9858 $x9750) $x9874)) (= $x4005 $x9874))))
-(let ((@x9597 (rewrite (= (and $x3927 (and $x3935 $x3936 $x3937 $x3783 $x3940 $x3942 $x3943)) $x9595))))
-(let (($x9587 (and $x3935 $x3936 $x3937 $x3783 $x3940 $x3942 $x3943)))
-(let (($x9579 (and $x3936 $x3937 $x3783 $x3940 $x3942 $x3943)))
-(let (($x9571 (and $x3937 $x3783 $x3940 $x3942 $x3943)))
-(let (($x9563 (and $x3783 $x3940 $x3942 $x3943)))
-(let (($x9548 (and $x3940 $x3942 $x3783 $x3943)))
-(let ((@x9539 (monotonicity (trans @x9533 (rewrite (= $x3945 $x3944)) (= $x3945 $x3944)) (= $x3946 (and $x3942 $x3944)))))
-(let ((@x9544 (trans @x9539 (rewrite (= (and $x3942 $x3944) (and $x3942 $x3783 $x3943))) (= $x3946 (and $x3942 $x3783 $x3943)))))
-(let ((@x9552 (trans (monotonicity @x9544 (= $x3947 (and $x3940 (and $x3942 $x3783 $x3943)))) (rewrite (= (and $x3940 (and $x3942 $x3783 $x3943)) $x9548)) (= $x3947 $x9548))))
-(let ((@x9559 (trans (monotonicity @x9552 (= $x3948 (and true $x9548))) (rewrite (= (and true $x9548) $x9548)) (= $x3948 $x9548))))
-(let ((@x9527 (trans (monotonicity @x8932 @x8932 (= $x3938 $x3938)) (rewrite (= $x3938 $x3783)) (= $x3938 $x3783))))
-(let ((@x9567 (trans (monotonicity @x9527 @x9559 (= $x3949 (and $x3783 $x9548))) (rewrite (= (and $x3783 $x9548) $x9563)) (= $x3949 $x9563))))
-(let ((@x9575 (trans (monotonicity @x9567 (= $x3950 (and $x3937 $x9563))) (rewrite (= (and $x3937 $x9563) $x9571)) (= $x3950 $x9571))))
-(let ((@x9583 (trans (monotonicity @x9575 (= $x3951 (and $x3936 $x9571))) (rewrite (= (and $x3936 $x9571) $x9579)) (= $x3951 $x9579))))
-(let ((@x9591 (trans (monotonicity @x9583 (= $x3952 (and $x3935 $x9579))) (rewrite (= (and $x3935 $x9579) $x9587)) (= $x3952 $x9587))))
-(let ((@x9599 (trans (monotonicity @x9591 (= $x3953 (and $x3927 $x9587))) @x9597 (= $x3953 $x9595))))
-(let ((@x9763 (trans (monotonicity @x9599 @x9754 (= $x3987 (=> $x9595 $x9750))) (rewrite (= (=> $x9595 $x9750) $x9759)) (= $x3987 $x9759))))
-(let ((@x9771 (trans (monotonicity @x9763 (= $x3988 (and $x3927 $x9759))) (rewrite (= (and $x3927 $x9759) $x9767)) (= $x3988 $x9767))))
-(let ((@x9780 (trans (monotonicity @x9771 (= $x3989 (=> $x3925 $x9767))) (rewrite (= (=> $x3925 $x9767) $x9776)) (= $x3989 $x9776))))
-(let ((@x9788 (trans (monotonicity @x9780 (= $x3990 (and $x3925 $x9776))) (rewrite (= (and $x3925 $x9776) $x9784)) (= $x3990 $x9784))))
-(let (($x9497 (not $x3992)))
-(let (($x9511 (and $x3783 $x3776 $x9497)))
-(let ((@x9502 (monotonicity (rewrite (= (< v_b_L_H_max_G_1$ ?x3929) $x9497)) @x9050 (= $x3931 (and $x9497 $x3784)))))
-(let ((@x9507 (trans @x9502 (rewrite (= (and $x9497 $x3784) (and $x9497 $x3783 $x3776))) (= $x3931 (and $x9497 $x3783 $x3776)))))
-(let ((@x9515 (trans (monotonicity @x8934 @x9507 (= $x3932 (and $x3784 (and $x9497 $x3783 $x3776)))) (rewrite (= (and $x3784 (and $x9497 $x3783 $x3776)) $x9511)) (= $x3932 $x9511))))
-(let ((@x9522 (trans (monotonicity @x9515 (= $x3933 (and true $x9511))) (rewrite (= (and true $x9511) $x9511)) (= $x3933 $x9511))))
-(let ((@x9797 (trans (monotonicity @x9522 @x9788 (= $x3991 (=> $x9511 $x9784))) (rewrite (= (=> $x9511 $x9784) $x9793)) (= $x3991 $x9793))))
-(let ((@x9496 (trans (monotonicity @x8934 (= $x3928 $x3928)) (rewrite (= $x3928 (and $x3923 $x3926 $x3783 $x3776))) (= $x3928 (and $x3923 $x3926 $x3783 $x3776)))))
-(let ((@x9884 (monotonicity @x9496 (monotonicity @x9797 @x9878 (= (and $x3991 $x4005) $x9879)) (= $x4007 (=> (and $x3923 $x3926 $x3783 $x3776) $x9879)))))
-(let ((@x9890 (trans @x9884 (rewrite (= (=> (and $x3923 $x3926 $x3783 $x3776) $x9879) $x9886)) (= $x4007 $x9886))))
-(let ((@x9898 (trans (monotonicity @x9890 (= $x4008 (and $x3927 $x9886))) (rewrite (= (and $x3927 $x9886) $x9894)) (= $x4008 $x9894))))
-(let ((@x9906 (trans (monotonicity @x9898 (= $x4009 (=> $x3925 $x9894))) (rewrite (= (=> $x3925 $x9894) $x9902)) (= $x4009 $x9902))))
-(let ((@x9914 (trans (monotonicity @x9906 (= $x4010 (and $x3925 $x9902))) (rewrite (= (and $x3925 $x9902) $x9910)) (= $x4010 $x9910))))
-(let (($x9465 (not $x4012)))
-(let (($x9479 (and $x3783 $x3776 $x9465)))
-(let ((@x9470 (monotonicity (rewrite (= (< v_b_L_H_p_G_0$ v_b_P_H_len$) $x9465)) @x9050 (= $x3919 (and $x9465 $x3784)))))
-(let ((@x9475 (trans @x9470 (rewrite (= (and $x9465 $x3784) (and $x9465 $x3783 $x3776))) (= $x3919 (and $x9465 $x3783 $x3776)))))
-(let ((@x9483 (trans (monotonicity @x8934 @x9475 (= $x3920 (and $x3784 (and $x9465 $x3783 $x3776)))) (rewrite (= (and $x3784 (and $x9465 $x3783 $x3776)) $x9479)) (= $x3920 $x9479))))
-(let ((@x9490 (trans (monotonicity @x9483 (= $x3921 (and true $x9479))) (rewrite (= (and true $x9479) $x9479)) (= $x3921 $x9479))))
-(let ((@x9923 (trans (monotonicity @x9490 @x9914 (= $x4011 (=> $x9479 $x9910))) (rewrite (= (=> $x9479 $x9910) $x9919)) (= $x4011 $x9919))))
-(let ((@x9443 (rewrite (= (and true $x9434) $x9434))))
-(let (($x9419 (and $x3886 $x3806 $x3699 $x3893 $x3894 $x3895 $x3896 $x3897 $x3898 $x3783 $x3776)))
-(let (($x9420 (= (and $x3886 (and $x3806 $x3699 $x3893 $x3894 $x3895 $x3896 $x3897 $x3898 $x3783 $x3776)) $x9419)))
-(let (($x9417 (= $x3910 (and $x3886 (and $x3806 $x3699 $x3893 $x3894 $x3895 $x3896 $x3897 $x3898 $x3783 $x3776)))))
-(let (($x9411 (and $x3806 $x3699 $x3893 $x3894 $x3895 $x3896 $x3897 $x3898 $x3783 $x3776)))
-(let ((@x9413 (rewrite (= (and $x3807 (and $x3893 $x3894 $x3895 $x3896 $x3897 $x3898 $x3783 $x3776)) $x9411))))
-(let (($x9403 (and $x3893 $x3894 $x3895 $x3896 $x3897 $x3898 $x3783 $x3776)))
-(let ((@x9405 (rewrite (= (and $x3893 (and $x3894 $x3895 $x3896 $x3897 $x3898 $x3783 $x3776)) $x9403))))
-(let (($x9395 (and $x3894 $x3895 $x3896 $x3897 $x3898 $x3783 $x3776)))
-(let (($x9387 (and $x3895 $x3896 $x3897 $x3898 $x3783 $x3776)))
-(let (($x9379 (and $x3896 $x3897 $x3898 $x3783 $x3776)))
-(let ((@x8840 (rewrite (= (and true true) true))))
-(let ((@x9359 (rewrite (= (= (b_S_statusmap$ v_b_S_s$) (b_S_statusmap$ v_b_S_s$)) true))))
-(let ((@x9361 (monotonicity (rewrite (= (= ?x3874 ?x3874) true)) @x9359 (= $x3902 (and true true)))))
-(let ((@x9365 (monotonicity (trans @x9361 @x8840 (= $x3902 true)) @x8934 (= $x3903 $x3808))))
-(let ((@x9370 (monotonicity (trans @x9365 @x9042 (= $x3903 $x3784)) (= $x3904 (and (and $x3897 $x3898) $x3784)))))
-(let ((@x9375 (trans @x9370 (rewrite (= (and (and $x3897 $x3898) $x3784) (and $x3897 $x3898 $x3783 $x3776))) (= $x3904 (and $x3897 $x3898 $x3783 $x3776)))))
-(let ((@x9383 (trans (monotonicity @x9375 (= $x3905 (and $x3896 (and $x3897 $x3898 $x3783 $x3776)))) (rewrite (= (and $x3896 (and $x3897 $x3898 $x3783 $x3776)) $x9379)) (= $x3905 $x9379))))
-(let ((@x9391 (trans (monotonicity @x9383 (= $x3906 (and $x3895 $x9379))) (rewrite (= (and $x3895 $x9379) $x9387)) (= $x3906 $x9387))))
-(let ((@x9399 (trans (monotonicity @x9391 (= $x3907 (and $x3894 $x9387))) (rewrite (= (and $x3894 $x9387) $x9395)) (= $x3907 $x9395))))
-(let ((@x9407 (trans (monotonicity @x9399 (= $x3908 (and $x3893 $x9395))) @x9405 (= $x3908 $x9403))))
-(let ((@x9415 (trans (monotonicity @x9407 (= $x3909 (and $x3807 $x9403))) @x9413 (= $x3909 $x9411))))
-(let ((@x9333 (rewrite (= (and true $x3886) $x3886))))
-(let (($x9322 (forall ((?v0 B_S_ptr$) )(!true :pattern ( (b_S_timestamp$ v_b_S_s$ ?v0) )))
-))
-(let (($x9320 (= (<= (b_S_timestamp$ v_b_S_s$ ?0) (b_S_timestamp$ v_b_S_s$ ?0)) true)))
-(let ((@x9328 (trans (quant-intro (rewrite $x9320) (= $x3885 $x9322)) (elim-unused (= $x9322 true)) (= $x3885 true))))
-(let ((@x9335 (trans (monotonicity @x9328 (= $x3887 (and true $x3886))) @x9333 (= $x3887 $x3886))))
-(let ((@x9337 (monotonicity (rewrite (= (<= ?x3713 ?x3713) true)) @x9335 (= $x3888 (and true $x3886)))))
-(let ((@x9423 (trans (monotonicity (trans @x9337 @x9333 (= $x3888 $x3886)) @x9415 $x9417) (rewrite $x9420) (= $x3910 $x9419))))
-(let (($x9311 (forall ((?v0 B_S_ptr$) )(!true :pattern ( (b_S_select_o_tm$ (b_S_typemap$ v_b_S_s$) ?v0) )))
-))
-(let (($x3862 (b_S_thread_n_local$ v_b_S_s$ ?0)))
-(let (($x3877 (and (= (b_S_select_o_tm$ ?x3874 ?0) (b_S_select_o_tm$ ?x3874 ?0)) $x3862)))
-(let (($x3878 (=> $x3862 $x3877)))
-(let ((@x9277 (rewrite (= (=> $x3862 $x3862) true))))
-(let ((@x9270 (rewrite (= (and true $x3862) $x3862))))
-(let (($x9301 (= (= (b_S_select_o_tm$ ?x3874 ?0) (b_S_select_o_tm$ ?x3874 ?0)) true)))
-(let ((@x9306 (trans (monotonicity (rewrite $x9301) (= $x3877 (and true $x3862))) @x9270 (= $x3877 $x3862))))
-(let ((@x9310 (trans (monotonicity @x9306 (= $x3878 (=> $x3862 $x3862))) @x9277 (= $x3878 true))))
-(let ((@x9317 (trans (quant-intro @x9310 (= $x3880 $x9311)) (elim-unused (= $x9311 true)) (= $x3880 true))))
-(let ((@x9341 (monotonicity @x9317 (trans @x9337 @x9333 (= $x3888 $x3886)) (= $x3889 (and true $x3886)))))
-(let (($x9257 (forall ((?v0 B_S_ptr$) )(!true :pattern ( (b_S_select_o_sm$ (b_S_statusmap$ v_b_S_s$) ?v0) )))
-))
-(let ((?x3858 (b_S_statusmap$ v_b_S_s$)))
-(let ((?x3859 (b_S_select_o_sm$ ?x3858 ?0)))
-(let (($x3871 (and (= ?x3859 ?x3859) $x3862)))
-(let (($x3872 (=> $x3862 $x3871)))
-(let ((@x9290 (monotonicity (rewrite (= (= ?x3859 ?x3859) true)) (= $x3871 (and true $x3862)))))
-(let ((@x9294 (monotonicity (trans @x9290 @x9270 (= $x3871 $x3862)) (= $x3872 (=> $x3862 $x3862)))))
-(let ((@x9300 (trans (quant-intro (trans @x9294 @x9277 (= $x3872 true)) (= $x3873 $x9257)) (elim-unused (= $x9257 true)) (= $x3873 true))))
-(let ((@x9345 (monotonicity @x9300 (trans @x9341 @x9333 (= $x3889 $x3886)) (= $x3890 (and true $x3886)))))
-(let (($x9280 (forall ((?v0 B_S_ptr$) )(!true :pattern ( (b_S_select_o_mem$ (b_S_memory$ v_b_S_s$) ?v0) )))
-))
-(let ((?x3864 (b_S_select_o_mem$ (b_S_memory$ v_b_S_s$) ?0)))
-(let (($x3866 (and (= ?x3864 ?x3864) $x3862)))
-(let (($x3867 (=> $x3862 $x3866)))
-(let ((@x9268 (monotonicity (rewrite (= (= ?x3864 ?x3864) true)) (= $x3866 (and true $x3862)))))
-(let ((@x9275 (monotonicity (trans @x9268 @x9270 (= $x3866 $x3862)) (= $x3867 (=> $x3862 $x3862)))))
-(let ((@x9286 (trans (quant-intro (trans @x9275 @x9277 (= $x3867 true)) (= $x3869 $x9280)) (elim-unused (= $x9280 true)) (= $x3869 true))))
-(let ((@x9349 (monotonicity @x9286 (trans @x9345 @x9333 (= $x3890 $x3886)) (= $x3891 (and true $x3886)))))
-(let (($x3855 (= (b_S_kind_n_of$ (b_S_typ$ (b_S_owner$ v_b_S_s$ ?0))) b_S_kind_n_thread$)))
-(let ((@x9259 (quant-intro (rewrite (= (=> (not $x3855) (not $x3855)) true)) (= $x3861 $x9257))))
-(let ((@x9353 (monotonicity (trans @x9259 (elim-unused (= $x9257 true)) (= $x3861 true)) (trans @x9349 @x9333 (= $x3891 $x3886)) (= $x3892 (and true $x3886)))))
-(let ((@x9426 (monotonicity (trans @x9353 @x9333 (= $x3892 $x3886)) @x9423 (= $x3911 (and $x3886 $x9419)))))
-(let ((@x9433 (monotonicity @x8934 (trans @x9426 (rewrite (= (and $x3886 $x9419) $x9419)) (= $x3911 $x9419)) (= $x3912 (and $x3784 $x9419)))))
-(let ((@x9441 (monotonicity (trans @x9433 (rewrite (= (and $x3784 $x9419) $x9434)) (= $x3912 $x9434)) (= $x3913 (and true $x9434)))))
-(let ((@x9448 (monotonicity @x8934 (trans @x9441 @x9443 (= $x3913 $x9434)) (= $x3914 (and $x3784 $x9434)))))
-(let ((@x9454 (monotonicity (trans @x9448 (rewrite (= (and $x3784 $x9434) $x9434)) (= $x3914 $x9434)) (= $x3915 (and true $x9434)))))
-(let ((@x9458 (monotonicity @x8934 (trans @x9454 @x9443 (= $x3915 $x9434)) (= $x3916 (and $x3784 $x9434)))))
-(let ((@x9462 (monotonicity (trans @x9458 (rewrite (= (and $x3784 $x9434) $x9434)) (= $x3916 $x9434)) (= $x3917 (and true $x9434)))))
-(let ((@x9973 (monotonicity (trans @x9462 @x9443 (= $x3917 $x9434)) (monotonicity @x9923 @x9967 (= (and $x4011 $x4019) $x9968)) (= $x4021 (=> $x9434 $x9968)))))
-(let ((@x9979 (trans @x9973 (rewrite (= (=> $x9434 $x9968) (or $x9974 $x9968))) (= $x4021 (or $x9974 $x9968)))))
-(let (($x9062 (and $x3783 $x3776 $x3806 $x3699)))
-(let ((@x9058 (trans (monotonicity @x9050 (= $x3810 (and $x3807 $x3784))) (rewrite (= (and $x3807 $x3784) (and $x3806 $x3699 $x3783 $x3776))) (= $x3810 (and $x3806 $x3699 $x3783 $x3776)))))
-(let ((@x9061 (monotonicity @x8934 @x9058 (= $x3811 (and $x3784 (and $x3806 $x3699 $x3783 $x3776))))))
-(let ((@x9066 (trans @x9061 (rewrite (= (and $x3784 (and $x3806 $x3699 $x3783 $x3776)) $x9062)) (= $x3811 $x9062))))
-(let ((@x9073 (trans (monotonicity @x9066 (= $x3812 (and true $x9062))) (rewrite (= (and true $x9062) $x9062)) (= $x3812 $x9062))))
-(let ((@x9080 (trans (monotonicity @x8934 @x9073 (= $x3813 (and $x3784 $x9062))) (rewrite (= (and $x3784 $x9062) $x9062)) (= $x3813 $x9062))))
-(let ((@x9083 (monotonicity (rewrite (= $x3805 false)) @x9080 (= $x3814 (and false $x9062)))))
-(let ((@x9087 (trans @x9083 (rewrite (= (and false $x9062) false)) (= $x3814 false))))
-(let ((@x9094 (trans (monotonicity @x8934 @x9087 (= $x3815 (and $x3784 false))) (rewrite (= (and $x3784 false) false)) (= $x3815 false))))
-(let ((@x9101 (trans (monotonicity @x9094 (= $x3816 (and true false))) (rewrite (= (and true false) false)) (= $x3816 false))))
-(let ((@x9254 (trans (monotonicity @x9101 @x9247 (= $x3851 (=> false $x9245))) (rewrite (= (=> false $x9245) true)) (= $x3851 true))))
-(let ((@x9986 (trans (monotonicity @x9254 @x9979 (= $x4022 (and true (or $x9974 $x9968)))) (rewrite (= (and true (or $x9974 $x9968)) (or $x9974 $x9968))) (= $x4022 (or $x9974 $x9968)))))
-(let (($x9017 (and $x3772 $x3773 $x3776 $x3777 $x3780 $x3781 $x3783 $x3785 $x8956 $x8960 $x3794)))
-(let (($x8916 (and $x8667 $x3769)))
-(let (($x9018 (= (and $x3774 (and $x3776 $x3777 $x3780 $x3781 $x3783 $x3785 $x8956 $x8960 $x3794)) $x9017)))
-(let (($x9015 (= $x3802 (and $x3774 (and $x3776 $x3777 $x3780 $x3781 $x3783 $x3785 $x8956 $x8960 $x3794)))))
-(let (($x9009 (and $x3776 $x3777 $x3780 $x3781 $x3783 $x3785 $x8956 $x8960 $x3794)))
-(let ((@x9011 (rewrite (= (and $x3778 (and $x3780 $x3781 $x3783 $x3776 $x3785 $x8956 $x8960 $x3794)) $x9009))))
-(let (($x9001 (and $x3780 $x3781 $x3783 $x3776 $x3785 $x8956 $x8960 $x3794)))
-(let (($x8993 (and $x3783 $x3776 $x3785 $x8956 $x8960 $x3794)))
-(let (($x8985 (and $x3785 $x8956 $x8960 $x3794 $x3783 $x3776)))
-(let (($x8977 (and $x8956 $x8960 $x3794 $x3783 $x3776)))
-(let (($x8964 (= (and (< v_b_SL_H_witness_G_0$ v_b_P_H_len$) $x3794) (and $x8960 $x3794))))
-(let ((@x8965 (monotonicity (rewrite (= (< v_b_SL_H_witness_G_0$ v_b_P_H_len$) $x8960)) $x8964)))
-(let ((@x8973 (trans (monotonicity @x8965 @x8934 (= $x3796 (and (and $x8960 $x3794) $x3784))) (rewrite (= (and (and $x8960 $x3794) $x3784) (and $x8960 $x3794 $x3783 $x3776))) (= $x3796 (and $x8960 $x3794 $x3783 $x3776)))))
-(let (($x3788 (<= ?x3765 v_b_L_H_max_G_1$)))
-(let (($x8951 (or (not (and $x1212 $x1344 (not (<= v_b_L_H_p_G_0$ ?0)))) $x3788)))
-(let (($x3787 (and $x1345 (< ?0 v_b_L_H_p_G_0$))))
-(let (($x3789 (=> $x3787 $x3788)))
-(let ((@x8953 (rewrite (= (=> (and $x1212 $x1344 (not (<= v_b_L_H_p_G_0$ ?0))) $x3788) $x8951))))
-(let (($x8936 (not (<= v_b_L_H_p_G_0$ ?0))))
-(let (($x8942 (and $x1212 $x1344 $x8936)))
-(let ((@x8941 (monotonicity @x5523 (rewrite (= (< ?0 v_b_L_H_p_G_0$) $x8936)) (= $x3787 (and $x1345 $x8936)))))
-(let ((@x8949 (monotonicity (trans @x8941 (rewrite (= (and $x1345 $x8936) $x8942)) (= $x3787 $x8942)) (= $x3789 (=> $x8942 $x3788)))))
-(let ((@x8976 (monotonicity (quant-intro (trans @x8949 @x8953 (= $x3789 $x8951)) (= $x3790 $x8956)) @x8973 (= $x3797 (and $x8956 (and $x8960 $x3794 $x3783 $x3776))))))
-(let ((@x8981 (trans @x8976 (rewrite (= (and $x8956 (and $x8960 $x3794 $x3783 $x3776)) $x8977)) (= $x3797 $x8977))))
-(let ((@x8989 (trans (monotonicity @x8981 (= $x3798 (and $x3785 $x8977))) (rewrite (= (and $x3785 $x8977) $x8985)) (= $x3798 $x8985))))
-(let ((@x8997 (trans (monotonicity @x8934 @x8989 (= $x3799 (and $x3784 $x8985))) (rewrite (= (and $x3784 $x8985) $x8993)) (= $x3799 $x8993))))
-(let ((@x9000 (monotonicity (monotonicity (rewrite (= $x3780 $x3780)) (= $x3782 $x3782)) @x8997 (= $x3800 (and $x3782 $x8993)))))
-(let ((@x9008 (monotonicity (monotonicity (rewrite (= $x3776 $x3776)) (= $x3778 $x3778)) (trans @x9000 (rewrite (= (and $x3782 $x8993) $x9001)) (= $x3800 $x9001)) (= $x3801 (and $x3778 $x9001)))))
-(let ((@x9016 (monotonicity (monotonicity (rewrite (= $x3772 $x3772)) (= $x3774 $x3774)) (trans @x9008 @x9011 (= $x3801 $x9009)) $x9015)))
-(let ((@x9024 (monotonicity (trans @x9016 (rewrite $x9018) (= $x3802 $x9017)) (= $x3803 (and true $x9017)))))
-(let ((@x9031 (monotonicity (monotonicity (rewrite (= $x3676 $x8667)) (= $x3770 $x8916)) (trans @x9024 (rewrite (= (and true $x9017) $x9017)) (= $x3803 $x9017)) (= $x3804 (and $x8916 $x9017)))))
-(let ((@x9989 (monotonicity (trans @x9031 (rewrite (= (and $x8916 $x9017) $x9032)) (= $x3804 $x9032)) @x9986 (= $x4023 (=> $x9032 (or $x9974 $x9968))))))
-(let ((@x9995 (trans @x9989 (rewrite (= (=> $x9032 (or $x9974 $x9968)) $x9991)) (= $x4023 $x9991))))
-(let ((@x9998 (monotonicity (monotonicity (rewrite (= $x3676 $x8667)) (= $x3770 $x8916)) @x9995 (= $x4024 (and $x8916 $x9991)))))
-(let (($x3766 (<= ?x3765 v_b_L_H_max_G_0$)))
-(let (($x8908 (or (not (and $x1212 $x1344 (not (<= 1 ?0)))) $x3766)))
-(let (($x3763 (and $x1345 (< ?0 1))))
-(let (($x3767 (=> $x3763 $x3766)))
-(let (($x8887 (<= 1 ?0)))
-(let (($x8888 (not $x8887)))
-(let (($x8899 (and $x1212 $x1344 $x8888)))
-(let ((@x8895 (trans (rewrite (= (< ?0 1) $x8888)) (monotonicity (rewrite (= $x8887 $x8887)) (= $x8888 $x8888)) (= (< ?0 1) $x8888))))
-(let ((@x8903 (trans (monotonicity @x5523 @x8895 (= $x3763 (and $x1345 $x8888))) (rewrite (= (and $x1345 $x8888) $x8899)) (= $x3763 $x8899))))
-(let ((@x8912 (trans (monotonicity @x8903 (= $x3767 (=> $x8899 $x3766))) (rewrite (= (=> $x8899 $x3766) $x8908)) (= $x3767 $x8908))))
-(let ((@x10006 (monotonicity (quant-intro @x8912 (= $x3768 $x8913)) (trans @x9998 (rewrite (= (and $x8916 $x9991) $x9999)) (= $x4024 $x9999)) (= $x4025 (=> $x8913 $x9999)))))
-(let ((@x10015 (monotonicity (quant-intro @x8912 (= $x3768 $x8913)) (trans @x10006 (rewrite (= (=> $x8913 $x9999) $x10008)) (= $x4025 $x10008)) (= (and $x3768 $x4025) $x10013))))
-(let ((@x10018 (monotonicity (rewrite (= $x3761 $x3761)) @x10015 (= $x4027 (=> $x3761 $x10013)))))
-(let ((@x10027 (monotonicity (rewrite (= $x3761 $x3761)) (trans @x10018 (rewrite (= (=> $x3761 $x10013) $x10020)) (= $x4027 $x10020)) (= (and $x3761 $x4027) $x10025))))
-(let ((@x8874 (rewrite (= (and $x3747 (and $x3748 $x3749 $x3750)) (and $x3747 $x3748 $x3749 $x3750)))))
-(let ((@x8838 (monotonicity (rewrite (= $x3752 true)) (rewrite (= $x3752 true)) (= $x3753 (and true true)))))
-(let ((@x8844 (monotonicity (rewrite (= $x3751 true)) (trans @x8838 @x8840 (= $x3753 true)) (= $x3754 (and true true)))))
-(let ((@x8848 (monotonicity (rewrite (= $x3751 true)) (trans @x8844 @x8840 (= $x3754 true)) (= $x3755 (and true true)))))
-(let ((@x8853 (monotonicity (trans @x8848 @x8840 (= $x3755 true)) (= $x3756 (and $x3750 true)))))
-(let ((@x8860 (monotonicity (trans @x8853 (rewrite (= (and $x3750 true) $x3750)) (= $x3756 $x3750)) (= (and $x3749 $x3756) (and $x3749 $x3750)))))
-(let ((@x8868 (trans (monotonicity @x8860 (= $x3758 (and $x3748 (and $x3749 $x3750)))) (rewrite (= (and $x3748 (and $x3749 $x3750)) (and $x3748 $x3749 $x3750))) (= $x3758 (and $x3748 $x3749 $x3750)))))
-(let ((@x8876 (trans (monotonicity @x8868 (= $x3759 (and $x3747 (and $x3748 $x3749 $x3750)))) @x8874 (= $x3759 (and $x3747 $x3748 $x3749 $x3750)))))
-(let ((@x8884 (trans (monotonicity @x8876 (= $x3760 (and $x3744 (and $x3747 $x3748 $x3749 $x3750)))) (rewrite (= (and $x3744 (and $x3747 $x3748 $x3749 $x3750)) $x8880)) (= $x3760 $x8880))))
-(let ((@x10036 (trans (monotonicity @x8884 @x10027 (= $x4029 (=> $x8880 $x10025))) (rewrite (= (=> $x8880 $x10025) $x10032)) (= $x4029 $x10032))))
-(let ((@x10044 (trans (monotonicity @x10036 (= $x4030 (and $x3744 $x10032))) (rewrite (= (and $x3744 $x10032) $x10040)) (= $x4030 $x10040))))
-(let ((@x10053 (trans (monotonicity @x10044 (= $x4031 (=> $x3742 $x10040))) (rewrite (= (=> $x3742 $x10040) $x10049)) (= $x4031 $x10049))))
-(let ((@x10061 (trans (monotonicity @x10053 (= $x4032 (and $x3742 $x10049))) (rewrite (= (and $x3742 $x10049) $x10057)) (= $x4032 $x10057))))
-(let ((@x10070 (trans (monotonicity @x10061 (= $x4033 (=> $x3738 $x10057))) (rewrite (= (=> $x3738 $x10057) $x10066)) (= $x4033 $x10066))))
-(let (($x8812 (and $x3667 $x3668 $x3671 $x3672 $x8658 $x8667 $x3683 $x3685 $x3686 $x3687 $x3690 $x3691 $x3697 $x3698 $x3699 $x8701 $x3708 $x3709 $x3711 $x3714 $x8707 $x3719 $x3720)))
-(let (($x8804 (and $x3671 $x3672 $x8658 $x8667 $x3683 $x3685 $x3686 $x3687 $x3690 $x3691 $x3697 $x3698 $x3699 $x8701 $x3708 $x3709 $x3711 $x3714 $x8707 $x3719 $x3720)))
-(let (($x8796 (and $x8658 $x8667 $x3683 $x3685 $x3686 $x3687 $x3690 $x3691 $x3697 $x3698 $x3699 $x8701 $x3708 $x3709 $x3711 $x3714 $x8707 $x3719 $x3720)))
-(let (($x8788 (and $x8667 $x3683 $x3685 $x3686 $x3687 $x3690 $x3691 $x3697 $x3698 $x3699 $x8701 $x3708 $x3709 $x3711 $x3714 $x8707 $x3719 $x3720)))
-(let (($x8780 (and $x3683 $x3685 $x3686 $x3687 $x3690 $x3691 $x3697 $x3698 $x3699 $x8701 $x3708 $x3709 $x3711 $x3714 $x8707 $x3719 $x3720)))
-(let (($x8765 (and $x3697 $x3698 $x3699 $x8701 $x3708 $x3709 $x3711 $x3714 $x8707 $x3719 $x3720)))
-(let (($x8692 (and $x3683 $x3685 $x3686 $x3687 $x3690 $x3691)))
-(let (($x8766 (= (and $x3697 (and $x3698 $x3699 $x8701 $x3708 $x3709 $x3711 $x3714 $x8707 $x3719 $x3720)) $x8765)))
-(let (($x8763 (= $x3728 (and $x3697 (and $x3698 $x3699 $x8701 $x3708 $x3709 $x3711 $x3714 $x8707 $x3719 $x3720)))))
-(let (($x8757 (and $x3698 $x3699 $x8701 $x3708 $x3709 $x3711 $x3714 $x8707 $x3719 $x3720)))
-(let (($x8758 (= (and (and $x3698 $x3699) (and $x8701 $x3708 $x3709 $x3711 $x3714 $x8707 $x3719 $x3720)) $x8757)))
-(let (($x8755 (= $x3727 (and (and $x3698 $x3699) (and $x8701 $x3708 $x3709 $x3711 $x3714 $x8707 $x3719 $x3720)))))
-(let (($x8749 (and $x8701 $x3708 $x3709 $x3711 $x3714 $x8707 $x3719 $x3720)))
-(let ((@x8751 (rewrite (= (and $x8701 (and $x3708 $x3709 $x3711 $x3714 $x8707 $x3719 $x3720)) $x8749))))
-(let (($x8741 (and $x3708 $x3709 $x3711 $x3714 $x8707 $x3719 $x3720)))
-(let ((@x8743 (rewrite (= (and (and $x3708 $x3709) (and $x3711 $x3714 $x8707 $x3719 $x3720)) $x8741))))
-(let (($x8733 (and $x3711 $x3714 $x8707 $x3719 $x3720)))
-(let ((@x8727 (rewrite (= (and $x3714 (and $x8707 $x3719 $x3720)) (and $x3714 $x8707 $x3719 $x3720)))))
-(let (($x8705 (= (= (b_S_in_n_writes_n_at$ v_b_H_wrTime_S_1_T_6_o_1$ ?0) false) (not (b_S_in_n_writes_n_at$ v_b_H_wrTime_S_1_T_6_o_1$ ?0)))))
-(let ((@x8716 (monotonicity (quant-intro (rewrite $x8705) (= $x3718 $x8707)) (monotonicity (rewrite (= $x3719 $x3719)) (= $x3721 $x3721)) (= $x3722 (and $x8707 $x3721)))))
-(let ((@x8721 (trans @x8716 (rewrite (= (and $x8707 $x3721) (and $x8707 $x3719 $x3720))) (= $x3722 (and $x8707 $x3719 $x3720)))))
-(let ((@x8729 (trans (monotonicity @x8721 (= $x3723 (and $x3714 (and $x8707 $x3719 $x3720)))) @x8727 (= $x3723 (and $x3714 $x8707 $x3719 $x3720)))))
-(let ((@x8737 (trans (monotonicity @x8729 (= $x3724 (and $x3711 (and $x3714 $x8707 $x3719 $x3720)))) (rewrite (= (and $x3711 (and $x3714 $x8707 $x3719 $x3720)) $x8733)) (= $x3724 $x8733))))
-(let ((@x8745 (trans (monotonicity @x8737 (= $x3725 (and (and $x3708 $x3709) $x8733))) @x8743 (= $x3725 $x8741))))
-(let (($x8699 (= (< (b_S_frame_n_level$ ?0) b_S_current_n_frame_n_level$) (not (<= b_S_current_n_frame_n_level$ (b_S_frame_n_level$ ?0))))))
-(let ((@x8748 (monotonicity (quant-intro (rewrite $x8699) (= $x3706 $x8701)) @x8745 (= $x3726 (and $x8701 $x8741)))))
-(let ((@x8761 (trans (monotonicity (trans @x8748 @x8751 (= $x3726 $x8749)) $x8755) (rewrite $x8758) (= $x3727 $x8757))))
-(let ((@x8772 (monotonicity (trans (monotonicity @x8761 $x8763) (rewrite $x8766) (= $x3728 $x8765)) (= $x3729 (and true $x8765)))))
-(let (($x8684 (and $x3685 $x3686 $x3687 $x3690 $x3691)))
-(let ((@x8678 (rewrite (= (and $x3686 (and $x3687 $x3690 $x3691)) (and $x3686 $x3687 $x3690 $x3691)))))
-(let ((@x8675 (monotonicity (rewrite (= (and $x3687 (and $x3690 $x3691)) (and $x3687 $x3690 $x3691))) (= $x3694 (and $x3686 (and $x3687 $x3690 $x3691))))))
-(let ((@x8683 (monotonicity (trans @x8675 @x8678 (= $x3694 (and $x3686 $x3687 $x3690 $x3691))) (= $x3695 (and $x3685 (and $x3686 $x3687 $x3690 $x3691))))))
-(let ((@x8688 (trans @x8683 (rewrite (= (and $x3685 (and $x3686 $x3687 $x3690 $x3691)) $x8684)) (= $x3695 $x8684))))
-(let ((@x8696 (trans (monotonicity @x8688 (= $x3696 (and $x3683 $x8684))) (rewrite (= (and $x3683 $x8684) $x8692)) (= $x3696 $x8692))))
-(let ((@x8779 (monotonicity @x8696 (trans @x8772 (rewrite (= (and true $x8765) $x8765)) (= $x3729 $x8765)) (= $x3730 (and $x8692 $x8765)))))
-(let ((@x8787 (monotonicity (rewrite (= $x3676 $x8667)) (trans @x8779 (rewrite (= (and $x8692 $x8765) $x8780)) (= $x3730 $x8780)) (= $x3731 (and $x8667 $x8780)))))
-(let ((@x8665 (trans (rewrite (= (< v_b_P_H_len$ 1099511627776) $x8658)) (monotonicity (rewrite (= $x8657 $x8657)) (= $x8658 $x8658)) (= (< v_b_P_H_len$ 1099511627776) $x8658))))
-(let ((@x8795 (monotonicity @x8665 (trans @x8787 (rewrite (= (and $x8667 $x8780) $x8788)) (= $x3731 $x8788)) (= $x3732 (and $x8658 $x8788)))))
-(let ((@x8803 (monotonicity (monotonicity (rewrite (= $x3671 $x3671)) (= $x3673 $x3673)) (trans @x8795 (rewrite (= (and $x8658 $x8788) $x8796)) (= $x3732 $x8796)) (= $x3733 (and $x3673 $x8796)))))
-(let ((@x8811 (monotonicity (monotonicity (rewrite (= $x3667 $x3667)) (= $x3669 $x3669)) (trans @x8803 (rewrite (= (and $x3673 $x8796) $x8804)) (= $x3733 $x8804)) (= $x3734 (and $x3669 $x8804)))))
-(let ((@x8819 (monotonicity (monotonicity (rewrite (= $x3663 $x3663)) (= $x3665 $x3665)) (trans @x8811 (rewrite (= (and $x3669 $x8804) $x8812)) (= $x3734 $x8812)) (= $x3735 (and $x3665 $x8812)))))
-(let ((@x8827 (monotonicity (trans @x8819 (rewrite (= (and $x3665 $x8812) $x8820)) (= $x3735 $x8820)) (= $x3736 (and true $x8820)))))
-(let ((@x10076 (monotonicity (trans @x8827 (rewrite (= (and true $x8820) $x8820)) (= $x3736 $x8820)) (monotonicity @x10070 (= (and $x3738 $x4033) $x10071)) (= $x4035 (=> $x8820 $x10071)))))
-(let ((@x10085 (monotonicity (trans @x10076 (rewrite (= (=> $x8820 $x10071) $x10078)) (= $x4035 $x10078)) (= $x4036 (not $x10078)))))
-(let ((@x10087 (not-or-elim (mp (asserted $x4036) @x10085 (not $x10078)) $x8820)))
-(let ((@x10095 (and-elim @x10087 $x8667)))
-(let (($x21235 (or $x12351 $x21232)))
-(let (($x21238 (not $x21235)))
-(let (($x16251 (not $x3743)))
-(let (($x16242 (not $x3740)))
-(let (($x21241 (or $x16242 $x16251 (not $x3747) (not $x3748) (not $x3749) (not $x3750) $x21238)))
-(let (($x21244 (not $x21241)))
-(let (($x23354 (= (b_S_kind_n_of$ (b_S_typ$ ?x23206)) b_S_kind_n_primitive$)))
-(let ((?x22173 (b_S_kind_n_of$ b_T_T_u1$)))
-(let (($x22174 (= ?x22173 b_S_kind_n_primitive$)))
-(let (($x3529 (b_S_is_n_primitive$ b_T_T_u1$)))
-(let (($x22181 (= $x3529 $x22174)))
-(let (($x12265 (forall ((?v0 B_S_ctype$) )(!(let (($x1179 (b_S_is_n_primitive$ ?v0)))
-(= $x1179 (= (b_S_kind_n_of$ ?v0) b_S_kind_n_primitive$))) :pattern ( (b_S_is_n_primitive$ ?v0) )))
-))
-(let (($x1179 (b_S_is_n_primitive$ ?0)))
-(let (($x12261 (= $x1179 (= (b_S_kind_n_of$ ?0) b_S_kind_n_primitive$))))
-(let (($x3575 (forall ((?v0 B_S_ctype$) )(!(let (($x1179 (b_S_is_n_primitive$ ?v0)))
-(= $x1179 (= (b_S_kind_n_of$ ?v0) b_S_kind_n_primitive$))) :pattern ( (b_S_is_n_primitive$ ?v0) )))
-))
-(let ((@x12264 (rewrite (= (= $x1179 (= (b_S_kind_n_of$ ?0) b_S_kind_n_primitive$)) $x12261))))
-(let ((@x16196 (mp~ (mp (asserted $x3575) (quant-intro @x12264 (= $x3575 $x12265)) $x12265) (nnf-pos (refl (~ $x12261 $x12261)) (~ $x12265 $x12265)) $x12265)))
-(let ((@x5093 (asserted $x3529)))
-(let ((@x23476 (unit-resolution (def-axiom (or (not $x22181) (not $x3529) $x22174)) @x5093 (or (not $x22181) $x22174))))
-(let ((@x23477 (unit-resolution @x23476 (unit-resolution ((_ quant-inst b_T_T_u1$) (or (not $x12265) $x22181)) @x16196 $x22181) $x22174)))
-(let ((@x23492 (unit-resolution (def-axiom (or (not $x23223) $x16242 $x23216)) @x23251 (or (not $x23223) $x23216))))
-(let ((@x23499 (unit-resolution @x23492 (unit-resolution ((_ quant-inst (b_S_idx$ ?x3680 0 b_T_T_u1$) b_T_T_u1$) (or (not $x20961) $x23223)) @x20966 $x23223) $x23216)))
-(let ((@x23922 (symm (unit-resolution @x23405 @x16076 @x23251 $x23207) (= ?x23206 ?x3739))))
-(let ((@x23778 (trans (monotonicity @x23922 (= (b_S_typ$ ?x23206) ?x23215)) @x23499 (= (b_S_typ$ ?x23206) b_T_T_u1$))))
-(let ((@x23574 (trans (monotonicity @x23778 (= (b_S_kind_n_of$ (b_S_typ$ ?x23206)) ?x22173)) @x23477 $x23354)))
-(let (($x23361 (not (b_S_closed$ v_b_S_s$ (b_S_ts_n_emb$ (b_S_select_o_tm$ ?x3874 ?x23206))))))
-(let ((?x23356 (b_S_select_o_tm$ ?x3874 ?x23206)))
-(let (($x23357 (b_S_ts_n_is_n_volatile$ ?x23356)))
-(let (($x23358 (not $x23357)))
-(let (($x23362 (or $x23358 $x23361)))
-(let ((@x24072 (monotonicity @x23922 (= ?x23356 (b_S_select_o_tm$ ?x3874 ?x3739)))))
-(let ((@x23530 (monotonicity @x24072 (= $x23357 (b_S_ts_n_is_n_volatile$ (b_S_select_o_tm$ ?x3874 ?x3739))))))
-(let ((@x23502 (symm @x23530 (= (b_S_ts_n_is_n_volatile$ (b_S_select_o_tm$ ?x3874 ?x3739)) $x23357))))
-(let ((@x23522 (monotonicity @x23502 (= (not (b_S_ts_n_is_n_volatile$ (b_S_select_o_tm$ ?x3874 ?x3739))) $x23358))))
-(let ((?x23179 (b_S_select_o_tm$ ?x3874 ?x3739)))
-(let (($x23303 (b_S_ts_n_is_n_volatile$ ?x23179)))
-(let (($x23260 (not $x23303)))
-(let (($x16245 (not $x3741)))
-(let (($x23304 (or $x16245 $x23303)))
-(let (($x23305 (not $x23304)))
-(let ((?x23296 (b_S_ptr$ ?x3678 v_b_P_H_arr$)))
-(let (($x23297 (b_S_set_n_in$ ?x23296 (b_S_domain$ v_b_S_s$ (b_S_ptr$ ?x3678 (b_S_ref$ ?x3682))))))
-(let ((?x21715 (b_S_ref$ ?x3682)))
-(let ((?x22684 (b_S_ptr$ ?x3678 ?x21715)))
-(let (($x23045 (b_S_set_n_in$ ?x22684 (b_S_domain$ v_b_S_s$ ?x22684))))
-(let ((@x23339 (monotonicity (symm @x23283 (= v_b_P_H_arr$ ?x3681)) (= ?x23296 ?x3682))))
-(let (($x22691 (= ?x3682 ?x22684)))
-(let (($x22699 (= (or (not $x8559) (or (not $x3686) $x22691)) (or (not $x8559) (not $x3686) $x22691))))
-(let ((@x22701 (mp ((_ quant-inst (b_S_ptr$ ?x3678 ?x3681) (b_S_array$ b_T_T_u1$ v_b_P_H_len$)) (or (not $x8559) (or (not $x3686) $x22691))) (rewrite $x22699) (or (not $x8559) (not $x3686) $x22691))))
-(let ((@x24449 (symm (unit-resolution @x22701 @x16076 (and-elim @x10087 $x3686) $x22691) (= ?x22684 ?x3682))))
-(let ((@x23394 (monotonicity (trans @x24449 (symm @x23339 (= ?x3682 ?x23296)) (= ?x22684 ?x23296)) (= $x23045 $x23297))))
-(let (($x23063 (forall ((?v3 B_S_ptr$) )(!(let ((?x3680 (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$)))
-(let ((?x3681 (b_S_ref$ ?x3680)))
-(let ((?x3678 (b_S_array$ b_T_T_u1$ v_b_P_H_len$)))
-(let ((?x3682 (b_S_ptr$ ?x3678 ?x3681)))
-(let ((?x21715 (b_S_ref$ ?x3682)))
-(let ((?x22684 (b_S_ptr$ ?x3678 ?x21715)))
-(let (($x23060 (b_S_set_n_in2$ ?v3 (b_S_ver_n_domain$ (b_S_read_n_version$ v_b_S_s$ ?x22684)))))
-(or (b_S_has_n_volatile_n_owns_n_set$ (b_S_typ$ ?x22684)) (not (b_S_set_n_in$ ?v3 (b_S_owns$ v_b_S_s$ ?x22684))) $x23060)))))))) :pattern ( (b_S_set_n_in$ ?v3 (b_S_owns$ v_b_S_s$ (b_S_ptr$ (b_S_array$ b_T_T_u1$ v_b_P_H_len$) (b_S_ref$ (b_S_ptr$ (b_S_array$ b_T_T_u1$ v_b_P_H_len$) (b_S_ref$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$))))))) )))
-))
-(let (($x22949 (b_S_closed$ v_b_S_s$ ?x22684)))
-(let (($x22973 (not $x22949)))
-(let (($x23066 (not (or (not $x23045) $x22973 (not $x23063)))))
-(let (($x23019 (b_S_in_n_domain$ v_b_S_s$ ?x22684 ?x22684)))
-(let (($x23018 (b_S_in_n_domain_n_lab$ v_b_S_s$ ?x22684 ?x22684 b_l_H_public$)))
-(let (($x23027 (= $x23018 $x23019)))
-(let (($x12066 (forall ((?v0 B_S_state$) (?v1 B_S_ptr$) (?v2 B_S_ptr$) (?v3 B_S_label$) )(!(let (($x3056 (b_S_in_n_domain_n_lab$ ?v0 ?v1 ?v2 ?v3)))
-(= $x3056 (b_S_in_n_domain$ ?v0 ?v1 ?v2))) :pattern ( (b_S_in_n_domain_n_lab$ ?v0 ?v1 ?v2 ?v3) )))
-))
-(let (($x3056 (b_S_in_n_domain_n_lab$ ?3 ?2 ?1 ?0)))
-(let (($x12062 (= $x3056 (b_S_in_n_domain$ ?3 ?2 ?1))))
-(let (($x3060 (forall ((?v0 B_S_state$) (?v1 B_S_ptr$) (?v2 B_S_ptr$) (?v3 B_S_label$) )(!(let (($x3056 (b_S_in_n_domain_n_lab$ ?v0 ?v1 ?v2 ?v3)))
-(= $x3056 (b_S_in_n_domain$ ?v0 ?v1 ?v2))) :pattern ( (b_S_in_n_domain_n_lab$ ?v0 ?v1 ?v2 ?v3) )))
-))
-(let ((@x12068 (quant-intro (rewrite (= (= $x3056 (b_S_in_n_domain$ ?3 ?2 ?1)) $x12062)) (= $x3060 $x12066))))
-(let ((@x15761 (mp~ (mp (asserted $x3060) @x12068 $x12066) (nnf-pos (refl (~ $x12062 $x12062)) (~ $x12066 $x12066)) $x12066)))
-(let (($x36 (= b_S_kind_n_primitive$ b_S_kind_n_array$)))
-(let (($x37 (not $x36)))
-(let (($x23052 (= $x37 (not (= (b_S_kind_n_of$ (b_S_typ$ ?x22684)) b_S_kind_n_primitive$)))))
-(let ((?x22935 (b_S_typ$ ?x22684)))
-(let ((?x23088 (b_S_kind_n_of$ ?x22935)))
-(let (($x23089 (= ?x23088 b_S_kind_n_primitive$)))
-(let ((?x3688 (b_S_kind_n_of$ ?x3678)))
-(let (($x22849 (= ?x3688 b_S_kind_n_array$)))
-(let (($x21816 (b_S_is_n_arraytype$ ?x3678)))
-(let (($x22850 (= $x21816 $x22849)))
-(let (($x12251 (forall ((?v0 B_S_ctype$) )(!(let (($x2733 (b_S_is_n_arraytype$ ?v0)))
-(= $x2733 (= (b_S_kind_n_of$ ?v0) b_S_kind_n_array$))) :pattern ( (b_S_is_n_arraytype$ ?v0) )))
-))
-(let (($x2733 (b_S_is_n_arraytype$ ?0)))
-(let (($x12247 (= $x2733 (= (b_S_kind_n_of$ ?0) b_S_kind_n_array$))))
-(let (($x3569 (forall ((?v0 B_S_ctype$) )(!(let (($x2733 (b_S_is_n_arraytype$ ?v0)))
-(= $x2733 (= (b_S_kind_n_of$ ?v0) b_S_kind_n_array$))) :pattern ( (b_S_is_n_arraytype$ ?v0) )))
-))
-(let ((@x12250 (rewrite (= (= $x2733 (= (b_S_kind_n_of$ ?0) b_S_kind_n_array$)) $x12247))))
-(let ((@x16186 (mp~ (mp (asserted $x3569) (quant-intro @x12250 (= $x3569 $x12251)) $x12251) (nnf-pos (refl (~ $x12247 $x12247)) (~ $x12251 $x12251)) $x12251)))
-(let (($x2482 (forall ((?v0 B_S_ctype$) (?v1 Int) )(!(let ((?x2267 (b_S_array$ ?v0 ?v1)))
-(b_S_is_n_arraytype$ ?x2267)) :pattern ( (b_S_array$ ?v0 ?v1) )))
-))
-(let ((?x2267 (b_S_array$ ?1 ?0)))
-(let (($x2481 (b_S_is_n_arraytype$ ?x2267)))
-(let ((@x15316 (mp~ (asserted $x2482) (nnf-pos (refl (~ $x2481 $x2481)) (~ $x2482 $x2482)) $x2482)))
-(let ((@x24927 (unit-resolution (def-axiom (or (not $x22850) (not $x21816) $x22849)) (unit-resolution ((_ quant-inst b_T_T_u1$ v_b_P_H_len$) (or (not $x2482) $x21816)) @x15316 $x21816) (or (not $x22850) $x22849))))
-(let ((@x24928 (unit-resolution @x24927 (unit-resolution ((_ quant-inst (b_S_array$ b_T_T_u1$ v_b_P_H_len$)) (or (not $x12251) $x22850)) @x16186 $x22850) $x22849)))
-(let ((@x24406 (unit-resolution ((_ quant-inst (b_S_array$ b_T_T_u1$ v_b_P_H_len$) (b_S_ref$ ?x3680)) (or (not $x20974) (= (b_S_typ$ ?x3682) ?x3678))) @x20979 (= (b_S_typ$ ?x3682) ?x3678))))
-(let ((@x23038 (trans (monotonicity @x24449 (= ?x22935 (b_S_typ$ ?x3682))) @x24406 (= ?x22935 ?x3678))))
-(let ((@x23042 (trans (monotonicity @x23038 (= ?x23088 ?x3688)) @x24928 (= ?x23088 b_S_kind_n_array$))))
-(let ((@x23031 (monotonicity @x23042 (= $x23089 (= b_S_kind_n_array$ b_S_kind_n_primitive$)))))
-(let ((@x23049 (trans @x23031 (commutativity (= (= b_S_kind_n_array$ b_S_kind_n_primitive$) $x36)) (= $x23089 $x36))))
-(let (($x45 (and (not (= b_S_kind_n_composite$ b_S_kind_n_array$)) (and (not (= b_S_kind_n_thread$ b_S_kind_n_array$)) true))))
-(let (($x47 (and $x37 (and (not (= b_S_kind_n_composite$ b_S_kind_n_thread$)) $x45))))
-(let (($x49 (and (not (= b_S_kind_n_primitive$ b_S_kind_n_composite$)) (and (not (= b_S_kind_n_primitive$ b_S_kind_n_thread$)) $x47))))
-(let ((@x4039 (and-elim (asserted $x49) (and (not (= b_S_kind_n_primitive$ b_S_kind_n_thread$)) $x47))))
-(let ((@x23078 (mp (and-elim (and-elim @x4039 $x47) $x37) (monotonicity (symm @x23049 (= $x36 $x23089)) $x23052) (not $x23089))))
-(let (($x23034 (not $x23019)))
-(let (($x23037 (not $x23018)))
-(let ((@x23072 (monotonicity (symm (monotonicity @x24449 @x24449 (= $x23018 $x3738)) (= $x3738 $x23018)) (= $x10065 $x23037))))
-(let ((@x23071 (unit-resolution (def-axiom (or (not $x23027) $x23018 $x23034)) (mp (hypothesis $x10065) @x23072 $x23037) (unit-resolution ((_ quant-inst v_b_S_s$ (b_S_ptr$ ?x3678 ?x21715) (b_S_ptr$ ?x3678 ?x21715) b_l_H_public$) (or (not $x12066) $x23027)) @x15761 $x23027) $x23034)))
-(let (($x23069 (b_S_is$ ?x22684 ?x22935)))
-(let ((@x23095 (mp (and-elim @x10087 $x3686) (symm (monotonicity @x24449 @x23038 (= $x23069 $x3686)) (= $x3686 $x23069)) $x23069)))
-(let (($x23086 (b_S_typed$ v_b_S_s$ ?x22684)))
-(let ((@x23099 (mp (and-elim @x10087 $x3687) (symm (monotonicity @x24449 (= $x23086 $x3687)) (= $x3687 $x23086)) $x23086)))
-(let ((@x10097 (and-elim @x10087 $x3685)))
-(let ((@x23104 (trans (monotonicity @x24449 (= (b_S_owner$ v_b_S_s$ ?x22684) ?x3684)) @x10097 (= (b_S_owner$ v_b_S_s$ ?x22684) b_S_me$))))
-(let ((@x23113 (mp (and-elim @x10087 $x3683) (symm (monotonicity @x24449 (= $x22949 $x3683)) (= $x3683 $x22949)) $x22949)))
-(let (($x22936 (b_S_is_n_non_n_primitive$ ?x22935)))
-(let ((@x23118 (mp (and-elim @x10087 $x3691) (symm (monotonicity @x23038 (= $x22936 $x3691)) (= $x3691 $x22936)) $x22936)))
-(let ((@x10104 (and-elim @x10087 $x3699)))
-(let (($x19623 (forall ((?v0 B_S_state$) (?v1 B_S_ptr$) )(!(let (($x3028 (b_S_in_n_domain$ ?v0 ?v1 ?v1)))
-(let (($x1001 (= (b_S_kind_n_of$ (b_S_typ$ ?v1)) b_S_kind_n_primitive$)))
-(let (($x1106 (b_S_typed$ ?v0 ?v1)))
-(let (($x8534 (not $x1106)))
-(let (($x1098 (b_S_closed$ ?v0 ?v1)))
-(let (($x3231 (not $x1098)))
-(or (not (b_S_full_n_stop$ ?v0)) $x3231 (not (= (b_S_owner$ ?v0 ?v1) b_S_me$)) (not (b_S_is$ ?v1 (b_S_typ$ ?v1))) $x8534 $x1001 (not (b_S_is_n_non_n_primitive$ (b_S_typ$ ?v1))) $x3028))))))) :pattern ( (b_S_in_n_domain$ ?v0 ?v1 ?v1) )))
-))
-(let (($x8148 (forall ((?v0 B_S_state$) (?v1 B_S_ptr$) )(!(let (($x3028 (b_S_in_n_domain$ ?v0 ?v1 ?v1)))
-(let ((?x999 (b_S_typ$ ?v1)))
-(let (($x1042 (b_S_is_n_non_n_primitive$ ?x999)))
-(let (($x1001 (= (b_S_kind_n_of$ ?x999) b_S_kind_n_primitive$)))
-(let (($x1024 (not $x1001)))
-(let (($x1106 (b_S_typed$ ?v0 ?v1)))
-(let (($x1105 (b_S_is$ ?v1 ?x999)))
-(let ((?x1103 (b_S_owner$ ?v0 ?v1)))
-(let (($x1104 (= ?x1103 b_S_me$)))
-(let (($x1098 (b_S_closed$ ?v0 ?v1)))
-(let (($x1172 (b_S_full_n_stop$ ?v0)))
-(let (($x8134 (and $x1172 $x1098 $x1104 $x1105 $x1106 $x1024 $x1042)))
-(let (($x8142 (not $x8134)))
-(or $x8142 $x3028)))))))))))))) :pattern ( (b_S_in_n_domain$ ?v0 ?v1 ?v1) )))
-))
-(let (($x3028 (b_S_in_n_domain$ ?1 ?0 ?0)))
-(let (($x1098 (b_S_closed$ ?1 ?0)))
-(let (($x3231 (not $x1098)))
-(let (($x19618 (or (not (b_S_full_n_stop$ ?1)) $x3231 (not $x1104) (not (b_S_is$ ?0 (b_S_typ$ ?0))) $x8534 $x1001 (not (b_S_is_n_non_n_primitive$ (b_S_typ$ ?0))) $x3028)))
-(let ((?x999 (b_S_typ$ ?0)))
-(let (($x1042 (b_S_is_n_non_n_primitive$ ?x999)))
-(let (($x1105 (b_S_is$ ?0 ?x999)))
-(let (($x1172 (b_S_full_n_stop$ ?1)))
-(let (($x8134 (and $x1172 $x1098 $x1104 $x1105 $x1106 $x1024 $x1042)))
-(let (($x8142 (not $x8134)))
-(let (($x8143 (or $x8142 $x3028)))
-(let (($x19604 (or (not $x1172) $x3231 (not $x1104) (not $x1105) $x8534 $x1001 (not $x1042))))
-(let ((@x19610 (monotonicity (rewrite (= $x8134 (not $x19604))) (= $x8142 (not (not $x19604))))))
-(let ((@x19617 (monotonicity (trans @x19610 (rewrite (= (not (not $x19604)) $x19604)) (= $x8142 $x19604)) (= $x8143 (or $x19604 $x3028)))))
-(let ((@x19625 (quant-intro (trans @x19617 (rewrite (= (or $x19604 $x3028) $x19618)) (= $x8143 $x19618)) (= $x8148 $x19623))))
-(let (($x3031 (forall ((?v0 B_S_state$) (?v1 B_S_ptr$) )(!(let (($x3028 (b_S_in_n_domain$ ?v0 ?v1 ?v1)))
-(let ((?x999 (b_S_typ$ ?v1)))
-(let (($x1042 (b_S_is_n_non_n_primitive$ ?x999)))
-(let (($x1001 (= (b_S_kind_n_of$ ?x999) b_S_kind_n_primitive$)))
-(let (($x1024 (not $x1001)))
-(let (($x1106 (b_S_typed$ ?v0 ?v1)))
-(let (($x1105 (b_S_is$ ?v1 ?x999)))
-(let (($x3024 (and $x1105 (and $x1106 (and $x1024 $x1042)))))
-(let ((?x1103 (b_S_owner$ ?v0 ?v1)))
-(let (($x1104 (= ?x1103 b_S_me$)))
-(let (($x3025 (and $x1104 $x3024)))
-(let (($x1098 (b_S_closed$ ?v0 ?v1)))
-(let (($x3026 (and $x1098 $x3025)))
-(let (($x1172 (b_S_full_n_stop$ ?v0)))
-(let (($x3027 (and $x1172 $x3026)))
-(=> $x3027 $x3028)))))))))))))))) :pattern ( (b_S_in_n_domain$ ?v0 ?v1 ?v1) )))
-))
-(let (($x3024 (and $x1105 (and $x1106 (and $x1024 $x1042)))))
-(let (($x3025 (and $x1104 $x3024)))
-(let (($x3026 (and $x1098 $x3025)))
-(let (($x3027 (and $x1172 $x3026)))
-(let (($x3029 (=> $x3027 $x3028)))
-(let (($x8126 (and $x1098 $x1104 $x1105 $x1106 $x1024 $x1042)))
-(let (($x8118 (and $x1104 $x1105 $x1106 $x1024 $x1042)))
-(let ((@x8112 (rewrite (= (and $x1105 (and $x1106 $x1024 $x1042)) (and $x1105 $x1106 $x1024 $x1042)))))
-(let ((@x8109 (monotonicity (rewrite (= (and $x1106 (and $x1024 $x1042)) (and $x1106 $x1024 $x1042))) (= $x3024 (and $x1105 (and $x1106 $x1024 $x1042))))))
-(let ((@x8117 (monotonicity (trans @x8109 @x8112 (= $x3024 (and $x1105 $x1106 $x1024 $x1042))) (= $x3025 (and $x1104 (and $x1105 $x1106 $x1024 $x1042))))))
-(let ((@x8122 (trans @x8117 (rewrite (= (and $x1104 (and $x1105 $x1106 $x1024 $x1042)) $x8118)) (= $x3025 $x8118))))
-(let ((@x8130 (trans (monotonicity @x8122 (= $x3026 (and $x1098 $x8118))) (rewrite (= (and $x1098 $x8118) $x8126)) (= $x3026 $x8126))))
-(let ((@x8138 (trans (monotonicity @x8130 (= $x3027 (and $x1172 $x8126))) (rewrite (= (and $x1172 $x8126) $x8134)) (= $x3027 $x8134))))
-(let ((@x8147 (trans (monotonicity @x8138 (= $x3029 (=> $x8134 $x3028))) (rewrite (= (=> $x8134 $x3028) $x8143)) (= $x3029 $x8143))))
-(let ((@x15729 (mp~ (mp (asserted $x3031) (quant-intro @x8147 (= $x3031 $x8148)) $x8148) (nnf-pos (refl (~ $x8143 $x8143)) (~ $x8148 $x8148)) $x8148)))
-(let (($x23087 (not $x23086)))
-(let (($x23085 (not $x23069)))
-(let (($x21687 (not $x3699)))
-(let (($x24394 (or (not $x19623) $x21687 $x22973 (not (= (b_S_owner$ v_b_S_s$ ?x22684) b_S_me$)) $x23085 $x23087 $x23089 (not $x22936) $x23019)))
-(let (($x23090 (or $x21687 $x22973 (not (= (b_S_owner$ v_b_S_s$ ?x22684) b_S_me$)) $x23085 $x23087 $x23089 (not $x22936) $x23019)))
-(let ((@x24401 (mp ((_ quant-inst v_b_S_s$ (b_S_ptr$ ?x3678 ?x21715)) (or (not $x19623) $x23090)) (rewrite (= (or (not $x19623) $x23090) $x24394)) $x24394)))
-(let ((@x23120 (unit-resolution @x24401 (mp @x15729 @x19625 $x19623) @x10104 @x23118 @x23113 @x23104 (or $x23085 $x23087 $x23089 $x23019))))
-(let ((@x23328 (mp (lemma (unit-resolution @x23120 @x23099 @x23095 @x23071 @x23078 false) $x3738) (symm (monotonicity @x24449 @x24449 (= $x23018 $x3738)) (= $x3738 $x23018)) $x23018)))
-(let ((@x23329 (unit-resolution (def-axiom (or (not $x23027) $x23037 $x23019)) @x23328 (unit-resolution ((_ quant-inst v_b_S_s$ (b_S_ptr$ ?x3678 ?x21715) (b_S_ptr$ ?x3678 ?x21715) b_l_H_public$) (or (not $x12066) $x23027)) @x15761 $x23027) $x23019)))
-(let (($x19663 (forall ((?v0 B_S_state$) (?v1 B_S_ptr$) (?v2 B_S_ptr$) )(!(let (($x19647 (forall ((?v3 B_S_ptr$) )(!(let (($x3038 (b_S_set_n_in2$ ?v3 (b_S_ver_n_domain$ (b_S_read_n_version$ ?v0 ?v2)))))
-(let ((?x2289 (b_S_typ$ ?v1)))
-(let (($x3032 (b_S_has_n_volatile_n_owns_n_set$ ?x2289)))
-(or $x3032 (not (b_S_set_n_in$ ?v3 (b_S_owns$ ?v0 ?v1))) $x3038)))) :pattern ( (b_S_set_n_in$ ?v3 (b_S_owns$ ?v0 ?v1)) )))
-))
-(let (($x19654 (or (not (b_S_set_n_in$ ?v1 (b_S_domain$ ?v0 ?v2))) (not (b_S_closed$ ?v0 ?v1)) (not $x19647))))
-(let (($x19655 (not $x19654)))
-(let (($x2979 (b_S_in_n_domain$ ?v0 ?v1 ?v2)))
-(let (($x8173 (not $x2979)))
-(or $x8173 $x19655)))))) :pattern ( (b_S_in_n_domain$ ?v0 ?v1 ?v2) )))
-))
-(let (($x8179 (forall ((?v0 B_S_state$) (?v1 B_S_ptr$) (?v2 B_S_ptr$) )(!(let (($x8156 (forall ((?v3 B_S_ptr$) )(!(let (($x3038 (b_S_set_n_in2$ ?v3 (b_S_ver_n_domain$ (b_S_read_n_version$ ?v0 ?v2)))))
-(let (($x3035 (b_S_set_n_in$ ?v3 (b_S_owns$ ?v0 ?v1))))
-(let (($x3036 (and (not (b_S_has_n_volatile_n_owns_n_set$ (b_S_typ$ ?v1))) $x3035)))
-(let (($x8152 (not $x3036)))
-(or $x8152 $x3038))))) :pattern ( (b_S_set_n_in$ ?v3 (b_S_owns$ ?v0 ?v1)) )))
-))
-(let (($x1136 (b_S_closed$ ?v0 ?v1)))
-(let (($x2963 (b_S_set_n_in$ ?v1 (b_S_domain$ ?v0 ?v2))))
-(let (($x8165 (and $x2963 $x1136 $x8156)))
-(let (($x2979 (b_S_in_n_domain$ ?v0 ?v1 ?v2)))
-(let (($x8173 (not $x2979)))
-(or $x8173 $x8165))))))) :pattern ( (b_S_in_n_domain$ ?v0 ?v1 ?v2) )))
-))
-(let (($x19647 (forall ((?v3 B_S_ptr$) )(!(let (($x3038 (b_S_set_n_in2$ ?v3 (b_S_ver_n_domain$ (b_S_read_n_version$ ?2 ?0)))))
-(let ((?x2289 (b_S_typ$ ?1)))
-(let (($x3032 (b_S_has_n_volatile_n_owns_n_set$ ?x2289)))
-(or $x3032 (not (b_S_set_n_in$ ?v3 (b_S_owns$ ?2 ?1))) $x3038)))) :pattern ( (b_S_set_n_in$ ?v3 (b_S_owns$ ?2 ?1)) )))
-))
-(let (($x19654 (or (not (b_S_set_n_in$ ?1 (b_S_domain$ ?2 ?0))) (not (b_S_closed$ ?2 ?1)) (not $x19647))))
-(let (($x19655 (not $x19654)))
-(let (($x2979 (b_S_in_n_domain$ ?2 ?1 ?0)))
-(let (($x8173 (not $x2979)))
-(let (($x8156 (forall ((?v3 B_S_ptr$) )(!(let (($x3038 (b_S_set_n_in2$ ?v3 (b_S_ver_n_domain$ (b_S_read_n_version$ ?2 ?0)))))
-(let (($x3035 (b_S_set_n_in$ ?v3 (b_S_owns$ ?2 ?1))))
-(let (($x3036 (and (not (b_S_has_n_volatile_n_owns_n_set$ (b_S_typ$ ?1))) $x3035)))
-(let (($x8152 (not $x3036)))
-(or $x8152 $x3038))))) :pattern ( (b_S_set_n_in$ ?v3 (b_S_owns$ ?2 ?1)) )))
-))
-(let (($x1136 (b_S_closed$ ?2 ?1)))
-(let (($x2963 (b_S_set_n_in$ ?1 (b_S_domain$ ?2 ?0))))
-(let (($x8165 (and $x2963 $x1136 $x8156)))
-(let (($x8174 (or $x8173 $x8165)))
-(let (($x3038 (b_S_set_n_in2$ ?0 (b_S_ver_n_domain$ (b_S_read_n_version$ ?3 ?1)))))
-(let ((?x2289 (b_S_typ$ ?2)))
-(let (($x3032 (b_S_has_n_volatile_n_owns_n_set$ ?x2289)))
-(let (($x19642 (or $x3032 (not (b_S_set_n_in$ ?0 (b_S_owns$ ?3 ?2))) $x3038)))
-(let (($x3035 (b_S_set_n_in$ ?0 (b_S_owns$ ?3 ?2))))
-(let (($x3036 (and (not $x3032) $x3035)))
-(let (($x8152 (not $x3036)))
-(let (($x8153 (or $x8152 $x3038)))
-(let ((@x19636 (rewrite (= (not (not (or $x3032 (not $x3035)))) (or $x3032 (not $x3035))))))
-(let ((@x19634 (monotonicity (rewrite (= $x3036 (not (or $x3032 (not $x3035))))) (= $x8152 (not (not (or $x3032 (not $x3035))))))))
-(let ((@x19641 (monotonicity (trans @x19634 @x19636 (= $x8152 (or $x3032 (not $x3035)))) (= $x8153 (or (or $x3032 (not $x3035)) $x3038)))))
-(let ((@x19646 (trans @x19641 (rewrite (= (or (or $x3032 (not $x3035)) $x3038) $x19642)) (= $x8153 $x19642))))
-(let ((@x19652 (monotonicity (quant-intro @x19646 (= $x8156 $x19647)) (= $x8165 (and $x2963 $x1136 $x19647)))))
-(let ((@x19659 (trans @x19652 (rewrite (= (and $x2963 $x1136 $x19647) $x19655)) (= $x8165 $x19655))))
-(let ((@x19665 (quant-intro (monotonicity @x19659 (= $x8174 (or $x8173 $x19655))) (= $x8179 $x19663))))
-(let ((@x15741 (monotonicity (refl (~ $x2963 $x2963)) (refl (~ $x1136 $x1136)) (nnf-pos (refl (~ $x8153 $x8153)) (~ $x8156 $x8156)) (~ $x8165 $x8165))))
-(let ((@x15745 (nnf-pos (monotonicity (refl (~ $x8173 $x8173)) @x15741 (~ $x8174 $x8174)) (~ $x8179 $x8179))))
-(let (($x3046 (forall ((?v0 B_S_state$) (?v1 B_S_ptr$) (?v2 B_S_ptr$) )(!(let (($x3041 (forall ((?v3 B_S_ptr$) )(!(let (($x3038 (b_S_set_n_in2$ ?v3 (b_S_ver_n_domain$ (b_S_read_n_version$ ?v0 ?v2)))))
-(let (($x3035 (b_S_set_n_in$ ?v3 (b_S_owns$ ?v0 ?v1))))
-(let (($x3036 (and (not (b_S_has_n_volatile_n_owns_n_set$ (b_S_typ$ ?v1))) $x3035)))
-(=> $x3036 $x3038)))) :pattern ( (b_S_set_n_in$ ?v3 (b_S_owns$ ?v0 ?v1)) )))
-))
-(let (($x1136 (b_S_closed$ ?v0 ?v1)))
-(let (($x2963 (b_S_set_n_in$ ?v1 (b_S_domain$ ?v0 ?v2))))
-(let (($x3043 (and $x2963 (and $x1136 $x3041))))
-(let (($x2979 (b_S_in_n_domain$ ?v0 ?v1 ?v2)))
-(=> $x2979 $x3043)))))) :pattern ( (b_S_in_n_domain$ ?v0 ?v1 ?v2) )))
-))
-(let (($x3041 (forall ((?v3 B_S_ptr$) )(!(let (($x3038 (b_S_set_n_in2$ ?v3 (b_S_ver_n_domain$ (b_S_read_n_version$ ?2 ?0)))))
-(let (($x3035 (b_S_set_n_in$ ?v3 (b_S_owns$ ?2 ?1))))
-(let (($x3036 (and (not (b_S_has_n_volatile_n_owns_n_set$ (b_S_typ$ ?1))) $x3035)))
-(=> $x3036 $x3038)))) :pattern ( (b_S_set_n_in$ ?v3 (b_S_owns$ ?2 ?1)) )))
-))
-(let (($x3043 (and $x2963 (and $x1136 $x3041))))
-(let (($x3044 (=> $x2979 $x3043)))
-(let ((@x8161 (monotonicity (quant-intro (rewrite (= (=> $x3036 $x3038) $x8153)) (= $x3041 $x8156)) (= (and $x1136 $x3041) (and $x1136 $x8156)))))
-(let ((@x8169 (trans (monotonicity @x8161 (= $x3043 (and $x2963 (and $x1136 $x8156)))) (rewrite (= (and $x2963 (and $x1136 $x8156)) $x8165)) (= $x3043 $x8165))))
-(let ((@x8178 (trans (monotonicity @x8169 (= $x3044 (=> $x2979 $x8165))) (rewrite (= (=> $x2979 $x8165) $x8174)) (= $x3044 $x8174))))
-(let ((@x15746 (mp~ (mp (asserted $x3046) (quant-intro @x8178 (= $x3046 $x8179)) $x8179) @x15745 $x8179)))
-(let ((@x24384 (rewrite (= (or (not $x19663) (or $x23034 $x23066)) (or (not $x19663) $x23034 $x23066)))))
-(let ((@x24402 (mp ((_ quant-inst v_b_S_s$ (b_S_ptr$ ?x3678 ?x21715) (b_S_ptr$ ?x3678 ?x21715)) (or (not $x19663) (or $x23034 $x23066))) @x24384 (or (not $x19663) $x23034 $x23066))))
-(let ((@x23335 (unit-resolution (unit-resolution @x24402 (mp @x15746 @x19665 $x19663) (or $x23034 $x23066)) @x23329 $x23066)))
-(let ((@x23336 (unit-resolution (def-axiom (or (or (not $x23045) $x22973 (not $x23063)) $x23045)) @x23335 $x23045)))
-(let (($x19385 (forall ((?v0 B_S_state$) (?v1 Int) (?v2 B_S_ptr$) (?v3 Int) (?v4 Int) (?v5 B_S_ctype$) )(!(let ((?x2903 (b_S_idx$ (b_S_ptr$ ?v5 ?v1) ?v4 ?v5)))
-(let ((?x2429 (b_S_typemap$ ?v0)))
-(let (($x19373 (or (not (b_S_typed$ ?v0 ?x2903)) (b_S_ts_n_is_n_volatile$ (b_S_select_o_tm$ ?x2429 ?x2903)))))
-(let (($x19374 (not $x19373)))
-(let (($x11257 (>= (+ ?v4 (* (- 1) ?v3)) 0)))
-(let (($x2898 (b_S_set_n_in$ (b_S_ptr$ (b_S_array$ ?v5 ?v3) ?v1) (b_S_domain$ ?v0 ?v2))))
-(or (not (b_S_full_n_stop$ ?v0)) (not (b_S_is_n_primitive$ ?v5)) (not $x2898) (not (>= ?v4 0)) $x11257 $x19374))))))) :pattern ( (b_S_set_n_in$ (b_S_ptr$ (b_S_array$ ?v5 ?v3) ?v1) (b_S_domain$ ?v0 ?v2)) (b_S_select_o_tm$ (b_S_typemap$ ?v0) (b_S_idx$ (b_S_ptr$ ?v5 ?v1) ?v4 ?v5)) (b_S_is_n_primitive$ ?v5) ) :pattern ( (b_S_set_n_in$ (b_S_ptr$ (b_S_array$ ?v5 ?v3) ?v1) (b_S_domain$ ?v0 ?v2)) (b_S_owner$ ?v0 (b_S_idx$ (b_S_ptr$ ?v5 ?v1) ?v4 ?v5)) (b_S_is_n_primitive$ ?v5) )))
-))
-(let (($x12034 (forall ((?v0 B_S_state$) (?v1 Int) (?v2 B_S_ptr$) (?v3 Int) (?v4 Int) (?v5 B_S_ctype$) )(!(let ((?x2903 (b_S_idx$ (b_S_ptr$ ?v5 ?v1) ?v4 ?v5)))
-(let ((?x2429 (b_S_typemap$ ?v0)))
-(let (($x2915 (and (b_S_typed$ ?v0 ?x2903) (not (b_S_ts_n_is_n_volatile$ (b_S_select_o_tm$ ?x2429 ?x2903))))))
-(let (($x10181 (>= ?v4 0)))
-(let (($x2898 (b_S_set_n_in$ (b_S_ptr$ (b_S_array$ ?v5 ?v3) ?v1) (b_S_domain$ ?v0 ?v2))))
-(let (($x1179 (b_S_is_n_primitive$ ?v5)))
-(let (($x2894 (b_S_full_n_stop$ ?v0)))
-(let (($x12018 (and $x2894 $x1179 $x2898 $x10181 (not (>= (+ ?v4 (* (- 1) ?v3)) 0)))))
-(let (($x12021 (not $x12018)))
-(or $x12021 $x2915)))))))))) :pattern ( (b_S_set_n_in$ (b_S_ptr$ (b_S_array$ ?v5 ?v3) ?v1) (b_S_domain$ ?v0 ?v2)) (b_S_select_o_tm$ (b_S_typemap$ ?v0) (b_S_idx$ (b_S_ptr$ ?v5 ?v1) ?v4 ?v5)) (b_S_is_n_primitive$ ?v5) ) :pattern ( (b_S_set_n_in$ (b_S_ptr$ (b_S_array$ ?v5 ?v3) ?v1) (b_S_domain$ ?v0 ?v2)) (b_S_owner$ ?v0 (b_S_idx$ (b_S_ptr$ ?v5 ?v1) ?v4 ?v5)) (b_S_is_n_primitive$ ?v5) )))
-))
-(let ((?x2903 (b_S_idx$ (b_S_ptr$ ?0 ?4) ?1 ?0)))
-(let ((?x2429 (b_S_typemap$ ?5)))
-(let (($x19373 (or (not (b_S_typed$ ?5 ?x2903)) (b_S_ts_n_is_n_volatile$ (b_S_select_o_tm$ ?x2429 ?x2903)))))
-(let (($x19374 (not $x19373)))
-(let (($x11257 (>= (+ ?1 (* (- 1) ?2)) 0)))
-(let (($x2898 (b_S_set_n_in$ (b_S_ptr$ (b_S_array$ ?0 ?2) ?4) (b_S_domain$ ?5 ?3))))
-(let (($x19380 (or (not (b_S_full_n_stop$ ?5)) (not $x1179) (not $x2898) (not (>= ?1 0)) $x11257 $x19374)))
-(let (($x2915 (and (b_S_typed$ ?5 ?x2903) (not (b_S_ts_n_is_n_volatile$ (b_S_select_o_tm$ ?x2429 ?x2903))))))
-(let (($x10181 (>= ?1 0)))
-(let (($x2894 (b_S_full_n_stop$ ?5)))
-(let (($x12018 (and $x2894 $x1179 $x2898 $x10181 (not $x11257))))
-(let (($x12021 (not $x12018)))
-(let (($x12031 (or $x12021 $x2915)))
-(let (($x19381 (= (or (or (not $x2894) (not $x1179) (not $x2898) (not $x10181) $x11257) $x19374) $x19380)))
-(let (($x19378 (= $x12031 (or (or (not $x2894) (not $x1179) (not $x2898) (not $x10181) $x11257) $x19374))))
-(let (($x19349 (or (not $x2894) (not $x1179) (not $x2898) (not $x10181) $x11257)))
-(let ((@x19355 (monotonicity (rewrite (= $x12018 (not $x19349))) (= $x12021 (not (not $x19349))))))
-(let ((@x19379 (monotonicity (trans @x19355 (rewrite (= (not (not $x19349)) $x19349)) (= $x12021 $x19349)) (rewrite (= $x2915 $x19374)) $x19378)))
-(let ((@x19387 (quant-intro (trans @x19379 (rewrite $x19381) (= $x12031 $x19380)) (= $x12034 $x19385))))
-(let (($x7948 (forall ((?v0 B_S_state$) (?v1 Int) (?v2 B_S_ptr$) (?v3 Int) (?v4 Int) (?v5 B_S_ctype$) )(!(let ((?x2903 (b_S_idx$ (b_S_ptr$ ?v5 ?v1) ?v4 ?v5)))
-(let ((?x2429 (b_S_typemap$ ?v0)))
-(let (($x2915 (and (b_S_typed$ ?v0 ?x2903) (not (b_S_ts_n_is_n_volatile$ (b_S_select_o_tm$ ?x2429 ?x2903))))))
-(let (($x1751 (<= ?v3 ?v4)))
-(let (($x7247 (not $x1751)))
-(let (($x1330 (<= 0 ?v4)))
-(let (($x2898 (b_S_set_n_in$ (b_S_ptr$ (b_S_array$ ?v5 ?v3) ?v1) (b_S_domain$ ?v0 ?v2))))
-(let (($x1179 (b_S_is_n_primitive$ ?v5)))
-(let (($x2894 (b_S_full_n_stop$ ?v0)))
-(let (($x7922 (and $x2894 $x1179 $x2898 $x1330 $x7247)))
-(or (not $x7922) $x2915))))))))))) :pattern ( (b_S_set_n_in$ (b_S_ptr$ (b_S_array$ ?v5 ?v3) ?v1) (b_S_domain$ ?v0 ?v2)) (b_S_select_o_tm$ (b_S_typemap$ ?v0) (b_S_idx$ (b_S_ptr$ ?v5 ?v1) ?v4 ?v5)) (b_S_is_n_primitive$ ?v5) ) :pattern ( (b_S_set_n_in$ (b_S_ptr$ (b_S_array$ ?v5 ?v3) ?v1) (b_S_domain$ ?v0 ?v2)) (b_S_owner$ ?v0 (b_S_idx$ (b_S_ptr$ ?v5 ?v1) ?v4 ?v5)) (b_S_is_n_primitive$ ?v5) )))
-))
-(let (($x7943 (or (not (and $x2894 $x1179 $x2898 (<= 0 ?1) (not (<= ?2 ?1)))) $x2915)))
-(let (($x12022 (= (not (and $x2894 $x1179 $x2898 (<= 0 ?1) (not (<= ?2 ?1)))) $x12021)))
-(let (($x1751 (<= ?2 ?1)))
-(let (($x7247 (not $x1751)))
-(let (($x1330 (<= 0 ?1)))
-(let (($x7922 (and $x2894 $x1179 $x2898 $x1330 $x7247)))
-(let ((@x12020 (monotonicity (rewrite (= $x1330 $x10181)) (monotonicity (rewrite (= $x1751 $x11257)) (= $x7247 (not $x11257))) (= $x7922 $x12018))))
-(let ((@x12036 (quant-intro (monotonicity (monotonicity @x12020 $x12022) (= $x7943 $x12031)) (= $x7948 $x12034))))
-(let (($x2920 (forall ((?v0 B_S_state$) (?v1 Int) (?v2 B_S_ptr$) (?v3 Int) (?v4 Int) (?v5 B_S_ctype$) )(!(let ((?x2903 (b_S_idx$ (b_S_ptr$ ?v5 ?v1) ?v4 ?v5)))
-(let ((?x2429 (b_S_typemap$ ?v0)))
-(let (($x2915 (and (b_S_typed$ ?v0 ?x2903) (not (b_S_ts_n_is_n_volatile$ (b_S_select_o_tm$ ?x2429 ?x2903))))))
-(let (($x1330 (<= 0 ?v4)))
-(let (($x2333 (and $x1330 (< ?v4 ?v3))))
-(let (($x2898 (b_S_set_n_in$ (b_S_ptr$ (b_S_array$ ?v5 ?v3) ?v1) (b_S_domain$ ?v0 ?v2))))
-(let (($x2899 (and $x2898 $x2333)))
-(let (($x1179 (b_S_is_n_primitive$ ?v5)))
-(let (($x2900 (and $x1179 $x2899)))
-(let (($x2894 (b_S_full_n_stop$ ?v0)))
-(let (($x2901 (and $x2894 $x2900)))
-(=> $x2901 $x2915)))))))))))) :pattern ( (b_S_set_n_in$ (b_S_ptr$ (b_S_array$ ?v5 ?v3) ?v1) (b_S_domain$ ?v0 ?v2)) (b_S_select_o_tm$ (b_S_typemap$ ?v0) (b_S_idx$ (b_S_ptr$ ?v5 ?v1) ?v4 ?v5)) (b_S_is_n_primitive$ ?v5) ) :pattern ( (b_S_set_n_in$ (b_S_ptr$ (b_S_array$ ?v5 ?v3) ?v1) (b_S_domain$ ?v0 ?v2)) (b_S_owner$ ?v0 (b_S_idx$ (b_S_ptr$ ?v5 ?v1) ?v4 ?v5)) (b_S_is_n_primitive$ ?v5) )))
-))
-(let (($x2333 (and $x1330 (< ?1 ?2))))
-(let (($x2899 (and $x2898 $x2333)))
-(let (($x2900 (and $x1179 $x2899)))
-(let (($x2901 (and $x2894 $x2900)))
-(let (($x2916 (=> $x2901 $x2915)))
-(let ((@x7916 (rewrite (= (and $x1179 (and $x2898 $x1330 $x7247)) (and $x1179 $x2898 $x1330 $x7247)))))
-(let ((@x7252 (monotonicity (rewrite (= $x1330 $x1330)) (rewrite (= (< ?1 ?2) $x7247)) (= $x2333 (and $x1330 $x7247)))))
-(let ((@x7910 (trans (monotonicity @x7252 (= $x2899 (and $x2898 (and $x1330 $x7247)))) (rewrite (= (and $x2898 (and $x1330 $x7247)) (and $x2898 $x1330 $x7247))) (= $x2899 (and $x2898 $x1330 $x7247)))))
-(let ((@x7918 (trans (monotonicity @x7910 (= $x2900 (and $x1179 (and $x2898 $x1330 $x7247)))) @x7916 (= $x2900 (and $x1179 $x2898 $x1330 $x7247)))))
-(let ((@x7926 (trans (monotonicity @x7918 (= $x2901 (and $x2894 (and $x1179 $x2898 $x1330 $x7247)))) (rewrite (= (and $x2894 (and $x1179 $x2898 $x1330 $x7247)) $x7922)) (= $x2901 $x7922))))
-(let ((@x7947 (trans (monotonicity @x7926 (= $x2916 (=> $x7922 $x2915))) (rewrite (= (=> $x7922 $x2915) $x7943)) (= $x2916 $x7943))))
-(let ((@x12037 (mp (mp (asserted $x2920) (quant-intro @x7947 (= $x2920 $x7948)) $x7948) @x12036 $x12034)))
-(let ((@x19388 (mp (mp~ @x12037 (nnf-pos (refl (~ $x12031 $x12031)) (~ $x12034 $x12034)) $x12034) @x19387 $x19385)))
-(let (($x23298 (not $x23297)))
-(let (($x22190 (not $x3529)))
-(let (($x23330 (not $x19385)))
-(let (($x23309 (or $x23330 $x21687 $x22190 $x23298 $x8666 $x23305)))
-(let (($x23302 (>= (+ 0 (* (- 1) v_b_P_H_len$)) 0)))
-(let (($x23300 (not (>= 0 0))))
-(let (($x23306 (or $x21687 $x22190 $x23298 $x23300 $x23302 $x23305)))
-(let (($x23310 (or $x23330 $x23306)))
-(let (($x23348 (or $x21687 $x22190 $x23298 $x8666 $x23305)))
-(let ((@x23277 (rewrite (= (+ 0 (* (- 1) v_b_P_H_len$)) (* (- 1) v_b_P_H_len$)))))
-(let ((@x23344 (trans (monotonicity @x23277 (= $x23302 (>= (* (- 1) v_b_P_H_len$) 0))) (rewrite (= (>= (* (- 1) v_b_P_H_len$) 0) $x8666)) (= $x23302 $x8666))))
-(let ((@x23275 (trans (monotonicity (rewrite (= (>= 0 0) true)) (= $x23300 $x3805)) (rewrite (= $x3805 false)) (= $x23300 false))))
-(let ((@x23347 (monotonicity @x23275 @x23344 (= $x23306 (or $x21687 $x22190 $x23298 false $x8666 $x23305)))))
-(let ((@x23308 (trans @x23347 (rewrite (= (or $x21687 $x22190 $x23298 false $x8666 $x23305) $x23348)) (= $x23306 $x23348))))
-(let ((@x23318 (trans (monotonicity @x23308 (= $x23310 (or $x23330 $x23348))) (rewrite (= (or $x23330 $x23348) $x23309)) (= $x23310 $x23309))))
-(let ((@x23396 (unit-resolution (mp ((_ quant-inst v_b_S_s$ v_b_P_H_arr$ (b_S_ptr$ ?x3678 ?x21715) v_b_P_H_len$ 0 b_T_T_u1$) $x23310) @x23318 $x23309) @x19388 @x5093 @x10095 @x10104 (mp @x23336 @x23394 $x23297) (hypothesis $x23304) false)))
-(let ((@x23503 (mp (unit-resolution (def-axiom (or $x23304 $x23260)) (lemma @x23396 $x23305) $x23260) @x23522 $x23358)))
-(let (($x23368 (= (b_S_owner$ v_b_S_s$ (b_S_ts_n_emb$ ?x23356)) b_S_me$)))
-(let (($x23370 (or $x23368 (b_S_in_n_wrapped_n_domain$ v_b_S_s$ (b_S_ts_n_emb$ ?x23356)))))
-(let (($x23366 (= (b_S_kind_n_of$ (b_S_typ$ (b_S_ts_n_emb$ ?x23356))) b_S_kind_n_primitive$)))
-(let (($x23363 (not $x23362)))
-(let (($x23355 (not $x23354)))
-(let (($x23372 (or $x23355 $x23363 $x23366 (not $x23370))))
-(let (($x23377 (or (= (b_S_owner$ v_b_S_s$ ?x23206) b_S_me$) (b_S_in_n_wrapped_n_domain$ v_b_S_s$ ?x23206))))
-(let (($x23373 (not $x23372)))
-(let (($x23382 (not (or $x23373 (not (or $x23354 (not $x23377)))))))
-(let (($x23383 (or (not (b_S_typed$ v_b_S_s$ ?x23206)) $x23382)))
-(let (($x23349 (b_S_thread_n_local$ v_b_S_s$ ?x23206)))
-(let (($x23385 (= $x23349 (not $x23383))))
-(let ((@x23535 (monotonicity (symm (monotonicity @x23922 (= $x23349 $x3743)) (= $x3743 $x23349)) (= $x16251 (not $x23349)))))
-(let ((@x23541 (unit-resolution (def-axiom (or (not $x23385) $x23349 $x23383)) (mp (hypothesis $x16251) @x23535 (not $x23349)) (unit-resolution ((_ quant-inst v_b_S_s$ (b_S_ptr$ b_T_T_u1$ ?x23186)) (or (not $x19790) $x23385)) @x19793 $x23385) $x23383)))
-(let (($x23350 (b_S_typed$ v_b_S_s$ ?x23206)))
-(let ((@x23928 (mp (unit-resolution (def-axiom (or $x23304 $x3741)) (lemma @x23396 $x23305) $x3741) (symm (monotonicity @x23922 (= $x23350 $x3741)) (= $x3741 $x23350)) $x23350)))
-(let ((@x23600 (unit-resolution (def-axiom (or (not $x23383) (not $x23350) $x23382)) @x23928 @x23541 $x23382)))
-(let ((@x23583 (unit-resolution (def-axiom (or (or $x23373 (not (or $x23354 (not $x23377)))) $x23372)) @x23600 $x23372)))
-(let ((?x24269 (b_S_ref$ ?x22684)))
-(let ((?x24283 (b_S_ptr$ b_T_T_u1$ ?x24269)))
-(let ((?x24260 (b_S_idx$ ?x22684 0 b_T_T_u1$)))
-(let (($x24286 (= ?x24260 ?x24283)))
-(let (($x24289 (not $x24286)))
-(let (($x24292 (or (not (b_S_extent_n_hint$ ?x24260 ?x22684)) $x24289)))
-(let (($x24232 (not $x24292)))
-(let (($x24310 (or $x23217 $x24232)))
-(let (($x24274 (or (not (b_S_extent_n_hint$ ?x24260 ?x22684)) (not (= ?x24260 (b_S_ptr$ b_T_T_u1$ (+ ?x24269 (* 0 ?x3652))))))))
-(let (($x24290 (= (not (= ?x24260 (b_S_ptr$ b_T_T_u1$ (+ ?x24269 (* 0 ?x3652))))) $x24289)))
-(let ((@x24278 (monotonicity (rewrite (= (* 0 ?x3652) 0)) (= (+ ?x24269 (* 0 ?x3652)) (+ ?x24269 0)))))
-(let ((@x24282 (trans @x24278 (rewrite (= (+ ?x24269 0) ?x24269)) (= (+ ?x24269 (* 0 ?x3652)) ?x24269))))
-(let ((@x24285 (monotonicity @x24282 (= (b_S_ptr$ b_T_T_u1$ (+ ?x24269 (* 0 ?x3652))) ?x24283))))
-(let ((@x24288 (monotonicity @x24285 (= (= ?x24260 (b_S_ptr$ b_T_T_u1$ (+ ?x24269 (* 0 ?x3652)))) $x24286))))
-(let ((@x24309 (monotonicity (monotonicity (monotonicity @x24288 $x24290) (= $x24274 $x24292)) (= (not $x24274) $x24232))))
-(let ((@x24303 (trans (monotonicity @x24309 (= (or $x23217 (not $x24274)) $x24310)) (rewrite (= $x24310 $x24310)) (= (or $x23217 (not $x24274)) $x24310))))
-(let ((@x24501 (unit-resolution (mp ((_ quant-inst (b_S_ptr$ ?x3678 ?x21715) 0 b_T_T_u1$) (or $x23217 (not $x24274))) @x24303 $x24310) @x18901 (hypothesis $x24292) false)))
-(let (($x24111 (= (b_S_ts_n_emb$ (b_S_select_o_tm$ ?x3874 (b_S_idx$ ?x23296 0 b_T_T_u1$))) ?x23296)))
-(let ((?x24137 (b_S_idx$ ?x23296 0 b_T_T_u1$)))
-(let ((?x24145 (b_S_select_o_tm$ ?x3874 ?x24137)))
-(let (($x24127 (or (not $x24111) (b_S_ts_n_is_n_volatile$ ?x24145) (not (b_S_ts_n_is_n_array_n_elt$ ?x24145)) (not (b_S_typed$ v_b_S_s$ ?x24137)))))
-(let (($x24130 (not $x24127)))
-(let (($x24131 (b_S_typed$ v_b_S_s$ ?x23296)))
-(let ((@x24253 (mp (and-elim @x10087 $x3687) (symm (monotonicity @x23339 (= $x24131 $x3687)) (= $x3687 $x24131)) $x24131)))
-(let (($x18682 (forall ((?v0 B_S_state$) (?v1 Int) (?v2 B_S_ctype$) (?v3 Int) (?v4 Int) )(!(let (($x2378 (b_S_typed$ ?v0 (b_S_idx$ (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) ?v4 ?v2))))
-(let ((?x2370 (b_S_typemap$ ?v0)))
-(let ((?x2372 (b_S_select_o_tm$ ?x2370 (b_S_idx$ (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) ?v4 ?v2))))
-(let (($x2377 (b_S_ts_n_is_n_array_n_elt$ ?x2372)))
-(let (($x18670 (or (not (= (b_S_ts_n_emb$ ?x2372) (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1))) (b_S_ts_n_is_n_volatile$ ?x2372) (not $x2377) (not $x2378))))
-(let (($x18671 (not $x18670)))
-(let (($x11071 (>= (+ ?v4 (* (- 1) ?v3)) 0)))
-(let (($x10138 (>= ?v4 0)))
-(let (($x10556 (not $x10138)))
-(or (not (b_S_typed$ ?v0 (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1))) $x10556 $x11071 $x18671)))))))))) :pattern ( (b_S_select_o_sm$ (b_S_statusmap$ ?v0) (b_S_idx$ (b_S_ptr$ ?v2 ?v1) ?v4 ?v2)) (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) ) :pattern ( (b_S_select_o_tm$ (b_S_typemap$ ?v0) (b_S_idx$ (b_S_ptr$ ?v2 ?v1) ?v4 ?v2)) (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) )))
-))
-(let (($x11697 (forall ((?v0 B_S_state$) (?v1 Int) (?v2 B_S_ctype$) (?v3 Int) (?v4 Int) )(!(let (($x2378 (b_S_typed$ ?v0 (b_S_idx$ (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) ?v4 ?v2))))
-(let ((?x2370 (b_S_typemap$ ?v0)))
-(let ((?x2372 (b_S_select_o_tm$ ?x2370 (b_S_idx$ (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) ?v4 ?v2))))
-(let (($x2377 (b_S_ts_n_is_n_array_n_elt$ ?x2372)))
-(let (($x2376 (not (b_S_ts_n_is_n_volatile$ ?x2372))))
-(let ((?x2367 (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1)))
-(let (($x2374 (= (b_S_ts_n_emb$ ?x2372) ?x2367)))
-(let (($x7338 (and $x2374 $x2376 $x2377 $x2378)))
-(let (($x10138 (>= ?v4 0)))
-(let (($x2368 (b_S_typed$ ?v0 ?x2367)))
-(let (($x11688 (and $x2368 $x10138 (not (>= (+ ?v4 (* (- 1) ?v3)) 0)))))
-(let (($x11691 (not $x11688)))
-(or $x11691 $x7338))))))))))))) :pattern ( (b_S_select_o_sm$ (b_S_statusmap$ ?v0) (b_S_idx$ (b_S_ptr$ ?v2 ?v1) ?v4 ?v2)) (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) ) :pattern ( (b_S_select_o_tm$ (b_S_typemap$ ?v0) (b_S_idx$ (b_S_ptr$ ?v2 ?v1) ?v4 ?v2)) (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) )))
-))
-(let (($x2378 (b_S_typed$ ?4 (b_S_idx$ (b_S_ptr$ (b_S_array$ ?2 ?1) ?3) ?0 ?2))))
-(let ((?x2370 (b_S_typemap$ ?4)))
-(let ((?x2372 (b_S_select_o_tm$ ?x2370 (b_S_idx$ (b_S_ptr$ (b_S_array$ ?2 ?1) ?3) ?0 ?2))))
-(let (($x2377 (b_S_ts_n_is_n_array_n_elt$ ?x2372)))
-(let (($x18670 (or (not (= (b_S_ts_n_emb$ ?x2372) (b_S_ptr$ (b_S_array$ ?2 ?1) ?3))) (b_S_ts_n_is_n_volatile$ ?x2372) (not $x2377) (not $x2378))))
-(let (($x18671 (not $x18670)))
-(let (($x11071 (>= (+ ?0 (* (- 1) ?1)) 0)))
-(let (($x10138 (>= ?0 0)))
-(let (($x10556 (not $x10138)))
-(let (($x18677 (or (not (b_S_typed$ ?4 (b_S_ptr$ (b_S_array$ ?2 ?1) ?3))) $x10556 $x11071 $x18671)))
-(let (($x2376 (not (b_S_ts_n_is_n_volatile$ ?x2372))))
-(let ((?x2367 (b_S_ptr$ (b_S_array$ ?2 ?1) ?3)))
-(let (($x2374 (= (b_S_ts_n_emb$ ?x2372) ?x2367)))
-(let (($x7338 (and $x2374 $x2376 $x2377 $x2378)))
-(let (($x2368 (b_S_typed$ ?4 ?x2367)))
-(let (($x11688 (and $x2368 $x10138 (not $x11071))))
-(let (($x11691 (not $x11688)))
-(let (($x11694 (or $x11691 $x7338)))
-(let (($x18656 (or (not $x2368) $x10556 $x11071)))
-(let ((@x18662 (monotonicity (rewrite (= $x11688 (not $x18656))) (= $x11691 (not (not $x18656))))))
-(let ((@x18676 (monotonicity (trans @x18662 (rewrite (= (not (not $x18656)) $x18656)) (= $x11691 $x18656)) (rewrite (= $x7338 $x18671)) (= $x11694 (or $x18656 $x18671)))))
-(let ((@x18684 (quant-intro (trans @x18676 (rewrite (= (or $x18656 $x18671) $x18677)) (= $x11694 $x18677)) (= $x11697 $x18682))))
-(let (($x7352 (forall ((?v0 B_S_state$) (?v1 Int) (?v2 B_S_ctype$) (?v3 Int) (?v4 Int) )(!(let (($x2378 (b_S_typed$ ?v0 (b_S_idx$ (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) ?v4 ?v2))))
-(let ((?x2370 (b_S_typemap$ ?v0)))
-(let ((?x2372 (b_S_select_o_tm$ ?x2370 (b_S_idx$ (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) ?v4 ?v2))))
-(let (($x2377 (b_S_ts_n_is_n_array_n_elt$ ?x2372)))
-(let (($x2376 (not (b_S_ts_n_is_n_volatile$ ?x2372))))
-(let ((?x2367 (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1)))
-(let (($x2374 (= (b_S_ts_n_emb$ ?x2372) ?x2367)))
-(let (($x7338 (and $x2374 $x2376 $x2377 $x2378)))
-(let (($x1660 (<= ?v3 ?v4)))
-(let (($x7169 (not $x1660)))
-(let (($x1212 (<= 0 ?v4)))
-(let (($x2368 (b_S_typed$ ?v0 ?x2367)))
-(let (($x7327 (and $x2368 $x1212 $x7169)))
-(or (not $x7327) $x7338)))))))))))))) :pattern ( (b_S_select_o_sm$ (b_S_statusmap$ ?v0) (b_S_idx$ (b_S_ptr$ ?v2 ?v1) ?v4 ?v2)) (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) ) :pattern ( (b_S_select_o_tm$ (b_S_typemap$ ?v0) (b_S_idx$ (b_S_ptr$ ?v2 ?v1) ?v4 ?v2)) (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) )))
-))
-(let ((@x11568 (monotonicity (rewrite (= (<= ?1 ?0) $x11071)) (= (not (<= ?1 ?0)) (not $x11071)))))
-(let ((@x10140 (rewrite (= $x1212 $x10138))))
-(let ((@x11690 (monotonicity @x10140 @x11568 (= (and $x2368 $x1212 (not (<= ?1 ?0))) $x11688))))
-(let ((@x11693 (monotonicity @x11690 (= (not (and $x2368 $x1212 (not (<= ?1 ?0)))) $x11691))))
-(let ((@x11696 (monotonicity @x11693 (= (or (not (and $x2368 $x1212 (not (<= ?1 ?0)))) $x7338) $x11694))))
-(let (($x2390 (forall ((?v0 B_S_state$) (?v1 Int) (?v2 B_S_ctype$) (?v3 Int) (?v4 Int) )(!(let (($x2378 (b_S_typed$ ?v0 (b_S_idx$ (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) ?v4 ?v2))))
-(let ((?x2370 (b_S_typemap$ ?v0)))
-(let ((?x2372 (b_S_select_o_tm$ ?x2370 (b_S_idx$ (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) ?v4 ?v2))))
-(let (($x2377 (b_S_ts_n_is_n_array_n_elt$ ?x2372)))
-(let (($x2376 (not (b_S_ts_n_is_n_volatile$ ?x2372))))
-(let ((?x2367 (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1)))
-(let (($x2374 (= (b_S_ts_n_emb$ ?x2372) ?x2367)))
-(let (($x2381 (and $x2374 (and $x2376 (and $x2377 $x2378)))))
-(let (($x1212 (<= 0 ?v4)))
-(let (($x2271 (and $x1212 (< ?v4 ?v3))))
-(let (($x2368 (b_S_typed$ ?v0 ?x2367)))
-(let (($x2369 (and $x2368 $x2271)))
-(=> $x2369 $x2381))))))))))))) :pattern ( (b_S_select_o_sm$ (b_S_statusmap$ ?v0) (b_S_idx$ (b_S_ptr$ ?v2 ?v1) ?v4 ?v2)) (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) ) :pattern ( (b_S_select_o_tm$ (b_S_typemap$ ?v0) (b_S_idx$ (b_S_ptr$ ?v2 ?v1) ?v4 ?v2)) (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) )))
-))
-(let (($x7347 (or (not (and $x2368 $x1212 (not (<= ?1 ?0)))) $x7338)))
-(let (($x2381 (and $x2374 (and $x2376 (and $x2377 $x2378)))))
-(let (($x2271 (and $x1212 (< ?0 ?1))))
-(let (($x2369 (and $x2368 $x2271)))
-(let (($x2382 (=> $x2369 $x2381)))
-(let ((@x7337 (monotonicity (rewrite (= (and $x2376 (and $x2377 $x2378)) (and $x2376 $x2377 $x2378))) (= $x2381 (and $x2374 (and $x2376 $x2377 $x2378))))))
-(let ((@x7342 (trans @x7337 (rewrite (= (and $x2374 (and $x2376 $x2377 $x2378)) $x7338)) (= $x2381 $x7338))))
-(let (($x1660 (<= ?1 ?0)))
-(let (($x7169 (not $x1660)))
-(let (($x7327 (and $x2368 $x1212 $x7169)))
-(let ((@x7174 (monotonicity @x5396 (rewrite (= (< ?0 ?1) $x7169)) (= $x2271 (and $x1212 $x7169)))))
-(let ((@x7331 (trans (monotonicity @x7174 (= $x2369 (and $x2368 (and $x1212 $x7169)))) (rewrite (= (and $x2368 (and $x1212 $x7169)) $x7327)) (= $x2369 $x7327))))
-(let ((@x7351 (trans (monotonicity @x7331 @x7342 (= $x2382 (=> $x7327 $x7338))) (rewrite (= (=> $x7327 $x7338) $x7347)) (= $x2382 $x7347))))
-(let ((@x11700 (mp (mp (asserted $x2390) (quant-intro @x7351 (= $x2390 $x7352)) $x7352) (quant-intro @x11696 (= $x7352 $x11697)) $x11697)))
-(let ((@x18685 (mp (mp~ @x11700 (nnf-pos (refl (~ $x11694 $x11694)) (~ $x11697 $x11697)) $x11697) @x18684 $x18682)))
-(let (($x24152 (not $x24131)))
-(let (($x24161 (not $x18682)))
-(let (($x24167 (or $x24161 $x24152 $x8666 $x24130)))
-(let (($x24132 (or $x24152 $x23300 $x23302 $x24130)))
-(let (($x24168 (or $x24161 $x24132)))
-(let ((@x24160 (trans (monotonicity @x23275 @x23344 (= $x24132 (or $x24152 false $x8666 $x24130))) (rewrite (= (or $x24152 false $x8666 $x24130) (or $x24152 $x8666 $x24130))) (= $x24132 (or $x24152 $x8666 $x24130)))))
-(let ((@x24169 (trans (monotonicity @x24160 (= $x24168 (or $x24161 (or $x24152 $x8666 $x24130)))) (rewrite (= (or $x24161 (or $x24152 $x8666 $x24130)) $x24167)) (= $x24168 $x24167))))
-(let ((@x24243 (unit-resolution (mp ((_ quant-inst v_b_S_s$ v_b_P_H_arr$ b_T_T_u1$ v_b_P_H_len$ 0) $x24168) @x24169 $x24167) @x18685 @x10095 (lemma (unit-resolution (hypothesis $x24152) @x24253 false) $x24131) (hypothesis $x24127) false)))
-(let ((@x24327 (unit-resolution ((_ quant-inst (b_S_array$ b_T_T_u1$ v_b_P_H_len$) (b_S_ref$ ?x3680)) (or (not $x20968) (= ?x21715 ?x3681))) @x20973 (= ?x21715 ?x3681))))
-(let ((@x24335 (trans (trans (monotonicity @x24449 (= ?x24269 ?x21715)) @x24327 (= ?x24269 ?x3681)) @x23283 (= ?x24269 v_b_P_H_arr$))))
-(let ((@x24339 (trans @x23339 (unit-resolution @x22701 @x16076 (and-elim @x10087 $x3686) $x22691) (= ?x23296 ?x22684))))
-(let ((@x24454 (trans (monotonicity @x24339 (= ?x24137 ?x24260)) (hypothesis $x24286) (= ?x24137 ?x24283))))
-(let ((@x24456 (trans (trans @x24454 (monotonicity @x24335 (= ?x24283 ?x3680)) (= ?x24137 ?x3680)) @x24358 (= ?x24137 ?x23203))))
-(let ((@x24458 (monotonicity (trans @x24456 (symm @x23269 (= ?x23203 ?x3739)) (= ?x24137 ?x3739)) (= ?x24145 ?x23179))))
-(let ((@x24492 (monotonicity (trans @x24072 (symm @x24458 (= ?x23179 ?x24145)) (= ?x23356 ?x24145)) (= (b_S_ts_n_emb$ ?x23356) (b_S_ts_n_emb$ ?x24145)))))
-(let ((@x24493 (trans @x24492 (unit-resolution (def-axiom (or $x24127 $x24111)) (lemma @x24243 $x24130) $x24111) (= (b_S_ts_n_emb$ ?x23356) ?x23296))))
-(let ((@x24496 (monotonicity (trans @x24493 @x23339 (= (b_S_ts_n_emb$ ?x23356) ?x3682)) (= (b_S_owner$ v_b_S_s$ (b_S_ts_n_emb$ ?x23356)) ?x3684))))
-(let ((@x24497 (unit-resolution (hypothesis (not $x23368)) (trans @x24496 @x10097 $x23368) false)))
-(let ((@x23585 (unit-resolution (lemma @x24497 (or $x24289 $x23368)) (unit-resolution (def-axiom (or $x24292 $x24286)) (lemma @x24501 $x24232) $x24286) $x23368)))
-(let (($x23511 (= (b_S_kind_n_of$ (b_S_typ$ (b_S_ts_n_emb$ ?x23179))) b_S_kind_n_primitive$)))
-(let (($x23504 (= (b_S_kind_n_of$ (b_S_typ$ (b_S_ts_n_emb$ ?x23179))) (b_S_kind_n_of$ (b_S_typ$ (b_S_ts_n_emb$ ?x23356))))))
-(let ((@x23496 (monotonicity (symm @x24072 (= ?x23179 ?x23356)) (= (b_S_ts_n_emb$ ?x23179) (b_S_ts_n_emb$ ?x23356)))))
-(let ((@x23773 (monotonicity @x23496 (= (b_S_typ$ (b_S_ts_n_emb$ ?x23179)) (b_S_typ$ (b_S_ts_n_emb$ ?x23356))))))
-(let (($x23514 (or $x23511 (not (b_S_is_n_non_n_primitive$ (b_S_typ$ (b_S_ts_n_emb$ ?x23179)))))))
-(let (($x19952 (forall ((?v0 B_S_type_n_state$) )(!(let (($x3400 (= (b_S_kind_n_of$ (b_S_typ$ (b_S_ts_n_emb$ ?v0))) b_S_kind_n_primitive$)))
-(let (($x19948 (or $x3400 (not (b_S_is_n_non_n_primitive$ (b_S_typ$ (b_S_ts_n_emb$ ?v0)))))))
-(not $x19948))) :pattern ( (b_S_ts_n_emb$ ?v0) )))
-))
-(let (($x3405 (forall ((?v0 B_S_type_n_state$) )(!(let (($x3400 (= (b_S_kind_n_of$ (b_S_typ$ (b_S_ts_n_emb$ ?v0))) b_S_kind_n_primitive$)))
-(and (not $x3400) (b_S_is_n_non_n_primitive$ (b_S_typ$ (b_S_ts_n_emb$ ?v0))))) :pattern ( (b_S_ts_n_emb$ ?v0) )))
-))
-(let (($x3400 (= (b_S_kind_n_of$ (b_S_typ$ (b_S_ts_n_emb$ ?0))) b_S_kind_n_primitive$)))
-(let (($x19948 (or $x3400 (not (b_S_is_n_non_n_primitive$ (b_S_typ$ (b_S_ts_n_emb$ ?0)))))))
-(let (($x3403 (and (not $x3400) (b_S_is_n_non_n_primitive$ (b_S_typ$ (b_S_ts_n_emb$ ?0))))))
-(let ((@x16056 (mp~ (asserted $x3405) (nnf-pos (refl (~ $x3403 $x3403)) (~ $x3405 $x3405)) $x3405)))
-(let ((@x19955 (mp @x16056 (quant-intro (rewrite (= $x3403 (not $x19948))) (= $x3405 $x19952)) $x19952)))
-(let ((@x23763 (unit-resolution ((_ quant-inst (b_S_select_o_tm$ ?x3874 ?x3739)) (or (not $x19952) (not $x23514))) @x19955 (not $x23514))))
-(let ((@x23521 (unit-resolution (unit-resolution (def-axiom (or $x23514 (not $x23511))) @x23763 (not $x23511)) (trans (monotonicity @x23773 $x23504) (hypothesis $x23366) $x23511) false)))
-(let ((@x23523 (unit-resolution (def-axiom (or $x23373 $x23355 $x23363 $x23366 (not $x23370))) (lemma @x23521 (not $x23366)) (unit-resolution (def-axiom (or $x23370 (not $x23368))) @x23585 $x23370) (or $x23373 $x23355 $x23363))))
-(let ((@x23543 (unit-resolution @x23523 @x23583 (unit-resolution (def-axiom (or $x23362 $x23357)) @x23503 $x23362) @x23574 false)))
-(let (($x21247 (or $x16242 $x16251 $x21244)))
-(let (($x21250 (not $x21247)))
-(let (($x21253 (or $x16242 $x16245 $x21250)))
-(let (($x21256 (not $x21253)))
-(let (($x21259 (or $x16242 $x16245 $x21256)))
-(let (($x21262 (not $x21259)))
-(let (($x21265 (or $x10065 $x21262)))
-(let (($x21268 (not $x21265)))
-(let (($x20335 (forall ((?v0 Int) )(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x3840 (= ?x3765 v_b_S_result_G_0$)))
-(let (($x12631 (>= (+ ?v0 (* (- 1) v_b_P_H_len$)) 0)))
-(let (($x14211 (<= ?v0 4294967295)))
-(let (($x17271 (not $x14211)))
-(let (($x10138 (>= ?v0 0)))
-(let (($x10556 (not $x10138)))
-(or $x10556 $x17271 $x12631 (not $x3840))))))))))
-))
-(let (($x20320 (forall ((?v0 Int) )(let ((?x12644 (* (- 1) v_b_S_result_G_0$)))
-(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x12646 (<= (+ ?x3765 ?x12644) 0)))
-(let (($x12631 (>= (+ ?v0 (* (- 1) v_b_P_H_len$)) 0)))
-(let (($x14211 (<= ?v0 4294967295)))
-(let (($x17271 (not $x14211)))
-(let (($x10138 (>= ?v0 0)))
-(let (($x10556 (not $x10138)))
-(or $x10556 $x17271 $x12631 $x12646))))))))))
-))
-(let (($x20344 (not (or (not $x20320) (not $x20335)))))
-(let (($x20349 (or $x20298 $x20344)))
-(let (($x20360 (or $x12456 $x20190 $x20219 (not $x3818) (not $x3820) (not $x3822) $x20358 (not $x20349))))
-(let (($x20361 (not $x20360)))
-(let (($x20126 (forall ((?v0 Int) )(let ((?x12534 (* (- 1) v_b_L_H_max_G_3$)))
-(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x12536 (<= (+ ?x3765 ?x12534) 0)))
-(let (($x12521 (>= (+ ?v0 (* (- 1) v_b_L_H_p_G_1$)) 0)))
-(let (($x14211 (<= ?v0 4294967295)))
-(let (($x17271 (not $x14211)))
-(let (($x10138 (>= ?v0 0)))
-(let (($x10556 (not $x10138)))
-(or $x10556 $x17271 $x12521 $x12536))))))))))
-))
-(let (($x20146 (not (or (not $x20126) $x20131))))
-(let (($x20151 (or $x20104 $x20146)))
-(let (($x20159 (not (or $x12518 (not $x20151)))))
-(let (($x20164 (or $x12518 $x20159)))
-(let (($x20175 (or $x16351 $x16354 $x20170 (not $x3960) (not (>= v_b_L_H_p_G_1$ 2)) $x20173 (not $x20164))))
-(let (($x20176 (not $x20175)))
-(let (($x20181 (or $x16351 $x16354 $x20176)))
-(let (($x20193 (not $x20181)))
-(let (($x20233 (not (or $x20190 $x20219 $x12476 $x20230 (not $x3994) $x20173 $x20193))))
-(let (($x20194 (or $x16330 $x16339 (not $x3935) (not $x3936) (not $x3937) $x20190 (not $x3940) (not $x3942) $x20173 $x20193)))
-(let (($x20195 (not $x20194)))
-(let (($x20200 (or $x16330 $x16339 $x20195)))
-(let (($x20208 (not (or $x16330 $x16333 (not $x20200)))))
-(let (($x20213 (or $x16330 $x16333 $x20208)))
-(let (($x20222 (not (or $x20190 $x20219 $x12471 (not $x20213)))))
-(let (($x20238 (or $x20222 $x20233)))
-(let (($x20246 (not (or $x16330 $x16339 $x20190 $x20219 (not $x20238)))))
-(let (($x20251 (or $x16330 $x16339 $x20246)))
-(let (($x20259 (not (or $x16330 $x16333 (not $x20251)))))
-(let (($x20264 (or $x16330 $x16333 $x20259)))
-(let (($x20272 (not (or $x20190 $x20219 $x12453 (not $x20264)))))
-(let (($x20366 (or $x20272 $x20361)))
-(let (($x20080 (forall ((?v0 Int) )(let ((?x12384 (* (- 1) v_b_L_H_max_G_1$)))
-(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x12425 (<= (+ ?x3765 ?x12384) 0)))
-(let (($x12411 (>= (+ ?v0 (* (- 1) v_b_L_H_p_G_0$)) 0)))
-(let (($x14211 (<= ?v0 4294967295)))
-(let (($x17271 (not $x14211)))
-(let (($x10138 (>= ?v0 0)))
-(let (($x10556 (not $x10138)))
-(or $x10556 $x17271 $x12411 $x12425))))))))))
-))
-(let (($x20389 (or $x8666 $x16288 (not (>= v_b_L_H_max_G_1$ 0)) (not (<= v_b_L_H_max_G_1$ 255)) $x20374 $x20375 (not (<= v_b_L_H_p_G_0$ 4294967295)) (not (>= (+ v_b_P_H_len$ (* (- 1) v_b_L_H_p_G_0$)) 0)) (not $x20080) $x12435 $x20379 $x20190 $x20219 (not $x3886) (not $x3806) (not $x3893) (not $x3894) (not $x3895) (not $x3896) (not $x3897) (not $x3898) (not $x20366))))
-(let (($x20390 (not $x20389)))
-(let (($x20395 (or $x8666 $x16288 $x20390)))
-(let (($x20058 (forall ((?v0 Int) )(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x12367 (>= (+ v_b_L_H_max_G_0$ (* (- 1) ?x3765)) 0)))
-(let (($x12354 (>= ?v0 1)))
-(let (($x14211 (<= ?v0 4294967295)))
-(let (($x17271 (not $x14211)))
-(let (($x10138 (>= ?v0 0)))
-(let (($x10556 (not $x10138)))
-(or $x10556 $x17271 $x12354 $x12367)))))))))
-))
-(let (($x20404 (not (or (not $x20058) (not $x20395)))))
-(let (($x20409 (or $x20036 $x20404)))
-(let (($x20417 (not (or $x12351 (not $x20409)))))
-(let (($x20422 (or $x12351 $x20417)))
-(let (($x20433 (or $x16242 $x16251 (not $x3747) (not $x3748) (not $x3749) (not $x3750) (not $x20422))))
-(let (($x20434 (not $x20433)))
-(let (($x20439 (or $x16242 $x16251 $x20434)))
-(let (($x20447 (not (or $x16242 $x16245 (not $x20439)))))
-(let (($x20452 (or $x16242 $x16245 $x20447)))
-(let (($x20460 (not (or $x10065 (not $x20452)))))
-(let (($x20465 (or $x10065 $x20460)))
-(let (($x12631 (>= (+ ?0 (* (- 1) v_b_P_H_len$)) 0)))
-(let (($x14211 (<= ?0 4294967295)))
-(let (($x17271 (not $x14211)))
-(let (($x20324 (or $x10556 $x17271 $x12631 (not $x3840))))
-(let ((@x21180 (monotonicity (quant-intro (refl (= $x20324 $x20324)) (= $x20335 $x21173)) (= (not $x20335) $x21178))))
-(let (($x12646 (<= (+ ?x3765 (* (- 1) v_b_S_result_G_0$)) 0)))
-(let (($x20315 (or $x10556 $x17271 $x12631 $x12646)))
-(let ((@x21172 (monotonicity (quant-intro (refl (= $x20315 $x20315)) (= $x20320 $x21165)) (= (not $x20320) (not $x21165)))))
-(let ((@x21186 (monotonicity (monotonicity @x21172 @x21180 (= (or (not $x20320) (not $x20335)) $x21181)) (= $x20344 $x21184))))
-(let ((@x21192 (monotonicity (monotonicity @x21186 (= $x20349 $x21187)) (= (not $x20349) $x21190))))
-(let (($x12536 (<= (+ ?x3765 ?x12534) 0)))
-(let (($x12521 (>= (+ ?0 (* (- 1) v_b_L_H_p_G_1$)) 0)))
-(let (($x20121 (or $x10556 $x17271 $x12521 $x12536)))
-(let ((@x21056 (monotonicity (quant-intro (refl (= $x20121 $x20121)) (= $x20126 $x21049)) (= (not $x20126) (not $x21049)))))
-(let ((@x21062 (monotonicity (monotonicity @x21056 (= (or (not $x20126) $x20131) $x21057)) (= $x20146 $x21060))))
-(let ((@x21068 (monotonicity (monotonicity @x21062 (= $x20151 $x21063)) (= (not $x20151) $x21066))))
-(let ((@x21074 (monotonicity (monotonicity @x21068 (= (or $x12518 (not $x20151)) $x21069)) (= $x20159 $x21072))))
-(let ((@x21080 (monotonicity (monotonicity @x21074 (= $x20164 $x21075)) (= (not $x20164) $x21078))))
-(let ((@x21089 (monotonicity (monotonicity (monotonicity @x21080 (= $x20175 $x21081)) (= $x20176 $x21084)) (= $x20181 $x21087))))
-(let ((@x21125 (monotonicity (monotonicity @x21089 (= $x20193 $x21090)) (= (or $x20190 $x20219 $x12476 $x20230 (not $x3994) $x20173 $x20193) $x21123))))
-(let ((@x21098 (monotonicity (monotonicity (monotonicity @x21089 (= $x20193 $x21090)) (= $x20194 $x21093)) (= $x20195 $x21096))))
-(let ((@x21104 (monotonicity (monotonicity @x21098 (= $x20200 $x21099)) (= (not $x20200) $x21102))))
-(let ((@x21110 (monotonicity (monotonicity @x21104 (= (or $x16330 $x16333 (not $x20200)) $x21105)) (= $x20208 $x21108))))
-(let ((@x21116 (monotonicity (monotonicity @x21110 (= $x20213 $x21111)) (= (not $x20213) $x21114))))
-(let ((@x21122 (monotonicity (monotonicity @x21116 (= (or $x20190 $x20219 $x12471 (not $x20213)) $x21117)) (= $x20222 $x21120))))
-(let ((@x21131 (monotonicity @x21122 (monotonicity @x21125 (= $x20233 $x21126)) (= $x20238 $x21129))))
-(let ((@x21137 (monotonicity (monotonicity @x21131 (= (not $x20238) $x21132)) (= (or $x16330 $x16339 $x20190 $x20219 (not $x20238)) $x21135))))
-(let ((@x21146 (monotonicity (monotonicity (monotonicity @x21137 (= $x20246 $x21138)) (= $x20251 $x21141)) (= (not $x20251) $x21144))))
-(let ((@x21152 (monotonicity (monotonicity @x21146 (= (or $x16330 $x16333 (not $x20251)) $x21147)) (= $x20259 $x21150))))
-(let ((@x21158 (monotonicity (monotonicity @x21152 (= $x20264 $x21153)) (= (not $x20264) $x21156))))
-(let ((@x21164 (monotonicity (monotonicity @x21158 (= (or $x20190 $x20219 $x12453 (not $x20264)) $x21159)) (= $x20272 $x21162))))
-(let ((@x21201 (monotonicity @x21164 (monotonicity (monotonicity @x21192 (= $x20360 $x21193)) (= $x20361 $x21196)) (= $x20366 $x21199))))
-(let (($x12425 (<= (+ ?x3765 (* (- 1) v_b_L_H_max_G_1$)) 0)))
-(let (($x12411 (>= (+ ?0 (* (- 1) v_b_L_H_p_G_0$)) 0)))
-(let (($x20075 (or $x10556 $x17271 $x12411 $x12425)))
-(let ((@x21048 (monotonicity (quant-intro (refl (= $x20075 $x20075)) (= $x20080 $x21041)) (= (not $x20080) $x21046))))
-(let ((@x21207 (monotonicity @x21048 (monotonicity @x21201 (= (not $x20366) $x21202)) (= $x20389 $x21205))))
-(let ((@x21216 (monotonicity (monotonicity (monotonicity @x21207 (= $x20390 $x21208)) (= $x20395 $x21211)) (= (not $x20395) $x21214))))
-(let (($x12367 (>= (+ v_b_L_H_max_G_0$ (* (- 1) ?x3765)) 0)))
-(let (($x12354 (>= ?0 1)))
-(let (($x20053 (or $x10556 $x17271 $x12354 $x12367)))
-(let ((@x21040 (monotonicity (quant-intro (refl (= $x20053 $x20053)) (= $x20058 $x21033)) (= (not $x20058) (not $x21033)))))
-(let ((@x21222 (monotonicity (monotonicity @x21040 @x21216 (= (or (not $x20058) (not $x20395)) $x21217)) (= $x20404 $x21220))))
-(let ((@x21228 (monotonicity (monotonicity @x21222 (= $x20409 $x21223)) (= (not $x20409) $x21226))))
-(let ((@x21234 (monotonicity (monotonicity @x21228 (= (or $x12351 (not $x20409)) $x21229)) (= $x20417 $x21232))))
-(let ((@x21240 (monotonicity (monotonicity @x21234 (= $x20422 $x21235)) (= (not $x20422) $x21238))))
-(let ((@x21249 (monotonicity (monotonicity (monotonicity @x21240 (= $x20433 $x21241)) (= $x20434 $x21244)) (= $x20439 $x21247))))
-(let ((@x21255 (monotonicity (monotonicity @x21249 (= (not $x20439) $x21250)) (= (or $x16242 $x16245 (not $x20439)) $x21253))))
-(let ((@x21264 (monotonicity (monotonicity (monotonicity @x21255 (= $x20447 $x21256)) (= $x20452 $x21259)) (= (not $x20452) $x21262))))
-(let ((@x21270 (monotonicity (monotonicity @x21264 (= (or $x10065 (not $x20452)) $x21265)) (= $x20460 $x21268))))
-(let (($x16498 (forall ((?v0 Int) )(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x3840 (= ?x3765 v_b_S_result_G_0$)))
-(let (($x12631 (>= (+ ?v0 (* (- 1) v_b_P_H_len$)) 0)))
-(let (($x12635 (not $x12631)))
-(let (($x14211 (<= ?v0 4294967295)))
-(let (($x10138 (>= ?v0 0)))
-(let (($x13747 (and $x10138 $x14211 $x12635 $x3840)))
-(not $x13747)))))))))
-))
-(let (($x13163 (forall ((?v0 Int) )(let ((?x12644 (* (- 1) v_b_S_result_G_0$)))
-(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x12646 (<= (+ ?x3765 ?x12644) 0)))
-(let (($x12631 (>= (+ ?v0 (* (- 1) v_b_P_H_len$)) 0)))
-(let (($x12635 (not $x12631)))
-(let (($x14211 (<= ?v0 4294967295)))
-(let (($x10138 (>= ?v0 0)))
-(let (($x13586 (and $x10138 $x14211 $x12635)))
-(let (($x13963 (not $x13586)))
-(or $x13963 $x12646)))))))))))
-))
-(let (($x16502 (and $x13163 $x16498)))
-(let (($x16743 (not $x16738)))
-(let (($x16746 (and $x16473 $x16474 $x16743)))
-(let (($x16749 (not $x16746)))
-(let (($x16765 (or $x16749 $x16760)))
-(let (($x16768 (not $x16765)))
-(let (($x16771 (or $x16768 $x16502)))
-(let (($x16777 (and $x12453 $x12404 $x12389 $x3818 $x3820 $x3822 $x3824 $x16771)))
-(let (($x12553 (not $x12550)))
-(let (($x12556 (and $x12553 $x3976)))
-(let (($x16388 (not $x12556)))
-(let (($x13130 (forall ((?v0 Int) )(let ((?x12534 (* (- 1) v_b_L_H_max_G_3$)))
-(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x12536 (<= (+ ?x3765 ?x12534) 0)))
-(let (($x12521 (>= (+ ?v0 (* (- 1) v_b_L_H_p_G_1$)) 0)))
-(let (($x12525 (not $x12521)))
-(let (($x14211 (<= ?v0 4294967295)))
-(let (($x10138 (>= ?v0 0)))
-(let (($x14023 (and $x10138 $x14211 $x12525)))
-(let (($x12802 (not $x14023)))
-(or $x12802 $x12536)))))))))))
-))
-(let (($x16391 (and $x13130 $x16388)))
-(let (($x16605 (not $x16600)))
-(let (($x16608 (and $x16366 $x16367 $x16605)))
-(let (($x16611 (not $x16608)))
-(let (($x16627 (or $x16611 $x16622)))
-(let (($x16630 (not $x16627)))
-(let (($x16633 (or $x16630 $x16391)))
-(let (($x16636 (and $x12514 $x16633)))
-(let (($x16639 (or $x12518 $x16636)))
-(let (($x12505 (>= v_b_L_H_p_G_1$ 2)))
-(let (($x16645 (and $x12494 $x13856 $x12500 $x3960 $x12505 $x12486 $x16639)))
-(let (($x16650 (or $x16351 $x16354 $x16645)))
-(let (($x16688 (and $x12404 $x12389 $x12471 $x3993 $x3994 $x12486 $x16650)))
-(let (($x16656 (and $x3923 $x3926 $x3935 $x3936 $x3937 $x12404 $x3940 $x3942 $x12486 $x16650)))
-(let (($x16661 (or $x16330 $x16339 $x16656)))
-(let (($x16667 (and $x3923 $x3924 $x16661)))
-(let (($x16672 (or $x16330 $x16333 $x16667)))
-(let (($x16678 (and $x12404 $x12389 $x12476 $x16672)))
-(let (($x16693 (or $x16678 $x16688)))
-(let (($x16699 (and $x3923 $x3926 $x12404 $x12389 $x16693)))
-(let (($x16704 (or $x16330 $x16339 $x16699)))
-(let (($x16710 (and $x3923 $x3924 $x16704)))
-(let (($x16715 (or $x16330 $x16333 $x16710)))
-(let (($x16721 (and $x12404 $x12389 $x12456 $x16715)))
-(let (($x16782 (or $x16721 $x16777)))
-(let (($x12438 (not $x12435)))
-(let (($x13341 (forall ((?v0 Int) )(let ((?x12384 (* (- 1) v_b_L_H_max_G_1$)))
-(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x12425 (<= (+ ?x3765 ?x12384) 0)))
-(let (($x12411 (>= (+ ?v0 (* (- 1) v_b_L_H_p_G_0$)) 0)))
-(let (($x12415 (not $x12411)))
-(let (($x14211 (<= ?v0 4294967295)))
-(let (($x10138 (>= ?v0 0)))
-(let (($x13128 (and $x10138 $x14211 $x12415)))
-(let (($x13111 (not $x13128)))
-(or $x13111 $x12425)))))))))))
-))
-(let (($x12407 (>= (+ v_b_P_H_len$ (* (- 1) v_b_L_H_p_G_0$)) 0)))
-(let (($x13193 (<= v_b_L_H_p_G_0$ 4294967295)))
-(let (($x12799 (<= v_b_L_H_max_G_1$ 255)))
-(let (($x12381 (>= v_b_L_H_max_G_1$ 0)))
-(let (($x16788 (and $x8667 $x3769 $x12381 $x12799 $x12834 $x12397 $x13193 $x12407 $x13341 $x12438 $x3794 $x12404 $x12389 $x3886 $x3806 $x3893 $x3894 $x3895 $x3896 $x3897 $x3898 $x16782)))
-(let (($x16793 (or $x8666 $x16288 $x16788)))
-(let (($x12941 (forall ((?v0 Int) )(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x12367 (>= (+ v_b_L_H_max_G_0$ (* (- 1) ?x3765)) 0)))
-(let (($x12354 (>= ?v0 1)))
-(let (($x12357 (not $x12354)))
-(let (($x14211 (<= ?v0 4294967295)))
-(let (($x10138 (>= ?v0 0)))
-(let (($x14020 (and $x10138 $x14211 $x12357)))
-(let (($x13679 (not $x14020)))
-(or $x13679 $x12367))))))))))
-))
-(let (($x16796 (and $x12941 $x16793)))
-(let (($x16268 (not (and (>= ?v0!13 0) (<= ?v0!13 4294967295) (not $x16265)))))
-(let (($x16274 (or $x16268 $x16273)))
-(let (($x16275 (not $x16274)))
-(let (($x16799 (or $x16275 $x16796)))
-(let (($x16802 (and $x12348 $x16799)))
-(let (($x16805 (or $x12351 $x16802)))
-(let (($x16811 (and $x3740 $x3743 $x3747 $x3748 $x3749 $x3750 $x16805)))
-(let (($x16816 (or $x16242 $x16251 $x16811)))
-(let (($x16822 (and $x3740 $x3741 $x16816)))
-(let (($x16827 (or $x16242 $x16245 $x16822)))
-(let (($x16830 (and $x3738 $x16827)))
-(let (($x16833 (or $x10065 $x16830)))
-(let (($x20369 (and $x8667 $x3769 $x12381 $x12799 $x12834 $x12397 $x13193 $x12407 $x20080 $x12438 $x3794 $x12404 $x12389 $x3886 $x3806 $x3893 $x3894 $x3895 $x3896 $x3897 $x3898 $x20366)))
-(let ((@x20330 (monotonicity (rewrite (= (and $x10138 $x14211 (not $x12631) $x3840) (not $x20324))) (= (not (and $x10138 $x14211 (not $x12631) $x3840)) (not (not $x20324))))))
-(let ((@x20334 (trans @x20330 (rewrite (= (not (not $x20324)) $x20324)) (= (not (and $x10138 $x14211 (not $x12631) $x3840)) $x20324))))
-(let (($x12635 (not $x12631)))
-(let (($x13586 (and $x10138 $x14211 $x12635)))
-(let (($x13963 (not $x13586)))
-(let (($x13836 (or $x13963 $x12646)))
-(let ((@x20307 (monotonicity (rewrite (= $x13586 (not (or $x10556 $x17271 $x12631)))) (= $x13963 (not (not (or $x10556 $x17271 $x12631)))))))
-(let ((@x20311 (trans @x20307 (rewrite (= (not (not (or $x10556 $x17271 $x12631))) (or $x10556 $x17271 $x12631))) (= $x13963 (or $x10556 $x17271 $x12631)))))
-(let ((@x20319 (trans (monotonicity @x20311 (= $x13836 (or (or $x10556 $x17271 $x12631) $x12646))) (rewrite (= (or (or $x10556 $x17271 $x12631) $x12646) $x20315)) (= $x13836 $x20315))))
-(let ((@x20340 (monotonicity (quant-intro @x20319 (= $x13163 $x20320)) (quant-intro @x20334 (= $x16498 $x20335)) (= $x16502 (and $x20320 $x20335)))))
-(let ((@x20285 (monotonicity (rewrite (= $x16746 (not (or $x20277 $x20278 $x16738)))) (= $x16749 (not (not (or $x20277 $x20278 $x16738)))))))
-(let ((@x20289 (trans @x20285 (rewrite (= (not (not (or $x20277 $x20278 $x16738))) (or $x20277 $x20278 $x16738))) (= $x16749 (or $x20277 $x20278 $x16738)))))
-(let ((@x20297 (trans (monotonicity @x20289 (= $x16765 (or (or $x20277 $x20278 $x16738) $x16760))) (rewrite (= (or (or $x20277 $x20278 $x16738) $x16760) $x20293)) (= $x16765 $x20293))))
-(let ((@x20351 (monotonicity (monotonicity @x20297 (= $x16768 $x20298)) (trans @x20340 (rewrite (= (and $x20320 $x20335) $x20344)) (= $x16502 $x20344)) (= $x16771 $x20349))))
-(let ((@x20354 (monotonicity @x20351 (= $x16777 (and $x12453 $x12404 $x12389 $x3818 $x3820 $x3822 $x3824 $x20349)))))
-(let ((@x20365 (trans @x20354 (rewrite (= (and $x12453 $x12404 $x12389 $x3818 $x3820 $x3822 $x3824 $x20349) $x20361)) (= $x16777 $x20361))))
-(let ((@x20140 (trans (monotonicity (rewrite (= $x12556 $x20131)) (= $x16388 (not $x20131))) (rewrite (= (not $x20131) $x20130)) (= $x16388 $x20130))))
-(let (($x12525 (not $x12521)))
-(let (($x14023 (and $x10138 $x14211 $x12525)))
-(let (($x12802 (not $x14023)))
-(let (($x13633 (or $x12802 $x12536)))
-(let ((@x20113 (monotonicity (rewrite (= $x14023 (not (or $x10556 $x17271 $x12521)))) (= $x12802 (not (not (or $x10556 $x17271 $x12521)))))))
-(let ((@x20117 (trans @x20113 (rewrite (= (not (not (or $x10556 $x17271 $x12521))) (or $x10556 $x17271 $x12521))) (= $x12802 (or $x10556 $x17271 $x12521)))))
-(let ((@x20125 (trans (monotonicity @x20117 (= $x13633 (or (or $x10556 $x17271 $x12521) $x12536))) (rewrite (= (or (or $x10556 $x17271 $x12521) $x12536) $x20121)) (= $x13633 $x20121))))
-(let ((@x20143 (monotonicity (quant-intro @x20125 (= $x13130 $x20126)) @x20140 (= $x16391 (and $x20126 $x20130)))))
-(let ((@x20091 (monotonicity (rewrite (= $x16608 (not (or $x20083 $x20084 $x16600)))) (= $x16611 (not (not (or $x20083 $x20084 $x16600)))))))
-(let ((@x20095 (trans @x20091 (rewrite (= (not (not (or $x20083 $x20084 $x16600))) (or $x20083 $x20084 $x16600))) (= $x16611 (or $x20083 $x20084 $x16600)))))
-(let ((@x20103 (trans (monotonicity @x20095 (= $x16627 (or (or $x20083 $x20084 $x16600) $x16622))) (rewrite (= (or (or $x20083 $x20084 $x16600) $x16622) $x20099)) (= $x16627 $x20099))))
-(let ((@x20153 (monotonicity (monotonicity @x20103 (= $x16630 $x20104)) (trans @x20143 (rewrite (= (and $x20126 $x20130) $x20146)) (= $x16391 $x20146)) (= $x16633 $x20151))))
-(let ((@x20163 (trans (monotonicity @x20153 (= $x16636 (and $x12514 $x20151))) (rewrite (= (and $x12514 $x20151) $x20159)) (= $x16636 $x20159))))
-(let ((@x20169 (monotonicity (monotonicity @x20163 (= $x16639 $x20164)) (= $x16645 (and $x12494 $x13856 $x12500 $x3960 $x12505 $x12486 $x20164)))))
-(let ((@x20180 (trans @x20169 (rewrite (= (and $x12494 $x13856 $x12500 $x3960 $x12505 $x12486 $x20164) $x20176)) (= $x16645 $x20176))))
-(let ((@x20229 (monotonicity (monotonicity @x20180 (= $x16650 $x20181)) (= $x16688 (and $x12404 $x12389 $x12471 $x3993 $x3994 $x12486 $x20181)))))
-(let ((@x20237 (trans @x20229 (rewrite (= (and $x12404 $x12389 $x12471 $x3993 $x3994 $x12486 $x20181) $x20233)) (= $x16688 $x20233))))
-(let ((@x20197 (rewrite (= (and $x3923 $x3926 $x3935 $x3936 $x3937 $x12404 $x3940 $x3942 $x12486 $x20181) $x20195))))
-(let ((@x20186 (monotonicity (monotonicity @x20180 (= $x16650 $x20181)) (= $x16656 (and $x3923 $x3926 $x3935 $x3936 $x3937 $x12404 $x3940 $x3942 $x12486 $x20181)))))
-(let ((@x20205 (monotonicity (monotonicity (trans @x20186 @x20197 (= $x16656 $x20195)) (= $x16661 $x20200)) (= $x16667 (and $x3923 $x3924 $x20200)))))
-(let ((@x20212 (trans @x20205 (rewrite (= (and $x3923 $x3924 $x20200) $x20208)) (= $x16667 $x20208))))
-(let ((@x20218 (monotonicity (monotonicity @x20212 (= $x16672 $x20213)) (= $x16678 (and $x12404 $x12389 $x12476 $x20213)))))
-(let ((@x20226 (trans @x20218 (rewrite (= (and $x12404 $x12389 $x12476 $x20213) $x20222)) (= $x16678 $x20222))))
-(let ((@x20243 (monotonicity (monotonicity @x20226 @x20237 (= $x16693 $x20238)) (= $x16699 (and $x3923 $x3926 $x12404 $x12389 $x20238)))))
-(let ((@x20250 (trans @x20243 (rewrite (= (and $x3923 $x3926 $x12404 $x12389 $x20238) $x20246)) (= $x16699 $x20246))))
-(let ((@x20256 (monotonicity (monotonicity @x20250 (= $x16704 $x20251)) (= $x16710 (and $x3923 $x3924 $x20251)))))
-(let ((@x20263 (trans @x20256 (rewrite (= (and $x3923 $x3924 $x20251) $x20259)) (= $x16710 $x20259))))
-(let ((@x20269 (monotonicity (monotonicity @x20263 (= $x16715 $x20264)) (= $x16721 (and $x12404 $x12389 $x12456 $x20264)))))
-(let ((@x20276 (trans @x20269 (rewrite (= (and $x12404 $x12389 $x12456 $x20264) $x20272)) (= $x16721 $x20272))))
-(let (($x12415 (not $x12411)))
-(let (($x13128 (and $x10138 $x14211 $x12415)))
-(let (($x13111 (not $x13128)))
-(let (($x12774 (or $x13111 $x12425)))
-(let ((@x20067 (monotonicity (rewrite (= $x13128 (not (or $x10556 $x17271 $x12411)))) (= $x13111 (not (not (or $x10556 $x17271 $x12411)))))))
-(let ((@x20071 (trans @x20067 (rewrite (= (not (not (or $x10556 $x17271 $x12411))) (or $x10556 $x17271 $x12411))) (= $x13111 (or $x10556 $x17271 $x12411)))))
-(let ((@x20079 (trans (monotonicity @x20071 (= $x12774 (or (or $x10556 $x17271 $x12411) $x12425))) (rewrite (= (or (or $x10556 $x17271 $x12411) $x12425) $x20075)) (= $x12774 $x20075))))
-(let ((@x20371 (monotonicity (quant-intro @x20079 (= $x13341 $x20080)) (monotonicity @x20276 @x20365 (= $x16782 $x20366)) (= $x16788 $x20369))))
-(let ((@x20397 (monotonicity (trans @x20371 (rewrite (= $x20369 $x20390)) (= $x16788 $x20390)) (= $x16793 $x20395))))
-(let (($x12357 (not $x12354)))
-(let (($x14020 (and $x10138 $x14211 $x12357)))
-(let (($x13679 (not $x14020)))
-(let (($x12918 (or $x13679 $x12367)))
-(let ((@x20045 (monotonicity (rewrite (= $x14020 (not (or $x10556 $x17271 $x12354)))) (= $x13679 (not (not (or $x10556 $x17271 $x12354)))))))
-(let ((@x20049 (trans @x20045 (rewrite (= (not (not (or $x10556 $x17271 $x12354))) (or $x10556 $x17271 $x12354))) (= $x13679 (or $x10556 $x17271 $x12354)))))
-(let ((@x20057 (trans (monotonicity @x20049 (= $x12918 (or (or $x10556 $x17271 $x12354) $x12367))) (rewrite (= (or (or $x10556 $x17271 $x12354) $x12367) $x20053)) (= $x12918 $x20053))))
-(let ((@x20400 (monotonicity (quant-intro @x20057 (= $x12941 $x20058)) @x20397 (= $x16796 (and $x20058 $x20395)))))
-(let (($x20017 (or (not (>= ?v0!13 0)) (not (<= ?v0!13 4294967295)) $x16265)))
-(let (($x20019 (= (and (>= ?v0!13 0) (<= ?v0!13 4294967295) (not $x16265)) (not $x20017))))
-(let ((@x20027 (trans (monotonicity (rewrite $x20019) (= $x16268 (not (not $x20017)))) (rewrite (= (not (not $x20017)) $x20017)) (= $x16268 $x20017))))
-(let ((@x20035 (trans (monotonicity @x20027 (= $x16274 (or $x20017 $x16273))) (rewrite (= (or $x20017 $x16273) $x20031)) (= $x16274 $x20031))))
-(let ((@x20411 (monotonicity (monotonicity @x20035 (= $x16275 $x20036)) (trans @x20400 (rewrite (= (and $x20058 $x20395) $x20404)) (= $x16796 $x20404)) (= $x16799 $x20409))))
-(let ((@x20421 (trans (monotonicity @x20411 (= $x16802 (and $x12348 $x20409))) (rewrite (= (and $x12348 $x20409) $x20417)) (= $x16802 $x20417))))
-(let ((@x20427 (monotonicity (monotonicity @x20421 (= $x16805 $x20422)) (= $x16811 (and $x3740 $x3743 $x3747 $x3748 $x3749 $x3750 $x20422)))))
-(let ((@x20438 (trans @x20427 (rewrite (= (and $x3740 $x3743 $x3747 $x3748 $x3749 $x3750 $x20422) $x20434)) (= $x16811 $x20434))))
-(let ((@x20444 (monotonicity (monotonicity @x20438 (= $x16816 $x20439)) (= $x16822 (and $x3740 $x3741 $x20439)))))
-(let ((@x20451 (trans @x20444 (rewrite (= (and $x3740 $x3741 $x20439) $x20447)) (= $x16822 $x20447))))
-(let ((@x20457 (monotonicity (monotonicity @x20451 (= $x16827 $x20452)) (= $x16830 (and $x3738 $x20452)))))
-(let ((@x20467 (monotonicity (trans @x20457 (rewrite (= (and $x3738 $x20452) $x20460)) (= $x16830 $x20460)) (= $x16833 $x20465))))
-(let (($x16483 (<= (+ ?x16481 (* (- 1) v_b_S_result_G_0$)) 0)))
-(let (($x16478 (and $x16473 $x16474 (not (>= (+ ?v0!15 (* (- 1) v_b_P_H_len$)) 0)))))
-(let (($x16485 (not (or (not $x16478) $x16483))))
-(let (($x16506 (or $x16485 $x16502)))
-(let (($x14268 (and $x12404 $x12389 $x3818 $x3820 $x3822 $x3824)))
-(let (($x14273 (not $x14268)))
-(let (($x16469 (not $x14273)))
-(let (($x12619 (and $x12404 $x12389 $x12453)))
-(let (($x12622 (not $x12619)))
-(let (($x16466 (not $x12622)))
-(let (($x16510 (and $x16466 $x16469 $x16506)))
-(let (($x16376 (<= (+ ?x16374 ?x12534) 0)))
-(let (($x16371 (and $x16366 $x16367 (not (>= (+ ?v0!14 (* (- 1) v_b_L_H_p_G_1$)) 0)))))
-(let (($x16378 (not (or (not $x16371) $x16376))))
-(let (($x16395 (or $x16378 $x16391)))
-(let (($x16362 (not $x12518)))
-(let (($x16399 (and $x16362 $x16395)))
-(let (($x16403 (or $x12518 $x16399)))
-(let (($x13815 (and $x12494 $x13856 $x12500 $x3960 $x12505 $x12486)))
-(let (($x13880 (not $x13815)))
-(let (($x16357 (not $x13880)))
-(let (($x16407 (and $x16357 $x16403)))
-(let (($x16411 (or $x16351 $x16354 $x16407)))
-(let (($x12592 (and $x12404 $x12389 $x12471 $x3993 $x3994 $x12486)))
-(let (($x12595 (not $x12592)))
-(let (($x16435 (not $x12595)))
-(let (($x16438 (and $x16435 $x16411)))
-(let (($x12488 (and $x3923 $x3926 $x3935 $x3936 $x3937 $x12404 $x3940 $x3942 $x12486)))
-(let (($x12491 (not $x12488)))
-(let (($x16348 (not $x12491)))
-(let (($x16415 (and $x16348 $x16411)))
-(let (($x16419 (or $x16330 $x16339 $x16415)))
-(let (($x16336 (not $x9775)))
-(let (($x16423 (and $x16336 $x16419)))
-(let (($x16427 (or $x16330 $x16333 $x16423)))
-(let (($x12479 (and $x12404 $x12389 $x12476)))
-(let (($x12482 (not $x12479)))
-(let (($x16345 (not $x12482)))
-(let (($x16431 (and $x16345 $x16427)))
-(let (($x16442 (or $x16431 $x16438)))
-(let (($x12465 (and $x3923 $x3926 $x12404 $x12389)))
-(let (($x12468 (not $x12465)))
-(let (($x16342 (not $x12468)))
-(let (($x16446 (and $x16342 $x16442)))
-(let (($x16450 (or $x16330 $x16339 $x16446)))
-(let (($x16454 (and $x16336 $x16450)))
-(let (($x16458 (or $x16330 $x16333 $x16454)))
-(let (($x12459 (and $x12404 $x12389 $x12456)))
-(let (($x12462 (not $x12459)))
-(let (($x16327 (not $x12462)))
-(let (($x16462 (and $x16327 $x16458)))
-(let (($x16514 (or $x16462 $x16510)))
-(let (($x14257 (and $x12404 $x12389 $x3886 $x3806 $x3893 $x3894 $x3895 $x3896 $x3897 $x3898)))
-(let (($x14262 (not $x14257)))
-(let (($x16324 (not $x14262)))
-(let (($x13242 (and $x8667 $x3769 $x12381 $x12799 $x12389 $x12834 $x12397 $x13193 $x12404 $x12407 $x13341 $x12438 $x3794)))
-(let (($x16518 (and $x13242 $x16324 $x16514)))
-(let (($x16285 (not $x8667)))
-(let (($x16522 (or $x16285 $x16288 $x16518)))
-(let (($x16526 (and $x12941 $x16522)))
-(let (($x16530 (or $x16275 $x16526)))
-(let (($x16259 (not $x12351)))
-(let (($x16534 (and $x16259 $x16530)))
-(let (($x16538 (or $x12351 $x16534)))
-(let (($x16254 (not $x10031)))
-(let (($x16542 (and $x16254 $x16538)))
-(let (($x16546 (or $x16242 $x16251 $x16542)))
-(let (($x16248 (not $x10048)))
-(let (($x16550 (and $x16248 $x16546)))
-(let (($x16554 (or $x16242 $x16245 $x16550)))
-(let (($x16239 (not $x10065)))
-(let (($x16558 (and $x16239 $x16554)))
-(let (($x16562 (or $x10065 $x16558)))
-(let (($x16753 (= (+ ?x16481 (* (- 1) v_b_S_result_G_0$)) (+ (* (- 1) v_b_S_result_G_0$) ?x16481))))
-(let ((@x16757 (monotonicity (rewrite $x16753) (= $x16483 (<= (+ (* (- 1) v_b_S_result_G_0$) ?x16481) 0)))))
-(let ((@x16764 (trans @x16757 (rewrite (= (<= (+ (* (- 1) v_b_S_result_G_0$) ?x16481) 0) $x16760)) (= $x16483 $x16760))))
-(let (($x16476 (>= (+ ?v0!15 (* (- 1) v_b_P_H_len$)) 0)))
-(let (($x16731 (= (+ ?v0!15 (* (- 1) v_b_P_H_len$)) (+ (* (- 1) v_b_P_H_len$) ?v0!15))))
-(let ((@x16735 (monotonicity (rewrite $x16731) (= $x16476 (>= (+ (* (- 1) v_b_P_H_len$) ?v0!15) 0)))))
-(let ((@x16742 (trans @x16735 (rewrite (= (>= (+ (* (- 1) v_b_P_H_len$) ?v0!15) 0) $x16738)) (= $x16476 $x16738))))
-(let ((@x16748 (monotonicity (monotonicity @x16742 (= (not $x16476) $x16743)) (= $x16478 $x16746))))
-(let ((@x16767 (monotonicity (monotonicity @x16748 (= (not $x16478) $x16749)) @x16764 (= (or (not $x16478) $x16483) $x16765))))
-(let ((@x16776 (monotonicity (rewrite (= $x16466 $x12619)) (rewrite (= $x16469 $x14268)) (monotonicity (monotonicity @x16767 (= $x16485 $x16768)) (= $x16506 $x16771)) (= $x16510 (and $x12619 $x14268 $x16771)))))
-(let ((@x16781 (trans @x16776 (rewrite (= (and $x12619 $x14268 $x16771) $x16777)) (= $x16510 $x16777))))
-(let ((@x16619 (monotonicity (rewrite (= (+ ?x16374 ?x12534) (+ ?x12534 ?x16374))) (= $x16376 (<= (+ ?x12534 ?x16374) 0)))))
-(let ((@x16626 (trans @x16619 (rewrite (= (<= (+ ?x12534 ?x16374) 0) $x16622)) (= $x16376 $x16622))))
-(let ((@x16602 (rewrite (= (>= (+ (* (- 1) v_b_L_H_p_G_1$) ?v0!14) 0) $x16600))))
-(let (($x16369 (>= (+ ?v0!14 (* (- 1) v_b_L_H_p_G_1$)) 0)))
-(let (($x16593 (= (+ ?v0!14 (* (- 1) v_b_L_H_p_G_1$)) (+ (* (- 1) v_b_L_H_p_G_1$) ?v0!14))))
-(let ((@x16597 (monotonicity (rewrite $x16593) (= $x16369 (>= (+ (* (- 1) v_b_L_H_p_G_1$) ?v0!14) 0)))))
-(let ((@x16607 (monotonicity (trans @x16597 @x16602 (= $x16369 $x16600)) (= (not $x16369) $x16605))))
-(let ((@x16613 (monotonicity (monotonicity @x16607 (= $x16371 $x16608)) (= (not $x16371) $x16611))))
-(let ((@x16632 (monotonicity (monotonicity @x16613 @x16626 (= (or (not $x16371) $x16376) $x16627)) (= $x16378 $x16630))))
-(let ((@x16638 (monotonicity (rewrite (= $x16362 $x12514)) (monotonicity @x16632 (= $x16395 $x16633)) (= $x16399 $x16636))))
-(let ((@x16644 (monotonicity (rewrite (= $x16357 $x13815)) (monotonicity @x16638 (= $x16403 $x16639)) (= $x16407 (and $x13815 $x16639)))))
-(let ((@x16652 (monotonicity (trans @x16644 (rewrite (= (and $x13815 $x16639) $x16645)) (= $x16407 $x16645)) (= $x16411 $x16650))))
-(let ((@x16687 (monotonicity (rewrite (= $x16435 $x12592)) @x16652 (= $x16438 (and $x12592 $x16650)))))
-(let ((@x16655 (monotonicity (rewrite (= $x16348 $x12488)) @x16652 (= $x16415 (and $x12488 $x16650)))))
-(let ((@x16663 (monotonicity (trans @x16655 (rewrite (= (and $x12488 $x16650) $x16656)) (= $x16415 $x16656)) (= $x16419 $x16661))))
-(let ((@x16666 (monotonicity (rewrite (= $x16336 $x3925)) @x16663 (= $x16423 (and $x3925 $x16661)))))
-(let ((@x16674 (monotonicity (trans @x16666 (rewrite (= (and $x3925 $x16661) $x16667)) (= $x16423 $x16667)) (= $x16427 $x16672))))
-(let ((@x16677 (monotonicity (rewrite (= $x16345 $x12479)) @x16674 (= $x16431 (and $x12479 $x16672)))))
-(let ((@x16695 (monotonicity (trans @x16677 (rewrite (= (and $x12479 $x16672) $x16678)) (= $x16431 $x16678)) (trans @x16687 (rewrite (= (and $x12592 $x16650) $x16688)) (= $x16438 $x16688)) (= $x16442 $x16693))))
-(let ((@x16698 (monotonicity (rewrite (= $x16342 $x12465)) @x16695 (= $x16446 (and $x12465 $x16693)))))
-(let ((@x16706 (monotonicity (trans @x16698 (rewrite (= (and $x12465 $x16693) $x16699)) (= $x16446 $x16699)) (= $x16450 $x16704))))
-(let ((@x16709 (monotonicity (rewrite (= $x16336 $x3925)) @x16706 (= $x16454 (and $x3925 $x16704)))))
-(let ((@x16717 (monotonicity (trans @x16709 (rewrite (= (and $x3925 $x16704) $x16710)) (= $x16454 $x16710)) (= $x16458 $x16715))))
-(let ((@x16720 (monotonicity (rewrite (= $x16327 $x12459)) @x16717 (= $x16462 (and $x12459 $x16715)))))
-(let ((@x16784 (monotonicity (trans @x16720 (rewrite (= (and $x12459 $x16715) $x16721)) (= $x16462 $x16721)) @x16781 (= $x16514 $x16782))))
-(let ((@x16787 (monotonicity (rewrite (= $x16324 $x14257)) @x16784 (= $x16518 (and $x13242 $x14257 $x16782)))))
-(let ((@x16792 (trans @x16787 (rewrite (= (and $x13242 $x14257 $x16782) $x16788)) (= $x16518 $x16788))))
-(let ((@x16798 (monotonicity (monotonicity (rewrite (= $x16285 $x8666)) @x16792 (= $x16522 $x16793)) (= $x16526 $x16796))))
-(let ((@x16804 (monotonicity (rewrite (= $x16259 $x12348)) (monotonicity @x16798 (= $x16530 $x16799)) (= $x16534 $x16802))))
-(let ((@x16810 (monotonicity (rewrite (= $x16254 $x8880)) (monotonicity @x16804 (= $x16538 $x16805)) (= $x16542 (and $x8880 $x16805)))))
-(let ((@x16818 (monotonicity (trans @x16810 (rewrite (= (and $x8880 $x16805) $x16811)) (= $x16542 $x16811)) (= $x16546 $x16816))))
-(let ((@x16821 (monotonicity (rewrite (= $x16248 $x3742)) @x16818 (= $x16550 (and $x3742 $x16816)))))
-(let ((@x16829 (monotonicity (trans @x16821 (rewrite (= (and $x3742 $x16816) $x16822)) (= $x16550 $x16822)) (= $x16554 $x16827))))
-(let ((@x16835 (monotonicity (monotonicity (rewrite (= $x16239 $x3738)) @x16829 (= $x16558 $x16830)) (= $x16562 $x16833))))
-(let (($x12742 (exists ((?v0 Int) )(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x3840 (= ?x3765 v_b_S_result_G_0$)))
-(let (($x12631 (>= (+ ?v0 (* (- 1) v_b_P_H_len$)) 0)))
-(let (($x12635 (not $x12631)))
-(let (($x14211 (<= ?v0 4294967295)))
-(let (($x10138 (>= ?v0 0)))
-(and $x10138 $x14211 $x12635 $x3840))))))))
-))
-(let (($x13974 (not $x13163)))
-(let (($x14165 (or $x13974 $x12742)))
-(let (($x13256 (and $x13163 $x14165)))
-(let (($x13521 (or $x12622 $x14273 $x13256)))
-(let (($x13025 (not $x13130)))
-(let (($x12874 (or $x13025 $x12556)))
-(let (($x13199 (and $x13130 $x12874)))
-(let (($x13574 (or $x12518 $x13199)))
-(let (($x13045 (and $x12514 $x13574)))
-(let (($x14132 (or $x13880 $x13045)))
-(let (($x13699 (and $x12494 $x13856 $x14132)))
-(let (($x13117 (or $x12595 $x13699)))
-(let (($x13338 (or $x12491 $x13699)))
-(let (($x13207 (and $x3923 $x3926 $x13338)))
-(let (($x14076 (or $x9775 $x13207)))
-(let (($x14119 (and $x3923 $x3924 $x14076)))
-(let (($x13844 (or $x12482 $x14119)))
-(let (($x13324 (and $x13844 $x13117)))
-(let (($x12957 (or $x12468 $x13324)))
-(let (($x13000 (and $x3923 $x3926 $x12957)))
-(let (($x13827 (or $x9775 $x13000)))
-(let (($x14170 (and $x3923 $x3924 $x13827)))
-(let (($x14053 (or $x12462 $x14170)))
-(let (($x13922 (and $x14053 $x13521)))
-(let (($x13591 (not $x13242)))
-(let (($x13357 (or $x13591 $x14262 $x13922)))
-(let (($x12756 (and $x8667 $x3769 $x13357)))
-(let (($x13900 (not $x12941)))
-(let (($x12819 (or $x13900 $x12756)))
-(let (($x13702 (and $x12941 $x12819)))
-(let (($x13223 (or $x12351 $x13702)))
-(let (($x12832 (and $x12348 $x13223)))
-(let (($x13861 (or $x10031 $x12832)))
-(let (($x12808 (and $x3740 $x3743 $x13861)))
-(let (($x13195 (or $x10048 $x12808)))
-(let (($x13550 (and $x3740 $x3741 $x13195)))
-(let (($x13361 (or $x10065 $x13550)))
-(let (($x13725 (not (and $x3738 $x13361))))
-(let ((@x16497 (refl (~ (not (and $x10138 $x14211 $x12635 $x3840)) (not (and $x10138 $x14211 $x12635 $x3840))))))
-(let ((@x16494 (nnf-neg (nnf-pos (refl (~ $x13836 $x13836)) (~ $x13163 $x13163)) (~ (not $x13974) $x13163))))
-(let ((@x16505 (nnf-neg @x16494 (nnf-neg @x16497 (~ (not $x12742) $x16498)) (~ (not $x14165) $x16502))))
-(let ((@x16513 (nnf-neg (refl (~ $x16466 $x16466)) (refl (~ $x16469 $x16469)) (nnf-neg (sk (~ $x13974 $x16485)) @x16505 (~ (not $x13256) $x16506)) (~ (not $x13521) $x16510))))
-(let ((@x16387 (nnf-neg (nnf-pos (refl (~ $x13633 $x13633)) (~ $x13130 $x13130)) (~ (not $x13025) $x13130))))
-(let ((@x16398 (nnf-neg (sk (~ $x13025 $x16378)) (nnf-neg @x16387 (refl (~ $x16388 $x16388)) (~ (not $x12874) $x16391)) (~ (not $x13199) $x16395))))
-(let ((@x16406 (nnf-neg (refl (~ $x12518 $x12518)) (nnf-neg (refl (~ $x16362 $x16362)) @x16398 (~ (not $x13574) $x16399)) (~ (not $x13045) $x16403))))
-(let ((@x16414 (nnf-neg (refl (~ $x16351 $x16351)) (refl (~ $x16354 $x16354)) (nnf-neg (refl (~ $x16357 $x16357)) @x16406 (~ (not $x14132) $x16407)) (~ (not $x13699) $x16411))))
-(let ((@x16332 (refl (~ $x16330 $x16330))))
-(let ((@x16422 (nnf-neg @x16332 (refl (~ $x16339 $x16339)) (nnf-neg (refl (~ $x16348 $x16348)) @x16414 (~ (not $x13338) $x16415)) (~ (not $x13207) $x16419))))
-(let ((@x16430 (nnf-neg @x16332 (refl (~ $x16333 $x16333)) (nnf-neg (refl (~ $x16336 $x16336)) @x16422 (~ (not $x14076) $x16423)) (~ (not $x14119) $x16427))))
-(let ((@x16445 (nnf-neg (nnf-neg (refl (~ $x16345 $x16345)) @x16430 (~ (not $x13844) $x16431)) (nnf-neg (refl (~ $x16435 $x16435)) @x16414 (~ (not $x13117) $x16438)) (~ (not $x13324) $x16442))))
-(let ((@x16453 (nnf-neg @x16332 (refl (~ $x16339 $x16339)) (nnf-neg (refl (~ $x16342 $x16342)) @x16445 (~ (not $x12957) $x16446)) (~ (not $x13000) $x16450))))
-(let ((@x16461 (nnf-neg @x16332 (refl (~ $x16333 $x16333)) (nnf-neg (refl (~ $x16336 $x16336)) @x16453 (~ (not $x13827) $x16454)) (~ (not $x14170) $x16458))))
-(let ((@x16517 (nnf-neg (nnf-neg (refl (~ $x16327 $x16327)) @x16461 (~ (not $x14053) $x16462)) @x16513 (~ (not $x13922) $x16514))))
-(let ((@x16320 (monotonicity (refl (~ $x8667 $x8667)) (refl (~ $x3769 $x3769)) (refl (~ $x12381 $x12381)) (refl (~ $x12799 $x12799)) (refl (~ $x12389 $x12389)) (refl (~ $x12834 $x12834)) (refl (~ $x12397 $x12397)) (refl (~ $x13193 $x13193)) (refl (~ $x12404 $x12404)) (refl (~ $x12407 $x12407)) (nnf-pos (refl (~ $x12774 $x12774)) (~ $x13341 $x13341)) (refl (~ $x12438 $x12438)) (refl (~ $x3794 $x3794)) (~ $x13242 $x13242))))
-(let ((@x16521 (nnf-neg (nnf-neg @x16320 (~ (not $x13591) $x13242)) (refl (~ $x16324 $x16324)) @x16517 (~ (not $x13357) $x16518))))
-(let ((@x16525 (nnf-neg (refl (~ $x16285 $x16285)) (refl (~ $x16288 $x16288)) @x16521 (~ (not $x12756) $x16522))))
-(let ((@x16284 (nnf-neg (nnf-pos (refl (~ $x12918 $x12918)) (~ $x12941 $x12941)) (~ (not $x13900) $x12941))))
-(let ((@x16533 (nnf-neg (sk (~ $x13900 $x16275)) (nnf-neg @x16284 @x16525 (~ (not $x12819) $x16526)) (~ (not $x13702) $x16530))))
-(let ((@x16541 (nnf-neg (refl (~ $x12351 $x12351)) (nnf-neg (refl (~ $x16259 $x16259)) @x16533 (~ (not $x13223) $x16534)) (~ (not $x12832) $x16538))))
-(let ((@x16549 (nnf-neg (refl (~ $x16242 $x16242)) (refl (~ $x16251 $x16251)) (nnf-neg (refl (~ $x16254 $x16254)) @x16541 (~ (not $x13861) $x16542)) (~ (not $x12808) $x16546))))
-(let ((@x16557 (nnf-neg (refl (~ $x16242 $x16242)) (refl (~ $x16245 $x16245)) (nnf-neg (refl (~ $x16248 $x16248)) @x16549 (~ (not $x13195) $x16550)) (~ (not $x13550) $x16554))))
-(let ((@x16564 (nnf-neg (refl (~ $x10065 $x10065)) (nnf-neg (refl (~ $x16239 $x16239)) @x16557 (~ (not $x13361) $x16558)) (~ $x13725 $x16562))))
-(let (($x12661 (exists ((?v0 Int) )(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x3840 (= ?x3765 v_b_S_result_G_0$)))
-(let (($x12631 (>= (+ ?v0 (* (- 1) v_b_P_H_len$)) 0)))
-(let (($x12635 (not $x12631)))
-(let ((?x10215 (* (- 1) b_S_max_o_u4$)))
-(let ((?x10220 (+ ?v0 ?x10215)))
-(let (($x10221 (<= ?x10220 0)))
-(let (($x10138 (>= ?v0 0)))
-(and $x10138 $x10221 $x12635 $x3840))))))))))
-))
-(let (($x12652 (forall ((?v0 Int) )(let ((?x12644 (* (- 1) v_b_S_result_G_0$)))
-(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x12646 (<= (+ ?x3765 ?x12644) 0)))
-(let (($x12631 (>= (+ ?v0 (* (- 1) v_b_P_H_len$)) 0)))
-(let (($x12635 (not $x12631)))
-(let ((?x10215 (* (- 1) b_S_max_o_u4$)))
-(let ((?x10220 (+ ?v0 ?x10215)))
-(let (($x10221 (<= ?x10220 0)))
-(let (($x10138 (>= ?v0 0)))
-(let (($x12638 (and $x10138 $x10221 $x12635)))
-(let (($x12641 (not $x12638)))
-(or $x12641 $x12646)))))))))))))
-))
-(let (($x12655 (not $x12652)))
-(let (($x12664 (or $x12655 $x12661)))
-(let (($x12667 (and $x12652 $x12664)))
-(let (($x14289 (or $x12622 $x14273 $x12667)))
-(let (($x12542 (forall ((?v0 Int) )(let ((?x12534 (* (- 1) v_b_L_H_max_G_3$)))
-(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x12536 (<= (+ ?x3765 ?x12534) 0)))
-(let (($x12521 (>= (+ ?v0 (* (- 1) v_b_L_H_p_G_1$)) 0)))
-(let (($x12525 (not $x12521)))
-(let ((?x10215 (* (- 1) b_S_max_o_u4$)))
-(let ((?x10220 (+ ?v0 ?x10215)))
-(let (($x10221 (<= ?x10220 0)))
-(let (($x10138 (>= ?v0 0)))
-(let (($x12528 (and $x10138 $x10221 $x12525)))
-(let (($x12531 (not $x12528)))
-(or $x12531 $x12536)))))))))))))
-))
-(let (($x12545 (not $x12542)))
-(let (($x12559 (or $x12545 $x12556)))
-(let (($x12562 (and $x12542 $x12559)))
-(let (($x12565 (or $x12518 $x12562)))
-(let (($x12568 (and $x12514 $x12565)))
-(let ((?x12400 (* (- 1) v_b_L_H_p_G_0$)))
-(let ((?x12401 (+ b_S_max_o_u4$ ?x12400)))
-(let (($x12497 (>= ?x12401 1)))
-(let (($x12508 (and $x12494 $x12497 $x12500 $x3960 $x12505 $x12486)))
-(let (($x12511 (not $x12508)))
-(let (($x12571 (or $x12511 $x12568)))
-(let (($x12574 (and $x12494 $x12497 $x12571)))
-(let (($x12598 (or $x12595 $x12574)))
-(let (($x12577 (or $x12491 $x12574)))
-(let (($x12580 (and $x3923 $x3926 $x12577)))
-(let (($x12583 (or $x9775 $x12580)))
-(let (($x12586 (and $x3923 $x3924 $x12583)))
-(let (($x12589 (or $x12482 $x12586)))
-(let (($x12601 (and $x12589 $x12598)))
-(let (($x12604 (or $x12468 $x12601)))
-(let (($x12607 (and $x3923 $x3926 $x12604)))
-(let (($x12610 (or $x9775 $x12607)))
-(let (($x12613 (and $x3923 $x3924 $x12610)))
-(let (($x12616 (or $x12462 $x12613)))
-(let (($x14294 (and $x12616 $x14289)))
-(let (($x12431 (forall ((?v0 Int) )(let ((?x12384 (* (- 1) v_b_L_H_max_G_1$)))
-(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x12425 (<= (+ ?x3765 ?x12384) 0)))
-(let (($x12411 (>= (+ ?v0 (* (- 1) v_b_L_H_p_G_0$)) 0)))
-(let (($x12415 (not $x12411)))
-(let ((?x10215 (* (- 1) b_S_max_o_u4$)))
-(let ((?x10220 (+ ?v0 ?x10215)))
-(let (($x10221 (<= ?x10220 0)))
-(let (($x10138 (>= ?v0 0)))
-(let (($x12418 (and $x10138 $x10221 $x12415)))
-(let (($x12421 (not $x12418)))
-(or $x12421 $x12425)))))))))))))
-))
-(let (($x12399 (>= ?x12401 0)))
-(let (($x12391 (>= (+ b_S_max_o_u4$ (* (- 1) v_b_SL_H_witness_G_0$)) 0)))
-(let (($x12383 (>= (+ b_S_max_o_u1$ (* (- 1) v_b_L_H_max_G_1$)) 0)))
-(let (($x12441 (and $x8667 $x3769 $x12381 $x12383 $x12389 $x12391 $x12397 $x12399 $x12404 $x12407 $x12431 $x12438 $x3794)))
-(let (($x12444 (not $x12441)))
-(let (($x14297 (or $x12444 $x14262 $x14294)))
-(let (($x14300 (and $x8667 $x3769 $x14297)))
-(let (($x12374 (forall ((?v0 Int) )(let ((?x3765 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
-(let (($x12367 (>= (+ v_b_L_H_max_G_0$ (* (- 1) ?x3765)) 0)))
-(let (($x12354 (>= ?v0 1)))
-(let (($x12357 (not $x12354)))
-(let ((?x10215 (* (- 1) b_S_max_o_u4$)))
-(let ((?x10220 (+ ?v0 ?x10215)))
-(let (($x10221 (<= ?x10220 0)))
-(let (($x10138 (>= ?v0 0)))
-(let (($x12360 (and $x10138 $x10221 $x12357)))
-(let (($x12363 (not $x12360)))
-(or $x12363 $x12367))))))))))))
-))
-(let (($x12377 (not $x12374)))
-(let (($x14303 (or $x12377 $x14300)))
-(let (($x14306 (and $x12374 $x14303)))
-(let (($x14309 (or $x12351 $x14306)))
-(let (($x14312 (and $x12348 $x14309)))
-(let (($x14315 (or $x10031 $x14312)))
-(let (($x14318 (and $x3740 $x3743 $x14315)))
-(let (($x14321 (or $x10048 $x14318)))
-(let (($x14324 (and $x3740 $x3741 $x14321)))
-(let (($x14327 (or $x10065 $x14324)))
-(let (($x14330 (and $x3738 $x14327)))
-(let (($x14333 (not $x14330)))
-(let (($x13747 (and $x10138 $x14211 $x12635 $x3840)))
-(let ((?x10215 (* (- 1) b_S_max_o_u4$)))
-(let ((?x10220 (+ ?0 ?x10215)))
-(let (($x10221 (<= ?x10220 0)))
-(let (($x12658 (and $x10138 $x10221 $x12635 $x3840)))
-(let ((?x2232 (* 65536 65536)))
-(let ((?x2237 (- ?x2232 1)))
-(let (($x2238 (= b_S_max_o_u4$ ?x2237)))
-(let ((@x7014 (monotonicity (rewrite (= (* (- 1) 1) (- 1))) (= (+ 4294967296 (* (- 1) 1)) (+ 4294967296 (- 1))))))
-(let ((@x7019 (trans @x7014 (rewrite (= (+ 4294967296 (- 1)) 4294967295)) (= (+ 4294967296 (* (- 1) 1)) 4294967295))))
-(let ((@x7011 (trans (monotonicity (rewrite (= ?x2232 4294967296)) (= ?x2237 (- 4294967296 1))) (rewrite (= (- 4294967296 1) (+ 4294967296 (* (- 1) 1)))) (= ?x2237 (+ 4294967296 (* (- 1) 1))))))
-(let ((@x7024 (monotonicity (trans @x7011 @x7019 (= ?x2237 4294967295)) (= $x2238 (= b_S_max_o_u4$ 4294967295)))))
-(let ((@x7025 (mp (asserted $x2238) @x7024 (= b_S_max_o_u4$ 4294967295))))
-(let ((@x13415 (trans (monotonicity @x7025 (= ?x10215 (* (- 1) 4294967295))) (rewrite (= (* (- 1) 4294967295) (- 4294967295))) (= ?x10215 (- 4294967295)))))
-(let ((@x12861 (trans (monotonicity @x13415 (= ?x10220 (+ ?0 (- 4294967295)))) (rewrite (= (+ ?0 (- 4294967295)) (+ (- 4294967295) ?0))) (= ?x10220 (+ (- 4294967295) ?0)))))
-(let ((@x13817 (trans (monotonicity @x12861 (= $x10221 (<= (+ (- 4294967295) ?0) 0))) (rewrite (= (<= (+ (- 4294967295) ?0) 0) $x14211)) (= $x10221 $x14211))))
-(let ((@x12741 (monotonicity (monotonicity @x13817 (= (and $x10138 $x10221 $x12635) $x13586)) (= (not (and $x10138 $x10221 $x12635)) $x13963))))
-(let ((@x12841 (quant-intro (monotonicity @x12741 (= (or (not (and $x10138 $x10221 $x12635)) $x12646) $x13836)) (= $x12652 $x13163))))
-(let ((@x12999 (monotonicity (monotonicity @x12841 (= $x12655 $x13974)) (quant-intro (monotonicity @x13817 (= $x12658 $x13747)) (= $x12661 $x12742)) (= $x12664 $x14165))))
-(let ((@x13331 (monotonicity (monotonicity @x12841 @x12999 (= $x12667 $x13256)) (= $x14289 $x13521))))
-(let ((@x13632 (monotonicity (monotonicity @x13817 (= (and $x10138 $x10221 $x12525) $x14023)) (= (not (and $x10138 $x10221 $x12525)) $x12802))))
-(let ((@x13024 (quant-intro (monotonicity @x13632 (= (or (not (and $x10138 $x10221 $x12525)) $x12536) $x13633)) (= $x12542 $x13130))))
-(let ((@x14205 (monotonicity @x13024 (monotonicity (monotonicity @x13024 (= $x12545 $x13025)) (= $x12559 $x12874)) (= $x12562 $x13199))))
-(let ((@x14110 (monotonicity (monotonicity @x7025 (= ?x12401 (+ 4294967295 ?x12400))) (= $x12497 (>= (+ 4294967295 ?x12400) 1)))))
-(let ((@x13814 (trans @x14110 (rewrite (= (>= (+ 4294967295 ?x12400) 1) $x13856)) (= $x12497 $x13856))))
-(let ((@x13698 (monotonicity (monotonicity (monotonicity @x13814 (= $x12508 $x13815)) (= $x12511 $x13880)) (monotonicity (monotonicity @x14205 (= $x12565 $x13574)) (= $x12568 $x13045)) (= $x12571 $x14132))))
-(let ((@x13379 (monotonicity (monotonicity @x13814 @x13698 (= $x12574 $x13699)) (= $x12598 $x13117))))
-(let ((@x13206 (monotonicity (monotonicity @x13814 @x13698 (= $x12574 $x13699)) (= $x12577 $x13338))))
-(let ((@x13797 (monotonicity (monotonicity (monotonicity @x13206 (= $x12580 $x13207)) (= $x12583 $x14076)) (= $x12586 $x14119))))
-(let ((@x12956 (monotonicity (monotonicity @x13797 (= $x12589 $x13844)) @x13379 (= $x12601 $x13324))))
-(let ((@x14003 (monotonicity (monotonicity (monotonicity @x12956 (= $x12604 $x12957)) (= $x12607 $x13000)) (= $x12610 $x13827))))
-(let ((@x13356 (monotonicity (monotonicity (monotonicity @x14003 (= $x12613 $x14170)) (= $x12616 $x14053)) @x13331 (= $x14294 $x13922))))
-(let ((@x13685 (monotonicity (monotonicity @x13817 (= (and $x10138 $x10221 $x12415) $x13128)) (= (not (and $x10138 $x10221 $x12415)) $x13111))))
-(let ((@x13593 (quant-intro (monotonicity @x13685 (= (or (not (and $x10138 $x10221 $x12415)) $x12425) $x12774)) (= $x12431 $x13341))))
-(let ((@x13192 (monotonicity (monotonicity @x7025 (= ?x12401 (+ 4294967295 ?x12400))) (= $x12399 (>= (+ 4294967295 ?x12400) 0)))))
-(let ((@x13397 (trans @x13192 (rewrite (= (>= (+ 4294967295 ?x12400) 0) $x13193)) (= $x12399 $x13193))))
-(let ((@x13988 (rewrite (= (>= (+ 4294967295 (* (- 1) v_b_SL_H_witness_G_0$)) 0) $x12834))))
-(let (($x13515 (= (+ b_S_max_o_u4$ (* (- 1) v_b_SL_H_witness_G_0$)) (+ 4294967295 (* (- 1) v_b_SL_H_witness_G_0$)))))
-(let ((@x12807 (monotonicity (monotonicity @x7025 $x13515) (= $x12391 (>= (+ 4294967295 (* (- 1) v_b_SL_H_witness_G_0$)) 0)))))
-(let (($x13742 (= (+ b_S_max_o_u1$ (* (- 1) v_b_L_H_max_G_1$)) (+ 255 (* (- 1) v_b_L_H_max_G_1$)))))
-(let ((@x12798 (monotonicity (monotonicity (asserted (= b_S_max_o_u1$ 255)) $x13742) (= $x12383 (>= (+ 255 (* (- 1) v_b_L_H_max_G_1$)) 0)))))
-(let ((@x13309 (trans @x12798 (rewrite (= (>= (+ 255 (* (- 1) v_b_L_H_max_G_1$)) 0) $x12799)) (= $x12383 $x12799))))
-(let ((@x13590 (monotonicity @x13309 (trans @x12807 @x13988 (= $x12391 $x12834)) @x13397 @x13593 (= $x12441 $x13242))))
-(let ((@x13983 (monotonicity (monotonicity @x13590 (= $x12444 $x13591)) @x13356 (= $x14297 $x13357))))
-(let ((@x13411 (monotonicity (monotonicity @x13817 (= (and $x10138 $x10221 $x12357) $x14020)) (= (not (and $x10138 $x10221 $x12357)) $x13679))))
-(let ((@x14159 (quant-intro (monotonicity @x13411 (= (or (not (and $x10138 $x10221 $x12357)) $x12367) $x12918)) (= $x12374 $x12941))))
-(let ((@x13693 (monotonicity (monotonicity @x14159 (= $x12377 $x13900)) (monotonicity @x13983 (= $x14300 $x12756)) (= $x14303 $x12819))))
-(let ((@x13179 (monotonicity (monotonicity @x14159 @x13693 (= $x14306 $x13702)) (= $x14309 $x13223))))
-(let ((@x13194 (monotonicity (monotonicity (monotonicity @x13179 (= $x14312 $x12832)) (= $x14315 $x13861)) (= $x14318 $x12808))))
-(let ((@x13761 (monotonicity (monotonicity (monotonicity @x13194 (= $x14321 $x13195)) (= $x14324 $x13550)) (= $x14327 $x13361))))
-(let ((@x13603 (monotonicity (monotonicity @x13761 (= $x14330 (and $x3738 $x13361))) (= $x14333 $x13725))))
-(let (($x12625 (and b_S_position_n_marker$ $x12404 $x12389 $x3818 $x3820 $x3822 $x3824)))
-(let (($x12628 (not $x12625)))
-(let (($x12670 (or $x12628 $x12667)))
-(let (($x12673 (and b_S_position_n_marker$ $x12670)))
-(let (($x12676 (or $x12622 $x12673)))
-(let (($x12679 (and $x12616 $x12676)))
-(let (($x12447 (and $x12404 $x12389 $x3886 $x3806 $x3699 $x3893 $x3894 $x3895 $x3896 $x3897 $x3898)))
-(let (($x12450 (not $x12447)))
-(let (($x12682 (or $x12444 $x12450 $x12679)))
-(let (($x12685 (and $x8667 $x3769 $x12682)))
-(let (($x12688 (or $x12377 $x12685)))
-(let (($x12691 (and $x12374 $x12688)))
-(let (($x12694 (or $x12351 $x12691)))
-(let (($x12697 (and $x12348 $x12694)))
-(let (($x12700 (or $x10031 $x12697)))
-(let (($x12703 (and $x3740 $x3743 $x12700)))
-(let (($x12706 (or $x10048 $x12703)))
-(let (($x12709 (and $x3740 $x3741 $x12706)))
-(let (($x12712 (or $x10065 $x12709)))
-(let (($x12715 (and $x3738 $x12712)))
-(let (($x12718 (not $x12715)))
-(let ((@x13981 (iff-true (asserted b_S_position_n_marker$) (= b_S_position_n_marker$ true))))
-(let ((@x14267 (monotonicity @x13981 (= $x12625 (and true $x12404 $x12389 $x3818 $x3820 $x3822 $x3824)))))
-(let ((@x14272 (trans @x14267 (rewrite (= (and true $x12404 $x12389 $x3818 $x3820 $x3822 $x3824) $x14268)) (= $x12625 $x14268))))
-(let ((@x14278 (monotonicity (monotonicity @x14272 (= $x12628 $x14273)) (= $x12670 (or $x14273 $x12667)))))
-(let ((@x14285 (trans (monotonicity @x13981 @x14278 (= $x12673 (and true (or $x14273 $x12667)))) (rewrite (= (and true (or $x14273 $x12667)) (or $x14273 $x12667))) (= $x12673 (or $x14273 $x12667)))))
-(let ((@x14293 (trans (monotonicity @x14285 (= $x12676 (or $x12622 (or $x14273 $x12667)))) (rewrite (= (or $x12622 (or $x14273 $x12667)) $x14289)) (= $x12676 $x14289))))
-(let (($x14258 (= (and $x12404 $x12389 $x3886 $x3806 true $x3893 $x3894 $x3895 $x3896 $x3897 $x3898) $x14257)))
-(let (($x14255 (= $x12447 (and $x12404 $x12389 $x3886 $x3806 true $x3893 $x3894 $x3895 $x3896 $x3897 $x3898))))
-(let ((@x14261 (trans (monotonicity (iff-true @x10104 (= $x3699 true)) $x14255) (rewrite $x14258) (= $x12447 $x14257))))
-(let ((@x14299 (monotonicity (monotonicity @x14261 (= $x12450 $x14262)) (monotonicity @x14293 (= $x12679 $x14294)) (= $x12682 $x14297))))
-(let ((@x14308 (monotonicity (monotonicity (monotonicity @x14299 (= $x12685 $x14300)) (= $x12688 $x14303)) (= $x12691 $x14306))))
-(let ((@x14317 (monotonicity (monotonicity (monotonicity @x14308 (= $x12694 $x14309)) (= $x12697 $x14312)) (= $x12700 $x14315))))
-(let ((@x14326 (monotonicity (monotonicity (monotonicity @x14317 (= $x12703 $x14318)) (= $x12706 $x14321)) (= $x12709 $x14324))))
-(let ((@x14335 (monotonicity (monotonicity (monotonicity @x14326 (= $x12712 $x14327)) (= $x12715 $x14330)) (= $x12718 $x14333))))
-(let ((@x12637 (monotonicity (rewrite (= (<= v_b_P_H_len$ ?0) $x12631)) (= $x9165 $x12635))))
-(let ((@x10223 (rewrite (= $x1344 $x10221))))
-(let ((@x12663 (quant-intro (monotonicity @x10140 @x10223 @x12637 (= $x9202 $x12658)) (= $x9207 $x12661))))
-(let ((@x12640 (monotonicity @x10140 @x10223 @x12637 (= (and $x1212 $x1344 $x9165) (and $x10138 $x10221 $x12635)))))
-(let ((@x12643 (monotonicity @x12640 (= (not (and $x1212 $x1344 $x9165)) (not (and $x10138 $x10221 $x12635))))))
-(let ((@x12651 (monotonicity @x12643 (rewrite (= $x3837 $x12646)) (= $x9180 (or (not (and $x10138 $x10221 $x12635)) $x12646)))))
-(let ((@x12657 (monotonicity (quant-intro @x12651 (= $x9185 $x12652)) (= (not $x9185) $x12655))))
-(let ((@x12669 (monotonicity (quant-intro @x12651 (= $x9185 $x12652)) (monotonicity @x12657 @x12663 (= $x9228 $x12664)) (= $x9233 $x12667))))
-(let ((@x12390 (rewrite (= $x3776 $x12389))))
-(let ((@x12406 (rewrite (= $x3783 $x12404))))
-(let ((@x12630 (monotonicity (monotonicity @x12406 @x12390 (= $x9159 $x12625)) (= (not $x9159) $x12628))))
-(let ((@x12675 (monotonicity (monotonicity @x12630 @x12669 (= $x9240 $x12670)) (= $x9245 $x12673))))
-(let ((@x12621 (monotonicity @x12406 @x12390 (rewrite (= $x4012 $x12453)) (= (and $x3783 $x3776 $x4012) $x12619))))
-(let ((@x12678 (monotonicity (monotonicity @x12621 (= (not (and $x3783 $x3776 $x4012)) $x12622)) @x12675 (= $x9963 $x12676))))
-(let ((@x12555 (monotonicity (rewrite (= (<= v_b_P_H_len$ v_b_SL_H_witness_G_1$) $x12550)) (= $x9687 $x12553))))
-(let ((@x12527 (monotonicity (rewrite (= (<= v_b_L_H_p_G_1$ ?0) $x12521)) (= $x9663 $x12525))))
-(let ((@x12533 (monotonicity (monotonicity @x10140 @x10223 @x12527 (= $x9669 (and $x10138 $x10221 $x12525))) (= (not $x9669) (not (and $x10138 $x10221 $x12525))))))
-(let ((@x12541 (monotonicity @x12533 (rewrite (= $x3970 $x12536)) (= $x9678 (or (not (and $x10138 $x10221 $x12525)) $x12536)))))
-(let ((@x12547 (monotonicity (quant-intro @x12541 (= $x9683 $x12542)) (= (not $x9683) $x12545))))
-(let ((@x12561 (monotonicity @x12547 (monotonicity @x12555 (= $x9690 $x12556)) (= $x9718 $x12559))))
-(let ((@x12567 (monotonicity (monotonicity (rewrite (= $x3967 $x12514)) (= (not $x3967) $x12518)) (monotonicity (quant-intro @x12541 (= $x9683 $x12542)) @x12561 (= $x9723 $x12562)) (= $x9730 $x12565))))
-(let ((@x12487 (rewrite (= $x3943 $x12486))))
-(let ((@x12510 (monotonicity (rewrite (= $x9606 $x12494)) (rewrite (= $x9615 $x12497)) (rewrite (= $x9623 $x12500)) (rewrite (= $x3961 $x12505)) @x12487 (= $x9657 $x12508))))
-(let ((@x12573 (monotonicity (monotonicity @x12510 (= (not $x9657) $x12511)) (monotonicity (rewrite (= $x3967 $x12514)) @x12567 (= $x9735 $x12568)) (= $x9742 $x12571))))
-(let ((@x12576 (monotonicity (rewrite (= $x9606 $x12494)) (rewrite (= $x9615 $x12497)) @x12573 (= $x9750 $x12574))))
-(let ((@x12594 (monotonicity @x12406 @x12390 (rewrite (= $x3992 $x12471)) @x12487 (= $x9858 $x12592))))
-(let ((@x12600 (monotonicity (monotonicity @x12594 (= (not $x9858) $x12595)) @x12576 (= $x9874 $x12598))))
-(let ((@x12493 (monotonicity (monotonicity @x12406 @x12487 (= $x9595 $x12488)) (= (not $x9595) $x12491))))
-(let ((@x12582 (monotonicity (monotonicity @x12493 @x12576 (= $x9759 $x12577)) (= $x9767 $x12580))))
-(let ((@x12481 (monotonicity @x12406 @x12390 (monotonicity (rewrite (= $x3992 $x12471)) (= $x9497 $x12476)) (= $x9511 $x12479))))
-(let ((@x12591 (monotonicity (monotonicity @x12481 (= (not $x9511) $x12482)) (monotonicity (monotonicity @x12582 (= $x9776 $x12583)) (= $x9784 $x12586)) (= $x9793 $x12589))))
-(let ((@x12470 (monotonicity (monotonicity @x12406 @x12390 (= (and $x3923 $x3926 $x3783 $x3776) $x12465)) (= (not (and $x3923 $x3926 $x3783 $x3776)) $x12468))))
-(let ((@x12606 (monotonicity @x12470 (monotonicity @x12591 @x12600 (= $x9879 $x12601)) (= $x9886 $x12604))))
-(let ((@x12615 (monotonicity (monotonicity (monotonicity @x12606 (= $x9894 $x12607)) (= $x9902 $x12610)) (= $x9910 $x12613))))
-(let ((@x12461 (monotonicity @x12406 @x12390 (monotonicity (rewrite (= $x4012 $x12453)) (= $x9465 $x12456)) (= $x9479 $x12459))))
-(let ((@x12618 (monotonicity (monotonicity @x12461 (= (not $x9479) $x12462)) @x12615 (= $x9919 $x12616))))
-(let ((@x12452 (monotonicity (monotonicity @x12406 @x12390 (= $x9434 $x12447)) (= $x9974 $x12450))))
-(let ((@x12440 (monotonicity (rewrite (= (<= v_b_P_H_len$ v_b_SL_H_witness_G_0$) $x12435)) (= $x8960 $x12438))))
-(let ((@x12417 (monotonicity (rewrite (= (<= v_b_L_H_p_G_0$ ?0) $x12411)) (= $x8936 $x12415))))
-(let ((@x12423 (monotonicity (monotonicity @x10140 @x10223 @x12417 (= $x8942 (and $x10138 $x10221 $x12415))) (= (not $x8942) (not (and $x10138 $x10221 $x12415))))))
-(let ((@x12430 (monotonicity @x12423 (rewrite (= $x3788 $x12425)) (= $x8951 (or (not (and $x10138 $x10221 $x12415)) $x12425)))))
-(let ((@x12443 (monotonicity (rewrite (= $x3772 $x12381)) (rewrite (= $x3773 $x12383)) @x12390 (rewrite (= $x3777 $x12391)) (rewrite (= $x3780 $x12397)) (rewrite (= $x3781 $x12399)) @x12406 (rewrite (= $x3785 $x12407)) (quant-intro @x12430 (= $x8956 $x12431)) @x12440 (= $x9032 $x12441))))
-(let ((@x12684 (monotonicity (monotonicity @x12443 (= (not $x9032) $x12444)) @x12452 (monotonicity @x12618 @x12678 (= $x9968 $x12679)) (= $x9991 $x12682))))
-(let ((@x12362 (monotonicity @x10140 @x10223 (monotonicity (rewrite (= $x8887 $x12354)) (= $x8888 $x12357)) (= $x8899 (and $x10138 $x10221 $x12357)))))
-(let ((@x12373 (monotonicity (monotonicity @x12362 (= (not $x8899) (not (and $x10138 $x10221 $x12357)))) (rewrite (= $x3766 $x12367)) (= $x8908 (or (not (and $x10138 $x10221 $x12357)) $x12367)))))
-(let ((@x12379 (monotonicity (quant-intro @x12373 (= $x8913 $x12374)) (= (not $x8913) $x12377))))
-(let ((@x12690 (monotonicity @x12379 (monotonicity @x12684 (= $x9999 $x12685)) (= $x10008 $x12688))))
-(let ((@x12696 (monotonicity (monotonicity (rewrite (= $x3761 $x12348)) (= (not $x3761) $x12351)) (monotonicity (quant-intro @x12373 (= $x8913 $x12374)) @x12690 (= $x10013 $x12691)) (= $x10020 $x12694))))
-(let ((@x12702 (monotonicity (monotonicity (rewrite (= $x3761 $x12348)) @x12696 (= $x10025 $x12697)) (= $x10032 $x12700))))
-(let ((@x12711 (monotonicity (monotonicity (monotonicity @x12702 (= $x10040 $x12703)) (= $x10049 $x12706)) (= $x10057 $x12709))))
-(let ((@x12720 (monotonicity (monotonicity (monotonicity @x12711 (= $x10066 $x12712)) (= $x10071 $x12715)) (= (not $x10071) $x12718))))
-(let ((@x12721 (mp (not-or-elim (mp (asserted $x4036) @x10085 (not $x10078)) (not $x10071)) @x12720 $x12718)))
-(let ((@x20468 (mp (mp (mp~ (mp (mp @x12721 @x14335 $x14333) @x13603 $x13725) @x16564 $x16562) @x16835 $x16833) @x20467 $x20465)))
-(let ((@x21274 (mp @x20468 (monotonicity @x21270 (= $x20465 (or $x10065 $x21268))) (or $x10065 $x21268))))
-(let ((@x24559 (unit-resolution @x21274 (lemma (unit-resolution @x23120 @x23099 @x23095 @x23071 @x23078 false) $x3738) $x21268)))
-(let ((@x24561 (unit-resolution (def-axiom (or $x21262 $x16242 $x16245 $x21256)) (unit-resolution (def-axiom (or $x21265 $x21259)) @x24559 $x21259) $x21259)))
-(let ((@x24567 (unit-resolution @x24561 (unit-resolution (def-axiom (or $x23304 $x3741)) (lemma @x23396 $x23305) $x3741) @x23251 $x21256)))
-(let ((@x24570 (unit-resolution (def-axiom (or $x21250 $x16242 $x16251 $x21244)) @x23251 (unit-resolution (def-axiom (or $x21253 $x21247)) @x24567 $x21247) (or $x16251 $x21244))))
-(let ((@x25304 (unit-resolution (def-axiom (or $x21241 $x21235)) (unit-resolution @x24570 (lemma @x23543 $x3743) $x21244) $x21235)))
-(let ((@x25314 (unit-resolution (unit-resolution (def-axiom (or $x21238 $x12351 $x21232)) @x25304 $x21235) (lemma ((_ th-lemma arith farkas 1 1) @x10095 (hypothesis $x12351) false) $x12348) $x21232)))
-(let (($x16266 (not $x16265)))
-(let ((@x24547 (hypothesis $x20036)))
-(let (($x16263 (>= ?v0!13 0)))
-(let ((@x24551 ((_ th-lemma arith eq-propagate 0 0) (unit-resolution (def-axiom (or $x20031 $x16263)) @x24547 $x16263) (unit-resolution (def-axiom (or $x20031 $x16266)) @x24547 $x16266) (= ?v0!13 0))))
-(let ((@x24574 (monotonicity (monotonicity @x24551 (= (b_S_idx$ ?x3680 ?v0!13 b_T_T_u1$) ?x3739)) (= ?x16270 ?x3746))))
-(let ((@x24572 (unit-resolution (def-axiom (or $x21241 $x3747)) (unit-resolution @x24570 (lemma @x23543 $x3743) $x21244) $x3747)))
-(let ((@x24591 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= v_b_L_H_max_G_0$ ?x16270)) $x16273)) (unit-resolution (def-axiom (or $x20031 (not $x16273))) @x24547 (not $x16273)) (trans @x24572 (symm @x24574 (= ?x3746 ?x16270)) (= v_b_L_H_max_G_0$ ?x16270)) false)))
-(let ((@x25316 (unit-resolution (def-axiom (or $x21226 $x20036 $x21220)) (lemma @x24591 $x20031) (unit-resolution (def-axiom (or $x21229 $x21223)) @x25314 $x21223) $x21220)))
-(let ((@x25324 (unit-resolution (def-axiom (or $x21214 $x8666 $x16288 $x21208)) @x10095 (or $x21214 $x16288 $x21208))))
-(let ((@x25326 (unit-resolution @x25324 (mp @x24572 (symm (commutativity (= $x3769 $x3747)) (= $x3747 $x3769)) $x3769) (or $x21214 $x21208))))
-(let ((@x25327 (unit-resolution @x25326 (unit-resolution (def-axiom (or $x21217 $x21211)) @x25316 $x21211) $x21208)))
-(let ((@x25328 (unit-resolution (def-axiom (or $x21205 $x12397)) @x25327 $x12397)))
-(let ((@x25333 (unit-resolution (def-axiom (or $x21205 $x21041)) @x25327 $x21041)))
-(let (($x23869 (<= (+ v_b_L_H_p_G_0$ (* (- 1) ?v0!15)) 0)))
-(let (($x23793 (<= (+ v_b_L_H_max_G_1$ (* (- 1) v_b_S_result_G_0$)) 0)))
-(let (($x23789 (= v_b_L_H_max_G_1$ v_b_S_result_G_0$)))
-(let ((@x24013 (symm (unit-resolution (def-axiom (or $x21193 $x3824)) (hypothesis $x21196) $x3824) $x23789)))
-(let (($x21519 (not $x16760)))
-(let ((@x23878 (trans (hypothesis $x3794) (symm (hypothesis $x3824) $x23789) (= ?x3793 v_b_S_result_G_0$))))
-(let (($x23841 (not (= ?x3793 v_b_S_result_G_0$))))
-(let (($x23846 (or $x21178 $x20219 $x20374 $x12435 $x23841)))
-(let (($x23737 (>= (+ v_b_SL_H_witness_G_0$ (* (- 1) v_b_P_H_len$)) 0)))
-(let (($x23847 (or $x21178 (or $x20219 $x20374 $x23737 $x23841))))
-(let (($x23747 (= (>= (+ (* (- 1) v_b_P_H_len$) v_b_SL_H_witness_G_0$) 0) $x12435)))
-(let (($x23745 (= $x23737 (>= (+ (* (- 1) v_b_P_H_len$) v_b_SL_H_witness_G_0$) 0))))
-(let (($x23742 (= (+ v_b_SL_H_witness_G_0$ (* (- 1) v_b_P_H_len$)) (+ (* (- 1) v_b_P_H_len$) v_b_SL_H_witness_G_0$))))
-(let ((@x23750 (trans (monotonicity (rewrite $x23742) $x23745) (rewrite $x23747) (= $x23737 $x12435))))
-(let ((@x23845 (monotonicity @x23750 (= (or $x20219 $x20374 $x23737 $x23841) (or $x20219 $x20374 $x12435 $x23841)))))
-(let ((@x23855 (trans (monotonicity @x23845 (= $x23847 (or $x21178 (or $x20219 $x20374 $x12435 $x23841)))) (rewrite (= (or $x21178 (or $x20219 $x20374 $x12435 $x23841)) $x23846)) (= $x23847 $x23846))))
-(let ((@x23883 (unit-resolution (mp ((_ quant-inst v_b_SL_H_witness_G_0$) $x23847) @x23855 $x23846) (hypothesis $x12834) (hypothesis $x12438) (hypothesis $x12389) (hypothesis $x21173) @x23878 false)))
-(let ((@x24019 (unit-resolution (lemma @x23883 (or $x21178 $x20374 $x12435 $x20219 $x20379 $x20358)) (unit-resolution (def-axiom (or $x21193 $x3824)) (hypothesis $x21196) $x3824) (hypothesis $x12438) (hypothesis $x12389) (hypothesis $x3794) (hypothesis $x12834) $x21178)))
-(let ((@x24021 (unit-resolution (def-axiom (or $x21190 $x20298 $x21184)) (unit-resolution (def-axiom (or $x21181 $x21173)) @x24019 $x21181) (unit-resolution (def-axiom (or $x21193 $x21187)) (hypothesis $x21196) $x21187) $x20298)))
-(let (($x24008 (or (not (>= (+ v_b_L_H_max_G_1$ (* (- 1) ?x16481)) 0)) $x16760 (not $x23793))))
-(let ((@x24005 ((_ th-lemma arith farkas -1 1 1) (hypothesis (>= (+ v_b_L_H_max_G_1$ (* (- 1) ?x16481)) 0)) (hypothesis $x21519) (hypothesis $x23793) false)))
-(let ((@x24023 (unit-resolution (lemma @x24005 $x24008) (unit-resolution (def-axiom (or $x20293 $x21519)) @x24021 $x21519) (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x23789) $x23793)) @x24013 $x23793) (not (>= (+ v_b_L_H_max_G_1$ (* (- 1) ?x16481)) 0)))))
-(let (($x23889 (>= (+ v_b_L_H_max_G_1$ (* (- 1) ?x16481)) 0)))
-(let (($x23897 (or $x21046 $x20277 $x20278 $x23869 $x23889)))
-(let (($x23835 (<= (+ ?x16481 (* (- 1) v_b_L_H_max_G_1$)) 0)))
-(let (($x23815 (>= (+ ?v0!15 ?x12400) 0)))
-(let (($x23898 (or $x21046 (or $x20277 $x20278 $x23815 $x23835))))
-(let (($x23874 (= (+ ?x16481 (* (- 1) v_b_L_H_max_G_1$)) (+ (* (- 1) v_b_L_H_max_G_1$) ?x16481))))
-(let ((@x23887 (monotonicity (rewrite $x23874) (= $x23835 (<= (+ (* (- 1) v_b_L_H_max_G_1$) ?x16481) 0)))))
-(let ((@x23893 (trans @x23887 (rewrite (= (<= (+ (* (- 1) v_b_L_H_max_G_1$) ?x16481) 0) $x23889)) (= $x23835 $x23889))))
-(let ((@x23867 (monotonicity (rewrite (= (+ ?v0!15 ?x12400) (+ ?x12400 ?v0!15))) (= $x23815 (>= (+ ?x12400 ?v0!15) 0)))))
-(let ((@x23872 (trans @x23867 (rewrite (= (>= (+ ?x12400 ?v0!15) 0) $x23869)) (= $x23815 $x23869))))
-(let ((@x23896 (monotonicity @x23872 @x23893 (= (or $x20277 $x20278 $x23815 $x23835) (or $x20277 $x20278 $x23869 $x23889)))))
-(let ((@x23906 (trans (monotonicity @x23896 (= $x23898 (or $x21046 (or $x20277 $x20278 $x23869 $x23889)))) (rewrite (= (or $x21046 (or $x20277 $x20278 $x23869 $x23889)) $x23897)) (= $x23898 $x23897))))
-(let ((@x24028 (unit-resolution (mp ((_ quant-inst ?v0!15) $x23898) @x23906 $x23897) (hypothesis $x21041) (unit-resolution (def-axiom (or $x20293 $x16473)) @x24021 $x16473) (unit-resolution (def-axiom (or $x20293 $x16474)) @x24021 $x16474) (or $x23869 $x23889))))
-(let ((@x24031 ((_ th-lemma arith farkas -1 1 1) (unit-resolution (def-axiom (or $x20293 $x16743)) @x24021 $x16743) (unit-resolution @x24028 @x24023 $x23869) (unit-resolution (def-axiom (or $x21193 $x12453)) (hypothesis $x21196) $x12453) false)))
-(let ((@x25334 (unit-resolution (lemma @x24031 (or $x21193 $x21046 $x12435 $x20219 $x20379 $x20374)) @x25333 (unit-resolution (def-axiom (or $x21205 $x12438)) @x25327 $x12438) (unit-resolution (def-axiom (or $x21205 $x12389)) @x25327 $x12389) (unit-resolution (def-axiom (or $x21205 $x3794)) @x25327 $x3794) (unit-resolution (def-axiom (or $x21205 $x12834)) @x25327 $x12834) $x21193)))
-(let ((@x25336 (unit-resolution (def-axiom (or $x21202 $x21162 $x21196)) (unit-resolution (def-axiom (or $x21205 $x21199)) @x25327 $x21199) @x25334 $x21162)))
-(let ((@x25337 (unit-resolution (def-axiom (or $x21159 $x12456)) @x25336 $x12456)))
-(let ((@x25341 (mp @x23336 (symm (monotonicity @x24339 (= $x23297 $x23045)) (= $x23045 $x23297)) $x23297)))
-(let (($x24098 (or $x23330 $x21687 $x22190 $x23298 $x20375 $x12453 $x24083)))
-(let (($x24080 (>= (+ v_b_L_H_p_G_0$ (* (- 1) v_b_P_H_len$)) 0)))
-(let (($x24099 (or $x23330 (or $x21687 $x22190 $x23298 $x20375 $x24080 $x24083))))
-(let (($x24096 (= (or $x21687 $x22190 $x23298 $x20375 $x24080 $x24083) (or $x21687 $x22190 $x23298 $x20375 $x12453 $x24083))))
-(let ((@x24092 (rewrite (= (>= (+ (* (- 1) v_b_P_H_len$) v_b_L_H_p_G_0$) 0) $x12453))))
-(let (($x24086 (= (+ v_b_L_H_p_G_0$ (* (- 1) v_b_P_H_len$)) (+ (* (- 1) v_b_P_H_len$) v_b_L_H_p_G_0$))))
-(let ((@x24090 (monotonicity (rewrite $x24086) (= $x24080 (>= (+ (* (- 1) v_b_P_H_len$) v_b_L_H_p_G_0$) 0)))))
-(let ((@x24103 (monotonicity (monotonicity (trans @x24090 @x24092 (= $x24080 $x12453)) $x24096) (= $x24099 (or $x23330 (or $x21687 $x22190 $x23298 $x20375 $x12453 $x24083))))))
-(let ((@x24107 (trans @x24103 (rewrite (= (or $x23330 (or $x21687 $x22190 $x23298 $x20375 $x12453 $x24083)) $x24098)) (= $x24099 $x24098))))
-(let ((@x24142 (unit-resolution (mp ((_ quant-inst v_b_S_s$ v_b_P_H_arr$ (b_S_ptr$ ?x3678 ?x21715) v_b_P_H_len$ v_b_L_H_p_G_0$ b_T_T_u1$) $x24099) @x24107 $x24098) @x19388 @x5093 @x10104 (hypothesis $x12397) (hypothesis $x12456) (hypothesis $x23297) (hypothesis $x24082) false)))
-(let ((@x25343 (unit-resolution (lemma @x24142 (or $x24083 $x20375 $x12453 $x23298)) @x25341 (or $x24083 $x20375 $x12453))))
-(let ((@x25345 (unit-resolution (def-axiom (or $x24082 $x3924)) (unit-resolution @x25343 @x25337 @x25328 $x24083) $x3924)))
-(let ((@x25354 (unit-resolution (hypothesis $x24195) (mp @x25345 (symm @x25350 (= $x3924 $x24194)) $x24194) false)))
-(let ((@x25215 (unit-resolution (def-axiom (or $x24228 $x24195 $x24226)) (unit-resolution (lemma @x25354 (or $x24194 (not $x23973))) @x25156 $x24194) (or $x24228 $x24226))))
-(let ((@x25214 (unit-resolution (def-axiom (or (not $x23994) $x16330 $x23984)) @x25032 (or (not $x23994) $x23984))))
-(let ((@x25219 (unit-resolution @x25214 (unit-resolution ((_ quant-inst (b_S_idx$ ?x3680 v_b_L_H_p_G_0$ b_T_T_u1$) b_T_T_u1$) (or (not $x20961) $x23994)) @x20966 $x23994) $x23984)))
-(let ((@x25248 (trans (monotonicity (symm @x25156 (= ?x23972 ?x3922)) (= (b_S_typ$ ?x23972) ?x23986)) @x25219 (= (b_S_typ$ ?x23972) b_T_T_u1$))))
-(let ((@x25302 (trans (monotonicity @x25248 (= (b_S_kind_n_of$ (b_S_typ$ ?x23972)) ?x22173)) @x23477 $x24198)))
-(let ((@x25229 (monotonicity (symm (monotonicity @x25156 (= ?x23936 ?x24200)) (= ?x24200 ?x23936)) (= $x24201 $x24081))))
-(let (($x24854 (not $x24081)))
-(let ((@x25388 (unit-resolution (def-axiom (or $x24082 $x24854)) (unit-resolution @x25343 @x25337 @x25328 $x24083) $x24854)))
-(let ((@x25238 (mp @x25388 (monotonicity (symm @x25229 (= $x24081 $x24201)) (= $x24854 $x24202)) $x24202)))
-(let ((?x25453 (+ ?x24037 ?x24269)))
-(let ((?x25458 (b_S_ptr$ b_T_T_u1$ ?x25453)))
-(let ((?x25435 (b_S_idx$ ?x22684 v_b_L_H_p_G_0$ b_T_T_u1$)))
-(let (($x25461 (= ?x25435 ?x25458)))
-(let (($x25464 (not $x25461)))
-(let (($x25467 (or (not (b_S_extent_n_hint$ ?x25435 ?x22684)) $x25464)))
-(let (($x25470 (not $x25467)))
-(let (($x25473 (or $x23217 $x25470)))
-(let (($x25447 (not (= ?x25435 (b_S_ptr$ b_T_T_u1$ (+ ?x24269 (* v_b_L_H_p_G_0$ ?x3652)))))))
-(let (($x25476 (= (or $x23217 (not (or (not (b_S_extent_n_hint$ ?x25435 ?x22684)) $x25447))) $x25473)))
-(let (($x25462 (= (= ?x25435 (b_S_ptr$ b_T_T_u1$ (+ ?x24269 (* v_b_L_H_p_G_0$ ?x3652)))) $x25461)))
-(let ((@x25452 (monotonicity (rewrite (= (* v_b_L_H_p_G_0$ ?x3652) ?x24037)) (= (+ ?x24269 (* v_b_L_H_p_G_0$ ?x3652)) (+ ?x24269 ?x24037)))))
-(let ((@x25457 (trans @x25452 (rewrite (= (+ ?x24269 ?x24037) ?x25453)) (= (+ ?x24269 (* v_b_L_H_p_G_0$ ?x3652)) ?x25453))))
-(let ((@x25460 (monotonicity @x25457 (= (b_S_ptr$ b_T_T_u1$ (+ ?x24269 (* v_b_L_H_p_G_0$ ?x3652))) ?x25458))))
-(let ((@x25469 (monotonicity (monotonicity (monotonicity @x25460 $x25462) (= $x25447 $x25464)) (= (or (not (b_S_extent_n_hint$ ?x25435 ?x22684)) $x25447) $x25467))))
-(let ((@x25472 (monotonicity @x25469 (= (not (or (not (b_S_extent_n_hint$ ?x25435 ?x22684)) $x25447)) $x25470))))
-(let ((@x25475 ((_ quant-inst (b_S_ptr$ ?x3678 ?x21715) v_b_L_H_p_G_0$ b_T_T_u1$) (or $x23217 (not (or (not (b_S_extent_n_hint$ ?x25435 ?x22684)) $x25447))))))
-(let ((@x25481 (mp @x25475 (trans (monotonicity @x25472 $x25476) (rewrite (= $x25473 $x25473)) $x25476) $x25473)))
-(let ((@x25407 (unit-resolution (def-axiom (or $x25467 $x25461)) (lemma (unit-resolution @x25481 @x18901 (hypothesis $x25467) false) $x25470) $x25461)))
-(let ((?x25308 (b_S_idx$ ?x23296 v_b_L_H_p_G_0$ b_T_T_u1$)))
-(let ((?x25309 (b_S_select_o_tm$ ?x3874 ?x25308)))
-(let (($x25310 (= (b_S_ts_n_emb$ ?x25309) ?x23296)))
-(let (($x25362 (or (not $x25310) (b_S_ts_n_is_n_volatile$ ?x25309) (not (b_S_ts_n_is_n_array_n_elt$ ?x25309)) (not (b_S_typed$ v_b_S_s$ ?x25308)))))
-(let (($x25363 (not $x25362)))
-(let (($x25293 (or $x24161 $x24152 $x20375 $x12453 $x25363)))
-(let (($x25294 (or $x24161 (or $x24152 $x20375 $x24080 $x25363))))
-(let ((@x25292 (monotonicity (trans @x24090 @x24092 (= $x24080 $x12453)) (= (or $x24152 $x20375 $x24080 $x25363) (or $x24152 $x20375 $x12453 $x25363)))))
-(let ((@x25384 (trans (monotonicity @x25292 (= $x25294 (or $x24161 (or $x24152 $x20375 $x12453 $x25363)))) (rewrite (= (or $x24161 (or $x24152 $x20375 $x12453 $x25363)) $x25293)) (= $x25294 $x25293))))
-(let ((@x25376 (unit-resolution (mp ((_ quant-inst v_b_S_s$ v_b_P_H_arr$ b_T_T_u1$ v_b_P_H_len$ v_b_L_H_p_G_0$) $x25294) @x25384 $x25293) @x18685 @x25328 @x25337 (lemma (unit-resolution (hypothesis $x24152) @x24253 false) $x24131) (hypothesis $x25362) false)))
-(let ((@x25585 (trans (trans @x23922 @x23269 (= ?x23206 ?x23203)) (symm @x24358 (= ?x23203 ?x3680)) (= ?x23206 ?x3680))))
-(let ((@x25593 (trans (symm @x25587 (= ?x24043 ?x23996)) (monotonicity @x25585 (= ?x23996 ?x3922)) (= ?x24043 ?x3922))))
-(let (($x25908 (>= (+ ?x24040 (* (- 1) (b_S_ref$ ?x24043))) 0)))
-(let ((?x25052 (+ ?x23612 ?x24037 (* (- 1) (b_S_ref$ ?x24043)))))
-(let (($x25064 (>= ?x25052 0)))
-(let (($x25050 (= ?x25052 0)))
-(let (($x21853 (not $x20968)))
-(let (($x25054 (or $x21853 $x25050)))
-(let ((@x25058 (monotonicity (rewrite (= (= (b_S_ref$ ?x24043) ?x24040) $x25050)) (= (or $x21853 (= (b_S_ref$ ?x24043) ?x24040)) $x25054))))
-(let ((@x25061 (trans @x25058 (rewrite (= $x25054 $x25054)) (= (or $x21853 (= (b_S_ref$ ?x24043) ?x24040)) $x25054))))
-(let ((@x25599 (unit-resolution (mp ((_ quant-inst b_T_T_u1$ (+ ?x23612 ?x24037)) (or $x21853 (= (b_S_ref$ ?x24043) ?x24040))) @x25061 $x25054) @x20973 $x25050)))
-(let ((@x25911 (unit-resolution ((_ th-lemma arith assign-bounds -1) (or $x25908 (not $x25064))) (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x25050) $x25064)) @x25599 $x25064) $x25908)))
-(let (($x25907 (<= (+ ?x24040 (* (- 1) (b_S_ref$ ?x24043))) 0)))
-(let (($x25063 (<= ?x25052 0)))
-(let ((@x25914 (unit-resolution ((_ th-lemma arith assign-bounds -1) (or $x25907 (not $x25063))) (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x25050) $x25063)) @x25599 $x25063) $x25907)))
-(let ((@x25925 (unit-resolution ((_ th-lemma arith triangle-eq) (or (= ?x24040 (b_S_ref$ ?x24043)) (not $x25907) (not $x25908))) @x25914 @x25911 (= ?x24040 (b_S_ref$ ?x24043)))))
-(let (($x25910 (>= (+ ?x24040 (* (- 1) ?x25453)) 0)))
-(let (($x23420 (<= (+ ?x21715 (* (- 1) ?x23186)) 0)))
-(let ((@x25567 (monotonicity (trans @x23269 (symm @x24358 (= ?x23203 ?x3680)) (= ?x3739 ?x3680)) (= ?x23186 ?x3681))))
-(let ((@x25574 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x21715 ?x23186)) $x23420)) (trans @x24327 (symm @x25567 (= ?x3681 ?x23186)) (= ?x21715 ?x23186)) $x23420)))
-(let (($x25491 (>= (+ ?x21715 (* (- 1) ?x24269)) 0)))
-(let ((@x25608 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x21715 ?x24269)) $x25491)) (symm (monotonicity @x24449 (= ?x24269 ?x21715)) (= ?x21715 ?x24269)) $x25491)))
-(let (($x24750 (<= (+ ?x23186 (* (- 1) ?x23612)) 0)))
-(let ((@x25581 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x23186 ?x23612)) $x24750)) (symm (monotonicity @x23922 (= ?x23612 ?x23186)) (= ?x23186 ?x23612)) $x24750)))
-(let ((@x25922 (unit-resolution ((_ th-lemma arith assign-bounds 1 -1 1) (or $x25910 (not $x24750) (not $x25491) (not $x23420))) @x25581 @x25608 @x25574 $x25910)))
-(let (($x25909 (<= (+ ?x24040 (* (- 1) ?x25453)) 0)))
-(let (($x23421 (>= (+ ?x21715 (* (- 1) ?x23186)) 0)))
-(let ((@x25619 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x21715 ?x23186)) $x23421)) (trans @x24327 (symm @x25567 (= ?x3681 ?x23186)) (= ?x21715 ?x23186)) $x23421)))
-(let (($x25490 (<= (+ ?x21715 (* (- 1) ?x24269)) 0)))
-(let ((@x25631 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x21715 ?x24269)) $x25490)) (symm (monotonicity @x24449 (= ?x24269 ?x21715)) (= ?x21715 ?x24269)) $x25490)))
-(let (($x24751 (>= (+ ?x23186 (* (- 1) ?x23612)) 0)))
-(let ((@x25622 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x23186 ?x23612)) $x24751)) (symm (monotonicity @x23922 (= ?x23612 ?x23186)) (= ?x23186 ?x23612)) $x24751)))
-(let ((@x25916 (unit-resolution ((_ th-lemma arith assign-bounds 1 -1 1) (or $x25909 (not $x24751) (not $x25490) (not $x23421))) @x25622 @x25631 @x25619 $x25909)))
-(let ((@x25951 (unit-resolution ((_ th-lemma arith triangle-eq) (or (= ?x24040 ?x25453) (not $x25909) (not $x25910))) @x25916 @x25922 (= ?x24040 ?x25453))))
-(let ((@x25927 (trans (trans (symm @x25951 (= ?x25453 ?x24040)) @x25925 (= ?x25453 (b_S_ref$ ?x24043))) (monotonicity @x25593 (= (b_S_ref$ ?x24043) ?x24124)) (= ?x25453 ?x24124))))
-(let ((@x25944 (trans (monotonicity @x24339 (= ?x25308 ?x25435)) (hypothesis $x25461) (= ?x25308 ?x25458))))
-(let ((@x25837 (monotonicity (trans @x25944 (monotonicity @x25927 (= ?x25458 ?x23972)) (= ?x25308 ?x23972)) (= ?x25309 ?x24200))))
-(let ((@x25955 (trans (monotonicity (symm @x25837 (= ?x24200 ?x25309)) (= ?x24203 (b_S_ts_n_emb$ ?x25309))) (unit-resolution (def-axiom (or $x25362 $x25310)) (lemma @x25376 $x25363) $x25310) (= ?x24203 ?x23296))))
-(let ((@x25957 (monotonicity (trans @x25955 @x23339 (= ?x24203 ?x3682)) (= (b_S_owner$ v_b_S_s$ ?x24203) ?x3684))))
-(let ((@x25971 (unit-resolution (hypothesis (not $x24212)) (trans @x25957 @x10097 $x24212) false)))
-(let ((@x25374 (unit-resolution (def-axiom (or $x24214 (not $x24212))) (unit-resolution (lemma @x25971 (or $x25464 $x24212)) @x25407 $x24212) $x24214)))
-(let (($x25207 (or (not $x19952) (not (or $x24210 (not (b_S_is_n_non_n_primitive$ (b_S_typ$ ?x24203))))))))
-(let ((@x25126 (unit-resolution ((_ quant-inst (b_S_select_o_tm$ ?x3874 ?x23972)) $x25207) @x19955 (hypothesis (or $x24210 (not (b_S_is_n_non_n_primitive$ (b_S_typ$ ?x24203))))) false)))
-(let ((@x25204 (lemma @x25126 (not (or $x24210 (not (b_S_is_n_non_n_primitive$ (b_S_typ$ ?x24203))))))))
-(let (($x25192 (or $x24210 (not (b_S_is_n_non_n_primitive$ (b_S_typ$ ?x24203))))))
-(let ((@x25299 (unit-resolution (def-axiom (or $x24217 $x24199 $x24207 $x24210 (not $x24214))) (unit-resolution (def-axiom (or $x25192 (not $x24210))) @x25204 (not $x24210)) @x25374 (or $x24217 $x24199 $x24207))))
-(let ((@x25300 (unit-resolution @x25299 (unit-resolution (def-axiom (or $x24206 $x24201)) @x25238 $x24206) @x25302 $x24217)))
-(let (($x25367 (or (or $x24217 (not (or $x24198 (not $x24221)))) (or $x24199 $x24207 $x24210 (not $x24214)))))
-(let ((@x25298 (unit-resolution (def-axiom $x25367) @x25300 (unit-resolution @x25215 @x25226 $x24226) false)))
-(let (($x25758 (>= (+ v_b_L_H_p_G_0$ (* (- 1) ?v0!14)) 0)))
-(let (($x25493 (not $x25758)))
-(let (($x26041 (= ?x3929 ?x16374)))
-(let (($x26045 (not $x26041)))
-(let (($x21439 (<= (+ v_b_L_H_max_G_1$ ?x12534) 0)))
-(let (($x21437 (= v_b_L_H_max_G_1$ v_b_L_H_max_G_3$)))
-(let ((@x23828 (mp (hypothesis $x3993) (symm (commutativity (= $x21437 $x3993)) (= $x3993 $x21437)) $x21437)))
-(let ((@x23799 (lemma (unit-resolution (hypothesis (not $x21437)) @x23828 false) (or $x20230 $x21437))))
-(let ((@x25753 (unit-resolution @x23799 (unit-resolution (def-axiom (or $x21123 $x3993)) (hypothesis $x21126) $x3993) $x21437)))
-(let (($x21321 (not $x16622)))
-(let (($x13842 (<= v_b_P_H_len$ 4294967295)))
-(let (($x12342 (>= (+ b_S_max_o_u4$ (* (- 1) v_b_P_H_len$)) 0)))
-(let (($x12813 (= (+ b_S_max_o_u4$ (* (- 1) v_b_P_H_len$)) (+ 4294967295 (* (- 1) v_b_P_H_len$)))))
-(let ((@x12767 (monotonicity (monotonicity @x7025 $x12813) (= $x12342 (>= (+ 4294967295 (* (- 1) v_b_P_H_len$)) 0)))))
-(let ((@x13004 (trans @x12767 (rewrite (= (>= (+ 4294967295 (* (- 1) v_b_P_H_len$)) 0) $x13842)) (= $x12342 $x13842))))
-(let ((@x13005 (mp (mp (and-elim @x10087 $x3720) (rewrite (= $x3720 $x12342)) $x12342) @x13004 $x13842)))
-(let ((@x25757 (unit-resolution ((_ th-lemma arith assign-bounds 1 -1) (or $x13856 (not $x13842) $x12453)) @x13005 (or $x13856 $x12453))))
-(let ((@x26039 (unit-resolution (def-axiom (or $x21090 $x16351 $x16354 $x21084)) (unit-resolution ((_ th-lemma arith farkas 1 1) (or $x20375 $x12494)) @x25328 $x12494) (unit-resolution @x25757 @x25337 $x13856) (or $x21090 $x21084))))
-(let ((@x25754 (unit-resolution @x26039 (unit-resolution (def-axiom (or $x21123 $x21087)) (hypothesis $x21126) $x21087) $x21084)))
-(let (($x21314 (>= (+ v_b_L_H_p_G_0$ (* (- 1) v_b_L_H_p_G_1$)) (- 1))))
-(let ((@x25773 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x20170 $x21314)) (unit-resolution (def-axiom (or $x21081 $x12500)) @x25754 $x12500) $x21314)))
-(let ((@x24365 (lemma ((_ th-lemma arith farkas -1 1 1) (hypothesis $x12518) (hypothesis $x12456) (hypothesis $x21314) false) (or $x12514 $x12453 (not $x21314)))))
-(let ((@x25776 (unit-resolution (unit-resolution @x24365 @x25337 (or $x12514 (not $x21314))) @x25773 $x12514)))
-(let ((@x25780 (unit-resolution (def-axiom (or $x21078 $x12518 $x21072)) @x25776 (unit-resolution (def-axiom (or $x21081 $x21075)) @x25754 $x21075) $x21072)))
-(let ((@x25788 (symm (unit-resolution (def-axiom (or $x21123 $x3993)) (hypothesis $x21126) $x3993) $x21437)))
-(let ((@x26009 (monotonicity (unit-resolution (def-axiom (or $x21123 $x3994)) (hypothesis $x21126) $x3994) (= ?x3974 (b_S_idx$ ?x3680 v_b_SL_H_witness_G_0$ b_T_T_u1$)))))
-(let ((@x25796 (trans (monotonicity @x26009 (= ?x3975 ?x3793)) (unit-resolution (def-axiom (or $x21205 $x3794)) @x25327 $x3794) (= ?x3975 v_b_L_H_max_G_1$))))
-(let (($x21444 (>= (+ v_b_SL_H_witness_G_0$ (* (- 1) v_b_SL_H_witness_G_1$)) 0)))
-(let (($x21441 (= v_b_SL_H_witness_G_0$ v_b_SL_H_witness_G_1$)))
-(let ((@x25805 (mp (unit-resolution (def-axiom (or $x21123 $x3994)) (hypothesis $x21126) $x3994) (symm (commutativity (= $x21441 $x3994)) (= $x3994 $x21441)) $x21441)))
-(let ((@x25039 (unit-resolution ((_ th-lemma arith assign-bounds -1 -1) (or $x12553 $x12435 (not $x21444))) (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x21441) $x21444)) @x25805 $x21444) (unit-resolution (def-axiom (or $x21205 $x12438)) @x25327 $x12438) $x12553)))
-(let ((@x24865 (unit-resolution (def-axiom (or $x20131 $x12550 (not $x3976))) @x25039 (trans @x25796 @x25788 $x3976) $x20131)))
-(let ((@x24882 (unit-resolution (def-axiom (or $x21066 $x20104 $x21060)) (unit-resolution (def-axiom (or $x21057 $x20130)) @x24865 $x21057) (unit-resolution (def-axiom (or $x21069 $x21063)) @x25780 $x21063) $x20104)))
-(let ((@x25939 ((_ th-lemma arith farkas 1 -1 -1 1) (hypothesis $x12471) (hypothesis $x21321) (hypothesis $x21439) (hypothesis (>= (+ ?x3929 ?x16620) 0)) false)))
-(let ((@x25943 (lemma @x25939 (or (not (>= (+ ?x3929 ?x16620) 0)) $x12476 $x16622 (not $x21439)))))
-(let ((@x23480 (unit-resolution @x25943 (unit-resolution (def-axiom (or $x21123 $x12471)) (hypothesis $x21126) $x12471) (unit-resolution (def-axiom (or $x20099 $x21321)) @x24882 $x21321) (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x21437) $x21439)) @x25753 $x21439) (not (>= (+ ?x3929 ?x16620) 0)))))
-(let ((@x25040 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x26045 (>= (+ ?x3929 ?x16620) 0))) @x23480 $x26045)))
-(let ((@x26053 (symm (hypothesis (= v_b_L_H_p_G_0$ ?v0!14)) (= ?v0!14 v_b_L_H_p_G_0$))))
-(let ((@x26057 (monotonicity (monotonicity @x26053 (= (b_S_idx$ ?x3680 ?v0!14 b_T_T_u1$) ?x3922)) (= ?x16374 ?x3929))))
-(let ((@x26062 (lemma (unit-resolution (hypothesis $x26045) (symm @x26057 $x26041) false) (or (not (= v_b_L_H_p_G_0$ ?v0!14)) $x26041))))
-(let (($x24388 (<= (+ v_b_L_H_p_G_0$ (* (- 1) ?v0!14)) 0)))
-(let (($x24400 (>= (+ v_b_L_H_max_G_1$ ?x16620) 0)))
-(let (($x25800 (not $x24400)))
-(let ((@x25043 (unit-resolution ((_ th-lemma arith assign-bounds -1 -1) (or $x25800 $x16622 (not $x21439))) (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x21437) $x21439)) @x25753 $x21439) (unit-resolution (def-axiom (or $x20099 $x21321)) @x24882 $x21321) $x25800)))
-(let (($x25270 (or $x21046 $x20083 $x20084 $x24388 $x24400)))
-(let (($x24379 (<= (+ ?x16374 (* (- 1) v_b_L_H_max_G_1$)) 0)))
-(let (($x24371 (>= (+ ?v0!14 ?x12400) 0)))
-(let (($x25240 (or $x21046 (or $x20083 $x20084 $x24371 $x24379))))
-(let (($x25224 (= (+ ?x16374 (* (- 1) v_b_L_H_max_G_1$)) (+ (* (- 1) v_b_L_H_max_G_1$) ?x16374))))
-(let ((@x25242 (monotonicity (rewrite $x25224) (= $x24379 (<= (+ (* (- 1) v_b_L_H_max_G_1$) ?x16374) 0)))))
-(let ((@x25266 (trans @x25242 (rewrite (= (<= (+ (* (- 1) v_b_L_H_max_G_1$) ?x16374) 0) $x24400)) (= $x24379 $x24400))))
-(let ((@x25195 (monotonicity (rewrite (= (+ ?v0!14 ?x12400) (+ ?x12400 ?v0!14))) (= $x24371 (>= (+ ?x12400 ?v0!14) 0)))))
-(let ((@x25223 (trans @x25195 (rewrite (= (>= (+ ?x12400 ?v0!14) 0) $x24388)) (= $x24371 $x24388))))
-(let ((@x25269 (monotonicity @x25223 @x25266 (= (or $x20083 $x20084 $x24371 $x24379) (or $x20083 $x20084 $x24388 $x24400)))))
-(let ((@x25287 (trans (monotonicity @x25269 (= $x25240 (or $x21046 (or $x20083 $x20084 $x24388 $x24400)))) (rewrite (= (or $x21046 (or $x20083 $x20084 $x24388 $x24400)) $x25270)) (= $x25240 $x25270))))
-(let ((@x25045 (unit-resolution (mp ((_ quant-inst ?v0!14) $x25240) @x25287 $x25270) @x25333 (unit-resolution (def-axiom (or $x20099 $x16366)) @x24882 $x16366) (unit-resolution (def-axiom (or $x20099 $x16367)) @x24882 $x16367) @x25043 $x24388)))
-(let ((@x25794 (unit-resolution ((_ th-lemma arith triangle-eq) (or (= v_b_L_H_p_G_0$ ?v0!14) (not $x24388) $x25493)) @x25045 (or (= v_b_L_H_p_G_0$ ?v0!14) $x25493))))
-(let ((@x25807 (unit-resolution @x25794 (unit-resolution @x26062 @x25040 (not (= v_b_L_H_p_G_0$ ?v0!14))) $x25493)))
-(let ((@x25542 ((_ th-lemma arith farkas -1 -1 1) (unit-resolution (def-axiom (or $x20099 $x16605)) @x24882 $x16605) @x25773 @x25807 false)))
-(let ((@x23800 (hypothesis $x21114)))
-(let ((@x23806 (unit-resolution (def-axiom (or $x21111 $x3923)) @x23800 $x3923)))
-(let ((@x23831 (unit-resolution (def-axiom (or $x21108 $x16330 $x16333 $x21102)) (unit-resolution (def-axiom (or $x21111 $x21105)) @x23800 $x21105) @x23806 (unit-resolution (def-axiom (or $x21111 $x3924)) @x23800 $x3924) $x21102)))
-(let ((@x23833 (unit-resolution (def-axiom (or $x21156 $x16330 $x16333 $x21150)) (unit-resolution (def-axiom (or $x21111 $x3924)) @x23800 $x3924) (hypothesis $x21153) @x23806 $x21150)))
-(let ((@x23933 (unit-resolution (def-axiom (or $x21132 $x21120 $x21126)) (unit-resolution (def-axiom (or $x21117 $x21111)) @x23800 $x21117) (hypothesis $x21123) $x21132)))
-(let ((@x23949 (unit-resolution (def-axiom (or $x21144 $x16330 $x16339 $x21138)) (unit-resolution (def-axiom (or $x21135 $x21129)) @x23933 $x21135) (unit-resolution (def-axiom (or $x21147 $x21141)) @x23833 $x21141) @x23806 (unit-resolution (def-axiom (or $x21099 $x3926)) @x23831 $x3926) false)))
-(let ((@x25705 (unit-resolution (lemma @x23949 (or $x21111 $x21126 $x21156)) (unit-resolution (def-axiom (or $x21159 $x21153)) @x25336 $x21153) (or $x21111 $x21126))))
-(let ((@x24823 (unit-resolution (def-axiom (or $x21114 $x16330 $x16333 $x21108)) @x25345 (or $x21114 $x16330 $x21108))))
-(let ((@x24804 (unit-resolution @x24823 (unit-resolution (def-axiom (or $x21105 $x21099)) (hypothesis $x21102) $x21105) (unit-resolution (def-axiom (or $x21099 $x3923)) (hypothesis $x21102) $x3923) (hypothesis $x21111) false)))
-(let ((@x25544 (unit-resolution (lemma @x24804 (or $x21099 $x21114)) (unit-resolution @x25705 (lemma @x25542 $x21123) $x21111) $x21099)))
-(let ((@x25545 (unit-resolution (def-axiom (or $x21102 $x16330 $x16339 $x21096)) @x25032 @x25544 (or $x16339 $x21096))))
-(let ((@x25499 (unit-resolution @x25545 (lemma @x25298 $x3926) $x21096)))
-(let ((@x24990 (symm (unit-resolution (def-axiom (or $x21093 $x3940)) @x25499 $x3940) (= v_b_L_H_max_G_2$ v_b_L_H_max_G_3$))))
-(let ((@x25684 (symm (unit-resolution (def-axiom (or $x21093 $x3935)) @x25499 $x3935) (= ?x3929 v_b_L_H_max_G_2$))))
-(let ((@x25702 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x3929 v_b_L_H_max_G_3$)) $x24191)) (trans @x25684 @x24990 (= ?x3929 v_b_L_H_max_G_3$)) $x24191)))
-(let ((@x25703 (unit-resolution @x26039 (unit-resolution (def-axiom (or $x21093 $x21087)) @x25499 $x21087) $x21084)))
-(let ((@x25694 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x20170 $x21314)) (unit-resolution (def-axiom (or $x21081 $x12500)) @x25703 $x12500) $x21314)))
-(let ((@x25722 (unit-resolution (unit-resolution @x24365 @x25337 (or $x12514 (not $x21314))) @x25694 $x12514)))
-(let ((@x25710 (unit-resolution (def-axiom (or $x21078 $x12518 $x21072)) @x25722 (unit-resolution (def-axiom (or $x21081 $x21075)) @x25703 $x21075) $x21072)))
-(let ((@x25723 (monotonicity (unit-resolution (def-axiom (or $x21093 $x3942)) @x25499 $x3942) (= ?x3974 ?x3922))))
-(let ((@x25707 (trans (monotonicity @x25723 (= ?x3975 ?x3929)) @x25684 (= ?x3975 v_b_L_H_max_G_2$))))
-(let (($x24188 (>= (+ v_b_L_H_p_G_0$ (* (- 1) v_b_SL_H_witness_G_1$)) 0)))
-(let ((@x25713 (symm (unit-resolution (def-axiom (or $x21093 $x3942)) @x25499 $x3942) (= v_b_L_H_p_G_0$ v_b_SL_H_witness_G_1$))))
-(let ((@x25747 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= v_b_L_H_p_G_0$ v_b_SL_H_witness_G_1$)) $x24188)) @x25713 $x24188)))
-(let ((@x25736 (unit-resolution ((_ th-lemma arith assign-bounds -1 -1) (or $x12553 $x12453 (not $x24188))) @x25337 (or $x12553 (not $x24188)))))
-(let ((@x25735 (unit-resolution (def-axiom (or $x20131 $x12550 (not $x3976))) (unit-resolution @x25736 @x25747 $x12553) (trans @x25707 @x24990 $x3976) $x20131)))
-(let ((@x25885 (unit-resolution (def-axiom (or $x21066 $x20104 $x21060)) (unit-resolution (def-axiom (or $x21057 $x20130)) @x25735 $x21057) (unit-resolution (def-axiom (or $x21069 $x21063)) @x25710 $x21063) $x20104)))
-(let (($x25930 (>= (+ ?x3929 ?x16620) 0)))
-(let (($x26036 (= v_b_L_H_p_G_0$ ?v0!14)))
-(let ((@x25738 (unit-resolution ((_ th-lemma arith assign-bounds -1 -1) (or $x25758 $x16600 (not $x21314))) (unit-resolution (def-axiom (or $x20099 $x16605)) @x25885 $x16605) @x25694 $x25758)))
-(let ((@x25737 (unit-resolution (def-axiom (or $x21156 $x16330 $x16333 $x21150)) (unit-resolution (def-axiom (or $x21159 $x21153)) @x25336 $x21153) @x25345 (or $x16330 $x21150))))
-(let ((@x25813 (unit-resolution (def-axiom (or $x21147 $x21141)) (unit-resolution @x25737 @x25032 $x21150) $x21141)))
-(let ((@x25840 (unit-resolution (def-axiom (or $x21144 $x16330 $x16339 $x21138)) @x25032 @x25813 (or $x16339 $x21138))))
-(let ((@x25839 (unit-resolution (def-axiom (or $x21135 $x21129)) (unit-resolution @x25840 (lemma @x25298 $x3926) $x21138) $x21129)))
-(let ((@x25838 (unit-resolution (def-axiom (or $x21132 $x21120 $x21126)) (lemma @x25542 $x21123) (or $x21132 $x21120))))
-(let ((@x25853 (unit-resolution (def-axiom (or $x21117 $x12476)) (unit-resolution @x25838 @x25839 $x21120) $x12476)))
-(let ((@x25814 (unit-resolution ((_ th-lemma arith assign-bounds 1 1 1) (or $x25800 $x16622 (not $x24191) $x12471)) (unit-resolution (def-axiom (or $x20099 $x21321)) @x25885 $x21321) @x25853 @x25702 $x25800)))
-(let ((@x25830 (unit-resolution (mp ((_ quant-inst ?v0!14) $x25240) @x25287 $x25270) @x25333 (unit-resolution (def-axiom (or $x20099 $x16366)) @x25885 $x16366) (unit-resolution (def-axiom (or $x20099 $x16367)) @x25885 $x16367) @x25814 $x24388)))
-(let ((@x25831 (unit-resolution @x26062 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x26036 (not $x24388) $x25493)) @x25830 @x25738 $x26036) $x26041)))
-((_ th-lemma arith farkas -1 1 1) (unit-resolution ((_ th-lemma arith triangle-eq) (or $x26045 $x25930)) @x25831 $x25930) (unit-resolution (def-axiom (or $x20099 $x21321)) @x25885 $x21321) @x25702 false))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))
-
+fd9e057047e121293775315a7cd162f9a4c8122a 2972 0
+unsat
+((set-logic <null>)
+(declare-fun ?v0!14 () Int)
+(declare-fun ?v0!15 () Int)
+(declare-fun ?v0!13 () Int)
+(proof
+(let ((?x10078 (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$)))
+(let ((?x10372 (b_S_idx$ ?x10078 v_b_SL_H_witness_G_1$ b_T_T_u1$)))
+(let ((?x10373 (b_S_read_n_u1$ v_b_S_s$ ?x10372)))
+(let (($x10374 (= ?x10373 v_b_L_H_max_G_3$)))
+(let (($x11647 (<= (+ v_b_P_H_len$ (* (- 1) v_b_SL_H_witness_G_1$)) 0)))
+(let (($x19412 (or $x11647 (not $x10374))))
+(let (($x19413 (not $x19412)))
+(let (($x19906 (forall ((?v0 Int) )(!(let ((?x11631 (* (- 1) v_b_L_H_max_G_3$)))
+(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x11633 (<= (+ ?x10163 ?x11631) 0)))
+(let (($x11615 (>= (+ ?v0 (* (- 1) v_b_L_H_p_G_1$)) 0)))
+(let (($x12168 (<= ?v0 4294967295)))
+(let (($x16553 (not $x12168)))
+(let (($x2815 (>= ?v0 0)))
+(let (($x3763 (not $x2815)))
+(or $x3763 $x16553 $x11615 $x11633))))))))) :pattern ( (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$) )))
+))
+(let (($x19911 (not $x19906)))
+(let (($x19914 (or $x19911 $x19413)))
+(let (($x19917 (not $x19914)))
+(let ((?x15633 (b_S_idx$ ?x10078 ?v0!14 b_T_T_u1$)))
+(let ((?x15634 (b_S_read_n_u1$ v_b_S_s$ ?x15633)))
+(let ((?x15891 (* (- 1) ?x15634)))
+(let (($x15893 (>= (+ v_b_L_H_max_G_3$ ?x15891) 0)))
+(let (($x15871 (<= (+ v_b_L_H_p_G_1$ (* (- 1) ?v0!14)) 0)))
+(let (($x15627 (<= ?v0!14 4294967295)))
+(let (($x19366 (not $x15627)))
+(let (($x15626 (>= ?v0!14 0)))
+(let (($x19365 (not $x15626)))
+(let (($x19381 (or $x19365 $x19366 $x15871 $x15893)))
+(let (($x19386 (not $x19381)))
+(let (($x19920 (or $x19386 $x19917)))
+(let (($x19923 (not $x19920)))
+(let ((?x11581 (* (- 1) v_b_L_H_p_G_1$)))
+(let ((?x11609 (+ v_b_P_H_len$ ?x11581)))
+(let (($x11608 (>= ?x11609 0)))
+(let (($x11612 (not $x11608)))
+(let (($x19926 (or $x11612 $x19923)))
+(let (($x19929 (not $x19926)))
+(let (($x19932 (or $x11612 $x19929)))
+(let (($x19935 (not $x19932)))
+(let (($x11536 (>= v_b_SL_H_witness_G_1$ 0)))
+(let (($x19455 (not $x11536)))
+(let (($x11578 (>= v_b_L_H_p_G_1$ 2)))
+(let (($x19454 (not $x11578)))
+(let (($x10358 (b_S_local_n_value_n_is$ v_b_S_s$ b_H_tok_S_1_T_16_o_24$ b_H_loc_o_p$ v_b_L_H_p_G_1$ b_T_T_u4$)))
+(let (($x19453 (not $x10358)))
+(let ((?x11582 (+ v_b_L_H_p_G_0$ ?x11581)))
+(let (($x11580 (= ?x11582 (- 1))))
+(let (($x19452 (not $x11580)))
+(let (($x13353 (<= v_b_L_H_p_G_0$ 4294967294)))
+(let (($x15614 (not $x13353)))
+(let (($x11570 (>= v_b_L_H_p_G_0$ (- 1))))
+(let (($x15611 (not $x11570)))
+(let (($x19938 (or $x15611 $x15614 $x19452 $x19453 $x19454 $x19455 $x19935)))
+(let (($x19941 (not $x19938)))
+(let (($x19944 (or $x15611 $x15614 $x19941)))
+(let (($x19947 (not $x19944)))
+(let (($x11429 (>= v_b_L_H_p_G_0$ 1)))
+(let (($x19474 (not $x11429)))
+(let (($x10392 (= v_b_SL_H_witness_G_1$ v_b_SL_H_witness_G_0$)))
+(let (($x19513 (not $x10392)))
+(let (($x10391 (= v_b_L_H_max_G_3$ v_b_L_H_max_G_1$)))
+(let (($x19512 (not $x10391)))
+(let (($x11432 (>= v_b_SL_H_witness_G_0$ 0)))
+(let (($x19501 (not $x11432)))
+(let ((?x10320 (b_S_idx$ ?x10078 v_b_L_H_p_G_0$ b_T_T_u1$)))
+(let ((?x10327 (b_S_read_n_u1$ v_b_S_s$ ?x10320)))
+(let ((?x11517 (* (- 1) ?x10327)))
+(let ((?x11518 (+ v_b_L_H_max_G_1$ ?x11517)))
+(let (($x11516 (>= ?x11518 0)))
+(let (($x11515 (not $x11516)))
+(let (($x19980 (or $x11515 $x19501 $x19512 $x19513 $x19474 $x19455 $x19947)))
+(let (($x19983 (not $x19980)))
+(let ((?x25039 (+ ?x10327 ?x15891)))
+(let (($x25041 (>= ?x25039 0)))
+(let (($x25038 (= ?x10327 ?x15634)))
+(let (($x25035 (= v_b_L_H_p_G_0$ ?v0!14)))
+(let (($x10340 (= v_b_SL_H_witness_G_1$ v_b_L_H_p_G_0$)))
+(let (($x19473 (not $x10340)))
+(let (($x10338 (= v_b_L_H_max_G_3$ v_b_L_H_max_G_2$)))
+(let (($x19472 (not $x10338)))
+(let (($x10335 (b_S_local_n_value_n_is$ v_b_S_s$ b_H_tok_S_1_T_24_o_47$ b_H_loc_o_witness$ v_b_L_H_p_G_0$ b_T_T_u4$)))
+(let (($x19471 (not $x10335)))
+(let (($x10334 (b_S_local_n_value_n_is$ v_b_S_s$ b_H_tok_S_1_T_23_o_7$ b_H_loc_o_max$ v_b_L_H_max_G_2$ b_T_T_u1$)))
+(let (($x19470 (not $x10334)))
+(let (($x10333 (= v_b_L_H_max_G_2$ ?x10327)))
+(let (($x19469 (not $x10333)))
+(let (($x10324 (b_S_thread_n_local$ v_b_S_s$ ?x10320)))
+(let (($x15599 (not $x10324)))
+(let (($x10321 (b_S_is$ ?x10320 b_T_T_u1$)))
+(let (($x15590 (not $x10321)))
+(let (($x19950 (or $x15590 $x15599 $x19469 $x19470 $x19471 $x19472 $x19473 $x19474 $x19455 $x19947)))
+(let (($x19953 (not $x19950)))
+(let (($x19956 (or $x15590 $x15599 $x19953)))
+(let (($x19959 (not $x19956)))
+(let (($x10322 (b_S_typed$ v_b_S_s$ ?x10320)))
+(let (($x15593 (not $x10322)))
+(let (($x19962 (or $x15590 $x15593 $x19959)))
+(let (($x19965 (not $x19962)))
+(let (($x19968 (or $x15590 $x15593 $x19965)))
+(let (($x19971 (not $x19968)))
+(let (($x19974 (or $x11516 $x19474 $x19501 $x19971)))
+(let (($x19977 (not $x19974)))
+(let (($x19986 (or $x19977 $x19983)))
+(let (($x19989 (not $x19986)))
+(let (($x19992 (or $x15590 $x15599 $x19474 $x19501 $x19989)))
+(let (($x19995 (not $x19992)))
+(let ((?x23404 (b_S_ref$ ?x10320)))
+(let ((?x23225 (b_S_ptr$ b_T_T_u1$ ?x23404)))
+(let ((?x24099 (b_S_typ$ ?x23225)))
+(let ((?x24100 (b_S_kind_n_of$ ?x24099)))
+(let (($x23805 (= ?x24100 b_S_kind_n_primitive$)))
+(let ((?x21472 (b_S_kind_n_of$ b_T_T_u1$)))
+(let (($x21473 (= ?x21472 b_S_kind_n_primitive$)))
+(let (($x9768 (b_S_is_n_primitive$ b_T_T_u1$)))
+(let (($x21480 (= $x9768 $x21473)))
+(let (($x9891 (forall ((?v0 B_S_ctype$) )(!(let ((?x9849 (b_S_kind_n_of$ ?v0)))
+(let (($x9883 (= ?x9849 b_S_kind_n_primitive$)))
+(let (($x2704 (b_S_is_n_primitive$ ?v0)))
+(= $x2704 $x9883)))) :pattern ( (b_S_is_n_primitive$ ?v0) )))
+))
+(let ((?x9849 (b_S_kind_n_of$ ?0)))
+(let (($x9883 (= ?x9849 b_S_kind_n_primitive$)))
+(let (($x2704 (b_S_is_n_primitive$ ?0)))
+(let (($x9888 (= $x2704 $x9883)))
+(let (($x9886 (forall ((?v0 B_S_ctype$) )(!(let ((?x9849 (b_S_kind_n_of$ ?v0)))
+(let (($x9883 (= ?x9849 b_S_kind_n_primitive$)))
+(let (($x2704 (b_S_is_n_primitive$ ?v0)))
+(= $x2704 $x9883)))) :pattern ( (b_S_is_n_primitive$ ?v0) )))
+))
+(let ((@x9896 (mp (asserted $x9886) (quant-intro (rewrite (= (= $x2704 $x9883) $x9888)) (= $x9886 $x9891)) $x9891)))
+(let ((@x15456 (mp~ @x9896 (nnf-pos (refl (~ $x9888 $x9888)) (~ $x9891 $x9891)) $x9891)))
+(let (($x21224 (not $x9891)))
+(let (($x21483 (or $x21224 $x21480)))
+(let ((@x21484 ((_ quant-inst b_T_T_u1$) $x21483)))
+(let ((@x9769 (asserted $x9768)))
+(let ((@x23544 (unit-resolution (def-axiom (or (not $x21480) (not $x9768) $x21473)) @x9769 (or (not $x21480) $x21473))))
+(let ((?x23241 (b_S_typ$ ?x10320)))
+(let (($x23242 (= ?x23241 b_T_T_u1$)))
+(let (($x23270 (= $x10321 $x23242)))
+(let (($x19828 (forall ((?v0 B_S_ptr$) (?v1 B_S_ctype$) )(!(let ((?x6636 (b_S_typ$ ?v0)))
+(let (($x7865 (= ?x6636 ?v1)))
+(let (($x9596 (b_S_is$ ?v0 ?v1)))
+(= $x9596 $x7865)))) :pattern ( (b_S_is$ ?v0 ?v1) )))
+))
+(let (($x9617 (forall ((?v0 B_S_ptr$) (?v1 B_S_ctype$) )(let ((?x6636 (b_S_typ$ ?v0)))
+(let (($x7865 (= ?x6636 ?v1)))
+(let (($x9596 (b_S_is$ ?v0 ?v1)))
+(= $x9596 $x7865)))))
+))
+(let ((?x6636 (b_S_typ$ ?1)))
+(let (($x7865 (= ?x6636 ?0)))
+(let (($x9596 (b_S_is$ ?1 ?0)))
+(let (($x9614 (= $x9596 $x7865)))
+(let (($x9611 (forall ((?v0 B_S_ptr$) (?v1 B_S_ctype$) )(let ((?x6636 (b_S_typ$ ?v0)))
+(let (($x7865 (= ?x6636 ?v1)))
+(let (($x9596 (b_S_is$ ?v0 ?v1)))
+(= $x9596 $x7865)))))
+))
+(let ((@x9622 (mp (asserted $x9611) (quant-intro (rewrite (= (= $x9596 $x7865) $x9614)) (= $x9611 $x9617)) $x9617)))
+(let ((@x19833 (mp (mp~ @x9622 (nnf-pos (refl (~ $x9614 $x9614)) (~ $x9617 $x9617)) $x9617) (quant-intro (refl (= $x9614 $x9614)) (= $x9617 $x19828)) $x19828)))
+(let (($x22002 (not $x19828)))
+(let (($x23990 (or $x22002 $x23270)))
+(let ((@x23870 ((_ quant-inst (b_S_idx$ ?x10078 v_b_L_H_p_G_0$ b_T_T_u1$) b_T_T_u1$) $x23990)))
+(let ((?x10045 (b_S_sizeof$ b_T_T_u1$)))
+(let ((?x23278 (* ?x10045 v_b_L_H_p_G_0$)))
+(let ((?x10079 (b_S_ref$ ?x10078)))
+(let ((?x24174 (+ ?x10079 ?x23278)))
+(let ((?x24198 (b_S_ptr$ b_T_T_u1$ ?x24174)))
+(let ((?x23028 (b_S_typ$ ?x24198)))
+(let (($x23029 (= ?x23028 b_T_T_u1$)))
+(let (($x19841 (forall ((?v0 B_S_ctype$) (?v1 Int) )(!(= (b_S_typ$ (b_S_ptr$ ?v0 ?v1)) ?v0) :pattern ( (b_S_ptr$ ?v0 ?v1) )))
+))
+(let (($x9659 (forall ((?v0 B_S_ctype$) (?v1 Int) )(= (b_S_typ$ (b_S_ptr$ ?v0 ?v1)) ?v0))
+))
+(let (($x9658 (= (b_S_typ$ (b_S_ptr$ ?1 ?0)) ?1)))
+(let ((@x15361 (mp~ (asserted $x9659) (nnf-pos (refl (~ $x9658 $x9658)) (~ $x9659 $x9659)) $x9659)))
+(let ((@x19846 (mp @x15361 (quant-intro (refl (= $x9658 $x9658)) (= $x9659 $x19841)) $x19841)))
+(let (($x24201 (= ?x10320 ?x24198)))
+(let (($x24214 (not $x24201)))
+(let (($x24067 (b_S_extent_n_hint$ ?x10320 ?x10078)))
+(let (($x24065 (not $x24067)))
+(let (($x24160 (or $x24065 $x24214)))
+(let (($x24161 (not $x24160)))
+(let (($x18180 (forall ((?v0 B_S_ptr$) (?v1 Int) (?v2 B_S_ctype$) )(!(let ((?x7205 (b_S_idx$ ?v0 ?v1 ?v2)))
+(let (($x7213 (= ?x7205 (b_S_ptr$ ?v2 (+ (b_S_ref$ ?v0) (* ?v1 (b_S_sizeof$ ?v2)))))))
+(not (or (not (b_S_extent_n_hint$ ?x7205 ?v0)) (not $x7213))))) :pattern ( (b_S_idx$ ?v0 ?v1 ?v2) )))
+))
+(let (($x7216 (forall ((?v0 B_S_ptr$) (?v1 Int) (?v2 B_S_ctype$) )(!(let ((?x7205 (b_S_idx$ ?v0 ?v1 ?v2)))
+(let (($x7213 (= ?x7205 (b_S_ptr$ ?v2 (+ (b_S_ref$ ?v0) (* ?v1 (b_S_sizeof$ ?v2)))))))
+(and (b_S_extent_n_hint$ ?x7205 ?v0) $x7213))) :pattern ( (b_S_idx$ ?v0 ?v1 ?v2) )))
+))
+(let ((?x7205 (b_S_idx$ ?2 ?1 ?0)))
+(let (($x7213 (= ?x7205 (b_S_ptr$ ?0 (+ (b_S_ref$ ?2) (* ?1 (b_S_sizeof$ ?0)))))))
+(let (($x7214 (and (b_S_extent_n_hint$ ?x7205 ?2) $x7213)))
+(let ((@x18179 (rewrite (= $x7214 (not (or (not (b_S_extent_n_hint$ ?x7205 ?2)) (not $x7213)))))))
+(let ((@x14561 (mp~ (asserted $x7216) (nnf-pos (refl (~ $x7214 $x7214)) (~ $x7216 $x7216)) $x7216)))
+(let ((@x18183 (mp @x14561 (quant-intro @x18179 (= $x7216 $x18180)) $x18180)))
+(let (($x22568 (not $x18180)))
+(let (($x24300 (or $x22568 $x24161)))
+(let (($x24080 (not (= ?x10320 (b_S_ptr$ b_T_T_u1$ (+ ?x10079 (* v_b_L_H_p_G_0$ ?x10045)))))))
+(let (($x24081 (not (or $x24065 $x24080))))
+(let (($x24202 (= (= ?x10320 (b_S_ptr$ b_T_T_u1$ (+ ?x10079 (* v_b_L_H_p_G_0$ ?x10045)))) $x24201)))
+(let ((@x24197 (monotonicity (rewrite (= (* v_b_L_H_p_G_0$ ?x10045) ?x23278)) (= (+ ?x10079 (* v_b_L_H_p_G_0$ ?x10045)) ?x24174))))
+(let ((@x24200 (monotonicity @x24197 (= (b_S_ptr$ b_T_T_u1$ (+ ?x10079 (* v_b_L_H_p_G_0$ ?x10045))) ?x24198))))
+(let ((@x24150 (monotonicity (monotonicity (monotonicity @x24200 $x24202) (= $x24080 $x24214)) (= (or $x24065 $x24080) $x24160))))
+(let ((@x24316 (monotonicity (monotonicity @x24150 (= $x24081 $x24161)) (= (or $x22568 $x24081) $x24300))))
+(let ((@x24299 (mp ((_ quant-inst (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) v_b_L_H_p_G_0$ b_T_T_u1$) (or $x22568 $x24081)) (trans @x24316 (rewrite (= $x24300 $x24300)) (= (or $x22568 $x24081) $x24300)) $x24300)))
+(let ((@x24341 (unit-resolution (def-axiom (or $x24160 $x24201)) (unit-resolution @x24299 @x18183 $x24161) $x24201)))
+(let ((@x24343 (trans (monotonicity @x24341 (= ?x23241 ?x23028)) (unit-resolution ((_ quant-inst b_T_T_u1$ (+ ?x10079 ?x23278)) (or (not $x19841) $x23029)) @x19846 $x23029) $x23242)))
+(let (($x23889 (not $x23242)))
+(let ((@x24337 (unit-resolution (def-axiom (or (not $x23270) $x10321 $x23889)) (hypothesis $x15590) (or (not $x23270) $x23889))))
+(let ((@x24344 (unit-resolution (unit-resolution @x24337 (unit-resolution @x23870 @x19833 $x23270) $x23889) @x24343 false)))
+(let ((@x24345 (lemma @x24344 $x10321)))
+(let ((@x25031 (unit-resolution (def-axiom (or (not $x23270) $x15590 $x23242)) @x24345 (or (not $x23270) $x23242))))
+(let (($x23227 (= ?x10320 ?x23225)))
+(let (($x9607 (forall ((?v0 B_S_ptr$) (?v1 B_S_ctype$) )(!(or (not (b_S_is$ ?v0 ?v1)) (= ?v0 (b_S_ptr$ ?v1 (b_S_ref$ ?v0)))) :pattern ( (b_S_is$ ?v0 ?v1) )))
+))
+(let (($x9604 (or (not $x9596) (= ?1 (b_S_ptr$ ?0 (b_S_ref$ ?1))))))
+(let (($x9601 (forall ((?v0 B_S_ptr$) (?v1 B_S_ctype$) )(!(let (($x9596 (b_S_is$ ?v0 ?v1)))
+(=> $x9596 (= ?v0 (b_S_ptr$ ?v1 (b_S_ref$ ?v0))))) :pattern ( (b_S_is$ ?v0 ?v1) )))
+))
+(let ((@x9606 (rewrite (= (=> $x9596 (= ?1 (b_S_ptr$ ?0 (b_S_ref$ ?1)))) $x9604))))
+(let ((@x15336 (mp~ (mp (asserted $x9601) (quant-intro @x9606 (= $x9601 $x9607)) $x9607) (nnf-pos (refl (~ $x9604 $x9604)) (~ $x9607 $x9607)) $x9607)))
+(let (($x21994 (not $x9607)))
+(let (($x24289 (or $x21994 $x15590 $x23227)))
+(let ((@x24294 (mp ((_ quant-inst (b_S_idx$ ?x10078 v_b_L_H_p_G_0$ b_T_T_u1$) b_T_T_u1$) (or $x21994 (or $x15590 $x23227))) (rewrite (= (or $x21994 (or $x15590 $x23227)) $x24289)) $x24289)))
+(let ((@x25262 (symm (unit-resolution @x24294 @x15336 @x24345 $x23227) (= ?x23225 ?x10320))))
+(let ((@x24694 (trans (monotonicity @x25262 (= ?x24099 ?x23241)) (unit-resolution @x25031 (unit-resolution @x23870 @x19833 $x23270) $x23242) (= ?x24099 b_T_T_u1$))))
+(let ((@x24696 (trans (monotonicity @x24694 (= ?x24100 ?x21472)) (unit-resolution @x23544 (unit-resolution @x21484 @x15456 $x21480) $x21473) $x23805)))
+(let ((?x10272 (b_S_typemap$ v_b_S_s$)))
+(let ((?x24217 (b_S_select_o_tm$ ?x10272 ?x23225)))
+(let ((?x24218 (b_S_ts_n_emb$ ?x24217)))
+(let (($x23797 (b_S_closed$ v_b_S_s$ ?x24218)))
+(let (($x23803 (not $x23797)))
+(let (($x23775 (b_S_ts_n_is_n_volatile$ ?x24217)))
+(let (($x23784 (not $x23775)))
+(let (($x23804 (or $x23784 $x23803)))
+(let ((@x24686 (monotonicity (monotonicity @x25262 (= ?x24217 (b_S_select_o_tm$ ?x10272 ?x10320))) (= $x23775 (b_S_ts_n_is_n_volatile$ (b_S_select_o_tm$ ?x10272 ?x10320))))))
+(let ((@x24702 (symm @x24686 (= (b_S_ts_n_is_n_volatile$ (b_S_select_o_tm$ ?x10272 ?x10320)) $x23775))))
+(let ((@x24701 (monotonicity @x24702 (= (not (b_S_ts_n_is_n_volatile$ (b_S_select_o_tm$ ?x10272 ?x10320))) $x23784))))
+(let ((?x23101 (b_S_select_o_tm$ ?x10272 ?x10320)))
+(let (($x23361 (b_S_ts_n_is_n_volatile$ ?x23101)))
+(let (($x23297 (not $x23361)))
+(let (($x23362 (or $x15593 $x23361)))
+(let (($x23363 (not $x23362)))
+(let (($x11901 (>= v_b_L_H_p_G_0$ 0)))
+(let (($x20030 (forall ((?v0 Int) )(!(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x10238 (= ?x10163 v_b_S_result_G_0$)))
+(let (($x11800 (>= (+ ?v0 (* (- 1) v_b_P_H_len$)) 0)))
+(let (($x12168 (<= ?v0 4294967295)))
+(let (($x16553 (not $x12168)))
+(let (($x2815 (>= ?v0 0)))
+(let (($x3763 (not $x2815)))
+(or $x3763 $x16553 $x11800 (not $x10238))))))))) :pattern ( (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$) )))
+))
+(let (($x20035 (not $x20030)))
+(let (($x20022 (forall ((?v0 Int) )(!(let ((?x11816 (* (- 1) v_b_S_result_G_0$)))
+(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x11818 (<= (+ ?x10163 ?x11816) 0)))
+(let (($x11800 (>= (+ ?v0 (* (- 1) v_b_P_H_len$)) 0)))
+(let (($x12168 (<= ?v0 4294967295)))
+(let (($x16553 (not $x12168)))
+(let (($x2815 (>= ?v0 0)))
+(let (($x3763 (not $x2815)))
+(or $x3763 $x16553 $x11800 $x11818))))))))) :pattern ( (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$) )))
+))
+(let (($x20027 (not $x20022)))
+(let (($x20038 (or $x20027 $x20035)))
+(let (($x20041 (not $x20038)))
+(let ((?x15743 (b_S_idx$ ?x10078 ?v0!15 b_T_T_u1$)))
+(let ((?x15744 (b_S_read_n_u1$ v_b_S_s$ ?x15743)))
+(let ((?x16029 (* (- 1) ?x15744)))
+(let (($x16031 (>= (+ v_b_S_result_G_0$ ?x16029) 0)))
+(let (($x16009 (<= (+ v_b_P_H_len$ (* (- 1) ?v0!15)) 0)))
+(let (($x15737 (<= ?v0!15 4294967295)))
+(let (($x19560 (not $x15737)))
+(let (($x15736 (>= ?v0!15 0)))
+(let (($x19559 (not $x15736)))
+(let (($x19575 (or $x19559 $x19560 $x16009 $x16031)))
+(let (($x19580 (not $x19575)))
+(let (($x20044 (or $x19580 $x20041)))
+(let (($x20047 (not $x20044)))
+(let (($x10222 (= v_b_S_result_G_0$ v_b_L_H_max_G_1$)))
+(let (($x19640 (not $x10222)))
+(let (($x10220 (= v_b_SL_H_witness_G_2$ v_b_SL_H_witness_G_0$)))
+(let (($x19639 (not $x10220)))
+(let (($x10218 (= v_b_L_H_p_G_2$ v_b_L_H_p_G_0$)))
+(let (($x19638 (not $x10218)))
+(let (($x10216 (= v_b_L_H_max_G_4$ v_b_L_H_max_G_1$)))
+(let (($x19637 (not $x10216)))
+(let (($x15729 (not b_S_position_n_marker$)))
+(let (($x20050 (or $x15729 $x19474 $x19501 $x19637 $x19638 $x19639 $x19640 $x20047)))
+(let (($x20053 (not $x20050)))
+(let (($x20056 (or $x15729 $x20053)))
+(let (($x20059 (not $x20056)))
+(let ((?x11484 (* (- 1) v_b_L_H_p_G_0$)))
+(let ((?x11485 (+ v_b_P_H_len$ ?x11484)))
+(let (($x11486 (<= ?x11485 0)))
+(let (($x11487 (not $x11486)))
+(let (($x20062 (or $x11487 $x19474 $x19501 $x20059)))
+(let (($x20065 (not $x20062)))
+(let (($x19998 (or $x15590 $x15599 $x19995)))
+(let (($x20001 (not $x19998)))
+(let (($x20004 (or $x15590 $x15593 $x20001)))
+(let (($x20007 (not $x20004)))
+(let (($x20010 (or $x15590 $x15593 $x20007)))
+(let (($x20013 (not $x20010)))
+(let (($x20016 (or $x11486 $x19474 $x19501 $x20013)))
+(let (($x20019 (not $x20016)))
+(let (($x20068 (or $x20019 $x20065)))
+(let (($x20071 (not $x20068)))
+(let ((?x2238 (b_S_ptr_n_to$ b_T_T_u1$)))
+(let (($x10296 (b_S_local_n_value_n_is_n_ptr$ v_b_S_s$ b_H_tok_S_1_T_16_o_3$ b_H_loc_o_arr$ ?x10078 ?x2238)))
+(let (($x19683 (not $x10296)))
+(let ((?x10105 (b_S_ptr_n_to_n_int$ ?x10078)))
+(let (($x10295 (b_S_local_n_value_n_is$ v_b_S_s$ b_H_tok_S_1_T_16_o_3$ b_H_loc_o_arr$ ?x10105 ?x2238)))
+(let (($x19682 (not $x10295)))
+(let (($x10294 (b_S_local_n_value_n_is$ v_b_S_s$ b_H_tok_S_1_T_16_o_3$ b_H_loc_o_len$ v_b_P_H_len$ b_T_T_u4$)))
+(let (($x19681 (not $x10294)))
+(let (($x10293 (b_S_local_n_value_n_is$ v_b_S_s$ b_H_tok_S_1_T_16_o_3$ b_H_loc_o_max$ v_b_L_H_max_G_1$ b_T_T_u1$)))
+(let (($x19680 (not $x10293)))
+(let (($x10292 (b_S_local_n_value_n_is$ v_b_S_s$ b_H_tok_S_1_T_16_o_3$ b_H_loc_o_witness$ v_b_SL_H_witness_G_0$ b_T_T_u4$)))
+(let (($x19679 (not $x10292)))
+(let (($x10291 (b_S_local_n_value_n_is$ v_b_S_s$ b_H_tok_S_1_T_16_o_3$ b_H_loc_o_p$ v_b_L_H_p_G_0$ b_T_T_u4$)))
+(let (($x19678 (not $x10291)))
+(let (($x10097 (b_S_full_n_stop$ v_b_S_s$)))
+(let (($x19677 (not $x10097)))
+(let (($x10204 (b_S_good_n_state_n_ext$ b_H_tok_S_1_T_16_o_3$ v_b_S_s$)))
+(let (($x19676 (not $x10204)))
+(let (($x10284 (b_S_call_n_transition$ v_b_S_s$ v_b_S_s$)))
+(let (($x19675 (not $x10284)))
+(let ((?x10190 (b_S_idx$ ?x10078 v_b_SL_H_witness_G_0$ b_T_T_u1$)))
+(let ((?x10191 (b_S_read_n_u1$ v_b_S_s$ ?x10190)))
+(let (($x10192 (= ?x10191 v_b_L_H_max_G_1$)))
+(let (($x19674 (not $x10192)))
+(let ((?x11865 (* (- 1) v_b_SL_H_witness_G_0$)))
+(let ((?x11866 (+ v_b_P_H_len$ ?x11865)))
+(let (($x11867 (<= ?x11866 0)))
+(let (($x19898 (forall ((?v0 Int) )(!(let ((?x11887 (* (- 1) v_b_L_H_max_G_1$)))
+(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x11889 (<= (+ ?x10163 ?x11887) 0)))
+(let (($x11871 (>= (+ ?v0 (* (- 1) v_b_L_H_p_G_0$)) 0)))
+(let (($x12168 (<= ?v0 4294967295)))
+(let (($x16553 (not $x12168)))
+(let (($x2815 (>= ?v0 0)))
+(let (($x3763 (not $x2815)))
+(or $x3763 $x16553 $x11871 $x11889))))))))) :pattern ( (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$) )))
+))
+(let (($x19903 (not $x19898)))
+(let (($x11898 (>= ?x11485 0)))
+(let (($x19672 (not $x11898)))
+(let (($x13326 (<= v_b_L_H_p_G_0$ 4294967295)))
+(let (($x19671 (not $x13326)))
+(let (($x19670 (not $x11901)))
+(let (($x13315 (<= v_b_SL_H_witness_G_0$ 4294967295)))
+(let (($x19669 (not $x13315)))
+(let (($x13304 (<= v_b_L_H_max_G_1$ 255)))
+(let (($x19668 (not $x13304)))
+(let (($x11911 (>= v_b_L_H_max_G_1$ 0)))
+(let (($x19667 (not $x11911)))
+(let ((?x10137 (b_S_idx$ ?x10078 0 b_T_T_u1$)))
+(let ((?x10144 (b_S_read_n_u1$ v_b_S_s$ ?x10137)))
+(let (($x10167 (= ?x10144 v_b_L_H_max_G_0$)))
+(let (($x15548 (not $x10167)))
+(let (($x11259 (<= v_b_P_H_len$ 0)))
+(let (($x20074 (or $x11259 $x15548 $x19667 $x19668 $x19669 $x19670 $x19671 $x19672 $x19903 $x11867 $x19674 $x19675 $x19676 $x19677 $x19678 $x19679 $x19680 $x19681 $x19682 $x19683 $x19474 $x19501 $x20071)))
+(let (($x20077 (not $x20074)))
+(let (($x20080 (or $x11259 $x15548 $x20077)))
+(let (($x20083 (not $x20080)))
+(let (($x19890 (forall ((?v0 Int) )(!(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x11404 (>= (+ v_b_L_H_max_G_0$ (* (- 1) ?x10163)) 0)))
+(let (($x11388 (>= ?v0 1)))
+(let (($x12168 (<= ?v0 4294967295)))
+(let (($x16553 (not $x12168)))
+(let (($x2815 (>= ?v0 0)))
+(let (($x3763 (not $x2815)))
+(or $x3763 $x16553 $x11388 $x11404)))))))) :pattern ( (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$) )))
+))
+(let (($x19895 (not $x19890)))
+(let (($x20086 (or $x19895 $x20083)))
+(let (($x20089 (not $x20086)))
+(let ((?x15529 (b_S_idx$ ?x10078 ?v0!13 b_T_T_u1$)))
+(let ((?x15530 (b_S_read_n_u1$ v_b_S_s$ ?x15529)))
+(let (($x15533 (>= (+ v_b_L_H_max_G_0$ (* (- 1) ?x15530)) 0)))
+(let (($x15525 (>= ?v0!13 1)))
+(let (($x15524 (<= ?v0!13 4294967295)))
+(let (($x19298 (not $x15524)))
+(let (($x15523 (>= ?v0!13 0)))
+(let (($x19297 (not $x15523)))
+(let (($x19313 (or $x19297 $x19298 $x15525 $x15533)))
+(let (($x20589 (not $x15533)))
+(let (($x19318 (not $x19313)))
+(let ((@x24016 (hypothesis $x19318)))
+(let (($x10141 (b_S_thread_n_local$ v_b_S_s$ ?x10137)))
+(let ((?x21175 (b_S_typ$ ?x10078)))
+(let ((?x22803 (b_S_kind_n_of$ ?x21175)))
+(let (($x22807 (= ?x22803 b_S_kind_n_primitive$)))
+(let (($x21176 (= ?x21175 b_T_T_u1$)))
+(let (($x21147 (not $x19841)))
+(let (($x21181 (or $x21147 $x21176)))
+(let ((@x21182 ((_ quant-inst b_T_T_u1$ v_b_P_H_arr$) $x21181)))
+(let ((@x23076 (trans (monotonicity (unit-resolution @x21182 @x19846 $x21176) (= ?x22803 ?x21472)) (unit-resolution @x23544 (unit-resolution @x21484 @x15456 $x21480) $x21473) $x22807)))
+(let ((?x22818 (b_S_select_o_tm$ ?x10272 ?x10078)))
+(let ((?x22903 (b_S_ts_n_emb$ ?x22818)))
+(let (($x22904 (b_S_closed$ v_b_S_s$ ?x22903)))
+(let (($x22902 (b_S_ts_n_is_n_volatile$ ?x22818)))
+(let (($x22897 (not $x22902)))
+(let (($x22906 (or $x22897 (not $x22904))))
+(let ((?x22478 (b_S_select_o_tm$ ?x10272 ?x10137)))
+(let ((?x22485 (b_S_ref$ ?x10137)))
+(let ((?x22505 (b_S_ptr$ b_T_T_u1$ ?x22485)))
+(let ((?x22655 (b_S_select_o_tm$ ?x10272 ?x22505)))
+(let (($x22506 (= ?x10137 ?x22505)))
+(let ((?x22553 (b_S_ptr$ b_T_T_u1$ ?x10079)))
+(let (($x22556 (= ?x10137 ?x22553)))
+(let (($x22559 (not $x22556)))
+(let (($x22523 (b_S_extent_n_hint$ ?x10137 ?x10078)))
+(let (($x22524 (not $x22523)))
+(let (($x22562 (or $x22524 $x22559)))
+(let (($x22565 (not $x22562)))
+(let (($x22569 (or $x22568 $x22565)))
+(let (($x22542 (or $x22524 (not (= ?x10137 (b_S_ptr$ b_T_T_u1$ (+ ?x10079 (* 0 ?x10045))))))))
+(let (($x22543 (not $x22542)))
+(let (($x22560 (= (not (= ?x10137 (b_S_ptr$ b_T_T_u1$ (+ ?x10079 (* 0 ?x10045))))) $x22559)))
+(let ((@x22548 (monotonicity (rewrite (= (* 0 ?x10045) 0)) (= (+ ?x10079 (* 0 ?x10045)) (+ ?x10079 0)))))
+(let ((@x22552 (trans @x22548 (rewrite (= (+ ?x10079 0) ?x10079)) (= (+ ?x10079 (* 0 ?x10045)) ?x10079))))
+(let ((@x22555 (monotonicity @x22552 (= (b_S_ptr$ b_T_T_u1$ (+ ?x10079 (* 0 ?x10045))) ?x22553))))
+(let ((@x22558 (monotonicity @x22555 (= (= ?x10137 (b_S_ptr$ b_T_T_u1$ (+ ?x10079 (* 0 ?x10045)))) $x22556))))
+(let ((@x22567 (monotonicity (monotonicity (monotonicity @x22558 $x22560) (= $x22542 $x22562)) (= $x22543 $x22565))))
+(let ((@x22576 (trans (monotonicity @x22567 (= (or $x22568 $x22543) $x22569)) (rewrite (= $x22569 $x22569)) (= (or $x22568 $x22543) $x22569))))
+(let ((@x22577 (mp ((_ quant-inst (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) 0 b_T_T_u1$) (or $x22568 $x22543)) @x22576 $x22569)))
+(let ((@x22581 (def-axiom (or $x22562 $x22556))))
+(let ((@x24124 (unit-resolution @x22581 (lemma (unit-resolution @x22577 @x18183 (hypothesis $x22562) false) $x22565) $x22556)))
+(let (($x21179 (= ?x10079 v_b_P_H_arr$)))
+(let (($x19835 (forall ((?v0 B_S_ctype$) (?v1 Int) )(!(= (b_S_ref$ (b_S_ptr$ ?v0 ?v1)) ?v1) :pattern ( (b_S_ptr$ ?v0 ?v1) )))
+))
+(let (($x9655 (forall ((?v0 B_S_ctype$) (?v1 Int) )(= (b_S_ref$ (b_S_ptr$ ?v0 ?v1)) ?v1))
+))
+(let (($x9654 (= (b_S_ref$ (b_S_ptr$ ?1 ?0)) ?0)))
+(let ((@x15356 (mp~ (asserted $x9655) (nnf-pos (refl (~ $x9654 $x9654)) (~ $x9655 $x9655)) $x9655)))
+(let ((@x19840 (mp @x15356 (quant-intro (refl (= $x9654 $x9654)) (= $x9655 $x19835)) $x19835)))
+(let (($x21152 (not $x19835)))
+(let (($x21184 (or $x21152 $x21179)))
+(let ((@x21185 ((_ quant-inst b_T_T_u1$ v_b_P_H_arr$) $x21184)))
+(let ((@x24511 (unit-resolution @x21185 @x19840 $x21179)))
+(let ((@x22852 (monotonicity @x24511 (= ?x22553 ?x10078))))
+(let ((@x24070 (monotonicity (trans (hypothesis $x22556) @x22852 (= ?x10137 ?x10078)) (= ?x22485 ?x10079))))
+(let ((@x22338 (symm (monotonicity (trans @x24070 @x24511 (= ?x22485 v_b_P_H_arr$)) (= ?x22505 ?x10078)) (= ?x10078 ?x22505))))
+(let ((@x22340 (unit-resolution (hypothesis (not $x22506)) (trans (trans (hypothesis $x22556) @x22852 (= ?x10137 ?x10078)) @x22338 $x22506) false)))
+(let ((@x23350 (unit-resolution (lemma @x22340 (or $x22559 $x22506)) @x24124 $x22506)))
+(let ((@x23663 (trans (symm @x22852 (= ?x10078 ?x22553)) (symm @x24124 (= ?x22553 ?x10137)) (= ?x10078 ?x10137))))
+(let ((@x22940 (trans (monotonicity (trans @x23663 @x23350 (= ?x10078 ?x22505)) (= ?x22818 ?x22655)) (symm (monotonicity @x23350 (= ?x22478 ?x22655)) (= ?x22655 ?x22478)) (= ?x22818 ?x22478))))
+(let ((@x23082 (symm (monotonicity @x22940 (= $x22902 (b_S_ts_n_is_n_volatile$ ?x22478))) (= (b_S_ts_n_is_n_volatile$ ?x22478) $x22902))))
+(let (($x22602 (b_S_ts_n_is_n_volatile$ ?x22478)))
+(let (($x22641 (not $x22602)))
+(let (($x10139 (b_S_typed$ v_b_S_s$ ?x10137)))
+(let (($x15505 (not $x10139)))
+(let (($x22603 (or $x15505 $x22602)))
+(let (($x22604 (not $x22603)))
+(let ((?x10076 (b_S_array$ b_T_T_u1$ v_b_P_H_len$)))
+(let ((?x10080 (b_S_ptr$ ?x10076 ?x10079)))
+(let ((?x21014 (b_S_ref$ ?x10080)))
+(let ((?x21983 (b_S_ptr$ ?x10076 ?x21014)))
+(let ((?x22343 (b_S_domain$ v_b_S_s$ ?x21983)))
+(let ((?x22595 (b_S_ptr$ ?x10076 v_b_P_H_arr$)))
+(let (($x22596 (b_S_set_n_in$ ?x22595 ?x22343)))
+(let ((@x24530 (monotonicity (symm @x24511 (= v_b_P_H_arr$ ?x10079)) (= ?x22595 ?x10080))))
+(let (($x21990 (= ?x10080 ?x21983)))
+(let (($x10084 (b_S_is$ ?x10080 ?x10076)))
+(let (($x11245 (>= (+ b_S_max_o_u4$ (* (- 1) v_b_P_H_len$)) 0)))
+(let (($x11243 (>= v_b_P_H_len$ 0)))
+(let (($x10439 (forall ((?v0 B_S_ptr$) )(!(let (($x10113 (b_S_in_n_writes_n_at$ v_b_H_wrTime_S_1_T_6_o_1$ ?v0)))
+(not $x10113)) :pattern ( (b_S_in_n_writes_n_at$ v_b_H_wrTime_S_1_T_6_o_1$ ?v0) )))
+))
+(let ((?x10111 (b_S_current_n_timestamp$ v_b_S_s$)))
+(let (($x10112 (= v_b_H_wrTime_S_1_T_6_o_1$ ?x10111)))
+(let (($x10109 (b_S_local_n_value_n_is$ v_b_S_s$ b_H_tok_S_1_T_6_o_1$ b_H_loc_o_len$ v_b_P_H_len$ b_T_T_u4$)))
+(let (($x10107 (b_S_local_n_value_n_is_n_ptr$ v_b_S_s$ b_H_tok_S_1_T_6_o_1$ b_H_loc_o_arr$ ?x10078 ?x2238)))
+(let (($x10106 (b_S_local_n_value_n_is$ v_b_S_s$ b_H_tok_S_1_T_6_o_1$ b_H_loc_o_arr$ ?x10105 ?x2238)))
+(let (($x11256 (forall ((?v0 B_S_pure_n_function$) )(!(let (($x11251 (>= (+ (b_S_frame_n_level$ ?v0) (* (- 1) b_S_current_n_frame_n_level$)) 0)))
+(not $x11251)) :pattern ( (b_S_frame_n_level$ ?v0) )))
+))
+(let (($x10096 (b_S_good_n_state_n_ext$ b_H_tok_S_1_T_6_o_1$ v_b_S_s$)))
+(let (($x10095 (b_S_function_n_entry$ v_b_S_s$)))
+(let (($x10089 (b_S_is_n_non_n_primitive$ ?x10076)))
+(let ((?x10086 (b_S_kind_n_of$ ?x10076)))
+(let (($x10087 (= ?x10086 b_S_kind_n_primitive$)))
+(let (($x10088 (not $x10087)))
+(let (($x10085 (b_S_typed$ v_b_S_s$ ?x10080)))
+(let ((?x10082 (b_S_owner$ v_b_S_s$ ?x10080)))
+(let (($x10083 (= ?x10082 b_S_me$)))
+(let (($x10081 (b_S_closed$ v_b_S_s$ ?x10080)))
+(let (($x11260 (not $x11259)))
+(let (($x11263 (>= v_b_P_H_len$ 1099511627776)))
+(let (($x11264 (not $x11263)))
+(let (($x11270 (>= (+ b_S_max_o_u4$ (* (- 1) v_b_SL_H_witness$)) 0)))
+(let (($x11268 (>= v_b_SL_H_witness$ 0)))
+(let (($x11278 (>= (+ b_S_max_o_u4$ (* (- 1) v_b_L_H_p$)) 0)))
+(let (($x11276 (>= v_b_L_H_p$ 0)))
+(let (($x11286 (>= (+ b_S_max_o_u1$ (* (- 1) v_b_L_H_max$)) 0)))
+(let (($x11284 (>= v_b_L_H_max$ 0)))
+(let (($x11342 (and $x11284 $x11286 $x11276 $x11278 $x11268 $x11270 $x11264 $x11260 $x10081 $x10083 $x10084 $x10085 $x10088 $x10089 $x10095 $x10096 $x10097 $x11256 $x10106 $x10107 $x10109 $x10112 $x10439 $x11243 $x11245)))
+(let (($x11844 (exists ((?v0 Int) )(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x10238 (= ?x10163 v_b_S_result_G_0$)))
+(let (($x11800 (>= (+ ?v0 (* (- 1) v_b_P_H_len$)) 0)))
+(let (($x11802 (not $x11800)))
+(let ((?x3113 (* (- 1) b_S_max_o_u4$)))
+(let ((?x3114 (+ ?v0 ?x3113)))
+(let (($x3115 (<= ?x3114 0)))
+(let (($x2815 (>= ?v0 0)))
+(and $x2815 $x3115 $x11802 $x10238))))))))))
+))
+(let (($x11824 (forall ((?v0 Int) )(let ((?x11816 (* (- 1) v_b_S_result_G_0$)))
+(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x11818 (<= (+ ?x10163 ?x11816) 0)))
+(let (($x11800 (>= (+ ?v0 (* (- 1) v_b_P_H_len$)) 0)))
+(let (($x11802 (not $x11800)))
+(let ((?x3113 (* (- 1) b_S_max_o_u4$)))
+(let ((?x3114 (+ ?v0 ?x3113)))
+(let (($x3115 (<= ?x3114 0)))
+(let (($x2815 (>= ?v0 0)))
+(let (($x11808 (and $x2815 $x3115 $x11802)))
+(let (($x11813 (not $x11808)))
+(or $x11813 $x11818)))))))))))))
+))
+(let (($x11827 (not $x11824)))
+(let (($x11847 (or $x11827 $x11844)))
+(let (($x11850 (and $x11824 $x11847)))
+(let (($x11792 (and b_S_position_n_marker$ $x11429 $x11432 $x10216 $x10218 $x10220 $x10222)))
+(let (($x11797 (not $x11792)))
+(let (($x11853 (or $x11797 $x11850)))
+(let (($x11856 (and b_S_position_n_marker$ $x11853)))
+(let (($x11772 (and $x11486 $x11429 $x11432)))
+(let (($x11777 (not $x11772)))
+(let (($x11859 (or $x11777 $x11856)))
+(let (($x11648 (not $x11647)))
+(let (($x11651 (and $x11648 $x10374)))
+(let (($x11639 (forall ((?v0 Int) )(let ((?x11631 (* (- 1) v_b_L_H_max_G_3$)))
+(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x11633 (<= (+ ?x10163 ?x11631) 0)))
+(let (($x11615 (>= (+ ?v0 (* (- 1) v_b_L_H_p_G_1$)) 0)))
+(let (($x11617 (not $x11615)))
+(let ((?x3113 (* (- 1) b_S_max_o_u4$)))
+(let ((?x3114 (+ ?v0 ?x3113)))
+(let (($x3115 (<= ?x3114 0)))
+(let (($x2815 (>= ?v0 0)))
+(let (($x11623 (and $x2815 $x3115 $x11617)))
+(let (($x11628 (not $x11623)))
+(or $x11628 $x11633)))))))))))))
+))
+(let (($x11642 (not $x11639)))
+(let (($x11654 (or $x11642 $x11651)))
+(let (($x11657 (and $x11639 $x11654)))
+(let (($x11660 (or $x11612 $x11657)))
+(let (($x11663 (and $x11608 $x11660)))
+(let ((?x11574 (+ b_S_max_o_u4$ ?x11484)))
+(let (($x11573 (>= ?x11574 1)))
+(let (($x11600 (and $x11570 $x11573 $x11580 $x10358 $x11578 $x11536)))
+(let (($x11605 (not $x11600)))
+(let (($x11666 (or $x11605 $x11663)))
+(let (($x11672 (and $x11570 $x11573 $x11666)))
+(let (($x11725 (and $x11516 $x11432 $x10391 $x10392 $x11429 $x11536)))
+(let (($x11730 (not $x11725)))
+(let (($x11733 (or $x11730 $x11672)))
+(let (($x11562 (and $x10321 $x10324 $x10333 $x10334 $x10335 $x10338 $x10340 $x11429 $x11536)))
+(let (($x11567 (not $x11562)))
+(let (($x11677 (or $x11567 $x11672)))
+(let (($x11683 (and $x10321 $x10324 $x11677)))
+(let (($x10323 (and $x10321 $x10322)))
+(let (($x11001 (not $x10323)))
+(let (($x11688 (or $x11001 $x11683)))
+(let (($x11694 (and $x10321 $x10322 $x11688)))
+(let (($x11527 (and $x11515 $x11429 $x11432)))
+(let (($x11532 (not $x11527)))
+(let (($x11699 (or $x11532 $x11694)))
+(let (($x11736 (and $x11699 $x11733)))
+(let (($x11507 (and $x10321 $x10324 $x11429 $x11432)))
+(let (($x11512 (not $x11507)))
+(let (($x11739 (or $x11512 $x11736)))
+(let (($x11745 (and $x10321 $x10324 $x11739)))
+(let (($x11750 (or $x11001 $x11745)))
+(let (($x11756 (and $x10321 $x10322 $x11750)))
+(let (($x11496 (and $x11487 $x11429 $x11432)))
+(let (($x11501 (not $x11496)))
+(let (($x11761 (or $x11501 $x11756)))
+(let (($x11862 (and $x11761 $x11859)))
+(let (($x11476 (and $x10284 $x10204 $x10097 $x10291 $x10292 $x10293 $x10294 $x10295 $x10296 $x11429 $x11432)))
+(let (($x11481 (not $x11476)))
+(let (($x11868 (not $x11867)))
+(let (($x11895 (forall ((?v0 Int) )(let ((?x11887 (* (- 1) v_b_L_H_max_G_1$)))
+(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x11889 (<= (+ ?x10163 ?x11887) 0)))
+(let (($x11871 (>= (+ ?v0 (* (- 1) v_b_L_H_p_G_0$)) 0)))
+(let (($x11873 (not $x11871)))
+(let ((?x3113 (* (- 1) b_S_max_o_u4$)))
+(let ((?x3114 (+ ?v0 ?x3113)))
+(let (($x3115 (<= ?x3114 0)))
+(let (($x2815 (>= ?v0 0)))
+(let (($x11879 (and $x2815 $x3115 $x11873)))
+(let (($x11884 (not $x11879)))
+(or $x11884 $x11889)))))))))))))
+))
+(let (($x11904 (>= ?x11574 0)))
+(let (($x11907 (>= (+ b_S_max_o_u4$ ?x11865) 0)))
+(let (($x11914 (>= (+ b_S_max_o_u1$ (* (- 1) v_b_L_H_max_G_1$)) 0)))
+(let (($x11957 (and $x11260 $x10167 $x11911 $x11914 $x11907 $x11901 $x11904 $x11898 $x11895 $x11868 $x10192 $x11429 $x11432)))
+(let (($x11962 (not $x11957)))
+(let (($x11971 (or $x11962 $x11481 $x11862)))
+(let (($x11979 (and $x11260 $x10167 $x11971)))
+(let (($x11411 (forall ((?v0 Int) )(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x11404 (>= (+ v_b_L_H_max_G_0$ (* (- 1) ?x10163)) 0)))
+(let (($x11388 (>= ?v0 1)))
+(let (($x11389 (not $x11388)))
+(let ((?x3113 (* (- 1) b_S_max_o_u4$)))
+(let ((?x3114 (+ ?v0 ?x3113)))
+(let (($x3115 (<= ?x3114 0)))
+(let (($x2815 (>= ?v0 0)))
+(let (($x11395 (and $x2815 $x3115 $x11389)))
+(let (($x11400 (not $x11395)))
+(or $x11400 $x11404))))))))))))
+))
+(let (($x11414 (not $x11411)))
+(let (($x11984 (or $x11414 $x11979)))
+(let (($x11987 (and $x11411 $x11984)))
+(let (($x11382 (>= v_b_P_H_len$ 1)))
+(let (($x11385 (not $x11382)))
+(let (($x11990 (or $x11385 $x11987)))
+(let (($x11993 (and $x11382 $x11990)))
+(let (($x10148 (b_S_local_n_value_n_is$ v_b_S_s$ b_H_tok_S_1_T_16_o_8$ b_H_loc_o_p$ 1 b_T_T_u4$)))
+(let (($x10147 (b_S_local_n_value_n_is$ v_b_S_s$ b_H_tok_S_1_T_14_o_3$ b_H_loc_o_witness$ 0 b_T_T_u4$)))
+(let (($x10146 (b_S_local_n_value_n_is$ v_b_S_s$ b_H_tok_S_1_T_12_o_3$ b_H_loc_o_max$ v_b_L_H_max_G_0$ b_T_T_u1$)))
+(let (($x10145 (= v_b_L_H_max_G_0$ ?x10144)))
+(let (($x10138 (b_S_is$ ?x10137 b_T_T_u1$)))
+(let (($x11374 (and $x10138 $x10141 $x10145 $x10146 $x10147 $x10148)))
+(let (($x11379 (not $x11374)))
+(let (($x11996 (or $x11379 $x11993)))
+(let (($x12002 (and $x10138 $x10141 $x11996)))
+(let (($x10140 (and $x10138 $x10139)))
+(let (($x11209 (not $x10140)))
+(let (($x12007 (or $x11209 $x12002)))
+(let (($x12013 (and $x10138 $x10139 $x12007)))
+(let (($x10136 (b_S_in_n_domain_n_lab$ v_b_S_s$ ?x10080 ?x10080 b_l_H_public$)))
+(let (($x11221 (not $x10136)))
+(let (($x12018 (or $x11221 $x12013)))
+(let (($x12021 (and $x10136 $x12018)))
+(let (($x12027 (not (or (not $x11342) $x12021))))
+(let (($x10242 (exists ((?v0 Int) )(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x10238 (= ?x10163 v_b_S_result_G_0$)))
+(let (($x10233 (< ?v0 v_b_P_H_len$)))
+(let (($x3097 (<= ?v0 b_S_max_o_u4$)))
+(let (($x2766 (<= 0 ?v0)))
+(and $x2766 (and $x3097 (and $x10233 $x10238)))))))))
+))
+(let (($x10244 (and $x10242 (=> $x10242 true))))
+(let (($x10237 (forall ((?v0 Int) )(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x10235 (<= ?x10163 v_b_S_result_G_0$)))
+(let (($x10233 (< ?v0 v_b_P_H_len$)))
+(let (($x3097 (<= ?v0 b_S_max_o_u4$)))
+(let (($x2766 (<= 0 ?v0)))
+(let (($x3098 (and $x2766 $x3097)))
+(let (($x10234 (and $x3098 $x10233)))
+(=> $x10234 $x10235)))))))))
+))
+(let (($x10245 (=> $x10237 $x10244)))
+(let (($x10227 (and true (and $x10216 (and $x10218 (and $x10220 (and $x10222 true)))))))
+(let (($x10174 (<= 0 v_b_SL_H_witness_G_0$)))
+(let (($x10181 (<= 1 v_b_L_H_p_G_0$)))
+(let (($x10182 (and $x10181 $x10174)))
+(let (($x10230 (and true (and $x10182 (and $x10182 $x10227)))))
+(let (($x10247 (=> (and b_S_position_n_marker$ (and $x10182 $x10230)) (and $x10237 $x10245))))
+(let (($x10248 (and b_S_position_n_marker$ $x10247)))
+(let (($x10206 (and true $x10182)))
+(let (($x10207 (and $x10182 $x10206)))
+(let (($x10411 (and $x10182 $x10207)))
+(let (($x10412 (and true $x10411)))
+(let (($x10413 (and $x10182 $x10412)))
+(let (($x10410 (<= v_b_P_H_len$ v_b_L_H_p_G_0$)))
+(let (($x10416 (and true (and $x10182 (and $x10410 $x10413)))))
+(let (($x10417 (=> $x10416 $x10248)))
+(let (($x10377 (=> (and (and (< v_b_SL_H_witness_G_1$ v_b_P_H_len$) $x10374) false) true)))
+(let (($x10375 (and (< v_b_SL_H_witness_G_1$ v_b_P_H_len$) $x10374)))
+(let (($x10378 (and $x10375 $x10377)))
+(let (($x10370 (forall ((?v0 Int) )(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x10368 (<= ?x10163 v_b_L_H_max_G_3$)))
+(let (($x3097 (<= ?v0 b_S_max_o_u4$)))
+(let (($x2766 (<= 0 ?v0)))
+(let (($x3098 (and $x2766 $x3097)))
+(let (($x10367 (and $x3098 (< ?v0 v_b_L_H_p_G_1$))))
+(=> $x10367 $x10368))))))))
+))
+(let (($x10379 (=> $x10370 $x10378)))
+(let (($x10365 (<= v_b_L_H_p_G_1$ v_b_P_H_len$)))
+(let (($x10381 (=> $x10365 (and $x10370 $x10379))))
+(let (($x10341 (<= 0 v_b_SL_H_witness_G_1$)))
+(let (($x10360 (and (<= 2 v_b_L_H_p_G_1$) $x10341)))
+(let (($x10363 (and (= v_b_L_H_p_G_1$ (+ v_b_L_H_p_G_0$ 1)) (and $x10358 (and $x10360 true)))))
+(let (($x10355 (and (<= 0 (+ v_b_L_H_p_G_0$ 1)) (<= (+ v_b_L_H_p_G_0$ 1) b_S_max_o_u4$))))
+(let (($x10383 (=> (and $x10355 $x10363) (and $x10365 $x10381))))
+(let (($x10384 (and $x10355 $x10383)))
+(let (($x10395 (and true (and $x10391 (and $x10392 (and true (and $x10181 $x10341)))))))
+(let (($x10398 (and true (and $x10182 (and $x10182 $x10395)))))
+(let (($x10390 (<= ?x10327 v_b_L_H_max_G_1$)))
+(let (($x10402 (and true (and $x10182 (and $x10390 (and $x10182 $x10398))))))
+(let (($x10403 (=> $x10402 $x10384)))
+(let (($x10346 (and true (and $x10338 (and $x10340 (and true (and $x10181 $x10341)))))))
+(let (($x10325 (and $x10321 $x10324)))
+(let (($x10351 (and $x10325 (and $x10333 (and $x10334 (and $x10335 (and (and $x10181 $x10181) $x10346)))))))
+(let (($x10385 (=> $x10351 $x10384)))
+(let (($x10387 (=> $x10323 (and $x10325 $x10385))))
+(let (($x10331 (and true (and $x10182 (and (< v_b_L_H_max_G_1$ ?x10327) $x10207)))))
+(let (($x10389 (=> $x10331 (and $x10323 $x10387))))
+(let (($x10326 (and $x10325 $x10182)))
+(let (($x10405 (=> $x10326 (and $x10389 $x10403))))
+(let (($x10407 (=> $x10323 (and $x10325 $x10405))))
+(let (($x10319 (and true (and $x10182 (and (< v_b_L_H_p_G_0$ v_b_P_H_len$) $x10207)))))
+(let (($x10409 (=> $x10319 (and $x10323 $x10407))))
+(let (($x10300 (and (= ?x10272 ?x10272) (= (b_S_statusmap$ v_b_S_s$) (b_S_statusmap$ v_b_S_s$)))))
+(let (($x10301 (and $x10300 $x10182)))
+(let (($x10297 (and $x10295 $x10296)))
+(let (($x10205 (and $x10204 $x10097)))
+(let (($x10307 (and $x10205 (and $x10291 (and $x10292 (and $x10293 (and $x10294 (and $x10297 $x10301))))))))
+(let (($x10283 (forall ((?v0 B_S_ptr$) )(!(let ((?x10280 (b_S_timestamp$ v_b_S_s$ ?v0)))
+(<= ?x10280 ?x10280)) :pattern ( (b_S_timestamp$ v_b_S_s$ ?v0) )))
+))
+(let (($x10286 (and (<= ?x10111 ?x10111) (and $x10283 $x10284))))
+(let (($x10278 (forall ((?v0 B_S_ptr$) )(!(let (($x10260 (b_S_thread_n_local$ v_b_S_s$ ?v0)))
+(let ((?x10272 (b_S_typemap$ v_b_S_s$)))
+(let ((?x10273 (b_S_select_o_tm$ ?x10272 ?v0)))
+(let (($x10275 (and (= ?x10273 ?x10273) $x10260)))
+(=> $x10260 $x10275))))) :pattern ( (b_S_select_o_tm$ (b_S_typemap$ v_b_S_s$) ?v0) )))
+))
+(let (($x10287 (and $x10278 $x10286)))
+(let (($x10271 (forall ((?v0 B_S_ptr$) )(!(let (($x10260 (b_S_thread_n_local$ v_b_S_s$ ?v0)))
+(let ((?x10256 (b_S_statusmap$ v_b_S_s$)))
+(let ((?x10257 (b_S_select_o_sm$ ?x10256 ?v0)))
+(let (($x10269 (and (= ?x10257 ?x10257) $x10260)))
+(=> $x10260 $x10269))))) :pattern ( (b_S_select_o_sm$ (b_S_statusmap$ v_b_S_s$) ?v0) )))
+))
+(let (($x10288 (and $x10271 $x10287)))
+(let (($x10267 (forall ((?v0 B_S_ptr$) )(!(let (($x10260 (b_S_thread_n_local$ v_b_S_s$ ?v0)))
+(let ((?x10261 (b_S_memory$ v_b_S_s$)))
+(let ((?x10262 (b_S_select_o_mem$ ?x10261 ?v0)))
+(let (($x10264 (and (= ?x10262 ?x10262) $x10260)))
+(=> $x10260 $x10264))))) :pattern ( (b_S_select_o_mem$ (b_S_memory$ v_b_S_s$) ?v0) )))
+))
+(let (($x10289 (and $x10267 $x10288)))
+(let (($x10259 (forall ((?v0 B_S_ptr$) )(!(let (($x10253 (= (b_S_kind_n_of$ (b_S_typ$ (b_S_owner$ v_b_S_s$ ?v0))) b_S_kind_n_thread$)))
+(=> (not $x10253) (not $x10253))) :pattern ( (b_S_select_o_sm$ (b_S_statusmap$ v_b_S_s$) ?v0) )))
+))
+(let (($x10290 (and $x10259 $x10289)))
+(let (($x10311 (and true (and $x10182 (and $x10290 (and $x10286 $x10307))))))
+(let (($x10313 (and true (and $x10182 $x10311))))
+(let (($x10315 (and true (and $x10182 $x10313))))
+(let (($x10419 (=> $x10315 (and $x10409 $x10417))))
+(let (($x10203 (not true)))
+(let (($x10212 (and $x10203 (and $x10182 (and true (and $x10182 (and $x10205 $x10207)))))))
+(let (($x10213 (and $x10182 $x10212)))
+(let (($x10214 (and true $x10213)))
+(let (($x10249 (=> $x10214 $x10248)))
+(let (($x10420 (and $x10249 $x10419)))
+(let (($x10194 (and (and (< v_b_SL_H_witness_G_0$ v_b_P_H_len$) $x10192) $x10182)))
+(let (($x10188 (forall ((?v0 Int) )(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x10186 (<= ?x10163 v_b_L_H_max_G_1$)))
+(let (($x3097 (<= ?v0 b_S_max_o_u4$)))
+(let (($x2766 (<= 0 ?v0)))
+(let (($x3098 (and $x2766 $x3097)))
+(let (($x10185 (and $x3098 (< ?v0 v_b_L_H_p_G_0$))))
+(=> $x10185 $x10186))))))))
+))
+(let (($x10183 (<= v_b_L_H_p_G_0$ v_b_P_H_len$)))
+(let (($x10180 (and (<= 0 v_b_L_H_p_G_0$) (<= v_b_L_H_p_G_0$ b_S_max_o_u4$))))
+(let (($x10176 (and $x10174 (<= v_b_SL_H_witness_G_0$ b_S_max_o_u4$))))
+(let (($x10172 (and (<= 0 v_b_L_H_max_G_1$) (<= v_b_L_H_max_G_1$ b_S_max_o_u1$))))
+(let (($x10200 (and $x10172 (and $x10176 (and $x10180 (and $x10182 (and $x10183 (and $x10188 $x10194))))))))
+(let (($x10201 (and true $x10200)))
+(let (($x10074 (< 0 v_b_P_H_len$)))
+(let (($x10168 (and $x10074 $x10167)))
+(let (($x10421 (=> (and $x10168 $x10201) $x10420)))
+(let (($x10166 (forall ((?v0 Int) )(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x10164 (<= ?x10163 v_b_L_H_max_G_0$)))
+(let (($x3097 (<= ?v0 b_S_max_o_u4$)))
+(let (($x2766 (<= 0 ?v0)))
+(let (($x3098 (and $x2766 $x3097)))
+(let (($x10161 (and $x3098 (< ?v0 1))))
+(=> $x10161 $x10164))))))))
+))
+(let (($x10423 (=> $x10166 (and $x10168 $x10421))))
+(let (($x10159 (<= 1 v_b_P_H_len$)))
+(let (($x10425 (=> $x10159 (and $x10166 $x10423))))
+(let (($x10149 (<= 1 1)))
+(let (($x10154 (and $x10148 (and $x10149 (and $x10149 (and (<= 0 0) (<= 0 0)))))))
+(let (($x10142 (and $x10138 $x10141)))
+(let (($x10427 (=> (and $x10142 (and $x10145 (and $x10146 (and $x10147 $x10154)))) (and $x10159 $x10425))))
+(let (($x10429 (=> $x10140 (and $x10142 $x10427))))
+(let (($x10431 (=> $x10136 (and $x10140 $x10429))))
+(let (($x10119 (and (<= 0 v_b_P_H_len$) (<= v_b_P_H_len$ b_S_max_o_u4$))))
+(let (($x10116 (forall ((?v0 B_S_ptr$) )(!(let (($x10113 (b_S_in_n_writes_n_at$ v_b_H_wrTime_S_1_T_6_o_1$ ?v0)))
+(= $x10113 false)) :pattern ( (b_S_in_n_writes_n_at$ v_b_H_wrTime_S_1_T_6_o_1$ ?v0) )))
+))
+(let (($x10108 (and $x10106 $x10107)))
+(let (($x10104 (forall ((?v0 B_S_pure_n_function$) )(!(let ((?x10100 (b_S_frame_n_level$ ?v0)))
+(< ?x10100 b_S_current_n_frame_n_level$)) :pattern ( (b_S_frame_n_level$ ?v0) )))
+))
+(let (($x10098 (and $x10096 $x10097)))
+(let (($x10125 (and $x10098 (and $x10104 (and $x10108 (and $x10109 (and $x10112 (and $x10116 $x10119))))))))
+(let (($x10127 (and true (and $x10095 $x10125))))
+(let (($x10094 (and $x10081 (and $x10083 (and $x10084 (and $x10085 (and $x10088 $x10089)))))))
+(let (($x10073 (< v_b_P_H_len$ 1099511627776)))
+(let (($x10071 (and (<= 0 v_b_SL_H_witness$) (<= v_b_SL_H_witness$ b_S_max_o_u4$))))
+(let (($x10067 (and (<= 0 v_b_L_H_p$) (<= v_b_L_H_p$ b_S_max_o_u4$))))
+(let (($x10063 (and (<= 0 v_b_L_H_max$) (<= v_b_L_H_max$ b_S_max_o_u1$))))
+(let (($x10133 (and $x10063 (and $x10067 (and $x10071 (and $x10073 (and $x10074 (and $x10094 $x10127))))))))
+(let (($x10134 (and true $x10133)))
+(let (($x10433 (=> $x10134 (and $x10136 $x10431))))
+(let (($x10434 (not $x10433)))
+(let (($x10649 (forall ((?v0 Int) )(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x10235 (<= ?x10163 v_b_S_result_G_0$)))
+(let (($x10233 (< ?v0 v_b_P_H_len$)))
+(let (($x3097 (<= ?v0 b_S_max_o_u4$)))
+(let (($x2766 (<= 0 ?v0)))
+(let (($x3098 (and $x2766 $x3097)))
+(let (($x10234 (and $x3098 $x10233)))
+(or (not $x10234) $x10235)))))))))
+))
+(let (($x10665 (or (not $x10649) $x10242)))
+(let (($x10670 (and $x10649 $x10665)))
+(let (($x10616 (and $x10216 (and $x10218 (and $x10220 $x10222)))))
+(let (($x10626 (and $x10182 $x10616)))
+(let (($x10629 (and $x10182 $x10626)))
+(let (($x10639 (and $x10182 $x10629)))
+(let (($x10642 (and b_S_position_n_marker$ $x10639)))
+(let (($x10677 (or (not $x10642) $x10670)))
+(let (($x10682 (and b_S_position_n_marker$ $x10677)))
+(let (($x11134 (or (not (and $x10182 (and $x10410 $x10182))) $x10682)))
+(let (($x10931 (forall ((?v0 Int) )(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x10368 (<= ?x10163 v_b_L_H_max_G_3$)))
+(let (($x3097 (<= ?v0 b_S_max_o_u4$)))
+(let (($x2766 (<= 0 ?v0)))
+(let (($x3098 (and $x2766 $x3097)))
+(let (($x10367 (and $x3098 (< ?v0 v_b_L_H_p_G_1$))))
+(or (not $x10367) $x10368))))))))
+))
+(let (($x10954 (or (not $x10931) $x10375)))
+(let (($x10959 (and $x10931 $x10954)))
+(let (($x10966 (or (not $x10365) $x10959)))
+(let (($x10971 (and $x10365 $x10966)))
+(let (($x10918 (and $x10358 $x10360)))
+(let ((?x10901 (+ 1 v_b_L_H_p_G_0$)))
+(let (($x10913 (= v_b_L_H_p_G_1$ ?x10901)))
+(let (($x10921 (and $x10913 $x10918)))
+(let (($x10907 (<= ?x10901 b_S_max_o_u4$)))
+(let (($x10904 (<= 0 ?x10901)))
+(let (($x10910 (and $x10904 $x10907)))
+(let (($x10924 (and $x10910 $x10921)))
+(let (($x10978 (or (not $x10924) $x10971)))
+(let (($x10983 (and $x10910 $x10978)))
+(let (($x10342 (and $x10181 $x10341)))
+(let (($x11019 (and $x10392 $x10342)))
+(let (($x11022 (and $x10391 $x11019)))
+(let (($x11032 (and $x10182 $x11022)))
+(let (($x11035 (and $x10182 $x11032)))
+(let (($x11045 (and $x10182 $x11035)))
+(let (($x11048 (and $x10390 $x11045)))
+(let (($x11051 (and $x10182 $x11048)))
+(let (($x11065 (or (not $x11051) $x10983)))
+(let (($x10873 (and $x10340 $x10342)))
+(let (($x10876 (and $x10338 $x10873)))
+(let (($x10886 (and $x10181 $x10876)))
+(let (($x10889 (and $x10335 $x10886)))
+(let (($x10892 (and $x10334 $x10889)))
+(let (($x10895 (and $x10333 $x10892)))
+(let (($x10898 (and $x10325 $x10895)))
+(let (($x10990 (or (not $x10898) $x10983)))
+(let (($x10995 (and $x10325 $x10990)))
+(let (($x11002 (or $x11001 $x10995)))
+(let (($x11007 (and $x10323 $x11002)))
+(let (($x11014 (or (not (and $x10182 (and (< v_b_L_H_max_G_1$ ?x10327) $x10182))) $x11007)))
+(let (($x11070 (and $x11014 $x11065)))
+(let (($x11077 (or (not $x10326) $x11070)))
+(let (($x11082 (and $x10325 $x11077)))
+(let (($x11088 (or $x11001 $x11082)))
+(let (($x11093 (and $x10323 $x11088)))
+(let (($x11100 (or (not (and $x10182 (and (< v_b_L_H_p_G_0$ v_b_P_H_len$) $x10182))) $x11093)))
+(let (($x11139 (and $x11100 $x11134)))
+(let (($x10789 (and $x10297 $x10182)))
+(let (($x10792 (and $x10294 $x10789)))
+(let (($x10795 (and $x10293 $x10792)))
+(let (($x10798 (and $x10292 $x10795)))
+(let (($x10801 (and $x10291 $x10798)))
+(let (($x10804 (and $x10205 $x10801)))
+(let (($x10807 (and $x10286 $x10804)))
+(let (($x10810 (and $x10286 $x10807)))
+(let (($x10813 (and $x10182 $x10810)))
+(let (($x10823 (and $x10182 $x10813)))
+(let (($x10833 (and $x10182 $x10823)))
+(let (($x11146 (or (not $x10833) $x11139)))
+(let (($x10529 (forall ((?v0 Int) )(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x10186 (<= ?x10163 v_b_L_H_max_G_1$)))
+(let (($x3097 (<= ?v0 b_S_max_o_u4$)))
+(let (($x2766 (<= 0 ?v0)))
+(let (($x3098 (and $x2766 $x3097)))
+(let (($x10185 (and $x3098 (< ?v0 v_b_L_H_p_G_0$))))
+(or (not $x10185) $x10186))))))))
+))
+(let (($x10532 (and $x10529 $x10194)))
+(let (($x10535 (and $x10183 $x10532)))
+(let (($x10538 (and $x10182 $x10535)))
+(let (($x10541 (and $x10180 $x10538)))
+(let (($x10544 (and $x10176 $x10541)))
+(let (($x10547 (and $x10172 $x10544)))
+(let (($x10557 (and $x10168 $x10547)))
+(let (($x11162 (or (not $x10557) $x11146)))
+(let (($x11167 (and $x10168 $x11162)))
+(let (($x10522 (forall ((?v0 Int) )(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x10164 (<= ?x10163 v_b_L_H_max_G_0$)))
+(let (($x3097 (<= ?v0 b_S_max_o_u4$)))
+(let (($x2766 (<= 0 ?v0)))
+(let (($x3098 (and $x2766 $x3097)))
+(let (($x10161 (and $x3098 (< ?v0 1))))
+(or (not $x10161) $x10164))))))))
+))
+(let (($x11174 (or (not $x10522) $x11167)))
+(let (($x11179 (and $x10522 $x11174)))
+(let (($x11186 (or (not $x10159) $x11179)))
+(let (($x11191 (and $x10159 $x11186)))
+(let (($x10150 (<= 0 0)))
+(let (($x10497 (and $x10149 $x10150)))
+(let (($x10500 (and $x10149 $x10497)))
+(let (($x10503 (and $x10148 $x10500)))
+(let (($x10506 (and $x10147 $x10503)))
+(let (($x10509 (and $x10146 $x10506)))
+(let (($x10512 (and $x10145 $x10509)))
+(let (($x10515 (and $x10142 $x10512)))
+(let (($x11198 (or (not $x10515) $x11191)))
+(let (($x11203 (and $x10142 $x11198)))
+(let (($x11210 (or $x11209 $x11203)))
+(let (($x11215 (and $x10140 $x11210)))
+(let (($x11222 (or $x11221 $x11215)))
+(let (($x11227 (and $x10136 $x11222)))
+(let (($x10442 (and $x10439 $x10119)))
+(let (($x10445 (and $x10112 $x10442)))
+(let (($x10448 (and $x10109 $x10445)))
+(let (($x10451 (and $x10108 $x10448)))
+(let (($x10454 (and $x10104 $x10451)))
+(let (($x10457 (and $x10098 $x10454)))
+(let (($x10460 (and $x10095 $x10457)))
+(let (($x10470 (and $x10094 $x10460)))
+(let (($x10473 (and $x10074 $x10470)))
+(let (($x10476 (and $x10073 $x10473)))
+(let (($x10479 (and $x10071 $x10476)))
+(let (($x10482 (and $x10067 $x10479)))
+(let (($x10485 (and $x10063 $x10482)))
+(let (($x11234 (or (not $x10485) $x11227)))
+(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ ?x10078 ?0 b_T_T_u1$))))
+(let (($x10238 (= ?x10163 v_b_S_result_G_0$)))
+(let (($x11800 (>= (+ ?0 (* (- 1) v_b_P_H_len$)) 0)))
+(let (($x11802 (not $x11800)))
+(let ((?x3113 (* (- 1) b_S_max_o_u4$)))
+(let ((?x3114 (+ ?0 ?x3113)))
+(let (($x3115 (<= ?x3114 0)))
+(let (($x2815 (>= ?0 0)))
+(let (($x11839 (and $x2815 $x3115 $x11802 $x10238)))
+(let (($x2766 (<= 0 ?0)))
+(let (($x10241 (and $x2766 (and (<= ?0 b_S_max_o_u4$) (and (< ?0 v_b_P_H_len$) $x10238)))))
+(let (($x11834 (= (and (<= ?0 b_S_max_o_u4$) (and (< ?0 v_b_P_H_len$) $x10238)) (and $x3115 (and $x11802 $x10238)))))
+(let ((@x11832 (monotonicity (rewrite (= (< ?0 v_b_P_H_len$) $x11802)) (= (and (< ?0 v_b_P_H_len$) $x10238) (and $x11802 $x10238)))))
+(let ((@x2814 (rewrite (= $x2766 $x2815))))
+(let ((@x11838 (monotonicity @x2814 (monotonicity (rewrite (= (<= ?0 b_S_max_o_u4$) $x3115)) @x11832 $x11834) (= $x10241 (and $x2815 (and $x3115 (and $x11802 $x10238)))))))
+(let ((@x11843 (trans @x11838 (rewrite (= (and $x2815 (and $x3115 (and $x11802 $x10238))) $x11839)) (= $x10241 $x11839))))
+(let (($x11818 (<= (+ ?x10163 (* (- 1) v_b_S_result_G_0$)) 0)))
+(let (($x11808 (and $x2815 $x3115 $x11802)))
+(let (($x11813 (not $x11808)))
+(let (($x11821 (or $x11813 $x11818)))
+(let (($x10235 (<= ?x10163 v_b_S_result_G_0$)))
+(let (($x10233 (< ?0 v_b_P_H_len$)))
+(let (($x3097 (<= ?0 b_S_max_o_u4$)))
+(let (($x3098 (and $x2766 $x3097)))
+(let (($x10234 (and $x3098 $x10233)))
+(let (($x10646 (or (not $x10234) $x10235)))
+(let ((@x3124 (monotonicity @x2814 (rewrite (= $x3097 $x3115)) (= $x3098 (and $x2815 $x3115)))))
+(let ((@x11807 (monotonicity @x3124 (rewrite (= $x10233 $x11802)) (= $x10234 (and (and $x2815 $x3115) $x11802)))))
+(let ((@x11812 (trans @x11807 (rewrite (= (and (and $x2815 $x3115) $x11802) $x11808)) (= $x10234 $x11808))))
+(let ((@x11823 (monotonicity (monotonicity @x11812 (= (not $x10234) $x11813)) (rewrite (= $x10235 $x11818)) (= $x10646 $x11821))))
+(let ((@x11829 (monotonicity (quant-intro @x11823 (= $x10649 $x11824)) (= (not $x10649) $x11827))))
+(let ((@x11852 (monotonicity (quant-intro @x11823 (= $x10649 $x11824)) (monotonicity @x11829 (quant-intro @x11843 (= $x10242 $x11844)) (= $x10665 $x11847)) (= $x10670 $x11850))))
+(let (($x11434 (and $x11429 $x11432)))
+(let (($x11793 (= (and b_S_position_n_marker$ (and $x11434 (and $x11434 (and $x11434 $x10616)))) $x11792)))
+(let (($x11790 (= $x10642 (and b_S_position_n_marker$ (and $x11434 (and $x11434 (and $x11434 $x10616)))))))
+(let ((@x11430 (rewrite (= $x10181 $x11429))))
+(let ((@x11436 (monotonicity @x11430 (rewrite (= $x10174 $x11432)) (= $x10182 $x11434))))
+(let ((@x11785 (monotonicity @x11436 (monotonicity @x11436 (= $x10626 (and $x11434 $x10616))) (= $x10629 (and $x11434 (and $x11434 $x10616))))))
+(let ((@x11788 (monotonicity @x11436 @x11785 (= $x10639 (and $x11434 (and $x11434 (and $x11434 $x10616)))))))
+(let ((@x11799 (monotonicity (trans (monotonicity @x11788 $x11790) (rewrite $x11793) (= $x10642 $x11792)) (= (not $x10642) $x11797))))
+(let ((@x11858 (monotonicity (monotonicity @x11799 @x11852 (= $x10677 $x11853)) (= $x10682 $x11856))))
+(let ((@x11768 (monotonicity (rewrite (= $x10410 $x11486)) @x11436 (= (and $x10410 $x10182) (and $x11486 $x11434)))))
+(let ((@x11771 (monotonicity @x11436 @x11768 (= (and $x10182 (and $x10410 $x10182)) (and $x11434 (and $x11486 $x11434))))))
+(let ((@x11776 (trans @x11771 (rewrite (= (and $x11434 (and $x11486 $x11434)) $x11772)) (= (and $x10182 (and $x10410 $x10182)) $x11772))))
+(let ((@x11861 (monotonicity (monotonicity @x11776 (= (not (and $x10182 (and $x10410 $x10182))) $x11777)) @x11858 (= $x11134 $x11859))))
+(let ((@x11653 (monotonicity (rewrite (= (< v_b_SL_H_witness_G_1$ v_b_P_H_len$) $x11648)) (= $x10375 $x11651))))
+(let (($x11633 (<= (+ ?x10163 (* (- 1) v_b_L_H_max_G_3$)) 0)))
+(let (($x11615 (>= (+ ?0 ?x11581) 0)))
+(let (($x11617 (not $x11615)))
+(let (($x11623 (and $x2815 $x3115 $x11617)))
+(let (($x11628 (not $x11623)))
+(let (($x11636 (or $x11628 $x11633)))
+(let (($x10368 (<= ?x10163 v_b_L_H_max_G_3$)))
+(let (($x10928 (or (not (and $x3098 (< ?0 v_b_L_H_p_G_1$))) $x10368)))
+(let ((@x11622 (monotonicity @x3124 (rewrite (= (< ?0 v_b_L_H_p_G_1$) $x11617)) (= (and $x3098 (< ?0 v_b_L_H_p_G_1$)) (and (and $x2815 $x3115) $x11617)))))
+(let ((@x11627 (trans @x11622 (rewrite (= (and (and $x2815 $x3115) $x11617) $x11623)) (= (and $x3098 (< ?0 v_b_L_H_p_G_1$)) $x11623))))
+(let ((@x11630 (monotonicity @x11627 (= (not (and $x3098 (< ?0 v_b_L_H_p_G_1$))) $x11628))))
+(let ((@x11641 (quant-intro (monotonicity @x11630 (rewrite (= $x10368 $x11633)) (= $x10928 $x11636)) (= $x10931 $x11639))))
+(let ((@x11656 (monotonicity (monotonicity @x11641 (= (not $x10931) $x11642)) @x11653 (= $x10954 $x11654))))
+(let ((@x11662 (monotonicity (monotonicity (rewrite (= $x10365 $x11608)) (= (not $x10365) $x11612)) (monotonicity @x11641 @x11656 (= $x10959 $x11657)) (= $x10966 $x11660))))
+(let (($x11601 (= (and (and $x11570 $x11573) (and $x11580 (and $x10358 (and $x11578 $x11536)))) $x11600)))
+(let (($x11598 (= $x10924 (and (and $x11570 $x11573) (and $x11580 (and $x10358 (and $x11578 $x11536)))))))
+(let ((@x11587 (monotonicity (rewrite (= (<= 2 v_b_L_H_p_G_1$) $x11578)) (rewrite (= $x10341 $x11536)) (= $x10360 (and $x11578 $x11536)))))
+(let ((@x11593 (monotonicity (rewrite (= $x10913 $x11580)) (monotonicity @x11587 (= $x10918 (and $x10358 (and $x11578 $x11536)))) (= $x10921 (and $x11580 (and $x10358 (and $x11578 $x11536)))))))
+(let ((@x11596 (monotonicity (rewrite (= $x10904 $x11570)) (rewrite (= $x10907 $x11573)) (= $x10910 (and $x11570 $x11573)))))
+(let ((@x11607 (monotonicity (trans (monotonicity @x11596 @x11593 $x11598) (rewrite $x11601) (= $x10924 $x11600)) (= (not $x10924) $x11605))))
+(let ((@x11668 (monotonicity @x11607 (monotonicity (rewrite (= $x10365 $x11608)) @x11662 (= $x10971 $x11663)) (= $x10978 $x11666))))
+(let ((@x11676 (trans (monotonicity @x11596 @x11668 (= $x10983 (and (and $x11570 $x11573) $x11666))) (rewrite (= (and (and $x11570 $x11573) $x11666) $x11672)) (= $x10983 $x11672))))
+(let (($x11716 (and $x11434 (and $x11434 (and $x11434 (and $x10391 (and $x10392 (and $x11429 $x11536))))))))
+(let (($x11714 (= $x11035 (and $x11434 (and $x11434 (and $x10391 (and $x10392 (and $x11429 $x11536))))))))
+(let ((@x11540 (monotonicity @x11430 (rewrite (= $x10341 $x11536)) (= $x10342 (and $x11429 $x11536)))))
+(let ((@x11709 (monotonicity (monotonicity @x11540 (= $x11019 (and $x10392 (and $x11429 $x11536)))) (= $x11022 (and $x10391 (and $x10392 (and $x11429 $x11536)))))))
+(let ((@x11712 (monotonicity @x11436 @x11709 (= $x11032 (and $x11434 (and $x10391 (and $x10392 (and $x11429 $x11536))))))))
+(let ((@x11721 (monotonicity (rewrite (= $x10390 $x11516)) (monotonicity @x11436 (monotonicity @x11436 @x11712 $x11714) (= $x11045 $x11716)) (= $x11048 (and $x11516 $x11716)))))
+(let ((@x11729 (trans (monotonicity @x11436 @x11721 (= $x11051 (and $x11434 (and $x11516 $x11716)))) (rewrite (= (and $x11434 (and $x11516 $x11716)) $x11725)) (= $x11051 $x11725))))
+(let ((@x11735 (monotonicity (monotonicity @x11729 (= (not $x11051) $x11730)) @x11676 (= $x11065 $x11733))))
+(let (($x11553 (and $x10334 (and $x10335 (and $x11429 (and $x10338 (and $x10340 (and $x11429 $x11536))))))))
+(let (($x11551 (= $x10889 (and $x10335 (and $x11429 (and $x10338 (and $x10340 (and $x11429 $x11536))))))))
+(let ((@x11546 (monotonicity (monotonicity @x11540 (= $x10873 (and $x10340 (and $x11429 $x11536)))) (= $x10876 (and $x10338 (and $x10340 (and $x11429 $x11536)))))))
+(let ((@x11549 (monotonicity @x11430 @x11546 (= $x10886 (and $x11429 (and $x10338 (and $x10340 (and $x11429 $x11536))))))))
+(let ((@x11558 (monotonicity (monotonicity (monotonicity @x11549 $x11551) (= $x10892 $x11553)) (= $x10895 (and $x10333 $x11553)))))
+(let ((@x11566 (trans (monotonicity @x11558 (= $x10898 (and $x10325 (and $x10333 $x11553)))) (rewrite (= (and $x10325 (and $x10333 $x11553)) $x11562)) (= $x10898 $x11562))))
+(let ((@x11679 (monotonicity (monotonicity @x11566 (= (not $x10898) $x11567)) @x11676 (= $x10990 $x11677))))
+(let ((@x11687 (trans (monotonicity @x11679 (= $x10995 (and $x10325 $x11677))) (rewrite (= (and $x10325 $x11677) $x11683)) (= $x10995 $x11683))))
+(let ((@x11693 (monotonicity (monotonicity @x11687 (= $x11002 $x11688)) (= $x11007 (and $x10323 $x11688)))))
+(let (($x10328 (< v_b_L_H_max_G_1$ ?x10327)))
+(let (($x10856 (and $x10328 $x10182)))
+(let (($x10859 (and $x10182 $x10856)))
+(let ((@x11523 (monotonicity (rewrite (= $x10328 $x11515)) @x11436 (= $x10856 (and $x11515 $x11434)))))
+(let ((@x11531 (trans (monotonicity @x11436 @x11523 (= $x10859 (and $x11434 (and $x11515 $x11434)))) (rewrite (= (and $x11434 (and $x11515 $x11434)) $x11527)) (= $x10859 $x11527))))
+(let ((@x11701 (monotonicity (monotonicity @x11531 (= (not $x10859) $x11532)) (trans @x11693 (rewrite (= (and $x10323 $x11688) $x11694)) (= $x11007 $x11694)) (= $x11014 $x11699))))
+(let ((@x11511 (trans (monotonicity @x11436 (= $x10326 (and $x10325 $x11434))) (rewrite (= (and $x10325 $x11434) $x11507)) (= $x10326 $x11507))))
+(let ((@x11741 (monotonicity (monotonicity @x11511 (= (not $x10326) $x11512)) (monotonicity @x11701 @x11735 (= $x11070 $x11736)) (= $x11077 $x11739))))
+(let ((@x11749 (trans (monotonicity @x11741 (= $x11082 (and $x10325 $x11739))) (rewrite (= (and $x10325 $x11739) $x11745)) (= $x11082 $x11745))))
+(let ((@x11755 (monotonicity (monotonicity @x11749 (= $x11088 $x11750)) (= $x11093 (and $x10323 $x11750)))))
+(let (($x11502 (= (not (and $x10182 (and (< v_b_L_H_p_G_0$ v_b_P_H_len$) $x10182))) $x11501)))
+(let (($x10316 (< v_b_L_H_p_G_0$ v_b_P_H_len$)))
+(let (($x10843 (and $x10316 $x10182)))
+(let (($x10846 (and $x10182 $x10843)))
+(let ((@x11492 (monotonicity (rewrite (= $x10316 $x11487)) @x11436 (= $x10843 (and $x11487 $x11434)))))
+(let ((@x11500 (trans (monotonicity @x11436 @x11492 (= $x10846 (and $x11434 (and $x11487 $x11434)))) (rewrite (= (and $x11434 (and $x11487 $x11434)) $x11496)) (= $x10846 $x11496))))
+(let ((@x11763 (monotonicity (monotonicity @x11500 $x11502) (trans @x11755 (rewrite (= (and $x10323 $x11750) $x11756)) (= $x11093 $x11756)) (= $x11100 $x11761))))
+(let (($x11452 (and $x10205 (and $x10291 (and $x10292 (and $x10293 (and $x10294 (and $x10297 $x11434))))))))
+(let (($x11458 (and true (and true $x10284))))
+(let (($x11477 (= (and $x11434 (and $x11434 (and $x11434 (and $x11458 (and $x11458 $x11452))))) $x11476)))
+(let (($x11474 (= $x10833 (and $x11434 (and $x11434 (and $x11434 (and $x11458 (and $x11458 $x11452))))))))
+(let (($x11450 (= $x10801 (and $x10291 (and $x10292 (and $x10293 (and $x10294 (and $x10297 $x11434))))))))
+(let ((@x11442 (monotonicity (monotonicity @x11436 (= $x10789 (and $x10297 $x11434))) (= $x10792 (and $x10294 (and $x10297 $x11434))))))
+(let ((@x11448 (monotonicity (monotonicity @x11442 (= $x10795 (and $x10293 (and $x10294 (and $x10297 $x11434))))) (= $x10798 (and $x10292 (and $x10293 (and $x10294 (and $x10297 $x11434))))))))
+(let (($x11419 (forall ((?v0 B_S_ptr$) )(!true :pattern ( (b_S_timestamp$ v_b_S_s$ ?v0) )))
+))
+(let (($x11417 (= (<= (b_S_timestamp$ v_b_S_s$ ?0) (b_S_timestamp$ v_b_S_s$ ?0)) true)))
+(let ((@x11425 (trans (quant-intro (rewrite $x11417) (= $x10283 $x11419)) (elim-unused (= $x11419 true)) (= $x10283 true))))
+(let ((@x11460 (monotonicity (rewrite (= (<= ?x10111 ?x10111) true)) (monotonicity @x11425 (= (and $x10283 $x10284) (and true $x10284))) (= $x10286 $x11458))))
+(let ((@x11463 (monotonicity @x11460 (monotonicity (monotonicity @x11448 $x11450) (= $x10804 $x11452)) (= $x10807 (and $x11458 $x11452)))))
+(let ((@x11469 (monotonicity @x11436 (monotonicity @x11460 @x11463 (= $x10810 (and $x11458 (and $x11458 $x11452)))) (= $x10813 (and $x11434 (and $x11458 (and $x11458 $x11452)))))))
+(let ((@x11472 (monotonicity @x11436 @x11469 (= $x10823 (and $x11434 (and $x11434 (and $x11458 (and $x11458 $x11452))))))))
+(let ((@x11483 (monotonicity (trans (monotonicity @x11436 @x11472 $x11474) (rewrite $x11477) (= $x10833 $x11476)) (= (not $x10833) $x11481))))
+(let ((@x11967 (monotonicity @x11483 (monotonicity @x11763 @x11861 (= $x11139 $x11862)) (= $x11146 (or $x11481 $x11862)))))
+(let (($x11936 (and (and $x11901 $x11904) (and $x11434 (and $x11898 (and $x11895 (and (and $x11868 $x10192) $x11434)))))))
+(let (($x11951 (and $x11260 $x10167)))
+(let (($x11958 (= (and $x11951 (and (and $x11911 $x11914) (and (and $x11432 $x11907) $x11936))) $x11957)))
+(let (($x11955 (= $x10557 (and $x11951 (and (and $x11911 $x11914) (and (and $x11432 $x11907) $x11936))))))
+(let (($x11931 (= $x10538 (and $x11434 (and $x11898 (and $x11895 (and (and $x11868 $x10192) $x11434)))))))
+(let (($x11919 (= (and (< v_b_SL_H_witness_G_0$ v_b_P_H_len$) $x10192) (and $x11868 $x10192))))
+(let ((@x11920 (monotonicity (rewrite (= (< v_b_SL_H_witness_G_0$ v_b_P_H_len$) $x11868)) $x11919)))
+(let (($x11889 (<= (+ ?x10163 (* (- 1) v_b_L_H_max_G_1$)) 0)))
+(let (($x11871 (>= (+ ?0 ?x11484) 0)))
+(let (($x11873 (not $x11871)))
+(let (($x11879 (and $x2815 $x3115 $x11873)))
+(let (($x11884 (not $x11879)))
+(let (($x11892 (or $x11884 $x11889)))
+(let (($x10186 (<= ?x10163 v_b_L_H_max_G_1$)))
+(let (($x10526 (or (not (and $x3098 (< ?0 v_b_L_H_p_G_0$))) $x10186)))
+(let ((@x11878 (monotonicity @x3124 (rewrite (= (< ?0 v_b_L_H_p_G_0$) $x11873)) (= (and $x3098 (< ?0 v_b_L_H_p_G_0$)) (and (and $x2815 $x3115) $x11873)))))
+(let ((@x11883 (trans @x11878 (rewrite (= (and (and $x2815 $x3115) $x11873) $x11879)) (= (and $x3098 (< ?0 v_b_L_H_p_G_0$)) $x11879))))
+(let ((@x11886 (monotonicity @x11883 (= (not (and $x3098 (< ?0 v_b_L_H_p_G_0$))) $x11884))))
+(let ((@x11897 (quant-intro (monotonicity @x11886 (rewrite (= $x10186 $x11889)) (= $x10526 $x11892)) (= $x10529 $x11895))))
+(let ((@x11926 (monotonicity @x11897 (monotonicity @x11920 @x11436 (= $x10194 (and (and $x11868 $x10192) $x11434))) (= $x10532 (and $x11895 (and (and $x11868 $x10192) $x11434))))))
+(let ((@x11929 (monotonicity (rewrite (= $x10183 $x11898)) @x11926 (= $x10535 (and $x11898 (and $x11895 (and (and $x11868 $x10192) $x11434)))))))
+(let ((@x11935 (monotonicity (rewrite (= (<= 0 v_b_L_H_p_G_0$) $x11901)) (rewrite (= (<= v_b_L_H_p_G_0$ b_S_max_o_u4$) $x11904)) (= $x10180 (and $x11901 $x11904)))))
+(let ((@x11941 (monotonicity (rewrite (= $x10174 $x11432)) (rewrite (= (<= v_b_SL_H_witness_G_0$ b_S_max_o_u4$) $x11907)) (= $x10176 (and $x11432 $x11907)))))
+(let ((@x11944 (monotonicity @x11941 (monotonicity @x11935 (monotonicity @x11436 @x11929 $x11931) (= $x10541 $x11936)) (= $x10544 (and (and $x11432 $x11907) $x11936)))))
+(let ((@x11947 (monotonicity (rewrite (= (<= 0 v_b_L_H_max_G_1$) $x11911)) (rewrite (= (<= v_b_L_H_max_G_1$ b_S_max_o_u1$) $x11914)) (= $x10172 (and $x11911 $x11914)))))
+(let ((@x11950 (monotonicity @x11947 @x11944 (= $x10547 (and (and $x11911 $x11914) (and (and $x11432 $x11907) $x11936))))))
+(let ((@x11956 (monotonicity (monotonicity (rewrite (= $x10074 $x11260)) (= $x10168 $x11951)) @x11950 $x11955)))
+(let ((@x11964 (monotonicity (trans @x11956 (rewrite $x11958) (= $x10557 $x11957)) (= (not $x10557) $x11962))))
+(let ((@x11975 (trans (monotonicity @x11964 @x11967 (= $x11162 (or $x11962 (or $x11481 $x11862)))) (rewrite (= (or $x11962 (or $x11481 $x11862)) $x11971)) (= $x11162 $x11971))))
+(let ((@x11978 (monotonicity (monotonicity (rewrite (= $x10074 $x11260)) (= $x10168 $x11951)) @x11975 (= $x11167 (and $x11951 $x11971)))))
+(let (($x11404 (>= (+ v_b_L_H_max_G_0$ (* (- 1) ?x10163)) 0)))
+(let (($x11388 (>= ?0 1)))
+(let (($x11389 (not $x11388)))
+(let (($x11395 (and $x2815 $x3115 $x11389)))
+(let (($x11400 (not $x11395)))
+(let (($x11408 (or $x11400 $x11404)))
+(let (($x10164 (<= ?x10163 v_b_L_H_max_G_0$)))
+(let (($x10519 (or (not (and $x3098 (< ?0 1))) $x10164)))
+(let ((@x11394 (monotonicity @x3124 (rewrite (= (< ?0 1) $x11389)) (= (and $x3098 (< ?0 1)) (and (and $x2815 $x3115) $x11389)))))
+(let ((@x11399 (trans @x11394 (rewrite (= (and (and $x2815 $x3115) $x11389) $x11395)) (= (and $x3098 (< ?0 1)) $x11395))))
+(let ((@x11410 (monotonicity (monotonicity @x11399 (= (not (and $x3098 (< ?0 1))) $x11400)) (rewrite (= $x10164 $x11404)) (= $x10519 $x11408))))
+(let ((@x11416 (monotonicity (quant-intro @x11410 (= $x10522 $x11411)) (= (not $x10522) $x11414))))
+(let ((@x11986 (monotonicity @x11416 (trans @x11978 (rewrite (= (and $x11951 $x11971) $x11979)) (= $x11167 $x11979)) (= $x11174 $x11984))))
+(let ((@x11992 (monotonicity (monotonicity (rewrite (= $x10159 $x11382)) (= (not $x10159) $x11385)) (monotonicity (quant-intro @x11410 (= $x10522 $x11411)) @x11986 (= $x11179 $x11987)) (= $x11186 $x11990))))
+(let (($x11368 (and $x10145 (and $x10146 (and $x10147 (and $x10148 (and true (and true true))))))))
+(let (($x11366 (= $x10509 (and $x10146 (and $x10147 (and $x10148 (and true (and true true))))))))
+(let ((@x11355 (monotonicity (rewrite (= $x10149 true)) (rewrite (= $x10150 true)) (= $x10497 (and true true)))))
+(let ((@x11358 (monotonicity (rewrite (= $x10149 true)) @x11355 (= $x10500 (and true (and true true))))))
+(let ((@x11361 (monotonicity @x11358 (= $x10503 (and $x10148 (and true (and true true)))))))
+(let ((@x11364 (monotonicity @x11361 (= $x10506 (and $x10147 (and $x10148 (and true (and true true))))))))
+(let ((@x11373 (monotonicity (monotonicity (monotonicity @x11364 $x11366) (= $x10512 $x11368)) (= $x10515 (and $x10142 $x11368)))))
+(let ((@x11381 (monotonicity (trans @x11373 (rewrite (= (and $x10142 $x11368) $x11374)) (= $x10515 $x11374)) (= (not $x10515) $x11379))))
+(let ((@x11998 (monotonicity @x11381 (monotonicity (rewrite (= $x10159 $x11382)) @x11992 (= $x11191 $x11993)) (= $x11198 $x11996))))
+(let ((@x12006 (trans (monotonicity @x11998 (= $x11203 (and $x10142 $x11996))) (rewrite (= (and $x10142 $x11996) $x12002)) (= $x11203 $x12002))))
+(let ((@x12012 (monotonicity (monotonicity @x12006 (= $x11210 $x12007)) (= $x11215 (and $x10140 $x12007)))))
+(let ((@x12020 (monotonicity (trans @x12012 (rewrite (= (and $x10140 $x12007) $x12013)) (= $x11215 $x12013)) (= $x11222 $x12018))))
+(let (($x11306 (and $x11256 (and $x10108 (and $x10109 (and $x10112 (and $x10439 (and $x11243 $x11245))))))))
+(let (($x11327 (and (and $x11268 $x11270) (and $x11264 (and $x11260 (and $x10094 (and $x10095 (and $x10098 $x11306))))))))
+(let ((@x11344 (rewrite (= (and (and $x11284 $x11286) (and (and $x11276 $x11278) $x11327)) $x11342))))
+(let (($x11322 (= $x10476 (and $x11264 (and $x11260 (and $x10094 (and $x10095 (and $x10098 $x11306))))))))
+(let (($x11304 (= $x10451 (and $x10108 (and $x10109 (and $x10112 (and $x10439 (and $x11243 $x11245))))))))
+(let ((@x11293 (monotonicity (rewrite (= (<= 0 v_b_P_H_len$) $x11243)) (rewrite (= (<= v_b_P_H_len$ b_S_max_o_u4$) $x11245)) (= $x10119 (and $x11243 $x11245)))))
+(let ((@x11299 (monotonicity (monotonicity @x11293 (= $x10442 (and $x10439 (and $x11243 $x11245)))) (= $x10445 (and $x10112 (and $x10439 (and $x11243 $x11245)))))))
+(let ((@x11302 (monotonicity @x11299 (= $x10448 (and $x10109 (and $x10112 (and $x10439 (and $x11243 $x11245))))))))
+(let (($x11251 (>= (+ (b_S_frame_n_level$ ?0) (* (- 1) b_S_current_n_frame_n_level$)) 0)))
+(let (($x11250 (not $x11251)))
+(let ((@x11255 (rewrite (= (< (b_S_frame_n_level$ ?0) b_S_current_n_frame_n_level$) $x11250))))
+(let ((@x11308 (monotonicity (quant-intro @x11255 (= $x10104 $x11256)) (monotonicity @x11302 $x11304) (= $x10454 $x11306))))
+(let ((@x11314 (monotonicity (monotonicity @x11308 (= $x10457 (and $x10098 $x11306))) (= $x10460 (and $x10095 (and $x10098 $x11306))))))
+(let ((@x11320 (monotonicity (rewrite (= $x10074 $x11260)) (monotonicity @x11314 (= $x10470 (and $x10094 (and $x10095 (and $x10098 $x11306))))) (= $x10473 (and $x11260 (and $x10094 (and $x10095 (and $x10098 $x11306))))))))
+(let ((@x11326 (monotonicity (rewrite (= (<= 0 v_b_SL_H_witness$) $x11268)) (rewrite (= (<= v_b_SL_H_witness$ b_S_max_o_u4$) $x11270)) (= $x10071 (and $x11268 $x11270)))))
+(let ((@x11329 (monotonicity @x11326 (monotonicity (rewrite (= $x10073 $x11264)) @x11320 $x11322) (= $x10479 $x11327))))
+(let ((@x11332 (monotonicity (rewrite (= (<= 0 v_b_L_H_p$) $x11276)) (rewrite (= (<= v_b_L_H_p$ b_S_max_o_u4$) $x11278)) (= $x10067 (and $x11276 $x11278)))))
+(let ((@x11338 (monotonicity (rewrite (= (<= 0 v_b_L_H_max$) $x11284)) (rewrite (= (<= v_b_L_H_max$ b_S_max_o_u1$) $x11286)) (= $x10063 (and $x11284 $x11286)))))
+(let ((@x11341 (monotonicity @x11338 (monotonicity @x11332 @x11329 (= $x10482 (and (and $x11276 $x11278) $x11327))) (= $x10485 (and (and $x11284 $x11286) (and (and $x11276 $x11278) $x11327))))))
+(let ((@x11349 (monotonicity (trans @x11341 @x11344 (= $x10485 $x11342)) (= (not $x10485) (not $x11342)))))
+(let ((@x12026 (monotonicity @x11349 (monotonicity @x12020 (= $x11227 $x12021)) (= $x11234 (or (not $x11342) $x12021)))))
+(let ((@x10656 (monotonicity (rewrite (= (=> $x10242 true) true)) (= $x10244 (and $x10242 true)))))
+(let ((@x10663 (monotonicity (quant-intro (rewrite (= (=> $x10234 $x10235) $x10646)) (= $x10237 $x10649)) (trans @x10656 (rewrite (= (and $x10242 true) $x10242)) (= $x10244 $x10242)) (= $x10245 (=> $x10649 $x10242)))))
+(let ((@x10672 (monotonicity (quant-intro (rewrite (= (=> $x10234 $x10235) $x10646)) (= $x10237 $x10649)) (trans @x10663 (rewrite (= (=> $x10649 $x10242) $x10665)) (= $x10245 $x10665)) (= (and $x10237 $x10245) $x10670))))
+(let (($x10614 (= (and $x10218 (and $x10220 (and $x10222 true))) (and $x10218 (and $x10220 $x10222)))))
+(let ((@x10612 (monotonicity (rewrite (= (and $x10222 true) $x10222)) (= (and $x10220 (and $x10222 true)) (and $x10220 $x10222)))))
+(let ((@x10618 (monotonicity (monotonicity @x10612 $x10614) (= (and $x10216 (and $x10218 (and $x10220 (and $x10222 true)))) $x10616))))
+(let ((@x10625 (trans (monotonicity @x10618 (= $x10227 (and true $x10616))) (rewrite (= (and true $x10616) $x10616)) (= $x10227 $x10616))))
+(let ((@x10631 (monotonicity (monotonicity @x10625 (= (and $x10182 $x10227) $x10626)) (= (and $x10182 (and $x10182 $x10227)) $x10629))))
+(let ((@x10638 (trans (monotonicity @x10631 (= $x10230 (and true $x10629))) (rewrite (= (and true $x10629) $x10629)) (= $x10230 $x10629))))
+(let ((@x10644 (monotonicity (monotonicity @x10638 (= (and $x10182 $x10230) $x10639)) (= (and b_S_position_n_marker$ (and $x10182 $x10230)) $x10642))))
+(let ((@x10681 (trans (monotonicity @x10644 @x10672 (= $x10247 (=> $x10642 $x10670))) (rewrite (= (=> $x10642 $x10670) $x10677)) (= $x10247 $x10677))))
+(let (($x11117 (and $x10410 $x10182)))
+(let (($x11120 (and $x10182 $x11117)))
+(let ((@x10568 (rewrite (= (and $x10182 $x10182) $x10182))))
+(let ((@x10563 (rewrite (= $x10206 $x10182))))
+(let ((@x10570 (trans (monotonicity @x10563 (= $x10207 (and $x10182 $x10182))) @x10568 (= $x10207 $x10182))))
+(let ((@x11108 (trans (monotonicity @x10570 (= $x10411 (and $x10182 $x10182))) @x10568 (= $x10411 $x10182))))
+(let ((@x11114 (monotonicity (trans (monotonicity @x11108 (= $x10412 $x10206)) @x10563 (= $x10412 $x10182)) (= $x10413 (and $x10182 $x10182)))))
+(let ((@x11119 (monotonicity (trans @x11114 @x10568 (= $x10413 $x10182)) (= (and $x10410 $x10413) $x11117))))
+(let ((@x11125 (monotonicity (monotonicity @x11119 (= (and $x10182 (and $x10410 $x10413)) $x11120)) (= $x10416 (and true $x11120)))))
+(let ((@x11132 (monotonicity (trans @x11125 (rewrite (= (and true $x11120) $x11120)) (= $x10416 $x11120)) (monotonicity @x10681 (= $x10248 $x10682)) (= $x10417 (=> $x11120 $x10682)))))
+(let ((@x10938 (monotonicity (rewrite (= (and $x10375 false) false)) (= $x10377 (=> false true)))))
+(let ((@x10942 (trans @x10938 (rewrite (= (=> false true) true)) (= $x10377 true))))
+(let ((@x10949 (trans (monotonicity @x10942 (= $x10378 (and $x10375 true))) (rewrite (= (and $x10375 true) $x10375)) (= $x10378 $x10375))))
+(let ((@x10933 (quant-intro (rewrite (= (=> (and $x3098 (< ?0 v_b_L_H_p_G_1$)) $x10368) $x10928)) (= $x10370 $x10931))))
+(let ((@x10958 (trans (monotonicity @x10933 @x10949 (= $x10379 (=> $x10931 $x10375))) (rewrite (= (=> $x10931 $x10375) $x10954)) (= $x10379 $x10954))))
+(let ((@x10964 (monotonicity (monotonicity @x10933 @x10958 (= (and $x10370 $x10379) $x10959)) (= $x10381 (=> $x10365 $x10959)))))
+(let ((@x10973 (monotonicity (trans @x10964 (rewrite (= (=> $x10365 $x10959) $x10966)) (= $x10381 $x10966)) (= (and $x10365 $x10381) $x10971))))
+(let ((@x10920 (monotonicity (rewrite (= (and $x10360 true) $x10360)) (= (and $x10358 (and $x10360 true)) $x10918))))
+(let ((@x10903 (rewrite (= (+ v_b_L_H_p_G_0$ 1) ?x10901))))
+(let ((@x10915 (monotonicity @x10903 (= (= v_b_L_H_p_G_1$ (+ v_b_L_H_p_G_0$ 1)) $x10913))))
+(let ((@x10909 (monotonicity @x10903 (= (<= (+ v_b_L_H_p_G_0$ 1) b_S_max_o_u4$) $x10907))))
+(let ((@x10912 (monotonicity (monotonicity @x10903 (= (<= 0 (+ v_b_L_H_p_G_0$ 1)) $x10904)) @x10909 (= $x10355 $x10910))))
+(let ((@x10926 (monotonicity @x10912 (monotonicity @x10915 @x10920 (= $x10363 $x10921)) (= (and $x10355 $x10363) $x10924))))
+(let ((@x10982 (trans (monotonicity @x10926 @x10973 (= $x10383 (=> $x10924 $x10971))) (rewrite (= (=> $x10924 $x10971) $x10978)) (= $x10383 $x10978))))
+(let ((@x11021 (monotonicity (rewrite (= (and true $x10342) $x10342)) (= (and $x10392 (and true $x10342)) $x11019))))
+(let ((@x11024 (monotonicity @x11021 (= (and $x10391 (and $x10392 (and true $x10342))) $x11022))))
+(let ((@x11031 (trans (monotonicity @x11024 (= $x10395 (and true $x11022))) (rewrite (= (and true $x11022) $x11022)) (= $x10395 $x11022))))
+(let ((@x11037 (monotonicity (monotonicity @x11031 (= (and $x10182 $x10395) $x11032)) (= (and $x10182 (and $x10182 $x10395)) $x11035))))
+(let ((@x11044 (trans (monotonicity @x11037 (= $x10398 (and true $x11035))) (rewrite (= (and true $x11035) $x11035)) (= $x10398 $x11035))))
+(let ((@x11050 (monotonicity (monotonicity @x11044 (= (and $x10182 $x10398) $x11045)) (= (and $x10390 (and $x10182 $x10398)) $x11048))))
+(let ((@x11056 (monotonicity (monotonicity @x11050 (= (and $x10182 (and $x10390 (and $x10182 $x10398))) $x11051)) (= $x10402 (and true $x11051)))))
+(let ((@x11063 (monotonicity (trans @x11056 (rewrite (= (and true $x11051) $x11051)) (= $x10402 $x11051)) (monotonicity @x10912 @x10982 (= $x10384 $x10983)) (= $x10403 (=> $x11051 $x10983)))))
+(let (($x10896 (= (and $x10333 (and $x10334 (and $x10335 (and (and $x10181 $x10181) $x10346)))) $x10895)))
+(let ((@x10875 (monotonicity (rewrite (= (and true $x10342) $x10342)) (= (and $x10340 (and true $x10342)) $x10873))))
+(let ((@x10878 (monotonicity @x10875 (= (and $x10338 (and $x10340 (and true $x10342))) $x10876))))
+(let ((@x10885 (trans (monotonicity @x10878 (= $x10346 (and true $x10876))) (rewrite (= (and true $x10876) $x10876)) (= $x10346 $x10876))))
+(let ((@x10888 (monotonicity (rewrite (= (and $x10181 $x10181) $x10181)) @x10885 (= (and (and $x10181 $x10181) $x10346) $x10886))))
+(let ((@x10894 (monotonicity (monotonicity @x10888 (= (and $x10335 (and (and $x10181 $x10181) $x10346)) $x10889)) (= (and $x10334 (and $x10335 (and (and $x10181 $x10181) $x10346))) $x10892))))
+(let ((@x10988 (monotonicity (monotonicity (monotonicity @x10894 $x10896) (= $x10351 $x10898)) (monotonicity @x10912 @x10982 (= $x10384 $x10983)) (= $x10385 (=> $x10898 $x10983)))))
+(let ((@x10997 (monotonicity (trans @x10988 (rewrite (= (=> $x10898 $x10983) $x10990)) (= $x10385 $x10990)) (= (and $x10325 $x10385) $x10995))))
+(let ((@x11006 (trans (monotonicity @x10997 (= $x10387 (=> $x10323 $x10995))) (rewrite (= (=> $x10323 $x10995) $x11002)) (= $x10387 $x11002))))
+(let ((@x10861 (monotonicity (monotonicity @x10570 (= (and $x10328 $x10207) $x10856)) (= (and $x10182 (and $x10328 $x10207)) $x10859))))
+(let ((@x10868 (trans (monotonicity @x10861 (= $x10331 (and true $x10859))) (rewrite (= (and true $x10859) $x10859)) (= $x10331 $x10859))))
+(let ((@x11012 (monotonicity @x10868 (monotonicity @x11006 (= (and $x10323 $x10387) $x11007)) (= $x10389 (=> $x10859 $x11007)))))
+(let ((@x11072 (monotonicity (trans @x11012 (rewrite (= (=> $x10859 $x11007) $x11014)) (= $x10389 $x11014)) (trans @x11063 (rewrite (= (=> $x11051 $x10983) $x11065)) (= $x10403 $x11065)) (= (and $x10389 $x10403) $x11070))))
+(let ((@x11081 (trans (monotonicity @x11072 (= $x10405 (=> $x10326 $x11070))) (rewrite (= (=> $x10326 $x11070) $x11077)) (= $x10405 $x11077))))
+(let ((@x11087 (monotonicity (monotonicity @x11081 (= (and $x10325 $x10405) $x11082)) (= $x10407 (=> $x10323 $x11082)))))
+(let ((@x11095 (monotonicity (trans @x11087 (rewrite (= (=> $x10323 $x11082) $x11088)) (= $x10407 $x11088)) (= (and $x10323 $x10407) $x11093))))
+(let ((@x10848 (monotonicity (monotonicity @x10570 (= (and $x10316 $x10207) $x10843)) (= (and $x10182 (and $x10316 $x10207)) $x10846))))
+(let ((@x10855 (trans (monotonicity @x10848 (= $x10319 (and true $x10846))) (rewrite (= (and true $x10846) $x10846)) (= $x10319 $x10846))))
+(let ((@x11104 (trans (monotonicity @x10855 @x11095 (= $x10409 (=> $x10846 $x11093))) (rewrite (= (=> $x10846 $x11093) $x11100)) (= $x10409 $x11100))))
+(let ((@x11141 (monotonicity @x11104 (trans @x11132 (rewrite (= (=> $x11120 $x10682) $x11134)) (= $x10417 $x11134)) (= (and $x10409 $x10417) $x11139))))
+(let (($x10802 (= (and $x10291 (and $x10292 (and $x10293 (and $x10294 (and $x10297 $x10301))))) $x10801)))
+(let ((@x10777 (rewrite (= (= (b_S_statusmap$ v_b_S_s$) (b_S_statusmap$ v_b_S_s$)) true))))
+(let ((@x10780 (monotonicity (rewrite (= (= ?x10272 ?x10272) true)) @x10777 (= $x10300 (and true true)))))
+(let ((@x10784 (trans @x10780 (rewrite (= (and true true) true)) (= $x10300 true))))
+(let ((@x10791 (monotonicity (trans (monotonicity @x10784 (= $x10301 $x10206)) @x10563 (= $x10301 $x10182)) (= (and $x10297 $x10301) $x10789))))
+(let ((@x10797 (monotonicity (monotonicity @x10791 (= (and $x10294 (and $x10297 $x10301)) $x10792)) (= (and $x10293 (and $x10294 (and $x10297 $x10301))) $x10795))))
+(let ((@x10800 (monotonicity @x10797 (= (and $x10292 (and $x10293 (and $x10294 (and $x10297 $x10301)))) $x10798))))
+(let ((@x10809 (monotonicity (monotonicity (monotonicity @x10800 $x10802) (= $x10307 $x10804)) (= (and $x10286 $x10307) $x10807))))
+(let ((@x10759 (rewrite (= (and true $x10286) $x10286))))
+(let (($x10748 (forall ((?v0 B_S_ptr$) )(!true :pattern ( (b_S_select_o_tm$ (b_S_typemap$ v_b_S_s$) ?v0) )))
+))
+(let (($x10260 (b_S_thread_n_local$ v_b_S_s$ ?0)))
+(let (($x10275 (and (= (b_S_select_o_tm$ ?x10272 ?0) (b_S_select_o_tm$ ?x10272 ?0)) $x10260)))
+(let (($x10276 (=> $x10260 $x10275)))
+(let ((@x10714 (rewrite (= (=> $x10260 $x10260) true))))
+(let ((@x10707 (rewrite (= (and true $x10260) $x10260))))
+(let (($x10738 (= (= (b_S_select_o_tm$ ?x10272 ?0) (b_S_select_o_tm$ ?x10272 ?0)) true)))
+(let ((@x10743 (trans (monotonicity (rewrite $x10738) (= $x10275 (and true $x10260))) @x10707 (= $x10275 $x10260))))
+(let ((@x10747 (trans (monotonicity @x10743 (= $x10276 (=> $x10260 $x10260))) @x10714 (= $x10276 true))))
+(let ((@x10754 (trans (quant-intro @x10747 (= $x10278 $x10748)) (elim-unused (= $x10748 true)) (= $x10278 true))))
+(let ((@x10761 (trans (monotonicity @x10754 (= $x10287 (and true $x10286))) @x10759 (= $x10287 $x10286))))
+(let (($x10694 (forall ((?v0 B_S_ptr$) )(!true :pattern ( (b_S_select_o_sm$ (b_S_statusmap$ v_b_S_s$) ?v0) )))
+))
+(let ((?x10256 (b_S_statusmap$ v_b_S_s$)))
+(let ((?x10257 (b_S_select_o_sm$ ?x10256 ?0)))
+(let (($x10269 (and (= ?x10257 ?x10257) $x10260)))
+(let (($x10270 (=> $x10260 $x10269)))
+(let ((@x10727 (monotonicity (rewrite (= (= ?x10257 ?x10257) true)) (= $x10269 (and true $x10260)))))
+(let ((@x10731 (monotonicity (trans @x10727 @x10707 (= $x10269 $x10260)) (= $x10270 (=> $x10260 $x10260)))))
+(let ((@x10737 (trans (quant-intro (trans @x10731 @x10714 (= $x10270 true)) (= $x10271 $x10694)) (elim-unused (= $x10694 true)) (= $x10271 true))))
+(let ((@x10765 (trans (monotonicity @x10737 @x10761 (= $x10288 (and true $x10286))) @x10759 (= $x10288 $x10286))))
+(let (($x10717 (forall ((?v0 B_S_ptr$) )(!true :pattern ( (b_S_select_o_mem$ (b_S_memory$ v_b_S_s$) ?v0) )))
+))
+(let ((?x10261 (b_S_memory$ v_b_S_s$)))
+(let ((?x10262 (b_S_select_o_mem$ ?x10261 ?0)))
+(let (($x10264 (and (= ?x10262 ?x10262) $x10260)))
+(let (($x10265 (=> $x10260 $x10264)))
+(let ((@x10705 (monotonicity (rewrite (= (= ?x10262 ?x10262) true)) (= $x10264 (and true $x10260)))))
+(let ((@x10712 (monotonicity (trans @x10705 @x10707 (= $x10264 $x10260)) (= $x10265 (=> $x10260 $x10260)))))
+(let ((@x10723 (trans (quant-intro (trans @x10712 @x10714 (= $x10265 true)) (= $x10267 $x10717)) (elim-unused (= $x10717 true)) (= $x10267 true))))
+(let ((@x10769 (trans (monotonicity @x10723 @x10765 (= $x10289 (and true $x10286))) @x10759 (= $x10289 $x10286))))
+(let (($x10253 (= (b_S_kind_n_of$ (b_S_typ$ (b_S_owner$ v_b_S_s$ ?0))) b_S_kind_n_thread$)))
+(let ((@x10696 (quant-intro (rewrite (= (=> (not $x10253) (not $x10253)) true)) (= $x10259 $x10694))))
+(let ((@x10771 (monotonicity (trans @x10696 (elim-unused (= $x10694 true)) (= $x10259 true)) @x10769 (= $x10290 (and true $x10286)))))
+(let ((@x10812 (monotonicity (trans @x10771 @x10759 (= $x10290 $x10286)) @x10809 (= (and $x10290 (and $x10286 $x10307)) $x10810))))
+(let ((@x10818 (monotonicity (monotonicity @x10812 (= (and $x10182 (and $x10290 (and $x10286 $x10307))) $x10813)) (= $x10311 (and true $x10813)))))
+(let ((@x10825 (monotonicity (trans @x10818 (rewrite (= (and true $x10813) $x10813)) (= $x10311 $x10813)) (= (and $x10182 $x10311) $x10823))))
+(let ((@x10832 (trans (monotonicity @x10825 (= $x10313 (and true $x10823))) (rewrite (= (and true $x10823) $x10823)) (= $x10313 $x10823))))
+(let ((@x10838 (monotonicity (monotonicity @x10832 (= (and $x10182 $x10313) $x10833)) (= $x10315 (and true $x10833)))))
+(let ((@x11144 (monotonicity (trans @x10838 (rewrite (= (and true $x10833) $x10833)) (= $x10315 $x10833)) @x11141 (= $x10419 (=> $x10833 $x11139)))))
+(let ((@x10591 (rewrite (= (and false (and $x10182 (and $x10182 (and $x10205 $x10182)))) false))))
+(let (($x10585 (= (and $x10182 (and true (and $x10182 (and $x10205 $x10207)))) (and $x10182 (and $x10182 (and $x10205 $x10182))))))
+(let (($x10574 (and $x10182 (and $x10205 $x10182))))
+(let (($x10210 (and true (and $x10182 (and $x10205 $x10207)))))
+(let ((@x10576 (monotonicity (monotonicity @x10570 (= (and $x10205 $x10207) (and $x10205 $x10182))) (= (and $x10182 (and $x10205 $x10207)) $x10574))))
+(let ((@x10583 (trans (monotonicity @x10576 (= $x10210 (and true $x10574))) (rewrite (= (and true $x10574) $x10574)) (= $x10210 $x10574))))
+(let ((@x10561 (rewrite (= $x10203 false))))
+(let ((@x10589 (monotonicity @x10561 (monotonicity @x10583 $x10585) (= $x10212 (and false (and $x10182 $x10574))))))
+(let ((@x10596 (monotonicity (trans @x10589 @x10591 (= $x10212 false)) (= $x10213 (and $x10182 false)))))
+(let ((@x10600 (trans @x10596 (rewrite (= (and $x10182 false) false)) (= $x10213 false))))
+(let ((@x10607 (trans (monotonicity @x10600 (= $x10214 (and true false))) (rewrite (= (and true false) false)) (= $x10214 false))))
+(let ((@x10687 (monotonicity @x10607 (monotonicity @x10681 (= $x10248 $x10682)) (= $x10249 (=> false $x10682)))))
+(let ((@x10691 (trans @x10687 (rewrite (= (=> false $x10682) true)) (= $x10249 true))))
+(let ((@x11153 (monotonicity @x10691 (trans @x11144 (rewrite (= (=> $x10833 $x11139) $x11146)) (= $x10419 $x11146)) (= $x10420 (and true $x11146)))))
+(let (($x10545 (= (and $x10176 (and $x10180 (and $x10182 (and $x10183 (and $x10188 $x10194))))) $x10544)))
+(let ((@x10531 (quant-intro (rewrite (= (=> (and $x3098 (< ?0 v_b_L_H_p_G_0$)) $x10186) $x10526)) (= $x10188 $x10529))))
+(let ((@x10537 (monotonicity (monotonicity @x10531 (= (and $x10188 $x10194) $x10532)) (= (and $x10183 (and $x10188 $x10194)) $x10535))))
+(let ((@x10543 (monotonicity (monotonicity @x10537 (= (and $x10182 (and $x10183 (and $x10188 $x10194))) $x10538)) (= (and $x10180 (and $x10182 (and $x10183 (and $x10188 $x10194)))) $x10541))))
+(let ((@x10552 (monotonicity (monotonicity (monotonicity @x10543 $x10545) (= $x10200 $x10547)) (= $x10201 (and true $x10547)))))
+(let ((@x10559 (monotonicity (trans @x10552 (rewrite (= (and true $x10547) $x10547)) (= $x10201 $x10547)) (= (and $x10168 $x10201) $x10557))))
+(let ((@x11160 (monotonicity @x10559 (trans @x11153 (rewrite (= (and true $x11146) $x11146)) (= $x10420 $x11146)) (= $x10421 (=> $x10557 $x11146)))))
+(let ((@x11169 (monotonicity (trans @x11160 (rewrite (= (=> $x10557 $x11146) $x11162)) (= $x10421 $x11162)) (= (and $x10168 $x10421) $x11167))))
+(let ((@x10524 (quant-intro (rewrite (= (=> (and $x3098 (< ?0 1)) $x10164) $x10519)) (= $x10166 $x10522))))
+(let ((@x11178 (trans (monotonicity @x10524 @x11169 (= $x10423 (=> $x10522 $x11167))) (rewrite (= (=> $x10522 $x11167) $x11174)) (= $x10423 $x11174))))
+(let ((@x11184 (monotonicity (monotonicity @x10524 @x11178 (= (and $x10166 $x10423) $x11179)) (= $x10425 (=> $x10159 $x11179)))))
+(let ((@x11193 (monotonicity (trans @x11184 (rewrite (= (=> $x10159 $x11179) $x11186)) (= $x10425 $x11186)) (= (and $x10159 $x10425) $x11191))))
+(let ((@x10499 (monotonicity (rewrite (= (and $x10150 $x10150) $x10150)) (= (and $x10149 (and $x10150 $x10150)) $x10497))))
+(let ((@x10505 (monotonicity (monotonicity @x10499 (= (and $x10149 (and $x10149 (and $x10150 $x10150))) $x10500)) (= $x10154 $x10503))))
+(let ((@x10511 (monotonicity (monotonicity @x10505 (= (and $x10147 $x10154) $x10506)) (= (and $x10146 (and $x10147 $x10154)) $x10509))))
+(let ((@x10517 (monotonicity (monotonicity @x10511 (= (and $x10145 (and $x10146 (and $x10147 $x10154))) $x10512)) (= (and $x10142 (and $x10145 (and $x10146 (and $x10147 $x10154)))) $x10515))))
+(let ((@x11202 (trans (monotonicity @x10517 @x11193 (= $x10427 (=> $x10515 $x11191))) (rewrite (= (=> $x10515 $x11191) $x11198)) (= $x10427 $x11198))))
+(let ((@x11208 (monotonicity (monotonicity @x11202 (= (and $x10142 $x10427) $x11203)) (= $x10429 (=> $x10140 $x11203)))))
+(let ((@x11217 (monotonicity (trans @x11208 (rewrite (= (=> $x10140 $x11203) $x11210)) (= $x10429 $x11210)) (= (and $x10140 $x10429) $x11215))))
+(let ((@x11226 (trans (monotonicity @x11217 (= $x10431 (=> $x10136 $x11215))) (rewrite (= (=> $x10136 $x11215) $x11222)) (= $x10431 $x11222))))
+(let (($x10483 (= (and $x10067 (and $x10071 (and $x10073 (and $x10074 (and $x10094 $x10127))))) $x10482)))
+(let (($x10455 (= (and $x10104 (and $x10108 (and $x10109 (and $x10112 (and $x10116 $x10119))))) $x10454)))
+(let (($x10113 (b_S_in_n_writes_n_at$ v_b_H_wrTime_S_1_T_6_o_1$ ?0)))
+(let (($x10436 (not $x10113)))
+(let ((@x10444 (monotonicity (quant-intro (rewrite (= (= $x10113 false) $x10436)) (= $x10116 $x10439)) (= (and $x10116 $x10119) $x10442))))
+(let ((@x10450 (monotonicity (monotonicity @x10444 (= (and $x10112 (and $x10116 $x10119)) $x10445)) (= (and $x10109 (and $x10112 (and $x10116 $x10119))) $x10448))))
+(let ((@x10453 (monotonicity @x10450 (= (and $x10108 (and $x10109 (and $x10112 (and $x10116 $x10119)))) $x10451))))
+(let ((@x10462 (monotonicity (monotonicity (monotonicity @x10453 $x10455) (= $x10125 $x10457)) (= (and $x10095 $x10125) $x10460))))
+(let ((@x10469 (trans (monotonicity @x10462 (= $x10127 (and true $x10460))) (rewrite (= (and true $x10460) $x10460)) (= $x10127 $x10460))))
+(let ((@x10475 (monotonicity (monotonicity @x10469 (= (and $x10094 $x10127) $x10470)) (= (and $x10074 (and $x10094 $x10127)) $x10473))))
+(let ((@x10481 (monotonicity (monotonicity @x10475 (= (and $x10073 (and $x10074 (and $x10094 $x10127))) $x10476)) (= (and $x10071 (and $x10073 (and $x10074 (and $x10094 $x10127)))) $x10479))))
+(let ((@x10490 (monotonicity (monotonicity (monotonicity @x10481 $x10483) (= $x10133 $x10485)) (= $x10134 (and true $x10485)))))
+(let ((@x11232 (monotonicity (trans @x10490 (rewrite (= (and true $x10485) $x10485)) (= $x10134 $x10485)) (monotonicity @x11226 (= (and $x10136 $x10431) $x11227)) (= $x10433 (=> $x10485 $x11227)))))
+(let ((@x11241 (monotonicity (trans @x11232 (rewrite (= (=> $x10485 $x11227) $x11234)) (= $x10433 $x11234)) (= $x10434 (not $x11234)))))
+(let ((@x12031 (trans @x11241 (monotonicity @x12026 (= (not $x11234) $x12027)) (= $x10434 $x12027))))
+(let ((@x12033 (not-or-elim (mp (asserted $x10434) @x12031 $x12027) $x11342)))
+(let ((@x12044 (and-elim @x12033 $x10084)))
+(let (($x21982 (not $x10084)))
+(let (($x21995 (or $x21994 $x21982 $x21990)))
+(let ((@x22000 (mp ((_ quant-inst (b_S_ptr$ ?x10076 ?x10079) (b_S_array$ b_T_T_u1$ v_b_P_H_len$)) (or $x21994 (or $x21982 $x21990))) (rewrite (= (or $x21994 (or $x21982 $x21990)) $x21995)) $x21995)))
+(let ((@x24520 (symm (unit-resolution @x22000 @x15336 @x12044 $x21990) (= ?x21983 ?x10080))))
+(let ((@x22795 (monotonicity (trans @x24520 (symm @x24530 (= ?x10080 ?x22595)) (= ?x21983 ?x22595)) (= (b_S_set_n_in$ ?x21983 ?x22343) $x22596))))
+(let (($x22344 (b_S_set_n_in$ ?x21983 ?x22343)))
+(let (($x22362 (forall ((?v3 B_S_ptr$) )(!(let ((?x10078 (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$)))
+(let ((?x10079 (b_S_ref$ ?x10078)))
+(let ((?x10076 (b_S_array$ b_T_T_u1$ v_b_P_H_len$)))
+(let ((?x10080 (b_S_ptr$ ?x10076 ?x10079)))
+(let ((?x21014 (b_S_ref$ ?x10080)))
+(let ((?x21983 (b_S_ptr$ ?x10076 ?x21014)))
+(let ((?x22357 (b_S_read_n_version$ v_b_S_s$ ?x21983)))
+(let ((?x22358 (b_S_ver_n_domain$ ?x22357)))
+(let ((?x22234 (b_S_typ$ ?x21983)))
+(let (($x22353 (b_S_has_n_volatile_n_owns_n_set$ ?x22234)))
+(or $x22353 (not (b_S_set_n_in$ ?v3 (b_S_owns$ v_b_S_s$ ?x21983))) (b_S_set_n_in2$ ?v3 ?x22358)))))))))))) :pattern ( (b_S_set_n_in$ ?v3 (b_S_owns$ v_b_S_s$ (b_S_ptr$ (b_S_array$ b_T_T_u1$ v_b_P_H_len$) (b_S_ref$ (b_S_ptr$ (b_S_array$ b_T_T_u1$ v_b_P_H_len$) (b_S_ref$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$))))))) )))
+))
+(let (($x22363 (not $x22362)))
+(let (($x22248 (b_S_closed$ v_b_S_s$ ?x21983)))
+(let (($x22272 (not $x22248)))
+(let (($x22352 (not $x22344)))
+(let (($x22364 (or $x22352 $x22272 $x22363)))
+(let (($x22365 (not $x22364)))
+(let (($x22318 (b_S_in_n_domain$ v_b_S_s$ ?x21983 ?x21983)))
+(let (($x22317 (b_S_in_n_domain_n_lab$ v_b_S_s$ ?x21983 ?x21983 b_l_H_public$)))
+(let (($x22326 (= $x22317 $x22318)))
+(let (($x8728 (forall ((?v0 B_S_state$) (?v1 B_S_ptr$) (?v2 B_S_ptr$) (?v3 B_S_label$) )(!(let (($x8719 (b_S_in_n_domain$ ?v0 ?v1 ?v2)))
+(let (($x8718 (b_S_in_n_domain_n_lab$ ?v0 ?v1 ?v2 ?v3)))
+(= $x8718 $x8719))) :pattern ( (b_S_in_n_domain_n_lab$ ?v0 ?v1 ?v2 ?v3) )))
+))
+(let (($x8719 (b_S_in_n_domain$ ?3 ?2 ?1)))
+(let (($x8718 (b_S_in_n_domain_n_lab$ ?3 ?2 ?1 ?0)))
+(let (($x8725 (= $x8718 $x8719)))
+(let (($x8723 (forall ((?v0 B_S_state$) (?v1 B_S_ptr$) (?v2 B_S_ptr$) (?v3 B_S_label$) )(!(let (($x8719 (b_S_in_n_domain$ ?v0 ?v1 ?v2)))
+(let (($x8718 (b_S_in_n_domain_n_lab$ ?v0 ?v1 ?v2 ?v3)))
+(= $x8718 $x8719))) :pattern ( (b_S_in_n_domain_n_lab$ ?v0 ?v1 ?v2 ?v3) )))
+))
+(let ((@x8733 (mp (asserted $x8723) (quant-intro (rewrite (= (= $x8718 $x8719) $x8725)) (= $x8723 $x8728)) $x8728)))
+(let ((@x15021 (mp~ @x8733 (nnf-pos (refl (~ $x8725 $x8725)) (~ $x8728 $x8728)) $x8728)))
+(let (($x22612 (or (not $x8728) $x22326)))
+(let ((@x22613 ((_ quant-inst v_b_S_s$ (b_S_ptr$ ?x10076 ?x21014) (b_S_ptr$ ?x10076 ?x21014) b_l_H_public$) $x22612)))
+(let (($x35 (= b_S_kind_n_primitive$ b_S_kind_n_array$)))
+(let (($x36 (not $x35)))
+(let (($x22500 (= $x36 (not (= (b_S_kind_n_of$ (b_S_typ$ ?x21983)) b_S_kind_n_primitive$)))))
+(let ((?x22234 (b_S_typ$ ?x21983)))
+(let ((?x22387 (b_S_kind_n_of$ ?x22234)))
+(let (($x22388 (= ?x22387 b_S_kind_n_primitive$)))
+(let (($x22148 (= ?x10086 b_S_kind_n_array$)))
+(let (($x21115 (b_S_is_n_arraytype$ ?x10076)))
+(let (($x22149 (= $x21115 $x22148)))
+(let (($x9869 (forall ((?v0 B_S_ctype$) )(!(let ((?x9849 (b_S_kind_n_of$ ?v0)))
+(let (($x9861 (= ?x9849 b_S_kind_n_array$)))
+(let (($x7848 (b_S_is_n_arraytype$ ?v0)))
+(= $x7848 $x9861)))) :pattern ( (b_S_is_n_arraytype$ ?v0) )))
+))
+(let (($x9861 (= ?x9849 b_S_kind_n_array$)))
+(let (($x7848 (b_S_is_n_arraytype$ ?0)))
+(let (($x9866 (= $x7848 $x9861)))
+(let (($x9864 (forall ((?v0 B_S_ctype$) )(!(let ((?x9849 (b_S_kind_n_of$ ?v0)))
+(let (($x9861 (= ?x9849 b_S_kind_n_array$)))
+(let (($x7848 (b_S_is_n_arraytype$ ?v0)))
+(= $x7848 $x9861)))) :pattern ( (b_S_is_n_arraytype$ ?v0) )))
+))
+(let ((@x9874 (mp (asserted $x9864) (quant-intro (rewrite (= (= $x7848 $x9861) $x9866)) (= $x9864 $x9869)) $x9869)))
+(let ((@x15446 (mp~ @x9874 (nnf-pos (refl (~ $x9866 $x9866)) (~ $x9869 $x9869)) $x9869)))
+(let (($x22159 (or (not $x9869) $x22149)))
+(let ((@x22160 ((_ quant-inst (b_S_array$ b_T_T_u1$ v_b_P_H_len$)) $x22159)))
+(let (($x7229 (forall ((?v0 B_S_ctype$) (?v1 Int) )(!(let ((?x6561 (b_S_array$ ?v0 ?v1)))
+(b_S_is_n_arraytype$ ?x6561)) :pattern ( (b_S_array$ ?v0 ?v1) )))
+))
+(let ((?x6561 (b_S_array$ ?1 ?0)))
+(let (($x7228 (b_S_is_n_arraytype$ ?x6561)))
+(let ((@x14576 (mp~ (asserted $x7229) (nnf-pos (refl (~ $x7228 $x7228)) (~ $x7229 $x7229)) $x7229)))
+(let (($x21122 (or (not $x7229) $x21115)))
+(let ((@x21123 ((_ quant-inst b_T_T_u1$ v_b_P_H_len$) $x21122)))
+(let ((@x22406 (unit-resolution (def-axiom (or (not $x22149) (not $x21115) $x22148)) (unit-resolution @x21123 @x14576 $x21115) (or (not $x22149) $x22148))))
+(let ((?x21180 (b_S_typ$ ?x10080)))
+(let (($x21183 (= ?x21180 ?x10076)))
+(let (($x21188 (or $x21147 $x21183)))
+(let ((@x21189 ((_ quant-inst (b_S_array$ b_T_T_u1$ v_b_P_H_len$) (b_S_ref$ ?x10078)) $x21188)))
+(let ((@x22414 (trans (monotonicity @x24520 (= ?x22234 ?x21180)) (unit-resolution @x21189 @x19846 $x21183) (= ?x22234 ?x10076))))
+(let ((@x22418 (trans (monotonicity @x22414 (= ?x22387 ?x10086)) (unit-resolution @x22406 (unit-resolution @x22160 @x15446 $x22149) $x22148) (= ?x22387 b_S_kind_n_array$))))
+(let ((@x22857 (monotonicity @x22418 (= $x22388 (= b_S_kind_n_array$ b_S_kind_n_primitive$)))))
+(let ((@x22934 (trans @x22857 (commutativity (= (= b_S_kind_n_array$ b_S_kind_n_primitive$) $x35)) (= $x22388 $x35))))
+(let (($x41 (= b_S_kind_n_thread$ b_S_kind_n_array$)))
+(let (($x42 (not $x41)))
+(let (($x39 (= b_S_kind_n_composite$ b_S_kind_n_array$)))
+(let (($x40 (not $x39)))
+(let (($x37 (= b_S_kind_n_composite$ b_S_kind_n_thread$)))
+(let (($x38 (not $x37)))
+(let (($x32 (= b_S_kind_n_primitive$ b_S_kind_n_thread$)))
+(let (($x33 (not $x32)))
+(let (($x29 (= b_S_kind_n_primitive$ b_S_kind_n_composite$)))
+(let (($x30 (not $x29)))
+(let (($x67 (and $x30 $x33 $x36 $x38 $x40 $x42)))
+(let (($x48 (and $x30 (and $x33 (and $x36 (and $x38 (and $x40 (and $x42 true))))))))
+(let (($x68 (= (and $x30 (and $x33 (and $x36 (and $x38 (and $x40 $x42))))) $x67)))
+(let (($x65 (= $x48 (and $x30 (and $x33 (and $x36 (and $x38 (and $x40 $x42))))))))
+(let (($x62 (= (and $x33 (and $x36 (and $x38 (and $x40 (and $x42 true))))) (and $x33 (and $x36 (and $x38 (and $x40 $x42)))))))
+(let (($x59 (= (and $x36 (and $x38 (and $x40 (and $x42 true)))) (and $x36 (and $x38 (and $x40 $x42))))))
+(let (($x56 (= (and $x38 (and $x40 (and $x42 true))) (and $x38 (and $x40 $x42)))))
+(let ((@x54 (monotonicity (rewrite (= (and $x42 true) $x42)) (= (and $x40 (and $x42 true)) (and $x40 $x42)))))
+(let ((@x66 (monotonicity (monotonicity (monotonicity (monotonicity @x54 $x56) $x59) $x62) $x65)))
+(let ((@x72 (mp (asserted $x48) (trans @x66 (rewrite $x68) (= $x48 $x67)) $x67)))
+(let ((@x75 (and-elim @x72 $x36)))
+(let (($x22333 (not $x22318)))
+(let (($x22336 (not $x22317)))
+(let ((@x22935 (monotonicity (symm (monotonicity @x24520 @x24520 (= $x22317 $x10136)) (= $x10136 $x22317)) (= $x11221 $x22336))))
+(let ((@x22938 (unit-resolution (def-axiom (or (not $x22326) $x22317 $x22333)) (mp (hypothesis $x11221) @x22935 $x22336) (unit-resolution @x22613 @x15021 $x22326) $x22333)))
+(let (($x22368 (b_S_is$ ?x21983 ?x22234)))
+(let ((@x22898 (mp @x12044 (symm (monotonicity @x24520 @x22414 (= $x22368 $x10084)) (= $x10084 $x22368)) $x22368)))
+(let (($x22385 (b_S_typed$ v_b_S_s$ ?x21983)))
+(let ((@x12045 (and-elim @x12033 $x10085)))
+(let ((@x22886 (mp @x12045 (symm (monotonicity @x24520 (= $x22385 $x10085)) (= $x10085 $x22385)) $x22385)))
+(let ((?x22243 (b_S_owner$ v_b_S_s$ ?x21983)))
+(let (($x22259 (= ?x22243 b_S_me$)))
+(let ((@x12043 (and-elim @x12033 $x10083)))
+(let ((@x12042 (and-elim @x12033 $x10081)))
+(let ((@x22429 (mp @x12042 (symm (monotonicity @x24520 (= $x22248 $x10081)) (= $x10081 $x22248)) $x22248)))
+(let (($x22235 (b_S_is_n_non_n_primitive$ ?x22234)))
+(let ((@x12047 (and-elim @x12033 $x10089)))
+(let ((@x22409 (mp @x12047 (symm (monotonicity @x22414 (= $x22235 $x10089)) (= $x10089 $x22235)) $x22235)))
+(let ((@x12050 (and-elim @x12033 $x10097)))
+(let (($x18905 (forall ((?v0 B_S_state$) (?v1 B_S_ptr$) )(!(let (($x8613 (b_S_in_n_domain$ ?v0 ?v1 ?v1)))
+(let ((?x2247 (b_S_typ$ ?v1)))
+(let (($x2351 (b_S_is_n_non_n_primitive$ ?x2247)))
+(let (($x9239 (not $x2351)))
+(let (($x2249 (= (b_S_kind_n_of$ ?x2247) b_S_kind_n_primitive$)))
+(let (($x2488 (b_S_typed$ ?v0 ?v1)))
+(let (($x9531 (not $x2488)))
+(let (($x2487 (b_S_is$ ?v1 ?x2247)))
+(let (($x16299 (not $x2487)))
+(let ((?x2484 (b_S_owner$ ?v0 ?v1)))
+(let (($x2486 (= ?x2484 b_S_me$)))
+(let (($x16298 (not $x2486)))
+(let (($x2471 (b_S_closed$ ?v0 ?v1)))
+(let (($x9185 (not $x2471)))
+(let (($x2687 (b_S_full_n_stop$ ?v0)))
+(let (($x16426 (not $x2687)))
+(or $x16426 $x9185 $x16298 $x16299 $x9531 $x2249 $x9239 $x8613))))))))))))))))) :pattern ( (b_S_in_n_domain$ ?v0 ?v1 ?v1) )))
+))
+(let (($x8634 (forall ((?v0 B_S_state$) (?v1 B_S_ptr$) )(!(let (($x8613 (b_S_in_n_domain$ ?v0 ?v1 ?v1)))
+(let ((?x2247 (b_S_typ$ ?v1)))
+(let (($x2351 (b_S_is_n_non_n_primitive$ ?x2247)))
+(let (($x2249 (= (b_S_kind_n_of$ ?x2247) b_S_kind_n_primitive$)))
+(let (($x2294 (not $x2249)))
+(let (($x2488 (b_S_typed$ ?v0 ?v1)))
+(let (($x2487 (b_S_is$ ?v1 ?x2247)))
+(let ((?x2484 (b_S_owner$ ?v0 ?v1)))
+(let (($x2486 (= ?x2484 b_S_me$)))
+(let (($x2471 (b_S_closed$ ?v0 ?v1)))
+(let (($x2687 (b_S_full_n_stop$ ?v0)))
+(let (($x8625 (and $x2687 $x2471 $x2486 $x2487 $x2488 $x2294 $x2351)))
+(let (($x8628 (not $x8625)))
+(or $x8628 $x8613)))))))))))))) :pattern ( (b_S_in_n_domain$ ?v0 ?v1 ?v1) )))
+))
+(let (($x8613 (b_S_in_n_domain$ ?1 ?0 ?0)))
+(let ((?x2247 (b_S_typ$ ?0)))
+(let (($x2351 (b_S_is_n_non_n_primitive$ ?x2247)))
+(let (($x9239 (not $x2351)))
+(let (($x2249 (= (b_S_kind_n_of$ ?x2247) b_S_kind_n_primitive$)))
+(let (($x2488 (b_S_typed$ ?1 ?0)))
+(let (($x9531 (not $x2488)))
+(let (($x2487 (b_S_is$ ?0 ?x2247)))
+(let (($x16299 (not $x2487)))
+(let ((?x2484 (b_S_owner$ ?1 ?0)))
+(let (($x2486 (= ?x2484 b_S_me$)))
+(let (($x16298 (not $x2486)))
+(let (($x2471 (b_S_closed$ ?1 ?0)))
+(let (($x9185 (not $x2471)))
+(let (($x2687 (b_S_full_n_stop$ ?1)))
+(let (($x16426 (not $x2687)))
+(let (($x18900 (or $x16426 $x9185 $x16298 $x16299 $x9531 $x2249 $x9239 $x8613)))
+(let (($x2294 (not $x2249)))
+(let (($x8625 (and $x2687 $x2471 $x2486 $x2487 $x2488 $x2294 $x2351)))
+(let (($x8628 (not $x8625)))
+(let (($x8631 (or $x8628 $x8613)))
+(let ((@x18902 (rewrite (= (or (or $x16426 $x9185 $x16298 $x16299 $x9531 $x2249 $x9239) $x8613) $x18900))))
+(let (($x18886 (or $x16426 $x9185 $x16298 $x16299 $x9531 $x2249 $x9239)))
+(let ((@x18892 (monotonicity (rewrite (= $x8625 (not $x18886))) (= $x8628 (not (not $x18886))))))
+(let ((@x18899 (monotonicity (trans @x18892 (rewrite (= (not (not $x18886)) $x18886)) (= $x8628 $x18886)) (= $x8631 (or $x18886 $x8613)))))
+(let (($x8616 (forall ((?v0 B_S_state$) (?v1 B_S_ptr$) )(!(let (($x8613 (b_S_in_n_domain$ ?v0 ?v1 ?v1)))
+(let ((?x2247 (b_S_typ$ ?v1)))
+(let (($x2351 (b_S_is_n_non_n_primitive$ ?x2247)))
+(let (($x2249 (= (b_S_kind_n_of$ ?x2247) b_S_kind_n_primitive$)))
+(let (($x2294 (not $x2249)))
+(let (($x2488 (b_S_typed$ ?v0 ?v1)))
+(let (($x2487 (b_S_is$ ?v1 ?x2247)))
+(let ((?x2484 (b_S_owner$ ?v0 ?v1)))
+(let (($x2486 (= ?x2484 b_S_me$)))
+(let (($x2471 (b_S_closed$ ?v0 ?v1)))
+(let (($x2687 (b_S_full_n_stop$ ?v0)))
+(let (($x8612 (and $x2687 (and $x2471 (and $x2486 (and $x2487 (and $x2488 (and $x2294 $x2351))))))))
+(=> $x8612 $x8613))))))))))))) :pattern ( (b_S_in_n_domain$ ?v0 ?v1 ?v1) )))
+))
+(let (($x8622 (forall ((?v0 B_S_state$) (?v1 B_S_ptr$) )(!(let (($x8613 (b_S_in_n_domain$ ?v0 ?v1 ?v1)))
+(let ((?x2247 (b_S_typ$ ?v1)))
+(let (($x2351 (b_S_is_n_non_n_primitive$ ?x2247)))
+(let (($x2249 (= (b_S_kind_n_of$ ?x2247) b_S_kind_n_primitive$)))
+(let (($x2294 (not $x2249)))
+(let (($x2488 (b_S_typed$ ?v0 ?v1)))
+(let (($x2487 (b_S_is$ ?v1 ?x2247)))
+(let ((?x2484 (b_S_owner$ ?v0 ?v1)))
+(let (($x2486 (= ?x2484 b_S_me$)))
+(let (($x2471 (b_S_closed$ ?v0 ?v1)))
+(let (($x2687 (b_S_full_n_stop$ ?v0)))
+(let (($x8612 (and $x2687 (and $x2471 (and $x2486 (and $x2487 (and $x2488 (and $x2294 $x2351))))))))
+(or (not $x8612) $x8613))))))))))))) :pattern ( (b_S_in_n_domain$ ?v0 ?v1 ?v1) )))
+))
+(let (($x8612 (and $x2687 (and $x2471 (and $x2486 (and $x2487 (and $x2488 (and $x2294 $x2351))))))))
+(let (($x8619 (or (not $x8612) $x8613)))
+(let ((@x8633 (monotonicity (monotonicity (rewrite (= $x8612 $x8625)) (= (not $x8612) $x8628)) (= $x8619 $x8631))))
+(let ((@x8638 (trans (quant-intro (rewrite (= (=> $x8612 $x8613) $x8619)) (= $x8616 $x8622)) (quant-intro @x8633 (= $x8622 $x8634)) (= $x8616 $x8634))))
+(let ((@x14989 (mp~ (mp (asserted $x8616) @x8638 $x8634) (nnf-pos (refl (~ $x8631 $x8631)) (~ $x8634 $x8634)) $x8634)))
+(let ((@x18908 (mp @x14989 (quant-intro (trans @x18899 @x18902 (= $x8631 $x18900)) (= $x8634 $x18905)) $x18905)))
+(let (($x22242 (not $x22235)))
+(let (($x22386 (not $x22385)))
+(let (($x22384 (not $x22368)))
+(let (($x24309 (or (not $x18905) $x19677 $x22272 (not $x22259) $x22384 $x22386 $x22388 $x22242 $x22318)))
+(let (($x24492 (= (or (not $x18905) (or $x19677 $x22272 (not $x22259) $x22384 $x22386 $x22388 $x22242 $x22318)) $x24309)))
+(let ((@x24028 ((_ quant-inst v_b_S_s$ (b_S_ptr$ ?x10076 ?x21014)) (or (not $x18905) (or $x19677 $x22272 (not $x22259) $x22384 $x22386 $x22388 $x22242 $x22318)))))
+(let ((@x24084 (mp @x24028 (rewrite $x24492) $x24309)))
+(let ((@x22410 (unit-resolution @x24084 @x18908 @x12050 @x22409 @x22429 (trans (monotonicity @x24520 (= ?x22243 ?x10082)) @x12043 $x22259) (or $x22384 $x22386 $x22388 $x22318))))
+(let ((@x22411 (unit-resolution @x22410 @x22886 @x22898 @x22938 (mp @x75 (monotonicity (symm @x22934 (= $x35 $x22388)) $x22500) (not $x22388)) false)))
+(let ((@x22434 (lemma @x22411 $x10136)))
+(let ((@x22687 (mp @x22434 (symm (monotonicity @x24520 @x24520 (= $x22317 $x10136)) (= $x10136 $x22317)) $x22317)))
+(let ((@x22688 (unit-resolution (def-axiom (or (not $x22326) $x22336 $x22318)) @x22687 (unit-resolution @x22613 @x15021 $x22326) $x22318)))
+(let (($x22366 (or $x22333 $x22365)))
+(let (($x18945 (forall ((?v0 B_S_state$) (?v1 B_S_ptr$) (?v2 B_S_ptr$) )(!(let (($x18929 (forall ((?v3 B_S_ptr$) )(!(let (($x8646 (b_S_set_n_in2$ ?v3 (b_S_ver_n_domain$ (b_S_read_n_version$ ?v0 ?v2)))))
+(let ((?x6628 (b_S_typ$ ?v1)))
+(let (($x8640 (b_S_has_n_volatile_n_owns_n_set$ ?x6628)))
+(or $x8640 (not (b_S_set_n_in$ ?v3 (b_S_owns$ ?v0 ?v1))) $x8646)))) :pattern ( (b_S_set_n_in$ ?v3 (b_S_owns$ ?v0 ?v1)) )))
+))
+(let (($x2554 (b_S_closed$ ?v0 ?v1)))
+(let (($x8955 (not $x2554)))
+(let (($x8428 (b_S_set_n_in$ ?v1 (b_S_domain$ ?v0 ?v2))))
+(let (($x18744 (not $x8428)))
+(let (($x18937 (not (or $x18744 $x8955 (not $x18929)))))
+(let (($x8461 (b_S_in_n_domain$ ?v0 ?v1 ?v2)))
+(let (($x8672 (not $x8461)))
+(or $x8672 $x18937))))))))) :pattern ( (b_S_in_n_domain$ ?v0 ?v1 ?v2) )))
+))
+(let (($x8687 (forall ((?v0 B_S_state$) (?v1 B_S_ptr$) (?v2 B_S_ptr$) )(!(let (($x8660 (forall ((?v3 B_S_ptr$) )(!(let (($x8646 (b_S_set_n_in2$ ?v3 (b_S_ver_n_domain$ (b_S_read_n_version$ ?v0 ?v2)))))
+(let (($x8643 (b_S_set_n_in$ ?v3 (b_S_owns$ ?v0 ?v1))))
+(let (($x8644 (and (not (b_S_has_n_volatile_n_owns_n_set$ (b_S_typ$ ?v1))) $x8643)))
+(let (($x8656 (not $x8644)))
+(or $x8656 $x8646))))) :pattern ( (b_S_set_n_in$ ?v3 (b_S_owns$ ?v0 ?v1)) )))
+))
+(let (($x2554 (b_S_closed$ ?v0 ?v1)))
+(let (($x8428 (b_S_set_n_in$ ?v1 (b_S_domain$ ?v0 ?v2))))
+(let (($x8681 (and $x8428 $x2554 $x8660)))
+(let (($x8461 (b_S_in_n_domain$ ?v0 ?v1 ?v2)))
+(let (($x8672 (not $x8461)))
+(or $x8672 $x8681))))))) :pattern ( (b_S_in_n_domain$ ?v0 ?v1 ?v2) )))
+))
+(let (($x18929 (forall ((?v3 B_S_ptr$) )(!(let (($x8646 (b_S_set_n_in2$ ?v3 (b_S_ver_n_domain$ (b_S_read_n_version$ ?2 ?0)))))
+(let ((?x6628 (b_S_typ$ ?1)))
+(let (($x8640 (b_S_has_n_volatile_n_owns_n_set$ ?x6628)))
+(or $x8640 (not (b_S_set_n_in$ ?v3 (b_S_owns$ ?2 ?1))) $x8646)))) :pattern ( (b_S_set_n_in$ ?v3 (b_S_owns$ ?2 ?1)) )))
+))
+(let (($x2554 (b_S_closed$ ?2 ?1)))
+(let (($x8955 (not $x2554)))
+(let (($x8428 (b_S_set_n_in$ ?1 (b_S_domain$ ?2 ?0))))
+(let (($x18744 (not $x8428)))
+(let (($x18937 (not (or $x18744 $x8955 (not $x18929)))))
+(let (($x8461 (b_S_in_n_domain$ ?2 ?1 ?0)))
+(let (($x8672 (not $x8461)))
+(let (($x8660 (forall ((?v3 B_S_ptr$) )(!(let (($x8646 (b_S_set_n_in2$ ?v3 (b_S_ver_n_domain$ (b_S_read_n_version$ ?2 ?0)))))
+(let (($x8643 (b_S_set_n_in$ ?v3 (b_S_owns$ ?2 ?1))))
+(let (($x8644 (and (not (b_S_has_n_volatile_n_owns_n_set$ (b_S_typ$ ?1))) $x8643)))
+(let (($x8656 (not $x8644)))
+(or $x8656 $x8646))))) :pattern ( (b_S_set_n_in$ ?v3 (b_S_owns$ ?2 ?1)) )))
+))
+(let (($x8681 (and $x8428 $x2554 $x8660)))
+(let (($x8684 (or $x8672 $x8681)))
+(let (($x8646 (b_S_set_n_in2$ ?0 (b_S_ver_n_domain$ (b_S_read_n_version$ ?3 ?1)))))
+(let ((?x6628 (b_S_typ$ ?2)))
+(let (($x8640 (b_S_has_n_volatile_n_owns_n_set$ ?x6628)))
+(let (($x18924 (or $x8640 (not (b_S_set_n_in$ ?0 (b_S_owns$ ?3 ?2))) $x8646)))
+(let (($x8643 (b_S_set_n_in$ ?0 (b_S_owns$ ?3 ?2))))
+(let (($x8644 (and (not $x8640) $x8643)))
+(let (($x8656 (not $x8644)))
+(let (($x8657 (or $x8656 $x8646)))
+(let ((@x18918 (rewrite (= (not (not (or $x8640 (not $x8643)))) (or $x8640 (not $x8643))))))
+(let ((@x18916 (monotonicity (rewrite (= $x8644 (not (or $x8640 (not $x8643))))) (= $x8656 (not (not (or $x8640 (not $x8643))))))))
+(let ((@x18923 (monotonicity (trans @x18916 @x18918 (= $x8656 (or $x8640 (not $x8643)))) (= $x8657 (or (or $x8640 (not $x8643)) $x8646)))))
+(let ((@x18928 (trans @x18923 (rewrite (= (or (or $x8640 (not $x8643)) $x8646) $x18924)) (= $x8657 $x18924))))
+(let ((@x18934 (monotonicity (quant-intro @x18928 (= $x8660 $x18929)) (= $x8681 (and $x8428 $x2554 $x18929)))))
+(let ((@x18941 (trans @x18934 (rewrite (= (and $x8428 $x2554 $x18929) $x18937)) (= $x8681 $x18937))))
+(let ((@x18947 (quant-intro (monotonicity @x18941 (= $x8684 (or $x8672 $x18937))) (= $x8687 $x18945))))
+(let ((@x15001 (monotonicity (refl (~ $x8428 $x8428)) (refl (~ $x2554 $x2554)) (nnf-pos (refl (~ $x8657 $x8657)) (~ $x8660 $x8660)) (~ $x8681 $x8681))))
+(let ((@x15005 (nnf-pos (monotonicity (refl (~ $x8672 $x8672)) @x15001 (~ $x8684 $x8684)) (~ $x8687 $x8687))))
+(let (($x8654 (forall ((?v0 B_S_state$) (?v1 B_S_ptr$) (?v2 B_S_ptr$) )(!(let (($x8649 (forall ((?v3 B_S_ptr$) )(!(let (($x8646 (b_S_set_n_in2$ ?v3 (b_S_ver_n_domain$ (b_S_read_n_version$ ?v0 ?v2)))))
+(let (($x8643 (b_S_set_n_in$ ?v3 (b_S_owns$ ?v0 ?v1))))
+(let (($x8644 (and (not (b_S_has_n_volatile_n_owns_n_set$ (b_S_typ$ ?v1))) $x8643)))
+(=> $x8644 $x8646)))) :pattern ( (b_S_set_n_in$ ?v3 (b_S_owns$ ?v0 ?v1)) )))
+))
+(let (($x2554 (b_S_closed$ ?v0 ?v1)))
+(let (($x8428 (b_S_set_n_in$ ?v1 (b_S_domain$ ?v0 ?v2))))
+(let (($x8461 (b_S_in_n_domain$ ?v0 ?v1 ?v2)))
+(=> $x8461 (and $x8428 (and $x2554 $x8649))))))) :pattern ( (b_S_in_n_domain$ ?v0 ?v1 ?v2) )))
+))
+(let (($x8678 (forall ((?v0 B_S_state$) (?v1 B_S_ptr$) (?v2 B_S_ptr$) )(!(let (($x8660 (forall ((?v3 B_S_ptr$) )(!(let (($x8646 (b_S_set_n_in2$ ?v3 (b_S_ver_n_domain$ (b_S_read_n_version$ ?v0 ?v2)))))
+(let (($x8643 (b_S_set_n_in$ ?v3 (b_S_owns$ ?v0 ?v1))))
+(let (($x8644 (and (not (b_S_has_n_volatile_n_owns_n_set$ (b_S_typ$ ?v1))) $x8643)))
+(let (($x8656 (not $x8644)))
+(or $x8656 $x8646))))) :pattern ( (b_S_set_n_in$ ?v3 (b_S_owns$ ?v0 ?v1)) )))
+))
+(let (($x2554 (b_S_closed$ ?v0 ?v1)))
+(let (($x8428 (b_S_set_n_in$ ?v1 (b_S_domain$ ?v0 ?v2))))
+(let (($x8666 (and $x8428 (and $x2554 $x8660))))
+(let (($x8461 (b_S_in_n_domain$ ?v0 ?v1 ?v2)))
+(let (($x8672 (not $x8461)))
+(or $x8672 $x8666))))))) :pattern ( (b_S_in_n_domain$ ?v0 ?v1 ?v2) )))
+))
+(let ((@x8686 (monotonicity (rewrite (= (and $x8428 (and $x2554 $x8660)) $x8681)) (= (or $x8672 (and $x8428 (and $x2554 $x8660))) $x8684))))
+(let (($x8666 (and $x8428 (and $x2554 $x8660))))
+(let (($x8673 (or $x8672 $x8666)))
+(let (($x8649 (forall ((?v3 B_S_ptr$) )(!(let (($x8646 (b_S_set_n_in2$ ?v3 (b_S_ver_n_domain$ (b_S_read_n_version$ ?2 ?0)))))
+(let (($x8643 (b_S_set_n_in$ ?v3 (b_S_owns$ ?2 ?1))))
+(let (($x8644 (and (not (b_S_has_n_volatile_n_owns_n_set$ (b_S_typ$ ?1))) $x8643)))
+(=> $x8644 $x8646)))) :pattern ( (b_S_set_n_in$ ?v3 (b_S_owns$ ?2 ?1)) )))
+))
+(let (($x8652 (=> $x8461 (and $x8428 (and $x2554 $x8649)))))
+(let ((@x8665 (monotonicity (quant-intro (rewrite (= (=> $x8644 $x8646) $x8657)) (= $x8649 $x8660)) (= (and $x2554 $x8649) (and $x2554 $x8660)))))
+(let ((@x8671 (monotonicity (monotonicity @x8665 (= (and $x8428 (and $x2554 $x8649)) $x8666)) (= $x8652 (=> $x8461 $x8666)))))
+(let ((@x8680 (quant-intro (trans @x8671 (rewrite (= (=> $x8461 $x8666) $x8673)) (= $x8652 $x8673)) (= $x8654 $x8678))))
+(let ((@x8692 (mp (asserted $x8654) (trans @x8680 (quant-intro @x8686 (= $x8678 $x8687)) (= $x8654 $x8687)) $x8687)))
+(let ((@x18948 (mp (mp~ @x8692 @x15005 $x8687) @x18947 $x18945)))
+(let (($x22607 (or (not $x18945) $x22333 $x22365)))
+(let ((@x22329 (mp ((_ quant-inst v_b_S_s$ (b_S_ptr$ ?x10076 ?x21014) (b_S_ptr$ ?x10076 ?x21014)) (or (not $x18945) $x22366)) (rewrite (= (or (not $x18945) $x22366) $x22607)) $x22607)))
+(let ((@x22691 (unit-resolution (def-axiom (or $x22364 $x22344)) (unit-resolution (unit-resolution @x22329 @x18948 $x22366) @x22688 $x22365) $x22344)))
+(let ((@x12041 (and-elim @x12033 $x11260)))
+(let (($x18667 (forall ((?v0 B_S_state$) (?v1 Int) (?v2 B_S_ptr$) (?v3 Int) (?v4 Int) (?v5 B_S_ctype$) )(!(let ((?x8245 (b_S_idx$ (b_S_ptr$ ?v5 ?v1) ?v4 ?v5)))
+(let ((?x7097 (b_S_typemap$ ?v0)))
+(let (($x18655 (or (not (b_S_typed$ ?v0 ?x8245)) (b_S_ts_n_is_n_volatile$ (b_S_select_o_tm$ ?x7097 ?x8245)))))
+(let (($x18656 (not $x18655)))
+(let (($x5403 (>= (+ ?v4 (* (- 1) ?v3)) 0)))
+(let (($x3057 (>= ?v4 0)))
+(let (($x16520 (not $x3057)))
+(let (($x8240 (b_S_set_n_in$ (b_S_ptr$ (b_S_array$ ?v5 ?v3) ?v1) (b_S_domain$ ?v0 ?v2))))
+(let (($x18630 (not $x8240)))
+(let (($x2704 (b_S_is_n_primitive$ ?v5)))
+(let (($x8855 (not $x2704)))
+(let (($x8236 (b_S_full_n_stop$ ?v0)))
+(let (($x18629 (not $x8236)))
+(or $x18629 $x8855 $x18630 $x16520 $x5403 $x18656)))))))))))))) :pattern ( (b_S_set_n_in$ (b_S_ptr$ (b_S_array$ ?v5 ?v3) ?v1) (b_S_domain$ ?v0 ?v2)) (b_S_select_o_tm$ (b_S_typemap$ ?v0) (b_S_idx$ (b_S_ptr$ ?v5 ?v1) ?v4 ?v5)) (b_S_is_n_primitive$ ?v5) ) :pattern ( (b_S_set_n_in$ (b_S_ptr$ (b_S_array$ ?v5 ?v3) ?v1) (b_S_domain$ ?v0 ?v2)) (b_S_owner$ ?v0 (b_S_idx$ (b_S_ptr$ ?v5 ?v1) ?v4 ?v5)) (b_S_is_n_primitive$ ?v5) )))
+))
+(let (($x8307 (forall ((?v0 B_S_state$) (?v1 Int) (?v2 B_S_ptr$) (?v3 Int) (?v4 Int) (?v5 B_S_ctype$) )(!(let ((?x8245 (b_S_idx$ (b_S_ptr$ ?v5 ?v1) ?v4 ?v5)))
+(let ((?x7097 (b_S_typemap$ ?v0)))
+(let (($x8291 (and (b_S_typed$ ?v0 ?x8245) (not (b_S_ts_n_is_n_volatile$ (b_S_select_o_tm$ ?x7097 ?x8245))))))
+(let (($x5403 (>= (+ ?v4 (* (- 1) ?v3)) 0)))
+(let (($x6757 (not $x5403)))
+(let (($x3057 (>= ?v4 0)))
+(let (($x8240 (b_S_set_n_in$ (b_S_ptr$ (b_S_array$ ?v5 ?v3) ?v1) (b_S_domain$ ?v0 ?v2))))
+(let (($x2704 (b_S_is_n_primitive$ ?v5)))
+(let (($x8236 (b_S_full_n_stop$ ?v0)))
+(let (($x8270 (and $x8236 $x2704 $x8240 $x3057 $x6757)))
+(let (($x8275 (not $x8270)))
+(or $x8275 $x8291)))))))))))) :pattern ( (b_S_set_n_in$ (b_S_ptr$ (b_S_array$ ?v5 ?v3) ?v1) (b_S_domain$ ?v0 ?v2)) (b_S_select_o_tm$ (b_S_typemap$ ?v0) (b_S_idx$ (b_S_ptr$ ?v5 ?v1) ?v4 ?v5)) (b_S_is_n_primitive$ ?v5) ) :pattern ( (b_S_set_n_in$ (b_S_ptr$ (b_S_array$ ?v5 ?v3) ?v1) (b_S_domain$ ?v0 ?v2)) (b_S_owner$ ?v0 (b_S_idx$ (b_S_ptr$ ?v5 ?v1) ?v4 ?v5)) (b_S_is_n_primitive$ ?v5) )))
+))
+(let ((?x8245 (b_S_idx$ (b_S_ptr$ ?0 ?4) ?1 ?0)))
+(let ((?x7097 (b_S_typemap$ ?5)))
+(let (($x18655 (or (not (b_S_typed$ ?5 ?x8245)) (b_S_ts_n_is_n_volatile$ (b_S_select_o_tm$ ?x7097 ?x8245)))))
+(let (($x18656 (not $x18655)))
+(let (($x5403 (>= (+ ?1 (* (- 1) ?2)) 0)))
+(let (($x3057 (>= ?1 0)))
+(let (($x16520 (not $x3057)))
+(let (($x8240 (b_S_set_n_in$ (b_S_ptr$ (b_S_array$ ?0 ?2) ?4) (b_S_domain$ ?5 ?3))))
+(let (($x18630 (not $x8240)))
+(let (($x8855 (not $x2704)))
+(let (($x8236 (b_S_full_n_stop$ ?5)))
+(let (($x18629 (not $x8236)))
+(let (($x18662 (or $x18629 $x8855 $x18630 $x16520 $x5403 $x18656)))
+(let (($x8291 (and (b_S_typed$ ?5 ?x8245) (not (b_S_ts_n_is_n_volatile$ (b_S_select_o_tm$ ?x7097 ?x8245))))))
+(let (($x6757 (not $x5403)))
+(let (($x8270 (and $x8236 $x2704 $x8240 $x3057 $x6757)))
+(let (($x8275 (not $x8270)))
+(let (($x8304 (or $x8275 $x8291)))
+(let (($x18631 (or $x18629 $x8855 $x18630 $x16520 $x5403)))
+(let ((@x18637 (monotonicity (rewrite (= $x8270 (not $x18631))) (= $x8275 (not (not $x18631))))))
+(let ((@x18661 (monotonicity (trans @x18637 (rewrite (= (not (not $x18631)) $x18631)) (= $x8275 $x18631)) (rewrite (= $x8291 $x18656)) (= $x8304 (or $x18631 $x18656)))))
+(let ((@x18669 (quant-intro (trans @x18661 (rewrite (= (or $x18631 $x18656) $x18662)) (= $x8304 $x18662)) (= $x8307 $x18667))))
+(let (($x8296 (forall ((?v0 B_S_state$) (?v1 Int) (?v2 B_S_ptr$) (?v3 Int) (?v4 Int) (?v5 B_S_ctype$) )(!(let ((?x8245 (b_S_idx$ (b_S_ptr$ ?v5 ?v1) ?v4 ?v5)))
+(let ((?x7097 (b_S_typemap$ ?v0)))
+(let (($x8291 (and (b_S_typed$ ?v0 ?x8245) (not (b_S_ts_n_is_n_volatile$ (b_S_select_o_tm$ ?x7097 ?x8245))))))
+(let (($x3027 (<= 0 ?v4)))
+(let (($x6740 (and $x3027 (< ?v4 ?v3))))
+(let (($x8240 (b_S_set_n_in$ (b_S_ptr$ (b_S_array$ ?v5 ?v3) ?v1) (b_S_domain$ ?v0 ?v2))))
+(let (($x2704 (b_S_is_n_primitive$ ?v5)))
+(let (($x8236 (b_S_full_n_stop$ ?v0)))
+(let (($x8243 (and $x8236 (and $x2704 (and $x8240 $x6740)))))
+(=> $x8243 $x8291)))))))))) :pattern ( (b_S_set_n_in$ (b_S_ptr$ (b_S_array$ ?v5 ?v3) ?v1) (b_S_domain$ ?v0 ?v2)) (b_S_select_o_tm$ (b_S_typemap$ ?v0) (b_S_idx$ (b_S_ptr$ ?v5 ?v1) ?v4 ?v5)) (b_S_is_n_primitive$ ?v5) ) :pattern ( (b_S_set_n_in$ (b_S_ptr$ (b_S_array$ ?v5 ?v3) ?v1) (b_S_domain$ ?v0 ?v2)) (b_S_owner$ ?v0 (b_S_idx$ (b_S_ptr$ ?v5 ?v1) ?v4 ?v5)) (b_S_is_n_primitive$ ?v5) )))
+))
+(let (($x8301 (forall ((?v0 B_S_state$) (?v1 Int) (?v2 B_S_ptr$) (?v3 Int) (?v4 Int) (?v5 B_S_ctype$) )(!(let ((?x8245 (b_S_idx$ (b_S_ptr$ ?v5 ?v1) ?v4 ?v5)))
+(let ((?x7097 (b_S_typemap$ ?v0)))
+(let (($x8291 (and (b_S_typed$ ?v0 ?x8245) (not (b_S_ts_n_is_n_volatile$ (b_S_select_o_tm$ ?x7097 ?x8245))))))
+(let (($x3027 (<= 0 ?v4)))
+(let (($x6740 (and $x3027 (< ?v4 ?v3))))
+(let (($x8240 (b_S_set_n_in$ (b_S_ptr$ (b_S_array$ ?v5 ?v3) ?v1) (b_S_domain$ ?v0 ?v2))))
+(let (($x2704 (b_S_is_n_primitive$ ?v5)))
+(let (($x8236 (b_S_full_n_stop$ ?v0)))
+(let (($x8243 (and $x8236 (and $x2704 (and $x8240 $x6740)))))
+(let (($x8254 (not $x8243)))
+(or $x8254 $x8291))))))))))) :pattern ( (b_S_set_n_in$ (b_S_ptr$ (b_S_array$ ?v5 ?v3) ?v1) (b_S_domain$ ?v0 ?v2)) (b_S_select_o_tm$ (b_S_typemap$ ?v0) (b_S_idx$ (b_S_ptr$ ?v5 ?v1) ?v4 ?v5)) (b_S_is_n_primitive$ ?v5) ) :pattern ( (b_S_set_n_in$ (b_S_ptr$ (b_S_array$ ?v5 ?v3) ?v1) (b_S_domain$ ?v0 ?v2)) (b_S_owner$ ?v0 (b_S_idx$ (b_S_ptr$ ?v5 ?v1) ?v4 ?v5)) (b_S_is_n_primitive$ ?v5) )))
+))
+(let (($x8243 (and $x8236 (and $x2704 (and $x8240 (and (<= 0 ?1) (< ?1 ?2)))))))
+(let (($x8254 (not $x8243)))
+(let (($x8298 (or $x8254 $x8291)))
+(let ((@x8272 (rewrite (= (and $x8236 (and $x2704 (and $x8240 (and $x3057 $x6757)))) $x8270))))
+(let (($x8265 (= (and $x2704 (and $x8240 (and (<= 0 ?1) (< ?1 ?2)))) (and $x2704 (and $x8240 (and $x3057 $x6757))))))
+(let (($x8262 (= (and $x8240 (and (<= 0 ?1) (< ?1 ?2))) (and $x8240 (and $x3057 $x6757)))))
+(let ((@x3058 (rewrite (= (<= 0 ?1) $x3057))))
+(let ((@x6762 (monotonicity @x3058 (rewrite (= (< ?1 ?2) $x6757)) (= (and (<= 0 ?1) (< ?1 ?2)) (and $x3057 $x6757)))))
+(let ((@x8269 (monotonicity (monotonicity (monotonicity @x6762 $x8262) $x8265) (= $x8243 (and $x8236 (and $x2704 (and $x8240 (and $x3057 $x6757))))))))
+(let ((@x8306 (monotonicity (monotonicity (trans @x8269 @x8272 (= $x8243 $x8270)) (= $x8254 $x8275)) (= $x8298 $x8304))))
+(let ((@x8311 (trans (quant-intro (rewrite (= (=> $x8243 $x8291) $x8298)) (= $x8296 $x8301)) (quant-intro @x8306 (= $x8301 $x8307)) (= $x8296 $x8307))))
+(let ((@x14905 (mp~ (mp (asserted $x8296) @x8311 $x8307) (nnf-pos (refl (~ $x8304 $x8304)) (~ $x8307 $x8307)) $x8307)))
+(let ((@x18670 (mp @x14905 @x18669 $x18667)))
+(let (($x22597 (not $x22596)))
+(let (($x21489 (not $x9768)))
+(let (($x22629 (not $x18667)))
+(let (($x22733 (or $x22629 $x19677 $x21489 $x22597 $x11259 $x22604)))
+(let (($x22601 (>= (+ 0 (* (- 1) v_b_P_H_len$)) 0)))
+(let (($x22599 (not (>= 0 0))))
+(let (($x22605 (or $x19677 $x21489 $x22597 $x22599 $x22601 $x22604)))
+(let (($x22734 (or $x22629 $x22605)))
+(let (($x22728 (or $x19677 $x21489 $x22597 $x11259 $x22604)))
+(let ((@x22717 (rewrite (= (+ 0 (* (- 1) v_b_P_H_len$)) (* (- 1) v_b_P_H_len$)))))
+(let ((@x22724 (trans (monotonicity @x22717 (= $x22601 (>= (* (- 1) v_b_P_H_len$) 0))) (rewrite (= (>= (* (- 1) v_b_P_H_len$) 0) $x11259)) (= $x22601 $x11259))))
+(let ((@x22715 (trans (monotonicity (rewrite (= (>= 0 0) true)) (= $x22599 $x10203)) @x10561 (= $x22599 false))))
+(let ((@x22727 (monotonicity @x22715 @x22724 (= $x22605 (or $x19677 $x21489 $x22597 false $x11259 $x22604)))))
+(let ((@x22732 (trans @x22727 (rewrite (= (or $x19677 $x21489 $x22597 false $x11259 $x22604) $x22728)) (= $x22605 $x22728))))
+(let ((@x22742 (trans (monotonicity @x22732 (= $x22734 (or $x22629 $x22728))) (rewrite (= (or $x22629 $x22728) $x22733)) (= $x22734 $x22733))))
+(let ((@x22743 (mp ((_ quant-inst v_b_S_s$ v_b_P_H_arr$ (b_S_ptr$ ?x10076 ?x21014) v_b_P_H_len$ 0 b_T_T_u1$) $x22734) @x22742 $x22733)))
+(let ((@x22761 (unit-resolution @x22743 @x18670 @x9769 @x12041 @x12050 (mp @x22691 @x22795 $x22596) (hypothesis $x22603) false)))
+(let ((@x22760 (lemma @x22761 $x22604)))
+(let ((@x23294 (mp (unit-resolution (def-axiom (or $x22603 $x22641)) @x22760 $x22641) (monotonicity @x23082 (= $x22641 $x22897)) $x22897)))
+(let (($x22894 (b_S_in_n_wrapped_n_domain$ v_b_S_s$ ?x22903)))
+(let ((?x22893 (b_S_owner$ v_b_S_s$ ?x22903)))
+(let (($x22888 (= ?x22893 b_S_me$)))
+(let (($x22895 (or $x22888 $x22894)))
+(let (($x22896 (not $x22895)))
+(let ((?x22890 (b_S_typ$ ?x22903)))
+(let ((?x22891 (b_S_kind_n_of$ ?x22890)))
+(let (($x22892 (= ?x22891 b_S_kind_n_primitive$)))
+(let (($x22889 (not $x22906)))
+(let (($x22817 (not $x22807)))
+(let (($x22900 (or $x22817 $x22889 $x22892 $x22896)))
+(let (($x22952 (b_S_in_n_wrapped_n_domain$ v_b_S_s$ ?x10078)))
+(let (($x22953 (= (b_S_owner$ v_b_S_s$ ?x10078) b_S_me$)))
+(let (($x22954 (or $x22953 $x22952)))
+(let (($x22941 (not $x22954)))
+(let (($x22942 (or $x22807 $x22941)))
+(let (($x22920 (not $x22942)))
+(let (($x22901 (not $x22900)))
+(let (($x22921 (or $x22901 $x22920)))
+(let (($x22923 (not $x22921)))
+(let (($x22799 (b_S_typed$ v_b_S_s$ ?x10078)))
+(let (($x22802 (not $x22799)))
+(let (($x22939 (or $x22802 $x22923)))
+(let (($x22943 (not $x22939)))
+(let (($x22801 (b_S_thread_n_local$ v_b_S_s$ ?x10078)))
+(let (($x22944 (= $x22801 $x22943)))
+(let (($x19072 (forall ((?v0 B_S_state$) (?v1 B_S_ptr$) )(!(let (($x9039 (b_S_in_n_wrapped_n_domain$ ?v0 ?v1)))
+(let ((?x2484 (b_S_owner$ ?v0 ?v1)))
+(let (($x2486 (= ?x2484 b_S_me$)))
+(let (($x2249 (= (b_S_kind_n_of$ (b_S_typ$ ?v1)) b_S_kind_n_primitive$)))
+(let ((?x2769 (b_S_typemap$ ?v0)))
+(let ((?x9020 (b_S_select_o_tm$ ?x2769 ?v1)))
+(let ((?x9024 (b_S_ts_n_emb$ ?x9020)))
+(let (($x9035 (or (= (b_S_owner$ ?v0 ?x9024) b_S_me$) (b_S_in_n_wrapped_n_domain$ ?v0 ?x9024))))
+(let (($x9022 (b_S_ts_n_is_n_volatile$ ?x9020)))
+(let (($x9023 (not $x9022)))
+(let (($x9027 (or $x9023 (not (b_S_closed$ ?v0 ?x9024)))))
+(let (($x2294 (not $x2249)))
+(let (($x19047 (or $x2294 (not $x9027) (= (b_S_kind_n_of$ (b_S_typ$ ?x9024)) b_S_kind_n_primitive$) (not $x9035))))
+(let (($x19056 (or (not $x19047) (not (or $x2249 (not (or $x2486 $x9039)))))))
+(let (($x2488 (b_S_typed$ ?v0 ?v1)))
+(let (($x9531 (not $x2488)))
+(let (($x19064 (not (or $x9531 (not $x19056)))))
+(let (($x9019 (b_S_thread_n_local$ ?v0 ?v1)))
+(= $x9019 $x19064))))))))))))))))))) :pattern ( (b_S_thread_n_local$ ?v0 ?v1) )))
+))
+(let (($x9066 (forall ((?v0 B_S_state$) (?v1 B_S_ptr$) )(!(let (($x9039 (b_S_in_n_wrapped_n_domain$ ?v0 ?v1)))
+(let ((?x2484 (b_S_owner$ ?v0 ?v1)))
+(let (($x2486 (= ?x2484 b_S_me$)))
+(let (($x2249 (= (b_S_kind_n_of$ (b_S_typ$ ?v1)) b_S_kind_n_primitive$)))
+(let (($x2294 (not $x2249)))
+(let (($x9041 (and $x2294 (or $x2486 $x9039))))
+(let ((?x2769 (b_S_typemap$ ?v0)))
+(let ((?x9020 (b_S_select_o_tm$ ?x2769 ?v1)))
+(let ((?x9024 (b_S_ts_n_emb$ ?x9020)))
+(let (($x9035 (or (= (b_S_owner$ ?v0 ?x9024) b_S_me$) (b_S_in_n_wrapped_n_domain$ ?v0 ?x9024))))
+(let (($x9022 (b_S_ts_n_is_n_volatile$ ?x9020)))
+(let (($x9023 (not $x9022)))
+(let (($x9027 (or $x9023 (not (b_S_closed$ ?v0 ?x9024)))))
+(let (($x9054 (and $x2249 $x9027 (not (= (b_S_kind_n_of$ (b_S_typ$ ?x9024)) b_S_kind_n_primitive$)) $x9035)))
+(let (($x9057 (or $x9054 $x9041)))
+(let (($x2488 (b_S_typed$ ?v0 ?v1)))
+(let (($x9060 (and $x2488 $x9057)))
+(let (($x9019 (b_S_thread_n_local$ ?v0 ?v1)))
+(= $x9019 $x9060))))))))))))))))))) :pattern ( (b_S_thread_n_local$ ?v0 ?v1) )))
+))
+(let ((?x2769 (b_S_typemap$ ?1)))
+(let ((?x9020 (b_S_select_o_tm$ ?x2769 ?0)))
+(let ((?x9024 (b_S_ts_n_emb$ ?x9020)))
+(let (($x9035 (or (= (b_S_owner$ ?1 ?x9024) b_S_me$) (b_S_in_n_wrapped_n_domain$ ?1 ?x9024))))
+(let (($x9022 (b_S_ts_n_is_n_volatile$ ?x9020)))
+(let (($x9023 (not $x9022)))
+(let (($x9027 (or $x9023 (not (b_S_closed$ ?1 ?x9024)))))
+(let (($x19047 (or $x2294 (not $x9027) (= (b_S_kind_n_of$ (b_S_typ$ ?x9024)) b_S_kind_n_primitive$) (not $x9035))))
+(let (($x19056 (or (not $x19047) (not (or $x2249 (not (or $x2486 (b_S_in_n_wrapped_n_domain$ ?1 ?0))))))))
+(let (($x19064 (not (or $x9531 (not $x19056)))))
+(let (($x9019 (b_S_thread_n_local$ ?1 ?0)))
+(let (($x9041 (and $x2294 (or $x2486 (b_S_in_n_wrapped_n_domain$ ?1 ?0)))))
+(let (($x9054 (and $x2249 $x9027 (not (= (b_S_kind_n_of$ (b_S_typ$ ?x9024)) b_S_kind_n_primitive$)) $x9035)))
+(let (($x9057 (or $x9054 $x9041)))
+(let (($x9060 (and $x2488 $x9057)))
+(let (($x9063 (= $x9019 $x9060)))
+(let (($x19054 (= $x9041 (not (or $x2249 (not (or $x2486 (b_S_in_n_wrapped_n_domain$ ?1 ?0))))))))
+(let ((@x19058 (monotonicity (rewrite (= $x9054 (not $x19047))) (rewrite $x19054) (= $x9057 $x19056))))
+(let ((@x19068 (trans (monotonicity @x19058 (= $x9060 (and $x2488 $x19056))) (rewrite (= (and $x2488 $x19056) $x19064)) (= $x9060 $x19064))))
+(let ((@x19074 (quant-intro (monotonicity @x19068 (= $x9063 (= $x9019 $x19064))) (= $x9066 $x19072))))
+(let (($x9046 (forall ((?v0 B_S_state$) (?v1 B_S_ptr$) )(!(let (($x9039 (b_S_in_n_wrapped_n_domain$ ?v0 ?v1)))
+(let ((?x2484 (b_S_owner$ ?v0 ?v1)))
+(let (($x2486 (= ?x2484 b_S_me$)))
+(let (($x2249 (= (b_S_kind_n_of$ (b_S_typ$ ?v1)) b_S_kind_n_primitive$)))
+(let (($x2294 (not $x2249)))
+(let (($x9041 (and $x2294 (or $x2486 $x9039))))
+(let ((?x2769 (b_S_typemap$ ?v0)))
+(let ((?x9020 (b_S_select_o_tm$ ?x2769 ?v1)))
+(let ((?x9024 (b_S_ts_n_emb$ ?x9020)))
+(let (($x9035 (or (= (b_S_owner$ ?v0 ?x9024) b_S_me$) (b_S_in_n_wrapped_n_domain$ ?v0 ?x9024))))
+(let (($x9036 (and (not (= (b_S_kind_n_of$ (b_S_typ$ ?x9024)) b_S_kind_n_primitive$)) $x9035)))
+(let (($x9022 (b_S_ts_n_is_n_volatile$ ?x9020)))
+(let (($x9023 (not $x9022)))
+(let (($x9027 (or $x9023 (not (b_S_closed$ ?v0 ?x9024)))))
+(let (($x2488 (b_S_typed$ ?v0 ?v1)))
+(let (($x9043 (and $x2488 (or (and $x2249 (and $x9027 $x9036)) $x9041))))
+(let (($x9019 (b_S_thread_n_local$ ?v0 ?v1)))
+(= $x9019 $x9043)))))))))))))))))) :pattern ( (b_S_thread_n_local$ ?v0 ?v1) )))
+))
+(let (($x9051 (forall ((?v0 B_S_state$) (?v1 B_S_ptr$) )(!(let (($x9039 (b_S_in_n_wrapped_n_domain$ ?v0 ?v1)))
+(let ((?x2484 (b_S_owner$ ?v0 ?v1)))
+(let (($x2486 (= ?x2484 b_S_me$)))
+(let (($x2249 (= (b_S_kind_n_of$ (b_S_typ$ ?v1)) b_S_kind_n_primitive$)))
+(let (($x2294 (not $x2249)))
+(let (($x9041 (and $x2294 (or $x2486 $x9039))))
+(let ((?x2769 (b_S_typemap$ ?v0)))
+(let ((?x9020 (b_S_select_o_tm$ ?x2769 ?v1)))
+(let ((?x9024 (b_S_ts_n_emb$ ?x9020)))
+(let (($x9035 (or (= (b_S_owner$ ?v0 ?x9024) b_S_me$) (b_S_in_n_wrapped_n_domain$ ?v0 ?x9024))))
+(let (($x9036 (and (not (= (b_S_kind_n_of$ (b_S_typ$ ?x9024)) b_S_kind_n_primitive$)) $x9035)))
+(let (($x9022 (b_S_ts_n_is_n_volatile$ ?x9020)))
+(let (($x9023 (not $x9022)))
+(let (($x9027 (or $x9023 (not (b_S_closed$ ?v0 ?x9024)))))
+(let (($x2488 (b_S_typed$ ?v0 ?v1)))
+(let (($x9043 (and $x2488 (or (and $x2249 (and $x9027 $x9036)) $x9041))))
+(let (($x9019 (b_S_thread_n_local$ ?v0 ?v1)))
+(= $x9019 $x9043)))))))))))))))))) :pattern ( (b_S_thread_n_local$ ?v0 ?v1) )))
+))
+(let (($x9036 (and (not (= (b_S_kind_n_of$ (b_S_typ$ ?x9024)) b_S_kind_n_primitive$)) $x9035)))
+(let (($x9043 (and $x2488 (or (and $x2249 (and $x9027 $x9036)) $x9041))))
+(let (($x9048 (= $x9019 $x9043)))
+(let ((@x9059 (monotonicity (rewrite (= (and $x2249 (and $x9027 $x9036)) $x9054)) (= (or (and $x2249 (and $x9027 $x9036)) $x9041) $x9057))))
+(let ((@x9068 (quant-intro (monotonicity (monotonicity @x9059 (= $x9043 $x9060)) (= $x9048 $x9063)) (= $x9051 $x9066))))
+(let ((@x9070 (trans (quant-intro (rewrite (= (= $x9019 $x9043) $x9048)) (= $x9046 $x9051)) @x9068 (= $x9046 $x9066))))
+(let ((@x15111 (mp~ (mp (asserted $x9046) @x9070 $x9066) (nnf-pos (refl (~ $x9063 $x9063)) (~ $x9066 $x9066)) $x9066)))
+(let ((@x19075 (mp @x15111 @x19074 $x19072)))
+(let (($x23521 (or (not $x19072) $x22944)))
+(let ((@x23524 ((_ quant-inst v_b_S_s$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$)) $x23521)))
+(let (($x23055 (not $x22801)))
+(let ((@x23295 (monotonicity (symm (monotonicity @x23663 (= $x22801 $x10141)) (= $x10141 $x22801)) (= (not $x10141) $x23055))))
+(let ((@x23090 (unit-resolution (def-axiom (or (not $x22944) $x22801 $x22939)) (mp (hypothesis (not $x10141)) @x23295 $x23055) (unit-resolution @x23524 @x19075 $x22944) $x22939)))
+(let ((@x23670 (mp (unit-resolution (def-axiom (or $x22603 $x10139)) @x22760 $x10139) (symm (monotonicity @x23663 (= $x22799 $x10139)) (= $x10139 $x22799)) $x22799)))
+(let ((@x23233 (unit-resolution (def-axiom (or $x22921 $x22900)) (unit-resolution (def-axiom (or $x22943 $x22802 $x22923)) @x23670 @x23090 $x22923) $x22900)))
+(let ((?x24419 (b_S_ref$ ?x21983)))
+(let ((?x24433 (b_S_ptr$ b_T_T_u1$ ?x24419)))
+(let ((?x24410 (b_S_idx$ ?x21983 0 b_T_T_u1$)))
+(let (($x24436 (= ?x24410 ?x24433)))
+(let (($x24439 (not $x24436)))
+(let (($x24411 (b_S_extent_n_hint$ ?x24410 ?x21983)))
+(let (($x24418 (not $x24411)))
+(let (($x24442 (or $x24418 $x24439)))
+(let (($x24445 (not $x24442)))
+(let (($x24448 (or $x22568 $x24445)))
+(let (($x24424 (or $x24418 (not (= ?x24410 (b_S_ptr$ b_T_T_u1$ (+ ?x24419 (* 0 ?x10045))))))))
+(let (($x24425 (not $x24424)))
+(let (($x24440 (= (not (= ?x24410 (b_S_ptr$ b_T_T_u1$ (+ ?x24419 (* 0 ?x10045))))) $x24439)))
+(let ((@x24428 (monotonicity (rewrite (= (* 0 ?x10045) 0)) (= (+ ?x24419 (* 0 ?x10045)) (+ ?x24419 0)))))
+(let ((@x24432 (trans @x24428 (rewrite (= (+ ?x24419 0) ?x24419)) (= (+ ?x24419 (* 0 ?x10045)) ?x24419))))
+(let ((@x24435 (monotonicity @x24432 (= (b_S_ptr$ b_T_T_u1$ (+ ?x24419 (* 0 ?x10045))) ?x24433))))
+(let ((@x24438 (monotonicity @x24435 (= (= ?x24410 (b_S_ptr$ b_T_T_u1$ (+ ?x24419 (* 0 ?x10045)))) $x24436))))
+(let ((@x24447 (monotonicity (monotonicity (monotonicity @x24438 $x24440) (= $x24424 $x24442)) (= $x24425 $x24445))))
+(let ((@x24455 (trans (monotonicity @x24447 (= (or $x22568 $x24425) $x24448)) (rewrite (= $x24448 $x24448)) (= (or $x22568 $x24425) $x24448))))
+(let ((@x24133 (unit-resolution (mp ((_ quant-inst (b_S_ptr$ ?x10076 ?x21014) 0 b_T_T_u1$) (or $x22568 $x24425)) @x24455 $x24448) @x18183 (hypothesis $x24442) false)))
+(let ((@x24460 (def-axiom (or $x24442 $x24436))))
+(let ((?x24245 (b_S_idx$ ?x22595 0 b_T_T_u1$)))
+(let ((?x24246 (b_S_select_o_tm$ ?x10272 ?x24245)))
+(let ((?x24247 (b_S_ts_n_emb$ ?x24246)))
+(let (($x24248 (= ?x24247 ?x22595)))
+(let (($x24257 (b_S_typed$ v_b_S_s$ ?x24245)))
+(let (($x24258 (not $x24257)))
+(let (($x24255 (b_S_ts_n_is_n_volatile$ ?x24246)))
+(let (($x24254 (not $x24248)))
+(let (($x23737 (or $x24254 $x24255 (not (b_S_ts_n_is_n_array_n_elt$ ?x24246)) $x24258)))
+(let (($x23791 (not $x23737)))
+(let (($x24240 (b_S_typed$ v_b_S_s$ ?x22595)))
+(let ((@x24353 (mp @x12045 (symm (monotonicity @x24530 (= $x24240 $x10085)) (= $x10085 $x24240)) $x24240)))
+(let ((@x24355 (lemma (unit-resolution (hypothesis (not $x24240)) @x24353 false) $x24240)))
+(let (($x17964 (forall ((?v0 B_S_state$) (?v1 Int) (?v2 B_S_ctype$) (?v3 Int) (?v4 Int) )(!(let (($x6905 (b_S_typed$ ?v0 (b_S_idx$ (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) ?v4 ?v2))))
+(let ((?x6897 (b_S_typemap$ ?v0)))
+(let ((?x6899 (b_S_select_o_tm$ ?x6897 (b_S_idx$ (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) ?v4 ?v2))))
+(let (($x6904 (b_S_ts_n_is_n_array_n_elt$ ?x6899)))
+(let (($x17952 (or (not (= (b_S_ts_n_emb$ ?x6899) (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1))) (b_S_ts_n_is_n_volatile$ ?x6899) (not $x6904) (not $x6905))))
+(let (($x17953 (not $x17952)))
+(let (($x4862 (>= (+ ?v4 (* (- 1) ?v3)) 0)))
+(let (($x2815 (>= ?v4 0)))
+(let (($x3763 (not $x2815)))
+(or (not (b_S_typed$ ?v0 (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1))) $x3763 $x4862 $x17953)))))))))) :pattern ( (b_S_select_o_sm$ (b_S_statusmap$ ?v0) (b_S_idx$ (b_S_ptr$ ?v2 ?v1) ?v4 ?v2)) (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) ) :pattern ( (b_S_select_o_tm$ (b_S_typemap$ ?v0) (b_S_idx$ (b_S_ptr$ ?v2 ?v1) ?v4 ?v2)) (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) )))
+))
+(let (($x6943 (forall ((?v0 B_S_state$) (?v1 Int) (?v2 B_S_ctype$) (?v3 Int) (?v4 Int) )(!(let (($x6905 (b_S_typed$ ?v0 (b_S_idx$ (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) ?v4 ?v2))))
+(let ((?x6897 (b_S_typemap$ ?v0)))
+(let ((?x6899 (b_S_select_o_tm$ ?x6897 (b_S_idx$ (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) ?v4 ?v2))))
+(let (($x6904 (b_S_ts_n_is_n_array_n_elt$ ?x6899)))
+(let ((?x6894 (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1)))
+(let (($x6901 (= (b_S_ts_n_emb$ ?x6899) ?x6894)))
+(let (($x6937 (and $x6901 (not (b_S_ts_n_is_n_volatile$ ?x6899)) $x6904 $x6905)))
+(let (($x4862 (>= (+ ?v4 (* (- 1) ?v3)) 0)))
+(let (($x6603 (not $x4862)))
+(let (($x2815 (>= ?v4 0)))
+(let (($x6895 (b_S_typed$ ?v0 ?x6894)))
+(let (($x6929 (and $x6895 $x2815 $x6603)))
+(let (($x6934 (not $x6929)))
+(or $x6934 $x6937)))))))))))))) :pattern ( (b_S_select_o_sm$ (b_S_statusmap$ ?v0) (b_S_idx$ (b_S_ptr$ ?v2 ?v1) ?v4 ?v2)) (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) ) :pattern ( (b_S_select_o_tm$ (b_S_typemap$ ?v0) (b_S_idx$ (b_S_ptr$ ?v2 ?v1) ?v4 ?v2)) (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) )))
+))
+(let (($x6905 (b_S_typed$ ?4 (b_S_idx$ (b_S_ptr$ (b_S_array$ ?2 ?1) ?3) ?0 ?2))))
+(let ((?x6897 (b_S_typemap$ ?4)))
+(let ((?x6899 (b_S_select_o_tm$ ?x6897 (b_S_idx$ (b_S_ptr$ (b_S_array$ ?2 ?1) ?3) ?0 ?2))))
+(let (($x6904 (b_S_ts_n_is_n_array_n_elt$ ?x6899)))
+(let (($x17952 (or (not (= (b_S_ts_n_emb$ ?x6899) (b_S_ptr$ (b_S_array$ ?2 ?1) ?3))) (b_S_ts_n_is_n_volatile$ ?x6899) (not $x6904) (not $x6905))))
+(let (($x17953 (not $x17952)))
+(let (($x4862 (>= (+ ?0 (* (- 1) ?1)) 0)))
+(let (($x3763 (not $x2815)))
+(let (($x17959 (or (not (b_S_typed$ ?4 (b_S_ptr$ (b_S_array$ ?2 ?1) ?3))) $x3763 $x4862 $x17953)))
+(let ((?x6894 (b_S_ptr$ (b_S_array$ ?2 ?1) ?3)))
+(let (($x6901 (= (b_S_ts_n_emb$ ?x6899) ?x6894)))
+(let (($x6937 (and $x6901 (not (b_S_ts_n_is_n_volatile$ ?x6899)) $x6904 $x6905)))
+(let (($x6603 (not $x4862)))
+(let (($x6895 (b_S_typed$ ?4 ?x6894)))
+(let (($x6929 (and $x6895 $x2815 $x6603)))
+(let (($x6934 (not $x6929)))
+(let (($x6940 (or $x6934 $x6937)))
+(let (($x17938 (or (not $x6895) $x3763 $x4862)))
+(let ((@x17944 (monotonicity (rewrite (= $x6929 (not $x17938))) (= $x6934 (not (not $x17938))))))
+(let ((@x17958 (monotonicity (trans @x17944 (rewrite (= (not (not $x17938)) $x17938)) (= $x6934 $x17938)) (rewrite (= $x6937 $x17953)) (= $x6940 (or $x17938 $x17953)))))
+(let ((@x17966 (quant-intro (trans @x17958 (rewrite (= (or $x17938 $x17953) $x17959)) (= $x6940 $x17959)) (= $x6943 $x17964))))
+(let (($x6917 (forall ((?v0 B_S_state$) (?v1 Int) (?v2 B_S_ctype$) (?v3 Int) (?v4 Int) )(!(let (($x6905 (b_S_typed$ ?v0 (b_S_idx$ (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) ?v4 ?v2))))
+(let ((?x6897 (b_S_typemap$ ?v0)))
+(let ((?x6899 (b_S_select_o_tm$ ?x6897 (b_S_idx$ (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) ?v4 ?v2))))
+(let (($x6904 (b_S_ts_n_is_n_array_n_elt$ ?x6899)))
+(let ((?x6894 (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1)))
+(let (($x6901 (= (b_S_ts_n_emb$ ?x6899) ?x6894)))
+(let (($x6908 (and $x6901 (and (not (b_S_ts_n_is_n_volatile$ ?x6899)) (and $x6904 $x6905)))))
+(let (($x2766 (<= 0 ?v4)))
+(let (($x6566 (and $x2766 (< ?v4 ?v3))))
+(let (($x6895 (b_S_typed$ ?v0 ?x6894)))
+(let (($x6896 (and $x6895 $x6566)))
+(=> $x6896 $x6908)))))))))))) :pattern ( (b_S_select_o_sm$ (b_S_statusmap$ ?v0) (b_S_idx$ (b_S_ptr$ ?v2 ?v1) ?v4 ?v2)) (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) ) :pattern ( (b_S_select_o_tm$ (b_S_typemap$ ?v0) (b_S_idx$ (b_S_ptr$ ?v2 ?v1) ?v4 ?v2)) (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) )))
+))
+(let (($x6923 (forall ((?v0 B_S_state$) (?v1 Int) (?v2 B_S_ctype$) (?v3 Int) (?v4 Int) )(!(let (($x6905 (b_S_typed$ ?v0 (b_S_idx$ (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) ?v4 ?v2))))
+(let ((?x6897 (b_S_typemap$ ?v0)))
+(let ((?x6899 (b_S_select_o_tm$ ?x6897 (b_S_idx$ (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) ?v4 ?v2))))
+(let (($x6904 (b_S_ts_n_is_n_array_n_elt$ ?x6899)))
+(let ((?x6894 (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1)))
+(let (($x6901 (= (b_S_ts_n_emb$ ?x6899) ?x6894)))
+(let (($x6908 (and $x6901 (and (not (b_S_ts_n_is_n_volatile$ ?x6899)) (and $x6904 $x6905)))))
+(let (($x2766 (<= 0 ?v4)))
+(let (($x6566 (and $x2766 (< ?v4 ?v3))))
+(let (($x6895 (b_S_typed$ ?v0 ?x6894)))
+(let (($x6896 (and $x6895 $x6566)))
+(or (not $x6896) $x6908)))))))))))) :pattern ( (b_S_select_o_sm$ (b_S_statusmap$ ?v0) (b_S_idx$ (b_S_ptr$ ?v2 ?v1) ?v4 ?v2)) (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) ) :pattern ( (b_S_select_o_tm$ (b_S_typemap$ ?v0) (b_S_idx$ (b_S_ptr$ ?v2 ?v1) ?v4 ?v2)) (b_S_ptr$ (b_S_array$ ?v2 ?v3) ?v1) )))
+))
+(let (($x6908 (and $x6901 (and (not (b_S_ts_n_is_n_volatile$ ?x6899)) (and $x6904 $x6905)))))
+(let (($x6920 (or (not (and $x6895 (and $x2766 (< ?0 ?1)))) $x6908)))
+(let (($x6566 (and $x2766 (< ?0 ?1))))
+(let (($x6896 (and $x6895 $x6566)))
+(let ((@x6608 (monotonicity @x2814 (rewrite (= (< ?0 ?1) $x6603)) (= $x6566 (and $x2815 $x6603)))))
+(let ((@x6933 (trans (monotonicity @x6608 (= $x6896 (and $x6895 (and $x2815 $x6603)))) (rewrite (= (and $x6895 (and $x2815 $x6603)) $x6929)) (= $x6896 $x6929))))
+(let ((@x6942 (monotonicity (monotonicity @x6933 (= (not $x6896) $x6934)) (rewrite (= $x6908 $x6937)) (= $x6920 $x6940))))
+(let ((@x6947 (trans (quant-intro (rewrite (= (=> $x6896 $x6908) $x6920)) (= $x6917 $x6923)) (quant-intro @x6942 (= $x6923 $x6943)) (= $x6917 $x6943))))
+(let ((@x14355 (mp~ (mp (asserted $x6917) @x6947 $x6943) (nnf-pos (refl (~ $x6940 $x6940)) (~ $x6943 $x6943)) $x6943)))
+(let ((@x17967 (mp @x14355 @x17966 $x17964)))
+(let (($x24241 (not $x24240)))
+(let (($x23110 (not $x17964)))
+(let (($x24183 (or $x23110 $x24241 $x11259 $x23791)))
+(let (($x23792 (or $x24241 $x22599 $x22601 $x23791)))
+(let (($x24184 (or $x23110 $x23792)))
+(let ((@x23271 (trans (monotonicity @x22715 @x22724 (= $x23792 (or $x24241 false $x11259 $x23791))) (rewrite (= (or $x24241 false $x11259 $x23791) (or $x24241 $x11259 $x23791))) (= $x23792 (or $x24241 $x11259 $x23791)))))
+(let ((@x23705 (trans (monotonicity @x23271 (= $x24184 (or $x23110 (or $x24241 $x11259 $x23791)))) (rewrite (= (or $x23110 (or $x24241 $x11259 $x23791)) $x24183)) (= $x24184 $x24183))))
+(let ((@x23755 (unit-resolution (mp ((_ quant-inst v_b_S_s$ v_b_P_H_arr$ b_T_T_u1$ v_b_P_H_len$ 0) $x24184) @x23705 $x24183) @x17967 @x12041 @x24355 (hypothesis $x23737) false)))
+(let (($x21186 (= ?x21014 ?x10079)))
+(let (($x21191 (or $x21152 $x21186)))
+(let ((@x21192 ((_ quant-inst (b_S_array$ b_T_T_u1$ v_b_P_H_len$) (b_S_ref$ ?x10078)) $x21191)))
+(let ((@x24524 (trans (monotonicity @x24520 (= ?x24419 ?x21014)) (unit-resolution @x21192 @x19840 $x21186) (= ?x24419 ?x10079))))
+(let ((@x24532 (trans @x24530 (unit-resolution @x22000 @x15336 @x12044 $x21990) (= ?x22595 ?x21983))))
+(let ((@x23632 (trans (monotonicity @x24532 (= ?x24245 ?x24410)) (hypothesis $x24436) (= ?x24245 ?x24433))))
+(let ((@x23628 (trans @x23632 (monotonicity (trans @x24524 @x24511 (= ?x24419 v_b_P_H_arr$)) (= ?x24433 ?x10078)) (= ?x24245 ?x10078))))
+(let ((@x23622 (trans (trans @x23628 (symm @x22852 (= ?x10078 ?x22553)) (= ?x24245 ?x22553)) (symm @x24124 (= ?x22553 ?x10137)) (= ?x24245 ?x10137))))
+(let ((@x23636 (symm (monotonicity (trans @x23622 @x23350 (= ?x24245 ?x22505)) (= ?x24246 ?x22655)) (= ?x22655 ?x24246))))
+(let ((@x23256 (monotonicity (monotonicity (trans @x23663 @x23350 (= ?x10078 ?x22505)) (= ?x22818 ?x22655)) (= ?x22903 (b_S_ts_n_emb$ ?x22655)))))
+(let ((@x23678 (trans @x23256 (monotonicity @x23636 (= (b_S_ts_n_emb$ ?x22655) ?x24247)) (= ?x22903 ?x24247))))
+(let ((@x23865 (trans @x23678 (unit-resolution (def-axiom (or $x23737 $x24248)) (lemma @x23755 $x23791) $x24248) (= ?x22903 ?x22595))))
+(let ((@x23912 (trans (monotonicity (trans @x23865 @x24530 (= ?x22903 ?x10080)) (= ?x22893 ?x10082)) @x12043 $x22888)))
+(let ((@x24132 (lemma (unit-resolution (hypothesis (not $x22888)) @x23912 false) (or $x24439 $x22888))))
+(let ((@x23115 (unit-resolution @x24132 (unit-resolution @x24460 (lemma @x24133 $x24445) $x24436) $x22888)))
+(let ((?x22658 (b_S_ts_n_emb$ ?x22655)))
+(let ((?x22663 (b_S_typ$ ?x22658)))
+(let ((?x22664 (b_S_kind_n_of$ ?x22663)))
+(let (($x22665 (= ?x22664 b_S_kind_n_primitive$)))
+(let ((@x23071 (monotonicity (monotonicity (symm @x23256 (= ?x22658 ?x22903)) (= ?x22663 ?x22890)) (= ?x22664 ?x22891))))
+(let (($x22946 (b_S_is_n_non_n_primitive$ ?x22663)))
+(let (($x23237 (not $x22946)))
+(let (($x23503 (or $x22665 $x23237)))
+(let (($x23504 (not $x23503)))
+(let (($x19234 (forall ((?v0 B_S_type_n_state$) )(!(let (($x9543 (= (b_S_kind_n_of$ (b_S_typ$ (b_S_ts_n_emb$ ?v0))) b_S_kind_n_primitive$)))
+(let (($x19230 (or $x9543 (not (b_S_is_n_non_n_primitive$ (b_S_typ$ (b_S_ts_n_emb$ ?v0)))))))
+(not $x19230))) :pattern ( (b_S_ts_n_emb$ ?v0) )))
+))
+(let (($x9548 (forall ((?v0 B_S_type_n_state$) )(!(let (($x9543 (= (b_S_kind_n_of$ (b_S_typ$ (b_S_ts_n_emb$ ?v0))) b_S_kind_n_primitive$)))
+(and (not $x9543) (b_S_is_n_non_n_primitive$ (b_S_typ$ (b_S_ts_n_emb$ ?v0))))) :pattern ( (b_S_ts_n_emb$ ?v0) )))
+))
+(let (($x9543 (= (b_S_kind_n_of$ (b_S_typ$ (b_S_ts_n_emb$ ?0))) b_S_kind_n_primitive$)))
+(let (($x19230 (or $x9543 (not (b_S_is_n_non_n_primitive$ (b_S_typ$ (b_S_ts_n_emb$ ?0)))))))
+(let (($x9546 (and (not $x9543) (b_S_is_n_non_n_primitive$ (b_S_typ$ (b_S_ts_n_emb$ ?0))))))
+(let ((@x15316 (mp~ (asserted $x9548) (nnf-pos (refl (~ $x9546 $x9546)) (~ $x9548 $x9548)) $x9548)))
+(let ((@x19237 (mp @x15316 (quant-intro (rewrite (= $x9546 (not $x19230))) (= $x9548 $x19234)) $x19234)))
+(let (($x23057 (or (not $x19234) $x23504)))
+(let ((@x23058 ((_ quant-inst (b_S_select_o_tm$ ?x10272 ?x22505)) $x23057)))
+(let ((@x23584 (unit-resolution (def-axiom (or $x23503 (not $x22665))) (unit-resolution @x23058 @x19237 $x23504) (not $x22665))))
+(let ((@x23060 (lemma (unit-resolution @x23584 (trans @x23071 (hypothesis $x22892) $x22665) false) (not $x22892))))
+(let ((@x23231 (unit-resolution (def-axiom (or $x22901 $x22817 $x22889 $x22892 $x22896)) @x23060 (unit-resolution (def-axiom (or $x22895 (not $x22888))) @x23115 $x22895) (or $x22901 $x22817 $x22889))))
+(let ((@x23406 (unit-resolution @x23231 @x23233 (unit-resolution (def-axiom (or $x22906 $x22902)) @x23294 $x22906) @x23076 false)))
+(let ((@x23403 (lemma @x23406 $x10141)))
+(let (($x20092 (or $x19318 $x20089)))
+(let (($x20095 (not $x20092)))
+(let (($x20098 (or $x11385 $x20095)))
+(let (($x20101 (not $x20098)))
+(let (($x20104 (or $x11385 $x20101)))
+(let (($x20107 (not $x20104)))
+(let (($x19727 (not $x10148)))
+(let (($x19726 (not $x10147)))
+(let (($x19725 (not $x10146)))
+(let (($x19724 (not $x10145)))
+(let (($x15511 (not $x10141)))
+(let (($x15502 (not $x10138)))
+(let (($x20110 (or $x15502 $x15511 $x19724 $x19725 $x19726 $x19727 $x20107)))
+(let (($x20113 (not $x20110)))
+(let (($x20116 (or $x15502 $x15511 $x20113)))
+(let (($x20119 (not $x20116)))
+(let (($x20122 (or $x15502 $x15505 $x20119)))
+(let (($x20125 (not $x20122)))
+(let (($x20128 (or $x15502 $x15505 $x20125)))
+(let (($x20131 (not $x20128)))
+(let (($x20134 (or $x11221 $x20131)))
+(let (($x20137 (not $x20134)))
+(let (($x20140 (or $x11221 $x20137)))
+(let (($x19617 (forall ((?v0 Int) )(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x10238 (= ?x10163 v_b_S_result_G_0$)))
+(let (($x11800 (>= (+ ?v0 (* (- 1) v_b_P_H_len$)) 0)))
+(let (($x12168 (<= ?v0 4294967295)))
+(let (($x16553 (not $x12168)))
+(let (($x2815 (>= ?v0 0)))
+(let (($x3763 (not $x2815)))
+(or $x3763 $x16553 $x11800 (not $x10238))))))))))
+))
+(let (($x19602 (forall ((?v0 Int) )(let ((?x11816 (* (- 1) v_b_S_result_G_0$)))
+(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x11818 (<= (+ ?x10163 ?x11816) 0)))
+(let (($x11800 (>= (+ ?v0 (* (- 1) v_b_P_H_len$)) 0)))
+(let (($x12168 (<= ?v0 4294967295)))
+(let (($x16553 (not $x12168)))
+(let (($x2815 (>= ?v0 0)))
+(let (($x3763 (not $x2815)))
+(or $x3763 $x16553 $x11800 $x11818))))))))))
+))
+(let (($x19626 (not (or (not $x19602) (not $x19617)))))
+(let (($x19631 (or $x19580 $x19626)))
+(let (($x19643 (not (or $x15729 $x19474 $x19501 $x19637 $x19638 $x19639 $x19640 (not $x19631)))))
+(let (($x19648 (or $x15729 $x19643)))
+(let (($x19656 (not (or $x11487 $x19474 $x19501 (not $x19648)))))
+(let (($x19408 (forall ((?v0 Int) )(let ((?x11631 (* (- 1) v_b_L_H_max_G_3$)))
+(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x11633 (<= (+ ?x10163 ?x11631) 0)))
+(let (($x11615 (>= (+ ?v0 (* (- 1) v_b_L_H_p_G_1$)) 0)))
+(let (($x12168 (<= ?v0 4294967295)))
+(let (($x16553 (not $x12168)))
+(let (($x2815 (>= ?v0 0)))
+(let (($x3763 (not $x2815)))
+(or $x3763 $x16553 $x11615 $x11633))))))))))
+))
+(let (($x19428 (not (or (not $x19408) $x19413))))
+(let (($x19433 (or $x19386 $x19428)))
+(let (($x19441 (not (or $x11612 (not $x19433)))))
+(let (($x19446 (or $x11612 $x19441)))
+(let (($x19458 (not (or $x15611 $x15614 $x19452 $x19453 $x19454 $x19455 (not $x19446)))))
+(let (($x19463 (or $x15611 $x15614 $x19458)))
+(let (($x19475 (not $x19463)))
+(let (($x19515 (not (or $x11515 $x19501 $x19512 $x19513 $x19474 $x19455 $x19475))))
+(let (($x19477 (not (or $x15590 $x15599 $x19469 $x19470 $x19471 $x19472 $x19473 $x19474 $x19455 $x19475))))
+(let (($x19482 (or $x15590 $x15599 $x19477)))
+(let (($x19490 (not (or $x15590 $x15593 (not $x19482)))))
+(let (($x19495 (or $x15590 $x15593 $x19490)))
+(let (($x19504 (not (or $x11516 $x19474 $x19501 (not $x19495)))))
+(let (($x19520 (or $x19504 $x19515)))
+(let (($x19528 (not (or $x15590 $x15599 $x19474 $x19501 (not $x19520)))))
+(let (($x19533 (or $x15590 $x15599 $x19528)))
+(let (($x19541 (not (or $x15590 $x15593 (not $x19533)))))
+(let (($x19546 (or $x15590 $x15593 $x19541)))
+(let (($x19554 (not (or $x11486 $x19474 $x19501 (not $x19546)))))
+(let (($x19661 (or $x19554 $x19656)))
+(let (($x19362 (forall ((?v0 Int) )(let ((?x11887 (* (- 1) v_b_L_H_max_G_1$)))
+(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x11889 (<= (+ ?x10163 ?x11887) 0)))
+(let (($x11871 (>= (+ ?v0 (* (- 1) v_b_L_H_p_G_0$)) 0)))
+(let (($x12168 (<= ?v0 4294967295)))
+(let (($x16553 (not $x12168)))
+(let (($x2815 (>= ?v0 0)))
+(let (($x3763 (not $x2815)))
+(or $x3763 $x16553 $x11871 $x11889))))))))))
+))
+(let (($x19685 (or $x11259 $x15548 $x19667 $x19668 $x19669 $x19670 $x19671 $x19672 (not $x19362) $x11867 $x19674 $x19675 $x19676 $x19677 $x19678 $x19679 $x19680 $x19681 $x19682 $x19683 $x19474 $x19501 (not $x19661))))
+(let (($x19686 (not $x19685)))
+(let (($x19691 (or $x11259 $x15548 $x19686)))
+(let (($x19340 (forall ((?v0 Int) )(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x11404 (>= (+ v_b_L_H_max_G_0$ (* (- 1) ?x10163)) 0)))
+(let (($x11388 (>= ?v0 1)))
+(let (($x12168 (<= ?v0 4294967295)))
+(let (($x16553 (not $x12168)))
+(let (($x2815 (>= ?v0 0)))
+(let (($x3763 (not $x2815)))
+(or $x3763 $x16553 $x11388 $x11404)))))))))
+))
+(let (($x19700 (not (or (not $x19340) (not $x19691)))))
+(let (($x19705 (or $x19318 $x19700)))
+(let (($x19713 (not (or $x11385 (not $x19705)))))
+(let (($x19718 (or $x11385 $x19713)))
+(let (($x19730 (not (or $x15502 $x15511 $x19724 $x19725 $x19726 $x19727 (not $x19718)))))
+(let (($x19735 (or $x15502 $x15511 $x19730)))
+(let (($x19743 (not (or $x15502 $x15505 (not $x19735)))))
+(let (($x19748 (or $x15502 $x15505 $x19743)))
+(let (($x19756 (not (or $x11221 (not $x19748)))))
+(let (($x19761 (or $x11221 $x19756)))
+(let (($x12168 (<= ?0 4294967295)))
+(let (($x16553 (not $x12168)))
+(let (($x19606 (or $x3763 $x16553 $x11800 (not $x10238))))
+(let ((@x20037 (monotonicity (quant-intro (refl (= $x19606 $x19606)) (= $x19617 $x20030)) (= (not $x19617) $x20035))))
+(let ((@x20026 (quant-intro (refl (= (or $x3763 $x16553 $x11800 $x11818) (or $x3763 $x16553 $x11800 $x11818))) (= $x19602 $x20022))))
+(let ((@x20040 (monotonicity (monotonicity @x20026 (= (not $x19602) $x20027)) @x20037 (= (or (not $x19602) (not $x19617)) $x20038))))
+(let ((@x20049 (monotonicity (monotonicity (monotonicity @x20040 (= $x19626 $x20041)) (= $x19631 $x20044)) (= (not $x19631) $x20047))))
+(let ((@x20052 (monotonicity @x20049 (= (or $x15729 $x19474 $x19501 $x19637 $x19638 $x19639 $x19640 (not $x19631)) $x20050))))
+(let ((@x20061 (monotonicity (monotonicity (monotonicity @x20052 (= $x19643 $x20053)) (= $x19648 $x20056)) (= (not $x19648) $x20059))))
+(let ((@x20067 (monotonicity (monotonicity @x20061 (= (or $x11487 $x19474 $x19501 (not $x19648)) $x20062)) (= $x19656 $x20065))))
+(let ((@x19910 (quant-intro (refl (= (or $x3763 $x16553 $x11615 $x11633) (or $x3763 $x16553 $x11615 $x11633))) (= $x19408 $x19906))))
+(let ((@x19916 (monotonicity (monotonicity @x19910 (= (not $x19408) $x19911)) (= (or (not $x19408) $x19413) $x19914))))
+(let ((@x19925 (monotonicity (monotonicity (monotonicity @x19916 (= $x19428 $x19917)) (= $x19433 $x19920)) (= (not $x19433) $x19923))))
+(let ((@x19931 (monotonicity (monotonicity @x19925 (= (or $x11612 (not $x19433)) $x19926)) (= $x19441 $x19929))))
+(let ((@x19937 (monotonicity (monotonicity @x19931 (= $x19446 $x19932)) (= (not $x19446) $x19935))))
+(let ((@x19940 (monotonicity @x19937 (= (or $x15611 $x15614 $x19452 $x19453 $x19454 $x19455 (not $x19446)) $x19938))))
+(let ((@x19949 (monotonicity (monotonicity (monotonicity @x19940 (= $x19458 $x19941)) (= $x19463 $x19944)) (= $x19475 $x19947))))
+(let ((@x19982 (monotonicity @x19949 (= (or $x11515 $x19501 $x19512 $x19513 $x19474 $x19455 $x19475) $x19980))))
+(let ((@x19952 (monotonicity @x19949 (= (or $x15590 $x15599 $x19469 $x19470 $x19471 $x19472 $x19473 $x19474 $x19455 $x19475) $x19950))))
+(let ((@x19961 (monotonicity (monotonicity (monotonicity @x19952 (= $x19477 $x19953)) (= $x19482 $x19956)) (= (not $x19482) $x19959))))
+(let ((@x19967 (monotonicity (monotonicity @x19961 (= (or $x15590 $x15593 (not $x19482)) $x19962)) (= $x19490 $x19965))))
+(let ((@x19973 (monotonicity (monotonicity @x19967 (= $x19495 $x19968)) (= (not $x19495) $x19971))))
+(let ((@x19979 (monotonicity (monotonicity @x19973 (= (or $x11516 $x19474 $x19501 (not $x19495)) $x19974)) (= $x19504 $x19977))))
+(let ((@x19988 (monotonicity @x19979 (monotonicity @x19982 (= $x19515 $x19983)) (= $x19520 $x19986))))
+(let ((@x19994 (monotonicity (monotonicity @x19988 (= (not $x19520) $x19989)) (= (or $x15590 $x15599 $x19474 $x19501 (not $x19520)) $x19992))))
+(let ((@x20003 (monotonicity (monotonicity (monotonicity @x19994 (= $x19528 $x19995)) (= $x19533 $x19998)) (= (not $x19533) $x20001))))
+(let ((@x20009 (monotonicity (monotonicity @x20003 (= (or $x15590 $x15593 (not $x19533)) $x20004)) (= $x19541 $x20007))))
+(let ((@x20015 (monotonicity (monotonicity @x20009 (= $x19546 $x20010)) (= (not $x19546) $x20013))))
+(let ((@x20021 (monotonicity (monotonicity @x20015 (= (or $x11486 $x19474 $x19501 (not $x19546)) $x20016)) (= $x19554 $x20019))))
+(let ((@x20073 (monotonicity (monotonicity @x20021 @x20067 (= $x19661 $x20068)) (= (not $x19661) $x20071))))
+(let ((@x19902 (quant-intro (refl (= (or $x3763 $x16553 $x11871 $x11889) (or $x3763 $x16553 $x11871 $x11889))) (= $x19362 $x19898))))
+(let ((@x20076 (monotonicity (monotonicity @x19902 (= (not $x19362) $x19903)) @x20073 (= $x19685 $x20074))))
+(let ((@x20085 (monotonicity (monotonicity (monotonicity @x20076 (= $x19686 $x20077)) (= $x19691 $x20080)) (= (not $x19691) $x20083))))
+(let ((@x19894 (quant-intro (refl (= (or $x3763 $x16553 $x11388 $x11404) (or $x3763 $x16553 $x11388 $x11404))) (= $x19340 $x19890))))
+(let ((@x20088 (monotonicity (monotonicity @x19894 (= (not $x19340) $x19895)) @x20085 (= (or (not $x19340) (not $x19691)) $x20086))))
+(let ((@x20097 (monotonicity (monotonicity (monotonicity @x20088 (= $x19700 $x20089)) (= $x19705 $x20092)) (= (not $x19705) $x20095))))
+(let ((@x20103 (monotonicity (monotonicity @x20097 (= (or $x11385 (not $x19705)) $x20098)) (= $x19713 $x20101))))
+(let ((@x20109 (monotonicity (monotonicity @x20103 (= $x19718 $x20104)) (= (not $x19718) $x20107))))
+(let ((@x20112 (monotonicity @x20109 (= (or $x15502 $x15511 $x19724 $x19725 $x19726 $x19727 (not $x19718)) $x20110))))
+(let ((@x20121 (monotonicity (monotonicity (monotonicity @x20112 (= $x19730 $x20113)) (= $x19735 $x20116)) (= (not $x19735) $x20119))))
+(let ((@x20127 (monotonicity (monotonicity @x20121 (= (or $x15502 $x15505 (not $x19735)) $x20122)) (= $x19743 $x20125))))
+(let ((@x20133 (monotonicity (monotonicity @x20127 (= $x19748 $x20128)) (= (not $x19748) $x20131))))
+(let ((@x20139 (monotonicity (monotonicity @x20133 (= (or $x11221 (not $x19748)) $x20134)) (= $x19756 $x20137))))
+(let (($x15761 (forall ((?v0 Int) )(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x10238 (= ?x10163 v_b_S_result_G_0$)))
+(let (($x11800 (>= (+ ?v0 (* (- 1) v_b_P_H_len$)) 0)))
+(let (($x11802 (not $x11800)))
+(let (($x12168 (<= ?v0 4294967295)))
+(let (($x2815 (>= ?v0 0)))
+(let (($x13448 (and $x2815 $x12168 $x11802 $x10238)))
+(not $x13448)))))))))
+))
+(let (($x13442 (forall ((?v0 Int) )(let ((?x11816 (* (- 1) v_b_S_result_G_0$)))
+(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x11818 (<= (+ ?x10163 ?x11816) 0)))
+(let (($x11800 (>= (+ ?v0 (* (- 1) v_b_P_H_len$)) 0)))
+(let (($x11802 (not $x11800)))
+(let (($x12168 (<= ?v0 4294967295)))
+(let (($x2815 (>= ?v0 0)))
+(let (($x13433 (and $x2815 $x12168 $x11802)))
+(let (($x13436 (not $x13433)))
+(or $x13436 $x11818)))))))))))
+))
+(let (($x15765 (and $x13442 $x15761)))
+(let (($x16014 (not $x16009)))
+(let (($x16017 (and $x15736 $x15737 $x16014)))
+(let (($x16020 (not $x16017)))
+(let (($x16036 (or $x16020 $x16031)))
+(let (($x16039 (not $x16036)))
+(let (($x16042 (or $x16039 $x15765)))
+(let (($x16048 (and b_S_position_n_marker$ $x11429 $x11432 $x10216 $x10218 $x10220 $x10222 $x16042)))
+(let (($x16053 (or $x15729 $x16048)))
+(let (($x16059 (and $x11486 $x11429 $x11432 $x16053)))
+(let (($x15648 (not $x11651)))
+(let (($x13373 (forall ((?v0 Int) )(let ((?x11631 (* (- 1) v_b_L_H_max_G_3$)))
+(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x11633 (<= (+ ?x10163 ?x11631) 0)))
+(let (($x11615 (>= (+ ?v0 (* (- 1) v_b_L_H_p_G_1$)) 0)))
+(let (($x11617 (not $x11615)))
+(let (($x12168 (<= ?v0 4294967295)))
+(let (($x2815 (>= ?v0 0)))
+(let (($x13364 (and $x2815 $x12168 $x11617)))
+(let (($x13367 (not $x13364)))
+(or $x13367 $x11633)))))))))))
+))
+(let (($x15651 (and $x13373 $x15648)))
+(let (($x15876 (not $x15871)))
+(let (($x15879 (and $x15626 $x15627 $x15876)))
+(let (($x15882 (not $x15879)))
+(let (($x15898 (or $x15882 $x15893)))
+(let (($x15901 (not $x15898)))
+(let (($x15904 (or $x15901 $x15651)))
+(let (($x15907 (and $x11608 $x15904)))
+(let (($x15910 (or $x11612 $x15907)))
+(let (($x15916 (and $x11570 $x13353 $x11580 $x10358 $x11578 $x11536 $x15910)))
+(let (($x15921 (or $x15611 $x15614 $x15916)))
+(let (($x15959 (and $x11516 $x11432 $x10391 $x10392 $x11429 $x11536 $x15921)))
+(let (($x15927 (and $x10321 $x10324 $x10333 $x10334 $x10335 $x10338 $x10340 $x11429 $x11536 $x15921)))
+(let (($x15932 (or $x15590 $x15599 $x15927)))
+(let (($x15938 (and $x10321 $x10322 $x15932)))
+(let (($x15943 (or $x15590 $x15593 $x15938)))
+(let (($x15949 (and $x11515 $x11429 $x11432 $x15943)))
+(let (($x15964 (or $x15949 $x15959)))
+(let (($x15970 (and $x10321 $x10324 $x11429 $x11432 $x15964)))
+(let (($x15975 (or $x15590 $x15599 $x15970)))
+(let (($x15981 (and $x10321 $x10322 $x15975)))
+(let (($x15986 (or $x15590 $x15593 $x15981)))
+(let (($x15992 (and $x11487 $x11429 $x11432 $x15986)))
+(let (($x16064 (or $x15992 $x16059)))
+(let (($x13340 (forall ((?v0 Int) )(let ((?x11887 (* (- 1) v_b_L_H_max_G_1$)))
+(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x11889 (<= (+ ?x10163 ?x11887) 0)))
+(let (($x11871 (>= (+ ?v0 (* (- 1) v_b_L_H_p_G_0$)) 0)))
+(let (($x11873 (not $x11871)))
+(let (($x12168 (<= ?v0 4294967295)))
+(let (($x2815 (>= ?v0 0)))
+(let (($x13331 (and $x2815 $x12168 $x11873)))
+(let (($x13334 (not $x13331)))
+(or $x13334 $x11889)))))))))))
+))
+(let (($x16070 (and $x11260 $x10167 $x11911 $x13304 $x13315 $x11901 $x13326 $x11898 $x13340 $x11868 $x10192 $x10284 $x10204 $x10097 $x10291 $x10292 $x10293 $x10294 $x10295 $x10296 $x11429 $x11432 $x16064)))
+(let (($x16075 (or $x11259 $x15548 $x16070)))
+(let (($x13292 (forall ((?v0 Int) )(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x11404 (>= (+ v_b_L_H_max_G_0$ (* (- 1) ?x10163)) 0)))
+(let (($x11388 (>= ?v0 1)))
+(let (($x11389 (not $x11388)))
+(let (($x12168 (<= ?v0 4294967295)))
+(let (($x2815 (>= ?v0 0)))
+(let (($x13283 (and $x2815 $x12168 $x11389)))
+(let (($x13286 (not $x13283)))
+(or $x13286 $x11404))))))))))
+))
+(let (($x16078 (and $x13292 $x16075)))
+(let (($x15528 (not (and $x15523 $x15524 (not $x15525)))))
+(let (($x15534 (or $x15528 $x15533)))
+(let (($x15535 (not $x15534)))
+(let (($x16081 (or $x15535 $x16078)))
+(let (($x16084 (and $x11382 $x16081)))
+(let (($x16087 (or $x11385 $x16084)))
+(let (($x16093 (and $x10138 $x10141 $x10145 $x10146 $x10147 $x10148 $x16087)))
+(let (($x16098 (or $x15502 $x15511 $x16093)))
+(let (($x16104 (and $x10138 $x10139 $x16098)))
+(let (($x16109 (or $x15502 $x15505 $x16104)))
+(let (($x16112 (and $x10136 $x16109)))
+(let (($x16115 (or $x11221 $x16112)))
+(let (($x19664 (and $x11260 $x10167 $x11911 $x13304 $x13315 $x11901 $x13326 $x11898 $x19362 $x11868 $x10192 $x10284 $x10204 $x10097 $x10291 $x10292 $x10293 $x10294 $x10295 $x10296 $x11429 $x11432 $x19661)))
+(let (($x19644 (= (and b_S_position_n_marker$ $x11429 $x11432 $x10216 $x10218 $x10220 $x10222 $x19631) $x19643)))
+(let (($x19635 (= $x16048 (and b_S_position_n_marker$ $x11429 $x11432 $x10216 $x10218 $x10220 $x10222 $x19631))))
+(let ((@x19612 (monotonicity (rewrite (= (and $x2815 $x12168 $x11802 $x10238) (not $x19606))) (= (not (and $x2815 $x12168 $x11802 $x10238)) (not (not $x19606))))))
+(let ((@x19616 (trans @x19612 (rewrite (= (not (not $x19606)) $x19606)) (= (not (and $x2815 $x12168 $x11802 $x10238)) $x19606))))
+(let ((@x19599 (rewrite (= (or (or $x3763 $x16553 $x11800) $x11818) (or $x3763 $x16553 $x11800 $x11818)))))
+(let (($x13433 (and $x2815 $x12168 $x11802)))
+(let (($x13436 (not $x13433)))
+(let (($x13439 (or $x13436 $x11818)))
+(let ((@x19589 (monotonicity (rewrite (= $x13433 (not (or $x3763 $x16553 $x11800)))) (= $x13436 (not (not (or $x3763 $x16553 $x11800)))))))
+(let ((@x19593 (trans @x19589 (rewrite (= (not (not (or $x3763 $x16553 $x11800))) (or $x3763 $x16553 $x11800))) (= $x13436 (or $x3763 $x16553 $x11800)))))
+(let ((@x19601 (trans (monotonicity @x19593 (= $x13439 (or (or $x3763 $x16553 $x11800) $x11818))) @x19599 (= $x13439 (or $x3763 $x16553 $x11800 $x11818)))))
+(let ((@x19622 (monotonicity (quant-intro @x19601 (= $x13442 $x19602)) (quant-intro @x19616 (= $x15761 $x19617)) (= $x15765 (and $x19602 $x19617)))))
+(let ((@x19567 (monotonicity (rewrite (= $x16017 (not (or $x19559 $x19560 $x16009)))) (= $x16020 (not (not (or $x19559 $x19560 $x16009)))))))
+(let ((@x19571 (trans @x19567 (rewrite (= (not (not (or $x19559 $x19560 $x16009))) (or $x19559 $x19560 $x16009))) (= $x16020 (or $x19559 $x19560 $x16009)))))
+(let ((@x19579 (trans (monotonicity @x19571 (= $x16036 (or (or $x19559 $x19560 $x16009) $x16031))) (rewrite (= (or (or $x19559 $x19560 $x16009) $x16031) $x19575)) (= $x16036 $x19575))))
+(let ((@x19633 (monotonicity (monotonicity @x19579 (= $x16039 $x19580)) (trans @x19622 (rewrite (= (and $x19602 $x19617) $x19626)) (= $x15765 $x19626)) (= $x16042 $x19631))))
+(let ((@x19650 (monotonicity (trans (monotonicity @x19633 $x19635) (rewrite $x19644) (= $x16048 $x19643)) (= $x16053 $x19648))))
+(let ((@x19660 (trans (monotonicity @x19650 (= $x16059 (and $x11486 $x11429 $x11432 $x19648))) (rewrite (= (and $x11486 $x11429 $x11432 $x19648) $x19656)) (= $x16059 $x19656))))
+(let ((@x19422 (trans (monotonicity (rewrite (= $x11651 $x19413)) (= $x15648 (not $x19413))) (rewrite (= (not $x19413) $x19412)) (= $x15648 $x19412))))
+(let ((@x19405 (rewrite (= (or (or $x3763 $x16553 $x11615) $x11633) (or $x3763 $x16553 $x11615 $x11633)))))
+(let (($x13364 (and $x2815 $x12168 $x11617)))
+(let (($x13367 (not $x13364)))
+(let (($x13370 (or $x13367 $x11633)))
+(let ((@x19395 (monotonicity (rewrite (= $x13364 (not (or $x3763 $x16553 $x11615)))) (= $x13367 (not (not (or $x3763 $x16553 $x11615)))))))
+(let ((@x19399 (trans @x19395 (rewrite (= (not (not (or $x3763 $x16553 $x11615))) (or $x3763 $x16553 $x11615))) (= $x13367 (or $x3763 $x16553 $x11615)))))
+(let ((@x19407 (trans (monotonicity @x19399 (= $x13370 (or (or $x3763 $x16553 $x11615) $x11633))) @x19405 (= $x13370 (or $x3763 $x16553 $x11615 $x11633)))))
+(let ((@x19425 (monotonicity (quant-intro @x19407 (= $x13373 $x19408)) @x19422 (= $x15651 (and $x19408 $x19412)))))
+(let ((@x19373 (monotonicity (rewrite (= $x15879 (not (or $x19365 $x19366 $x15871)))) (= $x15882 (not (not (or $x19365 $x19366 $x15871)))))))
+(let ((@x19377 (trans @x19373 (rewrite (= (not (not (or $x19365 $x19366 $x15871))) (or $x19365 $x19366 $x15871))) (= $x15882 (or $x19365 $x19366 $x15871)))))
+(let ((@x19385 (trans (monotonicity @x19377 (= $x15898 (or (or $x19365 $x19366 $x15871) $x15893))) (rewrite (= (or (or $x19365 $x19366 $x15871) $x15893) $x19381)) (= $x15898 $x19381))))
+(let ((@x19435 (monotonicity (monotonicity @x19385 (= $x15901 $x19386)) (trans @x19425 (rewrite (= (and $x19408 $x19412) $x19428)) (= $x15651 $x19428)) (= $x15904 $x19433))))
+(let ((@x19445 (trans (monotonicity @x19435 (= $x15907 (and $x11608 $x19433))) (rewrite (= (and $x11608 $x19433) $x19441)) (= $x15907 $x19441))))
+(let ((@x19451 (monotonicity (monotonicity @x19445 (= $x15910 $x19446)) (= $x15916 (and $x11570 $x13353 $x11580 $x10358 $x11578 $x11536 $x19446)))))
+(let ((@x19462 (trans @x19451 (rewrite (= (and $x11570 $x13353 $x11580 $x10358 $x11578 $x11536 $x19446) $x19458)) (= $x15916 $x19458))))
+(let ((@x19511 (monotonicity (monotonicity @x19462 (= $x15921 $x19463)) (= $x15959 (and $x11516 $x11432 $x10391 $x10392 $x11429 $x11536 $x19463)))))
+(let ((@x19519 (trans @x19511 (rewrite (= (and $x11516 $x11432 $x10391 $x10392 $x11429 $x11536 $x19463) $x19515)) (= $x15959 $x19515))))
+(let ((@x19479 (rewrite (= (and $x10321 $x10324 $x10333 $x10334 $x10335 $x10338 $x10340 $x11429 $x11536 $x19463) $x19477))))
+(let ((@x19468 (monotonicity (monotonicity @x19462 (= $x15921 $x19463)) (= $x15927 (and $x10321 $x10324 $x10333 $x10334 $x10335 $x10338 $x10340 $x11429 $x11536 $x19463)))))
+(let ((@x19487 (monotonicity (monotonicity (trans @x19468 @x19479 (= $x15927 $x19477)) (= $x15932 $x19482)) (= $x15938 (and $x10321 $x10322 $x19482)))))
+(let ((@x19494 (trans @x19487 (rewrite (= (and $x10321 $x10322 $x19482) $x19490)) (= $x15938 $x19490))))
+(let ((@x19500 (monotonicity (monotonicity @x19494 (= $x15943 $x19495)) (= $x15949 (and $x11515 $x11429 $x11432 $x19495)))))
+(let ((@x19508 (trans @x19500 (rewrite (= (and $x11515 $x11429 $x11432 $x19495) $x19504)) (= $x15949 $x19504))))
+(let ((@x19525 (monotonicity (monotonicity @x19508 @x19519 (= $x15964 $x19520)) (= $x15970 (and $x10321 $x10324 $x11429 $x11432 $x19520)))))
+(let ((@x19532 (trans @x19525 (rewrite (= (and $x10321 $x10324 $x11429 $x11432 $x19520) $x19528)) (= $x15970 $x19528))))
+(let ((@x19538 (monotonicity (monotonicity @x19532 (= $x15975 $x19533)) (= $x15981 (and $x10321 $x10322 $x19533)))))
+(let ((@x19545 (trans @x19538 (rewrite (= (and $x10321 $x10322 $x19533) $x19541)) (= $x15981 $x19541))))
+(let ((@x19551 (monotonicity (monotonicity @x19545 (= $x15986 $x19546)) (= $x15992 (and $x11487 $x11429 $x11432 $x19546)))))
+(let ((@x19558 (trans @x19551 (rewrite (= (and $x11487 $x11429 $x11432 $x19546) $x19554)) (= $x15992 $x19554))))
+(let ((@x19359 (rewrite (= (or (or $x3763 $x16553 $x11871) $x11889) (or $x3763 $x16553 $x11871 $x11889)))))
+(let (($x13331 (and $x2815 $x12168 $x11873)))
+(let (($x13334 (not $x13331)))
+(let (($x13337 (or $x13334 $x11889)))
+(let ((@x19349 (monotonicity (rewrite (= $x13331 (not (or $x3763 $x16553 $x11871)))) (= $x13334 (not (not (or $x3763 $x16553 $x11871)))))))
+(let ((@x19353 (trans @x19349 (rewrite (= (not (not (or $x3763 $x16553 $x11871))) (or $x3763 $x16553 $x11871))) (= $x13334 (or $x3763 $x16553 $x11871)))))
+(let ((@x19361 (trans (monotonicity @x19353 (= $x13337 (or (or $x3763 $x16553 $x11871) $x11889))) @x19359 (= $x13337 (or $x3763 $x16553 $x11871 $x11889)))))
+(let ((@x19666 (monotonicity (quant-intro @x19361 (= $x13340 $x19362)) (monotonicity @x19558 @x19660 (= $x16064 $x19661)) (= $x16070 $x19664))))
+(let ((@x19693 (monotonicity (trans @x19666 (rewrite (= $x19664 $x19686)) (= $x16070 $x19686)) (= $x16075 $x19691))))
+(let ((@x19337 (rewrite (= (or (or $x3763 $x16553 $x11388) $x11404) (or $x3763 $x16553 $x11388 $x11404)))))
+(let (($x13283 (and $x2815 $x12168 $x11389)))
+(let (($x13286 (not $x13283)))
+(let (($x13289 (or $x13286 $x11404)))
+(let ((@x19327 (monotonicity (rewrite (= $x13283 (not (or $x3763 $x16553 $x11388)))) (= $x13286 (not (not (or $x3763 $x16553 $x11388)))))))
+(let ((@x19331 (trans @x19327 (rewrite (= (not (not (or $x3763 $x16553 $x11388))) (or $x3763 $x16553 $x11388))) (= $x13286 (or $x3763 $x16553 $x11388)))))
+(let ((@x19339 (trans (monotonicity @x19331 (= $x13289 (or (or $x3763 $x16553 $x11388) $x11404))) @x19337 (= $x13289 (or $x3763 $x16553 $x11388 $x11404)))))
+(let ((@x19696 (monotonicity (quant-intro @x19339 (= $x13292 $x19340)) @x19693 (= $x16078 (and $x19340 $x19691)))))
+(let ((@x19305 (monotonicity (rewrite (= (and $x15523 $x15524 (not $x15525)) (not (or $x19297 $x19298 $x15525)))) (= $x15528 (not (not (or $x19297 $x19298 $x15525)))))))
+(let ((@x19309 (trans @x19305 (rewrite (= (not (not (or $x19297 $x19298 $x15525))) (or $x19297 $x19298 $x15525))) (= $x15528 (or $x19297 $x19298 $x15525)))))
+(let ((@x19317 (trans (monotonicity @x19309 (= $x15534 (or (or $x19297 $x19298 $x15525) $x15533))) (rewrite (= (or (or $x19297 $x19298 $x15525) $x15533) $x19313)) (= $x15534 $x19313))))
+(let ((@x19707 (monotonicity (monotonicity @x19317 (= $x15535 $x19318)) (trans @x19696 (rewrite (= (and $x19340 $x19691) $x19700)) (= $x16078 $x19700)) (= $x16081 $x19705))))
+(let ((@x19717 (trans (monotonicity @x19707 (= $x16084 (and $x11382 $x19705))) (rewrite (= (and $x11382 $x19705) $x19713)) (= $x16084 $x19713))))
+(let ((@x19723 (monotonicity (monotonicity @x19717 (= $x16087 $x19718)) (= $x16093 (and $x10138 $x10141 $x10145 $x10146 $x10147 $x10148 $x19718)))))
+(let ((@x19734 (trans @x19723 (rewrite (= (and $x10138 $x10141 $x10145 $x10146 $x10147 $x10148 $x19718) $x19730)) (= $x16093 $x19730))))
+(let ((@x19740 (monotonicity (monotonicity @x19734 (= $x16098 $x19735)) (= $x16104 (and $x10138 $x10139 $x19735)))))
+(let ((@x19747 (trans @x19740 (rewrite (= (and $x10138 $x10139 $x19735) $x19743)) (= $x16104 $x19743))))
+(let ((@x19753 (monotonicity (monotonicity @x19747 (= $x16109 $x19748)) (= $x16112 (and $x10136 $x19748)))))
+(let ((@x19763 (monotonicity (trans @x19753 (rewrite (= (and $x10136 $x19748) $x19756)) (= $x16112 $x19756)) (= $x16115 $x19761))))
+(let (($x15746 (<= (+ ?x15744 (* (- 1) v_b_S_result_G_0$)) 0)))
+(let (($x15741 (and $x15736 $x15737 (not (>= (+ ?v0!15 (* (- 1) v_b_P_H_len$)) 0)))))
+(let (($x15748 (not (or (not $x15741) $x15746))))
+(let (($x15769 (or $x15748 $x15765)))
+(let (($x15732 (not $x11797)))
+(let (($x15773 (and $x15732 $x15769)))
+(let (($x15777 (or $x15729 $x15773)))
+(let (($x15726 (not $x11777)))
+(let (($x15781 (and $x15726 $x15777)))
+(let (($x15636 (<= (+ ?x15634 (* (- 1) v_b_L_H_max_G_3$)) 0)))
+(let (($x15638 (not (or (not (and $x15626 $x15627 (not (>= (+ ?v0!14 ?x11581) 0)))) $x15636))))
+(let (($x15655 (or $x15638 $x15651)))
+(let (($x15622 (not $x11612)))
+(let (($x15659 (and $x15622 $x15655)))
+(let (($x15663 (or $x11612 $x15659)))
+(let (($x13358 (and $x11570 $x13353 $x11580 $x10358 $x11578 $x11536)))
+(let (($x13361 (not $x13358)))
+(let (($x15617 (not $x13361)))
+(let (($x15667 (and $x15617 $x15663)))
+(let (($x15671 (or $x15611 $x15614 $x15667)))
+(let (($x15695 (not $x11730)))
+(let (($x15698 (and $x15695 $x15671)))
+(let (($x15608 (not $x11567)))
+(let (($x15675 (and $x15608 $x15671)))
+(let (($x15679 (or $x15590 $x15599 $x15675)))
+(let (($x15596 (not $x11001)))
+(let (($x15683 (and $x15596 $x15679)))
+(let (($x15687 (or $x15590 $x15593 $x15683)))
+(let (($x15605 (not $x11532)))
+(let (($x15691 (and $x15605 $x15687)))
+(let (($x15702 (or $x15691 $x15698)))
+(let (($x15602 (not $x11512)))
+(let (($x15706 (and $x15602 $x15702)))
+(let (($x15710 (or $x15590 $x15599 $x15706)))
+(let (($x15714 (and $x15596 $x15710)))
+(let (($x15718 (or $x15590 $x15593 $x15714)))
+(let (($x15587 (not $x11501)))
+(let (($x15722 (and $x15587 $x15718)))
+(let (($x15785 (or $x15722 $x15781)))
+(let (($x15584 (not $x11481)))
+(let (($x13343 (and $x11260 $x10167 $x11911 $x13304 $x13315 $x11901 $x13326 $x11898 $x13340 $x11868 $x10192 $x11429 $x11432)))
+(let (($x15789 (and $x13343 $x15584 $x15785)))
+(let (($x15545 (not $x11260)))
+(let (($x15793 (or $x15545 $x15548 $x15789)))
+(let (($x15797 (and $x13292 $x15793)))
+(let (($x15801 (or $x15535 $x15797)))
+(let (($x15519 (not $x11385)))
+(let (($x15805 (and $x15519 $x15801)))
+(let (($x15809 (or $x11385 $x15805)))
+(let (($x15514 (not $x11379)))
+(let (($x15813 (and $x15514 $x15809)))
+(let (($x15817 (or $x15502 $x15511 $x15813)))
+(let (($x15508 (not $x11209)))
+(let (($x15821 (and $x15508 $x15817)))
+(let (($x15825 (or $x15502 $x15505 $x15821)))
+(let (($x15499 (not $x11221)))
+(let (($x15829 (and $x15499 $x15825)))
+(let (($x15833 (or $x11221 $x15829)))
+(let (($x16024 (= (+ ?x15744 (* (- 1) v_b_S_result_G_0$)) (+ (* (- 1) v_b_S_result_G_0$) ?x15744))))
+(let ((@x16028 (monotonicity (rewrite $x16024) (= $x15746 (<= (+ (* (- 1) v_b_S_result_G_0$) ?x15744) 0)))))
+(let ((@x16035 (trans @x16028 (rewrite (= (<= (+ (* (- 1) v_b_S_result_G_0$) ?x15744) 0) $x16031)) (= $x15746 $x16031))))
+(let (($x15739 (>= (+ ?v0!15 (* (- 1) v_b_P_H_len$)) 0)))
+(let (($x16002 (= (+ ?v0!15 (* (- 1) v_b_P_H_len$)) (+ (* (- 1) v_b_P_H_len$) ?v0!15))))
+(let ((@x16006 (monotonicity (rewrite $x16002) (= $x15739 (>= (+ (* (- 1) v_b_P_H_len$) ?v0!15) 0)))))
+(let ((@x16013 (trans @x16006 (rewrite (= (>= (+ (* (- 1) v_b_P_H_len$) ?v0!15) 0) $x16009)) (= $x15739 $x16009))))
+(let ((@x16019 (monotonicity (monotonicity @x16013 (= (not $x15739) $x16014)) (= $x15741 $x16017))))
+(let ((@x16038 (monotonicity (monotonicity @x16019 (= (not $x15741) $x16020)) @x16035 (= (or (not $x15741) $x15746) $x16036))))
+(let ((@x16047 (monotonicity (rewrite (= $x15732 $x11792)) (monotonicity (monotonicity @x16038 (= $x15748 $x16039)) (= $x15769 $x16042)) (= $x15773 (and $x11792 $x16042)))))
+(let ((@x16055 (monotonicity (trans @x16047 (rewrite (= (and $x11792 $x16042) $x16048)) (= $x15773 $x16048)) (= $x15777 $x16053))))
+(let ((@x16058 (monotonicity (rewrite (= $x15726 $x11772)) @x16055 (= $x15781 (and $x11772 $x16053)))))
+(let (($x15899 (= (or (not (and $x15626 $x15627 (not (>= (+ ?v0!14 ?x11581) 0)))) $x15636) $x15898)))
+(let (($x15886 (= (+ ?x15634 (* (- 1) v_b_L_H_max_G_3$)) (+ (* (- 1) v_b_L_H_max_G_3$) ?x15634))))
+(let ((@x15890 (monotonicity (rewrite $x15886) (= $x15636 (<= (+ (* (- 1) v_b_L_H_max_G_3$) ?x15634) 0)))))
+(let ((@x15897 (trans @x15890 (rewrite (= (<= (+ (* (- 1) v_b_L_H_max_G_3$) ?x15634) 0) $x15893)) (= $x15636 $x15893))))
+(let ((@x15868 (monotonicity (rewrite (= (+ ?v0!14 ?x11581) (+ ?x11581 ?v0!14))) (= (>= (+ ?v0!14 ?x11581) 0) (>= (+ ?x11581 ?v0!14) 0)))))
+(let ((@x15875 (trans @x15868 (rewrite (= (>= (+ ?x11581 ?v0!14) 0) $x15871)) (= (>= (+ ?v0!14 ?x11581) 0) $x15871))))
+(let ((@x15881 (monotonicity (monotonicity @x15875 (= (not (>= (+ ?v0!14 ?x11581) 0)) $x15876)) (= (and $x15626 $x15627 (not (>= (+ ?v0!14 ?x11581) 0))) $x15879))))
+(let ((@x15884 (monotonicity @x15881 (= (not (and $x15626 $x15627 (not (>= (+ ?v0!14 ?x11581) 0)))) $x15882))))
+(let ((@x15906 (monotonicity (monotonicity (monotonicity @x15884 @x15897 $x15899) (= $x15638 $x15901)) (= $x15655 $x15904))))
+(let ((@x15912 (monotonicity (monotonicity (rewrite (= $x15622 $x11608)) @x15906 (= $x15659 $x15907)) (= $x15663 $x15910))))
+(let ((@x15915 (monotonicity (rewrite (= $x15617 $x13358)) @x15912 (= $x15667 (and $x13358 $x15910)))))
+(let ((@x15923 (monotonicity (trans @x15915 (rewrite (= (and $x13358 $x15910) $x15916)) (= $x15667 $x15916)) (= $x15671 $x15921))))
+(let ((@x15958 (monotonicity (rewrite (= $x15695 $x11725)) @x15923 (= $x15698 (and $x11725 $x15921)))))
+(let ((@x15926 (monotonicity (rewrite (= $x15608 $x11562)) @x15923 (= $x15675 (and $x11562 $x15921)))))
+(let ((@x15934 (monotonicity (trans @x15926 (rewrite (= (and $x11562 $x15921) $x15927)) (= $x15675 $x15927)) (= $x15679 $x15932))))
+(let ((@x15937 (monotonicity (rewrite (= $x15596 $x10323)) @x15934 (= $x15683 (and $x10323 $x15932)))))
+(let ((@x15945 (monotonicity (trans @x15937 (rewrite (= (and $x10323 $x15932) $x15938)) (= $x15683 $x15938)) (= $x15687 $x15943))))
+(let ((@x15948 (monotonicity (rewrite (= $x15605 $x11527)) @x15945 (= $x15691 (and $x11527 $x15943)))))
+(let ((@x15966 (monotonicity (trans @x15948 (rewrite (= (and $x11527 $x15943) $x15949)) (= $x15691 $x15949)) (trans @x15958 (rewrite (= (and $x11725 $x15921) $x15959)) (= $x15698 $x15959)) (= $x15702 $x15964))))
+(let ((@x15969 (monotonicity (rewrite (= $x15602 $x11507)) @x15966 (= $x15706 (and $x11507 $x15964)))))
+(let ((@x15977 (monotonicity (trans @x15969 (rewrite (= (and $x11507 $x15964) $x15970)) (= $x15706 $x15970)) (= $x15710 $x15975))))
+(let ((@x15980 (monotonicity (rewrite (= $x15596 $x10323)) @x15977 (= $x15714 (and $x10323 $x15975)))))
+(let ((@x15988 (monotonicity (trans @x15980 (rewrite (= (and $x10323 $x15975) $x15981)) (= $x15714 $x15981)) (= $x15718 $x15986))))
+(let ((@x15991 (monotonicity (rewrite (= $x15587 $x11496)) @x15988 (= $x15722 (and $x11496 $x15986)))))
+(let ((@x16066 (monotonicity (trans @x15991 (rewrite (= (and $x11496 $x15986) $x15992)) (= $x15722 $x15992)) (trans @x16058 (rewrite (= (and $x11772 $x16053) $x16059)) (= $x15781 $x16059)) (= $x15785 $x16064))))
+(let ((@x16069 (monotonicity (rewrite (= $x15584 $x11476)) @x16066 (= $x15789 (and $x13343 $x11476 $x16064)))))
+(let ((@x16074 (trans @x16069 (rewrite (= (and $x13343 $x11476 $x16064) $x16070)) (= $x15789 $x16070))))
+(let ((@x16080 (monotonicity (monotonicity (rewrite (= $x15545 $x11259)) @x16074 (= $x15793 $x16075)) (= $x15797 $x16078))))
+(let ((@x16086 (monotonicity (rewrite (= $x15519 $x11382)) (monotonicity @x16080 (= $x15801 $x16081)) (= $x15805 $x16084))))
+(let ((@x16092 (monotonicity (rewrite (= $x15514 $x11374)) (monotonicity @x16086 (= $x15809 $x16087)) (= $x15813 (and $x11374 $x16087)))))
+(let ((@x16100 (monotonicity (trans @x16092 (rewrite (= (and $x11374 $x16087) $x16093)) (= $x15813 $x16093)) (= $x15817 $x16098))))
+(let ((@x16103 (monotonicity (rewrite (= $x15508 $x10140)) @x16100 (= $x15821 (and $x10140 $x16098)))))
+(let ((@x16111 (monotonicity (trans @x16103 (rewrite (= (and $x10140 $x16098) $x16104)) (= $x15821 $x16104)) (= $x15825 $x16109))))
+(let ((@x16117 (monotonicity (monotonicity (rewrite (= $x15499 $x10136)) @x16111 (= $x15829 $x16112)) (= $x15833 $x16115))))
+(let (($x13451 (exists ((?v0 Int) )(let ((?x10163 (b_S_read_n_u1$ v_b_S_s$ (b_S_idx$ (b_S_ptr$ b_T_T_u1$ v_b_P_H_arr$) ?v0 b_T_T_u1$))))
+(let (($x10238 (= ?x10163 v_b_S_result_G_0$)))
+(let (($x11800 (>= (+ ?v0 (* (- 1) v_b_P_H_len$)) 0)))
+(let (($x11802 (not $x11800)))
+(let (($x12168 (<= ?v0 4294967295)))
+(let (($x2815 (>= ?v0 0)))
+(and $x2815 $x12168 $x11802 $x10238))))))))
+))
+(let (($x13445 (not $x13442)))
+(let (($x13454 (or $x13445 $x13451)))
+(let (($x13457 (and $x13442 $x13454)))
+(let (($x13460 (or $x11797 $x13457)))
+(let (($x13463 (and b_S_position_n_marker$ $x13460)))
+(let (($x13466 (or $x11777 $x13463)))
+(let (($x13376 (not $x13373)))
+(let (($x13379 (or $x13376 $x11651)))
+(let (($x13382 (and $x13373 $x13379)))
+(let (($x13385 (or $x11612 $x13382)))
+(let (($x13388 (and $x11608 $x13385)))
+(let (($x13391 (or $x13361 $x13388)))
+(let (($x13394 (and $x11570 $x13353 $x13391)))
+(let (($x13412 (or $x11730 $x13394)))
+(let (($x13397 (or $x11567 $x13394)))
+(let (($x13400 (and $x10321 $x10324 $x13397)))
+(let (($x13403 (or $x11001 $x13400)))
+(let (($x13406 (and $x10321 $x10322 $x13403)))
+(let (($x13409 (or $x11532 $x13406)))
+(let (($x13415 (and $x13409 $x13412)))
+(let (($x13418 (or $x11512 $x13415)))
+(let (($x13421 (and $x10321 $x10324 $x13418)))
+(let (($x13424 (or $x11001 $x13421)))
+(let (($x13427 (and $x10321 $x10322 $x13424)))
+(let (($x13430 (or $x11501 $x13427)))
+(let (($x13469 (and $x13430 $x13466)))
+(let (($x13346 (not $x13343)))
+(let (($x13472 (or $x13346 $x11481 $x13469)))
+(let (($x13475 (and $x11260 $x10167 $x13472)))
+(let (($x13295 (not $x13292)))
+(let (($x13478 (or $x13295 $x13475)))
+(let (($x13481 (and $x13292 $x13478)))
+(let (($x13484 (or $x11385 $x13481)))
+(let (($x13487 (and $x11382 $x13484)))
+(let (($x13490 (or $x11379 $x13487)))
+(let (($x13493 (and $x10138 $x10141 $x13490)))
+(let (($x13496 (or $x11209 $x13493)))
+(let (($x13499 (and $x10138 $x10139 $x13496)))
+(let (($x13502 (or $x11221 $x13499)))
+(let (($x13508 (not (and $x10136 $x13502))))
+(let ((@x15760 (refl (~ (not (and $x2815 $x12168 $x11802 $x10238)) (not (and $x2815 $x12168 $x11802 $x10238))))))
+(let ((@x15757 (nnf-neg (nnf-pos (refl (~ $x13439 $x13439)) (~ $x13442 $x13442)) (~ (not $x13445) $x13442))))
+(let ((@x15768 (nnf-neg @x15757 (nnf-neg @x15760 (~ (not $x13451) $x15761)) (~ (not $x13454) $x15765))))
+(let ((@x15776 (nnf-neg (refl (~ $x15732 $x15732)) (nnf-neg (sk (~ $x13445 $x15748)) @x15768 (~ (not $x13457) $x15769)) (~ (not $x13460) $x15773))))
+(let ((@x15784 (nnf-neg (refl (~ $x15726 $x15726)) (nnf-neg (refl (~ $x15729 $x15729)) @x15776 (~ (not $x13463) $x15777)) (~ (not $x13466) $x15781))))
+(let ((@x15647 (nnf-neg (nnf-pos (refl (~ $x13370 $x13370)) (~ $x13373 $x13373)) (~ (not $x13376) $x13373))))
+(let ((@x15658 (nnf-neg (sk (~ $x13376 $x15638)) (nnf-neg @x15647 (refl (~ $x15648 $x15648)) (~ (not $x13379) $x15651)) (~ (not $x13382) $x15655))))
+(let ((@x15666 (nnf-neg (refl (~ $x11612 $x11612)) (nnf-neg (refl (~ $x15622 $x15622)) @x15658 (~ (not $x13385) $x15659)) (~ (not $x13388) $x15663))))
+(let ((@x15674 (nnf-neg (refl (~ $x15611 $x15611)) (refl (~ $x15614 $x15614)) (nnf-neg (refl (~ $x15617 $x15617)) @x15666 (~ (not $x13391) $x15667)) (~ (not $x13394) $x15671))))
+(let ((@x15592 (refl (~ $x15590 $x15590))))
+(let ((@x15682 (nnf-neg @x15592 (refl (~ $x15599 $x15599)) (nnf-neg (refl (~ $x15608 $x15608)) @x15674 (~ (not $x13397) $x15675)) (~ (not $x13400) $x15679))))
+(let ((@x15690 (nnf-neg @x15592 (refl (~ $x15593 $x15593)) (nnf-neg (refl (~ $x15596 $x15596)) @x15682 (~ (not $x13403) $x15683)) (~ (not $x13406) $x15687))))
+(let ((@x15705 (nnf-neg (nnf-neg (refl (~ $x15605 $x15605)) @x15690 (~ (not $x13409) $x15691)) (nnf-neg (refl (~ $x15695 $x15695)) @x15674 (~ (not $x13412) $x15698)) (~ (not $x13415) $x15702))))
+(let ((@x15713 (nnf-neg @x15592 (refl (~ $x15599 $x15599)) (nnf-neg (refl (~ $x15602 $x15602)) @x15705 (~ (not $x13418) $x15706)) (~ (not $x13421) $x15710))))
+(let ((@x15721 (nnf-neg @x15592 (refl (~ $x15593 $x15593)) (nnf-neg (refl (~ $x15596 $x15596)) @x15713 (~ (not $x13424) $x15714)) (~ (not $x13427) $x15718))))
+(let ((@x15788 (nnf-neg (nnf-neg (refl (~ $x15587 $x15587)) @x15721 (~ (not $x13430) $x15722)) @x15784 (~ (not $x13469) $x15785))))
+(let ((@x15580 (monotonicity (refl (~ $x11260 $x11260)) (refl (~ $x10167 $x10167)) (refl (~ $x11911 $x11911)) (refl (~ $x13304 $x13304)) (refl (~ $x13315 $x13315)) (refl (~ $x11901 $x11901)) (refl (~ $x13326 $x13326)) (refl (~ $x11898 $x11898)) (nnf-pos (refl (~ $x13337 $x13337)) (~ $x13340 $x13340)) (refl (~ $x11868 $x11868)) (refl (~ $x10192 $x10192)) (refl (~ $x11429 $x11429)) (refl (~ $x11432 $x11432)) (~ $x13343 $x13343))))
+(let ((@x15792 (nnf-neg (nnf-neg @x15580 (~ (not $x13346) $x13343)) (refl (~ $x15584 $x15584)) @x15788 (~ (not $x13472) $x15789))))
+(let ((@x15796 (nnf-neg (refl (~ $x15545 $x15545)) (refl (~ $x15548 $x15548)) @x15792 (~ (not $x13475) $x15793))))
+(let ((@x15544 (nnf-neg (nnf-pos (refl (~ $x13289 $x13289)) (~ $x13292 $x13292)) (~ (not $x13295) $x13292))))
+(let ((@x15804 (nnf-neg (sk (~ $x13295 $x15535)) (nnf-neg @x15544 @x15796 (~ (not $x13478) $x15797)) (~ (not $x13481) $x15801))))
+(let ((@x15812 (nnf-neg (refl (~ $x11385 $x11385)) (nnf-neg (refl (~ $x15519 $x15519)) @x15804 (~ (not $x13484) $x15805)) (~ (not $x13487) $x15809))))
+(let ((@x15820 (nnf-neg (refl (~ $x15502 $x15502)) (refl (~ $x15511 $x15511)) (nnf-neg (refl (~ $x15514 $x15514)) @x15812 (~ (not $x13490) $x15813)) (~ (not $x13493) $x15817))))
+(let ((@x15828 (nnf-neg (refl (~ $x15502 $x15502)) (refl (~ $x15505 $x15505)) (nnf-neg (refl (~ $x15508 $x15508)) @x15820 (~ (not $x13496) $x15821)) (~ (not $x13499) $x15825))))
+(let ((@x15835 (nnf-neg (refl (~ $x11221 $x11221)) (nnf-neg (refl (~ $x15499 $x15499)) @x15828 (~ (not $x13502) $x15829)) (~ $x13508 $x15833))))
+(let (($x6441 (= b_S_max_o_u4$ 4294967295)))
+(let ((@x6435 (monotonicity (rewrite (= (* 65536 65536) 4294967296)) (= (- (* 65536 65536) 1) (- 4294967296 1)))))
+(let ((@x6440 (trans @x6435 (rewrite (= (- 4294967296 1) 4294967295)) (= (- (* 65536 65536) 1) 4294967295))))
+(let ((@x6443 (monotonicity @x6440 (= (= b_S_max_o_u4$ (- (* 65536 65536) 1)) $x6441))))
+(let ((@x6446 (mp (asserted (= b_S_max_o_u4$ (- (* 65536 65536) 1))) @x6443 $x6441)))
+(let ((@x12140 (trans (monotonicity @x6446 (= ?x3113 (* (- 1) 4294967295))) (rewrite (= (* (- 1) 4294967295) (- 4294967295))) (= ?x3113 (- 4294967295)))))
+(let ((@x12164 (trans (monotonicity @x12140 (= ?x3114 (+ ?0 (- 4294967295)))) (rewrite (= (+ ?0 (- 4294967295)) (+ (- 4294967295) ?0))) (= ?x3114 (+ (- 4294967295) ?0)))))
+(let ((@x12172 (trans (monotonicity @x12164 (= $x3115 (<= (+ (- 4294967295) ?0) 0))) (rewrite (= (<= (+ (- 4294967295) ?0) 0) $x12168)) (= $x3115 $x12168))))
+(let ((@x13453 (quant-intro (monotonicity @x12172 (= $x11839 (and $x2815 $x12168 $x11802 $x10238))) (= $x11844 $x13451))))
+(let ((@x13441 (monotonicity (monotonicity (monotonicity @x12172 (= $x11808 $x13433)) (= $x11813 $x13436)) (= $x11821 $x13439))))
+(let ((@x13456 (monotonicity (monotonicity (quant-intro @x13441 (= $x11824 $x13442)) (= $x11827 $x13445)) @x13453 (= $x11847 $x13454))))
+(let ((@x13462 (monotonicity (monotonicity (quant-intro @x13441 (= $x11824 $x13442)) @x13456 (= $x11850 $x13457)) (= $x11853 $x13460))))
+(let ((@x13372 (monotonicity (monotonicity (monotonicity @x12172 (= $x11623 $x13364)) (= $x11628 $x13367)) (= $x11636 $x13370))))
+(let ((@x13381 (monotonicity (monotonicity (quant-intro @x13372 (= $x11639 $x13373)) (= $x11642 $x13376)) (= $x11654 $x13379))))
+(let ((@x13387 (monotonicity (monotonicity (quant-intro @x13372 (= $x11639 $x13373)) @x13381 (= $x11657 $x13382)) (= $x11660 $x13385))))
+(let ((@x13351 (monotonicity (monotonicity @x6446 (= ?x11574 (+ 4294967295 ?x11484))) (= $x11573 (>= (+ 4294967295 ?x11484) 1)))))
+(let ((@x13357 (trans @x13351 (rewrite (= (>= (+ 4294967295 ?x11484) 1) $x13353)) (= $x11573 $x13353))))
+(let ((@x13393 (monotonicity (monotonicity (monotonicity @x13357 (= $x11600 $x13358)) (= $x11605 $x13361)) (monotonicity @x13387 (= $x11663 $x13388)) (= $x11666 $x13391))))
+(let ((@x13414 (monotonicity (monotonicity @x13357 @x13393 (= $x11672 $x13394)) (= $x11733 $x13412))))
+(let ((@x13399 (monotonicity (monotonicity @x13357 @x13393 (= $x11672 $x13394)) (= $x11677 $x13397))))
+(let ((@x13408 (monotonicity (monotonicity (monotonicity @x13399 (= $x11683 $x13400)) (= $x11688 $x13403)) (= $x11694 $x13406))))
+(let ((@x13417 (monotonicity (monotonicity @x13408 (= $x11699 $x13409)) @x13414 (= $x11736 $x13415))))
+(let ((@x13426 (monotonicity (monotonicity (monotonicity @x13417 (= $x11739 $x13418)) (= $x11745 $x13421)) (= $x11750 $x13424))))
+(let ((@x13471 (monotonicity (monotonicity (monotonicity @x13426 (= $x11756 $x13427)) (= $x11761 $x13430)) (monotonicity (monotonicity @x13462 (= $x11856 $x13463)) (= $x11859 $x13466)) (= $x11862 $x13469))))
+(let ((@x13339 (monotonicity (monotonicity (monotonicity @x12172 (= $x11879 $x13331)) (= $x11884 $x13334)) (= $x11892 $x13337))))
+(let ((@x13325 (monotonicity (monotonicity @x6446 (= ?x11574 (+ 4294967295 ?x11484))) (= $x11904 (>= (+ 4294967295 ?x11484) 0)))))
+(let ((@x13330 (trans @x13325 (rewrite (= (>= (+ 4294967295 ?x11484) 0) $x13326)) (= $x11904 $x13326))))
+(let ((@x13314 (monotonicity (monotonicity @x6446 (= (+ b_S_max_o_u4$ ?x11865) (+ 4294967295 ?x11865))) (= $x11907 (>= (+ 4294967295 ?x11865) 0)))))
+(let ((@x13319 (trans @x13314 (rewrite (= (>= (+ 4294967295 ?x11865) 0) $x13315)) (= $x11907 $x13315))))
+(let (($x13299 (= (+ b_S_max_o_u1$ (* (- 1) v_b_L_H_max_G_1$)) (+ 255 (* (- 1) v_b_L_H_max_G_1$)))))
+(let (($x6449 (= b_S_max_o_u1$ 255)))
+(let ((@x6450 (asserted $x6449)))
+(let ((@x13303 (monotonicity (monotonicity @x6450 $x13299) (= $x11914 (>= (+ 255 (* (- 1) v_b_L_H_max_G_1$)) 0)))))
+(let ((@x13308 (trans @x13303 (rewrite (= (>= (+ 255 (* (- 1) v_b_L_H_max_G_1$)) 0) $x13304)) (= $x11914 $x13304))))
+(let ((@x13345 (monotonicity @x13308 @x13319 @x13330 (quant-intro @x13339 (= $x11895 $x13340)) (= $x11957 $x13343))))
+(let ((@x13474 (monotonicity (monotonicity @x13345 (= $x11962 $x13346)) @x13471 (= $x11971 $x13472))))
+(let ((@x13291 (monotonicity (monotonicity (monotonicity @x12172 (= $x11395 $x13283)) (= $x11400 $x13286)) (= $x11408 $x13289))))
+(let ((@x13480 (monotonicity (monotonicity (quant-intro @x13291 (= $x11411 $x13292)) (= $x11414 $x13295)) (monotonicity @x13474 (= $x11979 $x13475)) (= $x11984 $x13478))))
+(let ((@x13486 (monotonicity (monotonicity (quant-intro @x13291 (= $x11411 $x13292)) @x13480 (= $x11987 $x13481)) (= $x11990 $x13484))))
+(let ((@x13495 (monotonicity (monotonicity (monotonicity @x13486 (= $x11993 $x13487)) (= $x11996 $x13490)) (= $x12002 $x13493))))
+(let ((@x13504 (monotonicity (monotonicity (monotonicity @x13495 (= $x12007 $x13496)) (= $x12013 $x13499)) (= $x12018 $x13502))))
+(let ((@x13510 (monotonicity (monotonicity @x13504 (= $x12021 (and $x10136 $x13502))) (= (not $x12021) $x13508))))
+(let ((@x13511 (mp (not-or-elim (mp (asserted $x10434) @x12031 $x12027) (not $x12021)) @x13510 $x13508)))
+(let ((@x20143 (mp (mp (mp (mp~ @x13511 @x15835 $x15833) @x16117 $x16115) @x19763 $x19761) (monotonicity @x20139 (= $x19761 $x20140)) $x20140)))
+(let ((@x24002 (unit-resolution (def-axiom (or $x20134 $x20128)) (unit-resolution @x20143 @x22434 $x20137) $x20128)))
+(let ((?x22514 (b_S_typ$ ?x10137)))
+(let (($x22515 (= ?x22514 b_T_T_u1$)))
+(let ((@x22856 (trans (unit-resolution @x22581 (unit-resolution @x22577 @x18183 $x22565) $x22556) @x22852 (= ?x10137 ?x10078))))
+(let ((@x22875 (trans (monotonicity @x22856 (= ?x22514 ?x21175)) (unit-resolution @x21182 @x19846 $x21176) $x22515)))
+(let (($x22507 (not $x22515)))
+(let (($x22522 (= $x10138 $x22515)))
+(let (($x22949 (or $x22002 $x22522)))
+(let ((@x22487 ((_ quant-inst (b_S_idx$ ?x10078 0 b_T_T_u1$) b_T_T_u1$) $x22949)))
+(let ((@x22509 (unit-resolution (def-axiom (or (not $x22522) $x10138 $x22507)) (hypothesis $x15502) (or (not $x22522) $x22507))))
+(let ((@x22873 (unit-resolution (unit-resolution @x22509 (unit-resolution @x22487 @x19833 $x22522) $x22507) @x22875 false)))
+(let ((@x22876 (lemma @x22873 $x10138)))
+(let ((@x23964 (unit-resolution (def-axiom (or $x20131 $x15502 $x15505 $x20125)) (unit-resolution (def-axiom (or $x22603 $x10139)) @x22760 $x10139) @x22876 @x24002 $x20125)))
+(let ((?x22963 (* (- 1) ?x10144)))
+(let ((?x22964 (+ v_b_L_H_max_G_0$ ?x22963)))
+(let (($x22965 (>= ?x22964 0)))
+(let ((@x20962 (def-axiom (or $x20119 $x15502 $x15511 $x20113))))
+(let ((@x22988 (unit-resolution @x20962 (hypothesis $x10138) (hypothesis $x10141) (hypothesis $x20116) $x20113)))
+(let ((@x20944 (def-axiom (or $x20110 $x10145))))
+(let ((@x23016 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x19724 $x22965)) (unit-resolution @x20944 @x22988 $x10145) $x22965)))
+(let (($x22455 (or $x21994 $x15502 $x22506)))
+(let ((@x22447 (mp ((_ quant-inst (b_S_idx$ ?x10078 0 b_T_T_u1$) b_T_T_u1$) (or $x21994 (or $x15502 $x22506))) (rewrite (= (or $x21994 (or $x15502 $x22506)) $x22455)) $x22455)))
+(let ((@x23003 (monotonicity ((_ th-lemma arith eq-propagate 0 0) (hypothesis $x15523) (hypothesis (not $x15525)) (= ?v0!13 0)) (= ?x15529 ?x10137))))
+(let ((@x23005 (trans @x23003 (unit-resolution @x22447 @x15336 (hypothesis $x10138) $x22506) (= ?x15529 ?x22505))))
+(let (($x23008 (or (not (= ?x15530 (b_S_read_n_u1$ v_b_S_s$ ?x22505))) (<= (+ ?x15530 (* (- 1) (b_S_read_n_u1$ v_b_S_s$ ?x22505))) 0))))
+(let ((@x23010 (unit-resolution ((_ th-lemma arith triangle-eq) $x23008) (monotonicity @x23005 (= ?x15530 (b_S_read_n_u1$ v_b_S_s$ ?x22505))) (<= (+ ?x15530 (* (- 1) (b_S_read_n_u1$ v_b_S_s$ ?x22505))) 0))))
+(let ((?x22685 (b_S_read_n_u1$ v_b_S_s$ ?x22505)))
+(let ((?x22773 (* (- 1) ?x22685)))
+(let ((?x22835 (+ ?x10144 ?x22773)))
+(let (($x22839 (>= ?x22835 0)))
+(let (($x22834 (= ?x10144 ?x22685)))
+(let ((@x23011 (symm (unit-resolution @x22447 @x15336 (hypothesis $x10138) $x22506) (= ?x22505 ?x10137))))
+(let ((@x23020 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x22834) $x22839)) (symm (monotonicity @x23011 (= ?x22685 ?x10144)) $x22834) $x22839)))
+(let ((@x23023 (lemma ((_ th-lemma arith farkas 1 -1 -1 1) @x23020 @x23010 (hypothesis $x20589) @x23016 false) (or $x15502 $x15533 $x19297 $x15525 $x15511 $x20119))))
+(let ((@x24012 (unit-resolution @x23023 @x22876 (unit-resolution (def-axiom (or $x20122 $x20116)) @x23964 $x20116) (or $x15533 $x19297 $x15525 $x15511))))
+(let ((@x24203 (unit-resolution (unit-resolution @x24012 @x23403 (or $x15533 $x19297 $x15525)) (unit-resolution (def-axiom (or $x19313 (not $x15525))) @x24016 (not $x15525)) (unit-resolution (def-axiom (or $x19313 $x15523)) @x24016 $x15523) (unit-resolution (def-axiom (or $x19313 $x20589)) @x24016 $x20589) false)))
+(let ((@x24417 (unit-resolution @x20962 @x22876 (unit-resolution (def-axiom (or $x20122 $x20116)) @x23964 $x20116) (or $x15511 $x20113))))
+(let ((@x24506 (unit-resolution (def-axiom (or $x20110 $x20104)) (unit-resolution @x24417 @x23403 $x20113) $x20104)))
+(let ((@x24507 (unit-resolution (def-axiom (or $x20107 $x11385 $x20101)) (lemma ((_ th-lemma arith farkas 1 1) @x12041 (hypothesis $x11385) false) $x11382) @x24506 $x20101)))
+(let ((@x24462 (unit-resolution (def-axiom (or $x20095 $x19318 $x20089)) (unit-resolution (def-axiom (or $x20098 $x20092)) @x24507 $x20092) $x20092)))
+(let ((@x24496 (unit-resolution (def-axiom (or $x20086 $x20080)) (unit-resolution @x24462 (lemma @x24203 $x19313) $x20089) $x20080)))
+(let ((@x24578 (mp (unit-resolution @x20944 (unit-resolution @x24417 @x23403 $x20113) $x10145) (symm (commutativity (= $x10167 $x10145)) (= $x10145 $x10167)) $x10167)))
+(let ((@x24580 (unit-resolution (def-axiom (or $x20083 $x11259 $x15548 $x20077)) @x12041 (or $x20083 $x15548 $x20077))))
+(let ((@x24583 (unit-resolution (unit-resolution @x24580 @x24578 (or $x20083 $x20077)) @x24496 $x20077)))
+(let ((@x24576 (unit-resolution (def-axiom (or $x20074 $x11901)) @x24583 $x11901)))
+(let ((@x24314 (unit-resolution (def-axiom (or $x20074 $x10192)) @x24583 $x10192)))
+(let ((@x24415 (unit-resolution (def-axiom (or $x20074 $x11868)) @x24583 $x11868)))
+(let ((@x24499 (unit-resolution (def-axiom (or $x20074 $x19898)) @x24583 $x19898)))
+(let (($x23168 (<= (+ v_b_L_H_p_G_0$ (* (- 1) ?v0!15)) 0)))
+(let (($x23092 (<= (+ v_b_L_H_max_G_1$ (* (- 1) v_b_S_result_G_0$)) 0)))
+(let (($x23088 (= v_b_L_H_max_G_1$ v_b_S_result_G_0$)))
+(let ((@x9231 (asserted b_S_position_n_marker$)))
+(let ((@x23318 (unit-resolution (unit-resolution (def-axiom (or $x20059 $x15729 $x20053)) @x9231 (or $x20059 $x20053)) (unit-resolution (def-axiom (or $x20062 $x20056)) (hypothesis $x20065) $x20056) $x20053)))
+(let ((@x23324 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x23088) $x23092)) (symm (unit-resolution (def-axiom (or $x20050 $x10222)) @x23318 $x10222) $x23088) $x23092)))
+(let (($x20801 (not $x16031)))
+(let ((@x23175 (hypothesis $x10192)))
+(let ((@x23180 (hypothesis $x11868)))
+(let (($x23140 (not (= ?x10191 v_b_S_result_G_0$))))
+(let (($x23145 (or $x20035 $x19501 $x19669 $x11867 $x23140)))
+(let (($x23036 (>= (+ v_b_SL_H_witness_G_0$ (* (- 1) v_b_P_H_len$)) 0)))
+(let (($x23141 (or $x19501 $x19669 $x23036 $x23140)))
+(let (($x23146 (or $x20035 $x23141)))
+(let (($x23046 (= (>= (+ (* (- 1) v_b_P_H_len$) v_b_SL_H_witness_G_0$) 0) $x11867)))
+(let (($x23044 (= $x23036 (>= (+ (* (- 1) v_b_P_H_len$) v_b_SL_H_witness_G_0$) 0))))
+(let (($x23041 (= (+ v_b_SL_H_witness_G_0$ (* (- 1) v_b_P_H_len$)) (+ (* (- 1) v_b_P_H_len$) v_b_SL_H_witness_G_0$))))
+(let ((@x23049 (trans (monotonicity (rewrite $x23041) $x23044) (rewrite $x23046) (= $x23036 $x11867))))
+(let ((@x23150 (monotonicity (monotonicity @x23049 (= $x23141 (or $x19501 $x19669 $x11867 $x23140))) (= $x23146 (or $x20035 (or $x19501 $x19669 $x11867 $x23140))))))
+(let ((@x23154 (trans @x23150 (rewrite (= (or $x20035 (or $x19501 $x19669 $x11867 $x23140)) $x23145)) (= $x23146 $x23145))))
+(let ((@x23182 (unit-resolution (mp ((_ quant-inst v_b_SL_H_witness_G_0$) $x23146) @x23154 $x23145) (hypothesis $x13315) @x23180 (hypothesis $x11432) (hypothesis $x20030) (trans @x23175 (symm (hypothesis $x10222) $x23088) (= ?x10191 v_b_S_result_G_0$)) false)))
+(let ((@x23326 (unit-resolution (lemma @x23182 (or $x20035 $x19669 $x11867 $x19501 $x19674 $x19640)) (unit-resolution (def-axiom (or $x20050 $x10222)) @x23318 $x10222) @x23180 (hypothesis $x11432) @x23175 (hypothesis $x13315) $x20035)))
+(let ((@x23328 (unit-resolution (def-axiom (or $x20047 $x19580 $x20041)) (unit-resolution (def-axiom (or $x20038 $x20030)) @x23326 $x20038) (unit-resolution (def-axiom (or $x20050 $x20044)) @x23318 $x20044) $x19580)))
+(let ((@x23308 ((_ th-lemma arith farkas -1 1 1) (hypothesis (>= (+ v_b_L_H_max_G_1$ ?x16029) 0)) (hypothesis $x20801) (hypothesis $x23092) false)))
+(let ((@x23312 (lemma @x23308 (or (not (>= (+ v_b_L_H_max_G_1$ ?x16029) 0)) $x16031 (not $x23092)))))
+(let ((@x23330 (unit-resolution @x23312 (unit-resolution (def-axiom (or $x19575 $x20801)) @x23328 $x20801) @x23324 (not (>= (+ v_b_L_H_max_G_1$ ?x16029) 0)))))
+(let ((@x23333 (hypothesis $x19898)))
+(let (($x23188 (>= (+ v_b_L_H_max_G_1$ ?x16029) 0)))
+(let (($x23196 (or $x19903 $x19559 $x19560 $x23168 $x23188)))
+(let (($x23134 (<= (+ ?x15744 (* (- 1) v_b_L_H_max_G_1$)) 0)))
+(let (($x23114 (>= (+ ?v0!15 ?x11484) 0)))
+(let (($x23135 (or $x19559 $x19560 $x23114 $x23134)))
+(let (($x23197 (or $x19903 $x23135)))
+(let (($x23173 (= (+ ?x15744 (* (- 1) v_b_L_H_max_G_1$)) (+ (* (- 1) v_b_L_H_max_G_1$) ?x15744))))
+(let ((@x23186 (monotonicity (rewrite $x23173) (= $x23134 (<= (+ (* (- 1) v_b_L_H_max_G_1$) ?x15744) 0)))))
+(let ((@x23192 (trans @x23186 (rewrite (= (<= (+ (* (- 1) v_b_L_H_max_G_1$) ?x15744) 0) $x23188)) (= $x23134 $x23188))))
+(let ((@x23166 (monotonicity (rewrite (= (+ ?v0!15 ?x11484) (+ ?x11484 ?v0!15))) (= $x23114 (>= (+ ?x11484 ?v0!15) 0)))))
+(let ((@x23171 (trans @x23166 (rewrite (= (>= (+ ?x11484 ?v0!15) 0) $x23168)) (= $x23114 $x23168))))
+(let ((@x23201 (monotonicity (monotonicity @x23171 @x23192 (= $x23135 (or $x19559 $x19560 $x23168 $x23188))) (= $x23197 (or $x19903 (or $x19559 $x19560 $x23168 $x23188))))))
+(let ((@x23205 (trans @x23201 (rewrite (= (or $x19903 (or $x19559 $x19560 $x23168 $x23188)) $x23196)) (= $x23197 $x23196))))
+(let ((@x23335 (unit-resolution (mp ((_ quant-inst ?v0!15) $x23197) @x23205 $x23196) @x23333 (unit-resolution (def-axiom (or $x19575 $x15736)) @x23328 $x15736) (unit-resolution (def-axiom (or $x19575 $x15737)) @x23328 $x15737) (or $x23168 $x23188))))
+(let ((@x23338 ((_ th-lemma arith farkas -1 1 1) (unit-resolution (def-axiom (or $x19575 $x16014)) @x23328 $x16014) (unit-resolution @x23335 @x23330 $x23168) (unit-resolution (def-axiom (or $x20062 $x11486)) (hypothesis $x20065) $x11486) false)))
+(let ((@x24500 (unit-resolution (lemma @x23338 (or $x20062 $x19903 $x11867 $x19501 $x19674 $x19669)) @x24499 @x24415 (unit-resolution (def-axiom (or $x20074 $x11432)) @x24583 $x11432) @x24314 (unit-resolution (def-axiom (or $x20074 $x13315)) @x24583 $x13315) $x20062)))
+(let ((@x24502 (unit-resolution (def-axiom (or $x20071 $x20019 $x20065)) (unit-resolution (def-axiom (or $x20074 $x20068)) @x24583 $x20068) @x24500 $x20019)))
+(let ((@x24684 (unit-resolution (def-axiom (or $x20016 $x11487)) @x24502 $x11487)))
+(let ((@x24741 (mp @x22691 (symm (monotonicity @x24532 (= $x22596 $x22344)) (= $x22344 $x22596)) $x22596)))
+(let ((@x23420 (hypothesis $x11487)))
+(let (($x23378 (or $x22629 $x19677 $x21489 $x22597 $x19670 $x11486 $x23363)))
+(let (($x23360 (>= (+ v_b_L_H_p_G_0$ (* (- 1) v_b_P_H_len$)) 0)))
+(let (($x23364 (or $x19677 $x21489 $x22597 $x19670 $x23360 $x23363)))
+(let (($x23379 (or $x22629 $x23364)))
+(let ((@x23372 (rewrite (= (>= (+ (* (- 1) v_b_P_H_len$) v_b_L_H_p_G_0$) 0) $x11486))))
+(let (($x23366 (= (+ v_b_L_H_p_G_0$ (* (- 1) v_b_P_H_len$)) (+ (* (- 1) v_b_P_H_len$) v_b_L_H_p_G_0$))))
+(let ((@x23370 (monotonicity (rewrite $x23366) (= $x23360 (>= (+ (* (- 1) v_b_P_H_len$) v_b_L_H_p_G_0$) 0)))))
+(let ((@x23377 (monotonicity (trans @x23370 @x23372 (= $x23360 $x11486)) (= $x23364 (or $x19677 $x21489 $x22597 $x19670 $x11486 $x23363)))))
+(let ((@x23383 (monotonicity @x23377 (= $x23379 (or $x22629 (or $x19677 $x21489 $x22597 $x19670 $x11486 $x23363))))))
+(let ((@x23387 (trans @x23383 (rewrite (= (or $x22629 (or $x19677 $x21489 $x22597 $x19670 $x11486 $x23363)) $x23378)) (= $x23379 $x23378))))
+(let ((@x23388 (mp ((_ quant-inst v_b_S_s$ v_b_P_H_arr$ (b_S_ptr$ ?x10076 ?x21014) v_b_P_H_len$ v_b_L_H_p_G_0$ b_T_T_u1$) $x23379) @x23387 $x23378)))
+(let ((@x23422 (unit-resolution @x23388 @x18670 @x9769 @x12050 (hypothesis $x11901) @x23420 (hypothesis $x22596) (hypothesis $x23362) false)))
+(let ((@x24788 (unit-resolution (lemma @x23422 (or $x23363 $x19670 $x11486 $x22597)) @x24741 (or $x23363 $x19670 $x11486))))
+(let ((@x24697 (unit-resolution (def-axiom (or $x23362 $x23297)) (unit-resolution @x24788 @x24684 @x24576 $x23363) $x23297)))
+(let (($x23782 (b_S_in_n_wrapped_n_domain$ v_b_S_s$ ?x24218)))
+(let ((?x23727 (b_S_owner$ v_b_S_s$ ?x24218)))
+(let (($x23776 (= ?x23727 b_S_me$)))
+(let (($x23785 (or $x23776 $x23782)))
+(let (($x24475 (not $x23785)))
+(let ((?x23730 (b_S_typ$ ?x24218)))
+(let ((?x23768 (b_S_kind_n_of$ ?x23730)))
+(let (($x23769 (= ?x23768 b_S_kind_n_primitive$)))
+(let (($x23728 (not $x23804)))
+(let (($x23770 (not $x23805)))
+(let (($x24476 (or $x23770 $x23728 $x23769 $x24475)))
+(let (($x24627 (b_S_in_n_wrapped_n_domain$ v_b_S_s$ ?x23225)))
+(let (($x24478 (= (b_S_owner$ v_b_S_s$ ?x23225) b_S_me$)))
+(let (($x24943 (or $x24478 $x24627)))
+(let (($x25004 (not $x24943)))
+(let (($x24820 (or $x23805 $x25004)))
+(let (($x24623 (not $x24820)))
+(let (($x24474 (not $x24476)))
+(let (($x24809 (or $x24474 $x24623)))
+(let (($x24810 (not $x24809)))
+(let (($x24209 (b_S_typed$ v_b_S_s$ ?x23225)))
+(let (($x24210 (not $x24209)))
+(let (($x24817 (or $x24210 $x24810)))
+(let (($x24818 (not $x24817)))
+(let (($x23783 (b_S_thread_n_local$ v_b_S_s$ ?x23225)))
+(let (($x24819 (= $x23783 $x24818)))
+(let (($x24622 (or (not $x19072) $x24819)))
+(let ((@x24633 ((_ quant-inst v_b_S_s$ (b_S_ptr$ b_T_T_u1$ ?x23404)) $x24622)))
+(let (($x24628 (not $x23783)))
+(let ((@x24670 (monotonicity (symm (monotonicity @x25262 (= $x23783 $x10324)) (= $x10324 $x23783)) (= $x15599 $x24628))))
+(let ((@x24708 (unit-resolution (def-axiom (or (not $x24819) $x23783 $x24817)) (mp (hypothesis $x15599) @x24670 $x24628) (unit-resolution @x24633 @x19075 $x24819) $x24817)))
+(let ((@x24998 (unit-resolution (def-axiom (or $x23362 $x10322)) (unit-resolution @x24788 @x24684 @x24576 $x23363) $x10322)))
+(let ((@x24710 (mp @x24998 (symm (monotonicity @x25262 (= $x24209 $x10322)) (= $x10322 $x24209)) $x24209)))
+(let ((@x24724 (unit-resolution (def-axiom (or $x24809 $x24476)) (unit-resolution (def-axiom (or $x24818 $x24210 $x24810)) @x24710 @x24708 $x24810) $x24476)))
+(let ((?x24320 (b_S_idx$ ?x22595 v_b_L_H_p_G_0$ b_T_T_u1$)))
+(let ((?x24321 (b_S_select_o_tm$ ?x10272 ?x24320)))
+(let ((?x24322 (b_S_ts_n_emb$ ?x24321)))
+(let (($x24323 (= ?x24322 ?x22595)))
+(let (($x24328 (b_S_typed$ v_b_S_s$ ?x24320)))
+(let (($x24329 (not $x24328)))
+(let (($x24325 (b_S_ts_n_is_n_volatile$ ?x24321)))
+(let (($x24324 (not $x24323)))
+(let (($x24330 (or $x24324 $x24325 (not (b_S_ts_n_is_n_array_n_elt$ ?x24321)) $x24329)))
+(let (($x24331 (not $x24330)))
+(let (($x25071 (or $x23110 $x24241 $x19670 $x11486 $x24331)))
+(let (($x24332 (or $x24241 $x19670 $x23360 $x24331)))
+(let (($x25072 (or $x23110 $x24332)))
+(let ((@x25070 (monotonicity (trans @x23370 @x23372 (= $x23360 $x11486)) (= $x24332 (or $x24241 $x19670 $x11486 $x24331)))))
+(let ((@x25080 (trans (monotonicity @x25070 (= $x25072 (or $x23110 (or $x24241 $x19670 $x11486 $x24331)))) (rewrite (= (or $x23110 (or $x24241 $x19670 $x11486 $x24331)) $x25071)) (= $x25072 $x25071))))
+(let ((@x25137 (unit-resolution (mp ((_ quant-inst v_b_S_s$ v_b_P_H_arr$ b_T_T_u1$ v_b_P_H_len$ v_b_L_H_p_G_0$) $x25072) @x25080 $x25071) @x17967 @x24576 @x24684 @x24355 (hypothesis $x24330) false)))
+(let ((@x25083 (def-axiom (or $x24330 $x24323))))
+(let ((?x24315 (b_S_ref$ ?x24198)))
+(let ((?x24367 (* (- 1) ?x24315)))
+(let ((?x24368 (+ ?x10079 ?x23278 ?x24367)))
+(let (($x24402 (<= ?x24368 0)))
+(let (($x24365 (= ?x24368 0)))
+(let (($x24384 (or $x21152 $x24365)))
+(let ((@x24394 (monotonicity (rewrite (= (= ?x24315 ?x24174) $x24365)) (= (or $x21152 (= ?x24315 ?x24174)) $x24384))))
+(let ((@x24404 (trans @x24394 (rewrite (= $x24384 $x24384)) (= (or $x21152 (= ?x24315 ?x24174)) $x24384))))
+(let ((@x24403 (mp ((_ quant-inst b_T_T_u1$ (+ ?x10079 ?x23278)) (or $x21152 (= ?x24315 ?x24174))) @x24404 $x24384)))
+(let ((@x25241 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x24365) $x24402)) (unit-resolution @x24403 @x19840 $x24365) $x24402)))
+(let (($x24407 (>= ?x24368 0)))
+(let ((@x25244 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x24365) $x24407)) (unit-resolution @x24403 @x19840 $x24365) $x24407)))
+(let ((?x24925 (+ ?x23278 ?x24419)))
+(let (($x25226 (= ?x24174 ?x24925)))
+(let ((?x25227 (* (- 1) ?x24925)))
+(let ((?x25228 (+ ?x24174 ?x25227)))
+(let (($x25229 (<= ?x25228 0)))
+(let ((?x23747 (* (- 1) ?x21014)))
+(let ((?x23641 (+ ?x10079 ?x23747)))
+(let (($x24296 (<= ?x23641 0)))
+(let ((@x25085 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x10079 ?x21014)) $x24296)) (symm (unit-resolution @x21192 @x19840 $x21186) (= ?x10079 ?x21014)) $x24296)))
+(let ((?x25173 (* (- 1) ?x24419)))
+(let ((?x25174 (+ ?x21014 ?x25173)))
+(let (($x25175 (<= ?x25174 0)))
+(let ((@x25090 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x21014 ?x24419)) $x25175)) (symm (monotonicity @x24520 (= ?x24419 ?x21014)) (= ?x21014 ?x24419)) $x25175)))
+(let ((@x25103 (unit-resolution ((_ th-lemma arith assign-bounds -1 -1) (or $x25229 (not $x24296) (not $x25175))) @x25090 @x25085 $x25229)))
+(let (($x25230 (>= ?x25228 0)))
+(let (($x23809 (>= ?x23641 0)))
+(let ((@x25106 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x10079 ?x21014)) $x23809)) (symm (unit-resolution @x21192 @x19840 $x21186) (= ?x10079 ?x21014)) $x23809)))
+(let (($x25176 (>= ?x25174 0)))
+(let ((@x25109 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x21014 ?x24419)) $x25176)) (symm (monotonicity @x24520 (= ?x24419 ?x21014)) (= ?x21014 ?x24419)) $x25176)))
+(let ((@x25098 (unit-resolution ((_ th-lemma arith assign-bounds -1 -1) (or $x25230 (not $x23809) (not $x25176))) @x25109 @x25106 $x25230)))
+(let ((@x25111 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x25226 (not $x25229) (not $x25230))) @x25098 @x25103 (hypothesis (not $x25226)) false)))
+(let ((@x25182 (trans (symm (lemma @x25111 $x25226) (= ?x24925 ?x24174)) ((_ th-lemma arith eq-propagate -1 -1) @x25244 @x25241 (= ?x24174 ?x24315)) (= ?x24925 ?x24315))))
+(let ((@x25183 (trans @x25182 (monotonicity (symm @x24341 (= ?x24198 ?x10320)) (= ?x24315 ?x23404)) (= ?x24925 ?x23404))))
+(let ((?x24930 (b_S_ptr$ b_T_T_u1$ ?x24925)))
+(let ((?x24463 (b_S_idx$ ?x21983 v_b_L_H_p_G_0$ b_T_T_u1$)))
+(let (($x25146 (= ?x24463 ?x24930)))
+(let (($x25152 (or (not (b_S_extent_n_hint$ ?x24463 ?x21983)) (not $x25146))))
+(let (($x25155 (not $x25152)))
+(let (($x25158 (or $x22568 $x25155)))
+(let (($x24469 (not (= ?x24463 (b_S_ptr$ b_T_T_u1$ (+ ?x24419 (* v_b_L_H_p_G_0$ ?x10045)))))))
+(let (($x24471 (not (or (not (b_S_extent_n_hint$ ?x24463 ?x21983)) $x24469))))
+(let (($x25147 (= (= ?x24463 (b_S_ptr$ b_T_T_u1$ (+ ?x24419 (* v_b_L_H_p_G_0$ ?x10045)))) $x25146)))
+(let ((@x25139 (monotonicity (rewrite (= (* v_b_L_H_p_G_0$ ?x10045) ?x23278)) (= (+ ?x24419 (* v_b_L_H_p_G_0$ ?x10045)) (+ ?x24419 ?x23278)))))
+(let ((@x25143 (trans @x25139 (rewrite (= (+ ?x24419 ?x23278) ?x24925)) (= (+ ?x24419 (* v_b_L_H_p_G_0$ ?x10045)) ?x24925))))
+(let ((@x25145 (monotonicity @x25143 (= (b_S_ptr$ b_T_T_u1$ (+ ?x24419 (* v_b_L_H_p_G_0$ ?x10045))) ?x24930))))
+(let ((@x25154 (monotonicity (monotonicity (monotonicity @x25145 $x25147) (= $x24469 (not $x25146))) (= (or (not (b_S_extent_n_hint$ ?x24463 ?x21983)) $x24469) $x25152))))
+(let ((@x25162 (monotonicity (monotonicity @x25154 (= $x24471 $x25155)) (= (or $x22568 $x24471) $x25158))))
+(let ((@x25166 (mp ((_ quant-inst (b_S_ptr$ ?x10076 ?x21014) v_b_L_H_p_G_0$ b_T_T_u1$) (or $x22568 $x24471)) (trans @x25162 (rewrite (= $x25158 $x25158)) (= (or $x22568 $x24471) $x25158)) $x25158)))
+(let ((@x25257 (unit-resolution (def-axiom (or $x25152 $x25146)) (unit-resolution @x25166 @x18183 $x25155) $x25146)))
+(let ((@x25185 (trans (trans (monotonicity @x24532 (= ?x24320 ?x24463)) @x25257 (= ?x24320 ?x24930)) (monotonicity @x25183 (= ?x24930 ?x23225)) (= ?x24320 ?x23225))))
+(let ((@x25217 (symm (monotonicity (trans @x25185 @x25262 (= ?x24320 ?x10320)) (= ?x24321 ?x23101)) (= ?x23101 ?x24321))))
+(let ((@x25274 (monotonicity (monotonicity @x25262 (= ?x24217 ?x23101)) (= ?x24218 (b_S_ts_n_emb$ ?x23101)))))
+(let ((@x25219 (trans @x25274 (monotonicity @x25217 (= (b_S_ts_n_emb$ ?x23101) ?x24322)) (= ?x24218 ?x24322))))
+(let ((@x25221 (trans (trans @x25219 (hypothesis $x24323) (= ?x24218 ?x22595)) @x24530 (= ?x24218 ?x10080))))
+(let ((@x25293 (unit-resolution (hypothesis (not $x23776)) (trans (monotonicity @x25221 (= ?x23727 ?x10082)) @x12043 $x23776) false)))
+(let ((@x23976 (unit-resolution (lemma @x25293 (or $x24324 $x23776)) (unit-resolution @x25083 (lemma @x25137 $x24331) $x24323) $x23776)))
+(let ((?x23443 (b_S_ts_n_emb$ ?x23101)))
+(let ((?x23448 (b_S_typ$ ?x23443)))
+(let ((?x23449 (b_S_kind_n_of$ ?x23448)))
+(let (($x23450 (= ?x23449 b_S_kind_n_primitive$)))
+(let ((@x24651 (monotonicity (monotonicity (symm @x25274 (= ?x23443 ?x24218)) (= ?x23448 ?x23730)) (= ?x23449 ?x23768))))
+(let (($x23598 (b_S_is_n_non_n_primitive$ ?x23448)))
+(let (($x23599 (not $x23598)))
+(let (($x23602 (or $x23450 $x23599)))
+(let (($x23603 (not $x23602)))
+(let (($x24666 (or (not $x19234) $x23603)))
+(let ((@x24631 ((_ quant-inst (b_S_select_o_tm$ ?x10272 ?x10320)) $x24666)))
+(let ((@x24965 (unit-resolution (def-axiom (or $x23602 (not $x23450))) (unit-resolution @x24631 @x19237 $x23603) (not $x23450))))
+(let ((@x24645 (lemma (unit-resolution @x24965 (trans @x24651 (hypothesis $x23769) $x23450) false) (not $x23769))))
+(let ((@x24718 (unit-resolution (def-axiom (or $x24474 $x23770 $x23728 $x23769 $x24475)) @x24645 (unit-resolution (def-axiom (or $x23785 (not $x23776))) @x23976 $x23785) (or $x24474 $x23770 $x23728))))
+(let ((@x24717 (unit-resolution @x24718 @x24724 (unit-resolution (def-axiom (or $x23804 $x23775)) (mp @x24697 @x24701 $x23784) $x23804) @x24696 false)))
+(let ((@x20784 (def-axiom (or $x20013 $x15590 $x15593 $x20007))))
+(let ((@x24650 (unit-resolution (unit-resolution @x20784 @x24345 (or $x20013 $x15593 $x20007)) @x24998 (unit-resolution (def-axiom (or $x20016 $x20010)) @x24502 $x20010) $x20007)))
+(let ((@x20774 (def-axiom (or $x20004 $x19998))))
+(let ((@x20768 (def-axiom (or $x20001 $x15590 $x15599 $x19995))))
+(let ((@x25020 (unit-resolution (unit-resolution @x20768 @x24345 (or $x20001 $x15599 $x19995)) (unit-resolution @x20774 @x24650 $x19998) (or $x15599 $x19995))))
+(let ((@x23989 (hypothesis $x19980)))
+(let ((@x24787 (unit-resolution (def-axiom (or $x19959 $x15590 $x15599 $x19953)) @x24345 (or $x19959 $x15599 $x19953))))
+(let ((@x24655 (unit-resolution @x24787 (unit-resolution (def-axiom (or $x19992 $x10324)) (hypothesis $x19995) $x10324) (hypothesis $x19950) $x19959)))
+(let ((@x20748 (def-axiom (or $x19989 $x19977 $x19983))))
+(let ((@x24904 (unit-resolution @x20748 (unit-resolution (def-axiom (or $x19992 $x19986)) (hypothesis $x19995) $x19986) @x23989 $x19977)))
+(let ((@x20716 (def-axiom (or $x19974 $x19968))))
+(let ((@x24602 (unit-resolution (def-axiom (or $x19971 $x15590 $x15593 $x19965)) @x24345 (or $x19971 $x15593 $x19965))))
+(let ((@x24657 (unit-resolution @x24602 (unit-resolution @x20716 @x24904 $x19968) (unit-resolution (def-axiom (or $x19962 $x19956)) @x24655 $x19962) @x24998 false)))
+(let ((@x24972 (unit-resolution (lemma @x24657 (or $x19992 $x19983 $x19953)) @x23989 (unit-resolution @x25020 (lemma @x24717 $x10324) $x19995) $x19953)))
+(let (($x13277 (<= v_b_P_H_len$ 4294967295)))
+(let (($x13272 (= (+ b_S_max_o_u4$ (* (- 1) v_b_P_H_len$)) (+ 4294967295 (* (- 1) v_b_P_H_len$)))))
+(let ((@x13276 (monotonicity (monotonicity @x6446 $x13272) (= $x11245 (>= (+ 4294967295 (* (- 1) v_b_P_H_len$)) 0)))))
+(let ((@x13281 (trans @x13276 (rewrite (= (>= (+ 4294967295 (* (- 1) v_b_P_H_len$)) 0) $x13277)) (= $x11245 $x13277))))
+(let ((@x13282 (mp (and-elim @x12033 $x11245) @x13281 $x13277)))
+(let ((@x25068 (unit-resolution ((_ th-lemma arith assign-bounds 1 -1) (or $x13353 (not $x13277) $x11486)) @x13282 (or $x13353 $x11486))))
+(let ((@x25023 (unit-resolution (def-axiom (or $x19947 $x15611 $x15614 $x19941)) (unit-resolution ((_ th-lemma arith farkas 1 1) (or $x19670 $x11570)) @x24576 $x11570) (unit-resolution @x25068 @x24684 $x13353) (or $x19947 $x19941))))
+(let ((@x25021 (unit-resolution @x25023 (unit-resolution (def-axiom (or $x19950 $x19944)) @x24972 $x19944) $x19941)))
+(let ((@x20652 (def-axiom (or $x19938 $x19932))))
+(let (($x20596 (>= ?x11582 (- 1))))
+(let ((@x25129 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x19452 $x20596)) (unit-resolution (def-axiom (or $x19938 $x11580)) @x25021 $x11580) $x20596)))
+(let ((@x25134 (unit-resolution ((_ th-lemma arith assign-bounds -1 -1) (or $x11608 $x11486 (not $x20596))) @x24684 (or $x11608 (not $x20596)))))
+(let ((@x20638 (def-axiom (or $x19935 $x11612 $x19929))))
+(let ((@x25133 (unit-resolution @x20638 (unit-resolution @x25134 @x25129 $x11608) (unit-resolution @x20652 @x25021 $x19932) $x19929)))
+(let ((@x20630 (def-axiom (or $x19926 $x19920))))
+(let ((@x25121 (symm (unit-resolution (def-axiom (or $x19950 $x10338)) @x24972 $x10338) (= v_b_L_H_max_G_2$ v_b_L_H_max_G_3$))))
+(let ((@x25118 (symm (unit-resolution (def-axiom (or $x19950 $x10333)) @x24972 $x10333) (= ?x10327 v_b_L_H_max_G_2$))))
+(let ((@x25171 (monotonicity (unit-resolution (def-axiom (or $x19950 $x10340)) @x24972 $x10340) (= ?x10372 ?x10320))))
+(let ((@x25190 (trans (monotonicity @x25171 (= ?x10373 ?x10327)) @x25118 (= ?x10373 v_b_L_H_max_G_2$))))
+(let (($x24861 (>= (+ v_b_L_H_p_G_0$ (* (- 1) v_b_SL_H_witness_G_1$)) 0)))
+(let ((@x25188 (symm (unit-resolution (def-axiom (or $x19950 $x10340)) @x24972 $x10340) (= v_b_L_H_p_G_0$ v_b_SL_H_witness_G_1$))))
+(let ((@x25200 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= v_b_L_H_p_G_0$ v_b_SL_H_witness_G_1$)) $x24861)) @x25188 $x24861)))
+(let ((@x20614 (def-axiom (or $x19413 $x11647 (not $x10374)))))
+(let ((@x25206 (unit-resolution @x20614 (unit-resolution ((_ th-lemma arith assign-bounds -1 -1) (or $x11648 (not $x24861) $x11486)) @x25200 @x24684 $x11648) (trans @x25190 @x25121 $x10374) $x19413)))
+(let ((@x20618 (def-axiom (or $x19914 $x19412))))
+(let ((@x20626 (def-axiom (or $x19923 $x19386 $x19917))))
+(let ((@x25210 (unit-resolution @x20626 (unit-resolution @x20618 @x25206 $x19914) (unit-resolution @x20630 @x25133 $x19920) $x19386)))
+(let (($x24182 (>= (+ v_b_L_H_max_G_1$ ?x15891) 0)))
+(let (($x24206 (not $x24182)))
+(let ((?x11631 (* (- 1) v_b_L_H_max_G_3$)))
+(let ((?x20720 (+ v_b_L_H_max_G_1$ ?x11631)))
+(let (($x20721 (<= ?x20720 0)))
+(let (($x24870 (<= (+ ?x10327 ?x11631) 0)))
+(let ((@x25195 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not (= ?x10327 v_b_L_H_max_G_3$)) $x24870)) (trans @x25118 @x25121 (= ?x10327 v_b_L_H_max_G_3$)) $x24870)))
+(let ((@x20758 (def-axiom (or $x19992 $x19986))))
+(let ((@x25198 (unit-resolution @x20758 (unit-resolution @x25020 (lemma @x24717 $x10324) $x19995) $x19986)))
+(let ((@x25214 (unit-resolution (def-axiom (or $x19974 $x11515)) (unit-resolution @x20748 @x23989 @x25198 $x19977) $x11515)))
+(let ((@x24170 (hypothesis $x20721)))
+(let (($x20603 (not $x15893)))
+(let ((@x24171 (hypothesis $x20603)))
+(let ((@x24211 (lemma ((_ th-lemma arith farkas -1 1 1) (hypothesis $x24182) @x24171 @x24170 false) (or $x24206 $x15893 (not $x20721)))))
+(let ((@x25131 (unit-resolution @x24211 (unit-resolution (def-axiom (or $x19381 $x20603)) @x25210 $x20603) (unit-resolution ((_ th-lemma arith assign-bounds 1 1) (or $x20721 (not $x24870) $x11516)) @x25214 @x25195 $x20721) $x24206)))
+(let ((?x15869 (* (- 1) ?v0!14)))
+(let ((?x23656 (+ v_b_L_H_p_G_0$ ?x15869)))
+(let (($x24586 (>= ?x23656 0)))
+(let ((@x24735 (hypothesis $x20596)))
+(let ((@x24001 (unit-resolution ((_ th-lemma arith assign-bounds -1 -1) (or $x24586 $x15871 (not $x20596))) (hypothesis $x15876) @x24735 $x24586)))
+(let (($x23657 (<= ?x23656 0)))
+(let (($x24913 (or $x19903 $x19365 $x19366 $x23657 $x24182)))
+(let (($x23648 (<= (+ ?x15634 (* (- 1) v_b_L_H_max_G_1$)) 0)))
+(let (($x23640 (>= (+ ?v0!14 ?x11484) 0)))
+(let (($x23649 (or $x19365 $x19366 $x23640 $x23648)))
+(let (($x24853 (or $x19903 $x23649)))
+(let (($x24880 (= (+ ?x15634 (* (- 1) v_b_L_H_max_G_1$)) (+ (* (- 1) v_b_L_H_max_G_1$) ?x15634))))
+(let ((@x24024 (monotonicity (rewrite $x24880) (= $x23648 (<= (+ (* (- 1) v_b_L_H_max_G_1$) ?x15634) 0)))))
+(let ((@x24867 (trans @x24024 (rewrite (= (<= (+ (* (- 1) v_b_L_H_max_G_1$) ?x15634) 0) $x24182)) (= $x23648 $x24182))))
+(let ((@x24020 (monotonicity (rewrite (= (+ ?v0!14 ?x11484) (+ ?x11484 ?v0!14))) (= $x23640 (>= (+ ?x11484 ?v0!14) 0)))))
+(let ((@x24881 (trans @x24020 (rewrite (= (>= (+ ?x11484 ?v0!14) 0) $x23657)) (= $x23640 $x23657))))
+(let ((@x24935 (monotonicity (monotonicity @x24881 @x24867 (= $x23649 (or $x19365 $x19366 $x23657 $x24182))) (= $x24853 (or $x19903 (or $x19365 $x19366 $x23657 $x24182))))))
+(let ((@x24917 (trans @x24935 (rewrite (= (or $x19903 (or $x19365 $x19366 $x23657 $x24182)) $x24913)) (= $x24853 $x24913))))
+(let ((@x24941 (unit-resolution (mp ((_ quant-inst ?v0!14) $x24853) @x24917 $x24913) @x23333 (unit-resolution (def-axiom (or $x19381 $x15626)) (hypothesis $x19386) $x15626) (unit-resolution (def-axiom (or $x19381 $x15627)) (hypothesis $x19386) $x15627) (hypothesis $x24206) $x23657)))
+(let ((@x24757 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x25035 (not $x23657) (not $x24586))) @x24941 @x24001 (hypothesis (not $x25035)) false)))
+(let ((@x24761 (lemma @x24757 (or $x19381 $x25035 $x19903 $x24182 $x15871 (not $x20596)))))
+(let ((@x25179 (unit-resolution (unit-resolution @x24761 @x24499 (or $x19381 $x25035 $x24182 $x15871 (not $x20596))) @x25131 @x25129 (unit-resolution (def-axiom (or $x19381 $x15876)) @x25210 $x15876) @x25210 $x25035)))
+(let ((@x25060 (monotonicity (symm (hypothesis $x25035) (= ?v0!14 v_b_L_H_p_G_0$)) (= ?x15633 ?x10320))))
+(let ((@x25064 (unit-resolution (hypothesis (not $x25038)) (symm (monotonicity @x25060 (= ?x15634 ?x10327)) $x25038) false)))
+(let ((@x25067 (lemma @x25064 (or (not $x25035) $x25038))))
+(let ((@x25052 ((_ th-lemma arith triangle-eq) (or (not $x25038) $x25041))))
+(let ((@x25298 ((_ th-lemma arith farkas -1 -1 1) (unit-resolution (def-axiom (or $x19381 $x20603)) @x25210 $x20603) @x25195 (unit-resolution @x25052 (unit-resolution @x25067 @x25179 $x25038) $x25041) false)))
+(let ((@x25299 (lemma @x25298 $x19983)))
+(let ((@x24908 (unit-resolution @x25023 (unit-resolution (def-axiom (or $x19980 $x19944)) @x25299 $x19944) $x19941)))
+(let ((@x24947 (unit-resolution ((_ th-lemma arith triangle-eq) (or $x19452 $x20596)) (unit-resolution (def-axiom (or $x19938 $x11580)) @x24908 $x11580) $x20596)))
+(let ((@x24954 (unit-resolution @x20638 (unit-resolution @x25134 @x24947 $x11608) (unit-resolution @x20652 @x24908 $x19932) $x19929)))
+(let (($x20719 (= v_b_L_H_max_G_1$ v_b_L_H_max_G_3$)))
+(let ((@x25006 (mp (unit-resolution (def-axiom (or $x19980 $x10391)) @x25299 $x10391) (symm (commutativity (= $x20719 $x10391)) (= $x10391 $x20719)) $x20719)))
+(let (($x25065 (not $x25035)))
+(let (($x25044 (not $x25038)))
+(let (($x25049 (not $x25041)))
+(let ((@x25051 (lemma ((_ th-lemma arith farkas 1 -1 -1 1) (hypothesis $x25041) @x24170 @x24171 (hypothesis $x11516) false) (or $x25049 (not $x20721) $x15893 $x11515))))
+(let ((@x24891 (unit-resolution @x25051 (unit-resolution (def-axiom (or $x19980 $x11516)) (hypothesis $x19983) $x11516) @x24171 @x24170 $x25049)))
+(let ((@x24597 (unit-resolution @x20638 (unit-resolution ((_ th-lemma arith assign-bounds -1 -1) (or $x11608 $x11486 (not $x20596))) @x24735 @x23420 $x11608) (hypothesis $x19932) $x19929)))
+(let ((@x24892 (symm (unit-resolution (def-axiom (or $x19980 $x10391)) (hypothesis $x19983) $x10391) $x20719)))
+(let ((@x24061 (monotonicity (unit-resolution (def-axiom (or $x19980 $x10392)) (hypothesis $x19983) $x10392) (= ?x10372 ?x10190))))
+(let ((@x24887 (trans (monotonicity @x24061 (= ?x10373 ?x10191)) @x23175 (= ?x10373 v_b_L_H_max_G_1$))))
+(let ((?x11645 (* (- 1) v_b_SL_H_witness_G_1$)))
+(let ((?x20724 (+ v_b_SL_H_witness_G_0$ ?x11645)))
+(let (($x20726 (>= ?x20724 0)))
+(let (($x20723 (= v_b_SL_H_witness_G_0$ v_b_SL_H_witness_G_1$)))
+(let ((@x24982 (mp (unit-resolution (def-axiom (or $x19980 $x10392)) (hypothesis $x19983) $x10392) (symm (commutativity (= $x20723 $x10392)) (= $x10392 $x20723)) $x20723)))
+(let ((@x24888 (lemma ((_ th-lemma arith farkas 1 -1 1) (hypothesis $x20726) (hypothesis $x11647) @x23180 false) (or $x11648 (not $x20726) $x11867))))
+(let ((@x24648 (unit-resolution @x24888 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x20723) $x20726)) @x24982 $x20726) @x23180 $x11648)))
+(let ((@x24798 (unit-resolution @x20618 (unit-resolution @x20614 @x24648 (trans @x24887 @x24892 $x10374) $x19413) $x19914)))
+(let ((@x20602 (def-axiom (or $x19381 $x15876))))
+(let ((@x25013 (unit-resolution @x20602 (unit-resolution @x20626 @x24798 (unit-resolution @x20630 @x24597 $x19920) $x19386) $x15876)))
+(let ((@x25017 (unit-resolution @x24761 @x25013 (unit-resolution @x20626 @x24798 (unit-resolution @x20630 @x24597 $x19920) $x19386) @x23333 (unit-resolution @x24211 @x24171 @x24170 $x24206) (unit-resolution @x25067 (unit-resolution @x25052 @x24891 $x25044) $x25065) @x24735 false)))
+(let ((@x24056 (lemma @x25017 (or $x19980 $x19903 (not $x20596) $x11867 $x15893 (not $x20721) $x19935 $x11486 $x19674))))
+(let ((@x24843 (unit-resolution @x24056 @x24499 @x24415 @x24684 @x24314 (or $x19980 (not $x20596) $x15893 (not $x20721) $x19935))))
+(let ((@x24844 (unit-resolution @x24843 (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x20719) $x20721)) @x25006 $x20721) @x25299 @x24947 (unit-resolution @x20652 @x24908 $x19932) $x15893)))
+(let ((@x20605 (def-axiom (or $x19381 $x20603))))
+(let ((@x25302 (monotonicity (unit-resolution (def-axiom (or $x19980 $x10392)) @x25299 $x10392) (= ?x10372 ?x10190))))
+(let ((@x25305 (trans (monotonicity @x25302 (= ?x10373 ?x10191)) @x24314 (= ?x10373 v_b_L_H_max_G_1$))))
+(let ((@x25306 (trans @x25305 (symm (unit-resolution (def-axiom (or $x19980 $x10391)) @x25299 $x10391) $x20719) $x10374)))
+(let ((@x25307 (mp (unit-resolution (def-axiom (or $x19980 $x10392)) @x25299 $x10392) (symm (commutativity (= $x20723 $x10392)) (= $x10392 $x20723)) $x20723)))
+(let ((@x25311 (unit-resolution (unit-resolution @x24888 @x24415 (or $x11648 (not $x20726))) (unit-resolution ((_ th-lemma arith triangle-eq) (or (not $x20723) $x20726)) @x25307 $x20726) $x11648)))
+(unit-resolution @x20626 (unit-resolution @x20618 (unit-resolution @x20614 @x25311 @x25306 $x19413) $x19914) (unit-resolution @x20605 @x24844 $x19381) (unit-resolution @x20630 @x24954 $x19920) false))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))))
+
--- a/src/HOL/Tools/SMT2/smt2_systems.ML	Tue Jun 03 16:22:01 2014 +0200
+++ b/src/HOL/Tools/SMT2/smt2_systems.ML	Tue Jun 03 16:27:31 2014 +0200
@@ -125,6 +125,7 @@
 
   fun z3_options ctxt =
     ["smt.random_seed=" ^ string_of_int (Config.get ctxt SMT2_Config.random_seed),
+     "smt.refine_inj_axioms=false",
      "-T:" ^ string_of_int (Real.ceil (Config.get ctxt SMT2_Config.timeout)),
      "-smt2"]