src/HOL/Complex/ex/MIR.thy
changeset 24249 1f60b45c5f97
parent 23997 a23d0b4b1c1f
child 24336 fff40259f336
equal deleted inserted replaced
24248:d276e4b53d6b 24249:1f60b45c5f97
  5776 
  5776 
  5777 definition
  5777 definition
  5778   "test5 (u\<Colon>unit) = mircfrqe (A(E(And (Ge(Sub (Bound 1) (Bound 0))) (Eq (Add (Floor (Bound 1)) (Floor (Neg(Bound 0))))))))"
  5778   "test5 (u\<Colon>unit) = mircfrqe (A(E(And (Ge(Sub (Bound 1) (Bound 0))) (Eq (Add (Floor (Bound 1)) (Floor (Neg(Bound 0))))))))"
  5779 
  5779 
  5780 code_gen mircfrqe mirlfrqe test1 test2 test3 test4 test5
  5780 code_gen mircfrqe mirlfrqe test1 test2 test3 test4 test5
  5781   in SML to Mir
  5781   in SML module_name Mir
  5782 
  5782 
  5783 code_gen mircfrqe mirlfrqe in SML to Mir file "raw_mir.ML"
  5783 (*code_gen mircfrqe mirlfrqe
       
  5784   in SML module_name Mir file "raw_mir.ML"*)
  5784 
  5785 
  5785 ML "set Toplevel.timing"
  5786 ML "set Toplevel.timing"
  5786 ML "Mir.test1 ()"
  5787 ML "Mir.test1 ()"
  5787 ML "Mir.test2 ()"
  5788 ML "Mir.test2 ()"
  5788 ML "Mir.test3 ()"
  5789 ML "Mir.test3 ()"