src/HOL/Decision_Procs/MIR.thy
changeset 51272 9c8d63b4b6be
parent 51143 0a2371e7ced3
child 51369 960b0ca9ae5d
equal deleted inserted replaced
51271:e8d2ecf6aaac 51272:9c8d63b4b6be
  5500   "problem3 = A (And (Le (Sub (Floor (Bound 0)) (Bound 0))) (Le (Add (Bound 0) (Floor (Neg (Bound 0))))))"
  5500   "problem3 = A (And (Le (Sub (Floor (Bound 0)) (Bound 0))) (Le (Add (Bound 0) (Floor (Neg (Bound 0))))))"
  5501 
  5501 
  5502 definition
  5502 definition
  5503   "problem4 = E (And (Ge (Sub (Bound 1) (Bound 0))) (Eq (Add (Floor (Bound 1)) (Floor (Neg (Bound 0))))))"
  5503   "problem4 = E (And (Ge (Sub (Bound 1) (Bound 0))) (Eq (Add (Floor (Bound 1)) (Floor (Neg (Bound 0))))))"
  5504 
  5504 
  5505 ML {*
  5505 ML_val {* @{code mircfrqe} @{code problem1} *}
  5506   Par_List.map (fn e => e ())
  5506 ML_val {* @{code mirlfrqe} @{code problem1} *}
  5507    [fn () => @{code mircfrqe} @{code problem1},
  5507 ML_val {* @{code mircfrqe} @{code problem2} *}
  5508     fn () => @{code mirlfrqe} @{code problem1},
  5508 ML_val {* @{code mirlfrqe} @{code problem2} *}
  5509     fn () => @{code mircfrqe} @{code problem2},
  5509 ML_val {* @{code mircfrqe} @{code problem3} *}
  5510     fn () => @{code mirlfrqe} @{code problem2},
  5510 ML_val {* @{code mirlfrqe} @{code problem3} *}
  5511     fn () => @{code mircfrqe} @{code problem3},
  5511 ML_val {* @{code mircfrqe} @{code problem4} *}
  5512     fn () => @{code mirlfrqe} @{code problem3},
  5512 ML_val {* @{code mirlfrqe} @{code problem4} *}
  5513     fn () => @{code mircfrqe} @{code problem4},
  5513 
  5514     fn () => @{code mirlfrqe} @{code problem4}]
       
  5515 *}
       
  5516 
  5514 
  5517 (*code_reflect Mir
  5515 (*code_reflect Mir
  5518   functions mircfrqe mirlfrqe
  5516   functions mircfrqe mirlfrqe
  5519   file "mir.ML"*)
  5517   file "mir.ML"*)
  5520 
  5518