src/HOL/Mirabelle/ex/Ex.thy
author wenzelm
Sat, 28 Jul 2012 20:36:25 +0200
changeset 48589 fb446a780d50
child 62573 27f90319a499
permissions -rw-r--r--
separate session HOL-Mirabelle-ex -- cannot run isolated shell scripts within build tool;

theory Ex imports Pure
begin

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

end