24.04.2013 Views

Verification of Parameterised FPGA Circuit Descriptions with Layout ...

Verification of Parameterised FPGA Circuit Descriptions with Layout ...

Verification of Parameterised FPGA Circuit Descriptions with Layout ...

SHOW MORE
SHOW LESS

Create successful ePaper yourself

Turn your PDF publications into a flip-book with our unique Google optimized e-Paper software.

APPENDIX B. THEORETICAL BASIS FOR LAYOUT REASONING 206<br />

theorem min_max_corres: "!! (a::int) (b::int). min a b = - (max (-a) (-b))"<br />

apply (simp add: max_def min_def)<br />

done<br />

section {* minf function and correspondance <strong>with</strong> maxf *}<br />

consts<br />

minf :: "(int*int*(int=>int))=>int"<br />

recdef minf "measure (%(b, t, f). nat(t+1-b))"<br />

"minf (bot, top, fun) = (if (top < bot) then 0<br />

else (<br />

case (top = bot) <strong>of</strong> True =><br />

fun top<br />

| False => (<br />

let one = fun top in<br />

let two = minf (bot, top - 1, fun) in<br />

min one two)<br />

))"<br />

theorem minf_maxf_corres: "!! (f::int=>int) b t. minf(b,t,f) = - maxf (b,t,% x.- f x)<br />

"<br />

apply (case_tac "b

Hooray! Your file is uploaded and ready to be published.

Saved successfully!

Ooh no, something went wrong!