src/HOL/SAT.thy
changeset 60758 d8d85a8172b5
parent 58889 5b7a9633cfa8
child 63962 83a625d06e91
--- a/src/HOL/SAT.thy	Sat Jul 18 21:44:18 2015 +0200
+++ b/src/HOL/SAT.thy	Sat Jul 18 22:58:50 2015 +0200
@@ -5,7 +5,7 @@
 Basic setup for the 'sat' and 'satx' tactics.
 *)
 
-section {* Reconstructing external resolution proofs for propositional logic *}
+section \<open>Reconstructing external resolution proofs for propositional logic\<close>
 
 theory SAT
 imports HOL
@@ -15,10 +15,10 @@
 ML_file "Tools/sat_solver.ML"
 ML_file "Tools/sat.ML"
 
-method_setup sat = {* Scan.succeed (SIMPLE_METHOD' o SAT.sat_tac) *}
+method_setup sat = \<open>Scan.succeed (SIMPLE_METHOD' o SAT.sat_tac)\<close>
   "SAT solver"
 
-method_setup satx = {* Scan.succeed (SIMPLE_METHOD' o SAT.satx_tac) *}
+method_setup satx = \<open>Scan.succeed (SIMPLE_METHOD' o SAT.satx_tac)\<close>
   "SAT solver (with definitional CNF)"
 
 end