changeset 62589 | b5783412bfed |
parent 62573 | 27f90319a499 |
child 63167 | 0909deb8059b |
--- a/src/HOL/Mirabelle/ex/Ex.thy Thu Mar 10 12:11:50 2016 +0100 +++ b/src/HOL/Mirabelle/ex/Ex.thy Thu Mar 10 17:30:04 2016 +0100 @@ -3,7 +3,7 @@ ML {* val rc = Isabelle_System.bash - "cd \"$ISABELLE_HOME/src/HOL/Library\"; \"$ISABELLE_TOOL\" mirabelle arith Inner_Product.thy"; + "cd \"$ISABELLE_HOME/src/HOL/Library\"; isabelle mirabelle arith Inner_Product.thy"; if rc <> 0 then error ("Mirabelle example failed: " ^ string_of_int rc) else (); *} -- "some arbitrary small test case"