src/HOL/Boogie/Examples/Boogie_Dijkstra.thy
changeset 40163 a462d5207aa6
parent 36081 70deefb6c093
child 40513 1204d268464f
--- a/src/HOL/Boogie/Examples/Boogie_Dijkstra.thy	Tue Oct 26 11:45:12 2010 +0200
+++ b/src/HOL/Boogie/Examples/Boogie_Dijkstra.thy	Tue Oct 26 11:46:19 2010 +0200
@@ -83,9 +83,9 @@
 
 declare [[smt_certificates="~~/src/HOL/Boogie/Examples/Boogie_Dijkstra.certs"]]
 declare [[smt_fixed=true]]
+declare [[smt_oracle=false]]
 
 boogie_vc Dijkstra
-  using [[z3_proofs=true]]
   by boogie
 
 boogie_end