src/HOL/IMP/Abs_Int2_ivl.thy
changeset 49188 22f7e7b68f50
parent 47613 e72e44cee6f2
child 49396 73fb17ed2e08
--- a/src/HOL/IMP/Abs_Int2_ivl.thy	Thu Sep 06 08:59:50 2012 -0700
+++ b/src/HOL/IMP/Abs_Int2_ivl.thy	Fri Sep 07 07:20:55 2012 +0200
@@ -261,6 +261,7 @@
 value "show_acom (steps test2_ivl 0)"
 value "show_acom (steps test2_ivl 1)"
 value "show_acom (steps test2_ivl 2)"
+value "show_acom (steps test2_ivl 3)"
 
 text{* Fixed point reached in 2 steps.
  Not so if the start value of x is known: *}
@@ -271,6 +272,7 @@
 value "show_acom (steps test3_ivl 2)"
 value "show_acom (steps test3_ivl 3)"
 value "show_acom (steps test3_ivl 4)"
+value "show_acom (steps test3_ivl 5)"
 
 text{* Takes as many iterations as the actual execution. Would diverge if
 loop did not terminate. Worse still, as the following example shows: even if