src/HOL/Mirabelle/ex/Ex.thy
changeset 62573 27f90319a499
parent 48589 fb446a780d50
child 62589 b5783412bfed
equal deleted inserted replaced
62572:acd17a6ce17d 62573:27f90319a499
     1 theory Ex imports Pure
     1 theory Ex imports Pure
     2 begin
     2 begin
     3 
     3 
     4 ML {*
     4 ML {*
     5   val rc = Isabelle_System.bash
     5   val rc = Isabelle_System.bash
     6     "cd \"$ISABELLE_HOME/src/HOL/Library\"; \"$ISABELLE_TOOL\" mirabelle -q arith Inner_Product.thy";
     6     "cd \"$ISABELLE_HOME/src/HOL/Library\"; \"$ISABELLE_TOOL\" mirabelle arith Inner_Product.thy";
     7   if rc <> 0 then error ("Mirabelle example failed: " ^ string_of_int rc)
     7   if rc <> 0 then error ("Mirabelle example failed: " ^ string_of_int rc)
     8   else ();
     8   else ();
     9 *} -- "some arbitrary small test case"
     9 *} -- "some arbitrary small test case"
    10 
    10 
    11 end
    11 end