src/HOL/Mirabelle/ex/Ex.thy
changeset 67443 3abf6a722518
parent 63971 da89140186e2
child 69043 57a76e4728ed
equal deleted inserted replaced
67442:f075640b8868 67443:3abf6a722518
     4 ML \<open>
     4 ML \<open>
     5   val rc = Isabelle_System.bash
     5   val rc = Isabelle_System.bash
     6     "cd \"$ISABELLE_HOME/src/HOL/Analysis\"; isabelle mirabelle arith Inner_Product.thy";
     6     "cd \"$ISABELLE_HOME/src/HOL/Analysis\"; isabelle 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 \<close> \<comment> "some arbitrary small test case"
     9 \<close> \<comment> \<open>some arbitrary small test case\<close>
    10 
    10 
    11 end
    11 end
    12 
    12