src/HOL/Mirabelle/ex/Ex.thy
changeset 69043 57a76e4728ed
parent 67443 3abf6a722518
equal deleted inserted replaced
69042:6e9df530b441 69043:57a76e4728ed
     1 theory Ex imports Pure
     1 theory Ex imports Pure
     2 begin
     2 begin
     3 
     3 
     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\"; if isabelle build -n \"$MIRABELLE_LOGIC\"; then isabelle mirabelle arith Inner_Product.thy; fi";
     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> \<open>some arbitrary small test case\<close>
     9 \<close> \<comment> \<open>some arbitrary small test case\<close>
    10 
    10 
    11 end
    11 end