src/HOL/Mirabelle/ex/Ex.thy
author haftmann
Wed, 25 Dec 2013 15:52:25 +0100
changeset 54861 00d551179872
parent 48589 fb446a780d50
child 62573 27f90319a499
permissions -rw-r--r--
postponed min/max lemmas until abstract lattice is available

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