src/Sequents/T.thy
changeset 60770 240563fbf41d
parent 54742 7a86358a3c0b
child 61385 538100cc4399
--- a/src/Sequents/T.thy	Thu Jul 23 14:20:51 2015 +0200
+++ b/src/Sequents/T.thy	Thu Jul 23 14:25:05 2015 +0200
@@ -30,7 +30,7 @@
    "[| $E |L> $E';  $F |L> $F';  $G |R> $G';
                $E', P, $F'|-         $G'|] ==> $E, <>P, $F |-          $G"
 
-ML {*
+ML \<open>
 structure T_Prover = Modal_ProverFun
 (
   val rewrite_rls = @{thms rewrite_rls}
@@ -40,9 +40,9 @@
   val aside_rls = [@{thm lstar0}, @{thm lstar1}, @{thm lstar2}, @{thm rstar0},
     @{thm rstar1}, @{thm rstar2}]
 )
-*}
+\<close>
 
-method_setup T_solve = {* Scan.succeed (fn ctxt => SIMPLE_METHOD (T_Prover.solve_tac ctxt 2)) *}
+method_setup T_solve = \<open>Scan.succeed (fn ctxt => SIMPLE_METHOD (T_Prover.solve_tac ctxt 2))\<close>
 
 
 (* Theorems of system T from Hughes and Cresswell and Hailpern, LNCS 129 *)