src/HOL/Boogie/Examples/Boogie_Max.thy
changeset 52722 2c81f7baf8c4
parent 52721 6bafe21b13b2
child 52724 f547266a9338
--- a/src/HOL/Boogie/Examples/Boogie_Max.thy	Tue Jul 23 13:14:14 2013 +0200
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,50 +0,0 @@
-(*  Title:      HOL/Boogie/Examples/Boogie_Max.thy
-    Author:     Sascha Boehme, TU Muenchen
-*)
-
-header {* Boogie example: get the greatest element of a list *}
-
-theory Boogie_Max
-imports Boogie
-begin
-
-text {*
-We prove correct the verification condition generated from the following
-Boogie code:
-
-\begin{verbatim}
-procedure max(array : [int]int, length : int)
-  returns (max : int);
-  requires (0 < length);
-  ensures (forall i: int :: 0 <= i && i < length ==> array[i] <= max);
-  ensures (exists i: int :: 0 <= i && i < length ==> array[i] == max);
-
-implementation max(array : [int]int, length : int) returns (max : int)
-{
-  var p : int, k : int;
-  max := array[0];
-  k := 0;
-  p := 1;
-  while (p < length)
-    invariant (forall i: int :: 0 <= i && i < p ==> array[i] <= max);
-    invariant (array[k] == max);
-  {
-    if (array[p] > max) { max := array[p]; k := p; }
-    p := p + 1;
-  }
-}
-\end{verbatim}
-*}
-
-boogie_open "Boogie_Max.b2i"
-
-declare [[smt_oracle = false]]
-declare [[smt_certificates = "Boogie_Max.certs"]]
-declare [[smt_read_only_certificates = true]]
-
-boogie_vc max
-  by boogie
-
-boogie_end
-
-end