src/HOL/IMP/Abs_Int3.thy
changeset 49399 a9d9f3483b71
parent 49396 73fb17ed2e08
child 49496 2694d1615eef
equal deleted inserted replaced
49398:0fa4389c04f9 49399:a9d9f3483b71
   381 ..
   381 ..
   382 
   382 
   383 
   383 
   384 subsubsection "Tests"
   384 subsubsection "Tests"
   385 
   385 
   386 (* FIXME dirty trick to get around some problem with the code generator *)
   386 (* Trick to make the code generator happy. *)
   387 lemma [code]: "equal_class.equal (x::'a st) y = equal_class.equal x y"
   387 lemma [code]: "equal_class.equal (x::'a st) y = equal_class.equal x y"
   388 by(rule refl)
   388 by(rule refl)
   389 
   389 
   390 definition "step_up_ivl n =
   390 definition "step_up_ivl n =
   391   ((\<lambda>C. C \<nabla> step_ivl (top(strip C)) C)^^n)"
   391   ((\<lambda>C. C \<nabla> step_ivl (top(strip C)) C)^^n)"