src/HOL/Complex/ex/MIR.thy
changeset 24348 c708ea5b109a
parent 24336 fff40259f336
child 24473 acd19ea21fbb
equal deleted inserted replaced
24347:245ff8661b8c 24348:c708ea5b109a
  5770   "test4 (u\<Colon>unit) = mirlfrqe (A (Iff (Eq (Add (Floor (Bound 0)) (Floor (Neg (Bound 0))))) (Eq (Sub (Floor (Bound 0)) (Bound 0)))))"
  5770   "test4 (u\<Colon>unit) = mirlfrqe (A (Iff (Eq (Add (Floor (Bound 0)) (Floor (Neg (Bound 0))))) (Eq (Sub (Floor (Bound 0)) (Bound 0)))))"
  5771 
  5771 
  5772 definition
  5772 definition
  5773   "test5 (u\<Colon>unit) = mircfrqe (A(E(And (Ge(Sub (Bound 1) (Bound 0))) (Eq (Add (Floor (Bound 1)) (Floor (Neg(Bound 0))))))))"
  5773   "test5 (u\<Colon>unit) = mircfrqe (A(E(And (Ge(Sub (Bound 1) (Bound 0))) (Eq (Add (Floor (Bound 1)) (Floor (Neg(Bound 0))))))))"
  5774 
  5774 
  5775 code_gen mircfrqe mirlfrqe test1 test2 test3 test4 test5
  5775 export_code mircfrqe mirlfrqe test1 test2 test3 test4 test5
  5776   in SML module_name Mir
  5776   in SML module_name Mir
  5777 
  5777 
  5778 (*code_gen mircfrqe mirlfrqe
  5778 (*export_code mircfrqe mirlfrqe
  5779   in SML module_name Mir file "raw_mir.ML"*)
  5779   in SML module_name Mir file "raw_mir.ML"*)
  5780 
  5780 
  5781 ML "set Toplevel.timing"
  5781 ML "set Toplevel.timing"
  5782 ML "Mir.test1 ()"
  5782 ML "Mir.test1 ()"
  5783 ML "Mir.test2 ()"
  5783 ML "Mir.test2 ()"