src/HOL/Mirabelle/ex/Ex.thy
author wenzelm
Wed, 09 Mar 2016 19:30:09 +0100
changeset 62573 27f90319a499
parent 48589 fb446a780d50
child 62589 b5783412bfed
permissions -rw-r--r--
isabelle.Build uses ML_Process directly; isabelle_process is for batch mode only; removed unused feeder (already part of "isabelle console");

theory Ex imports Pure
begin

ML {*
  val rc = Isabelle_System.bash
    "cd \"$ISABELLE_HOME/src/HOL/Library\"; \"$ISABELLE_TOOL\" mirabelle arith Inner_Product.thy";
  if rc <> 0 then error ("Mirabelle example failed: " ^ string_of_int rc)
  else ();
*} -- "some arbitrary small test case"

end