src/HOL/Mirabelle/ex/Ex.thy
author traytel
Thu, 12 Sep 2013 11:23:49 +0200
changeset 53560 4b5f42cfa244
parent 48589 fb446a780d50
child 62573 27f90319a499
permissions -rw-r--r--
removed unused/inlinable theorems

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