src/HOL/Boogie/Examples/Boogie_Max.thy
changeset 33445 f0c78a28e18e
parent 33424 a3b002e2cd55
child 33663 a84fd6385832
--- a/src/HOL/Boogie/Examples/Boogie_Max.thy	Thu Nov 05 14:41:37 2009 +0100
+++ b/src/HOL/Boogie/Examples/Boogie_Max.thy	Thu Nov 05 14:48:40 2009 +0100
@@ -41,9 +41,9 @@
 text {*
 Approach 1: Discharge the verification condition fully automatically by SMT:
 *}
-boogie_vc b_max
+boogie_vc max
   unfolding labels
-  using [[smt_cert="~~/src/HOL/Boogie/Examples/cert/Boogie_b_max"]]
+  using [[smt_cert="~~/src/HOL/Boogie/Examples/cert/Boogie_max"]]
   using [[z3_proofs=true]]
   by (smt boogie)
 
@@ -53,7 +53,7 @@
 explicit proof. This approach is most useful in an interactive debug-and-fix
 mode. 
 *}
-boogie_vc b_max
+boogie_vc max
 proof (split_vc (verbose) try: fast simp)
   print_cases
   case L_14_5c