src/ZF/UNITY/Constrains.thy
changeset 60770 240563fbf41d
parent 60754 02924903a6fd
child 68233 5e0e9376b2b0
--- a/src/ZF/UNITY/Constrains.thy	Thu Jul 23 14:20:51 2015 +0200
+++ b/src/ZF/UNITY/Constrains.thy	Thu Jul 23 14:25:05 2015 +0200
@@ -3,7 +3,7 @@
     Copyright   2001  University of Cambridge
 *)
 
-section{*Weak Safety Properties*}
+section\<open>Weak Safety Properties\<close>
 
 theory Constrains
 imports UNITY
@@ -457,7 +457,7 @@
 named_theorems program "program definitions"
 
 ML
-{*
+\<open>
 (*Combines two invariance ASSUMPTIONS into one.  USEFUL??*)
 fun Always_Int_tac ctxt =
   dresolve_tac ctxt @{thms Always_Int_I} THEN'
@@ -494,14 +494,14 @@
   resolve_tac ctxt @{thms AlwaysI} i THEN
   force_tac ctxt i
   THEN constrains_tac ctxt i;
-*}
+\<close>
 
-method_setup safety = {*
-  Scan.succeed (SIMPLE_METHOD' o constrains_tac) *}
+method_setup safety = \<open>
+  Scan.succeed (SIMPLE_METHOD' o constrains_tac)\<close>
   "for proving safety properties"
 
-method_setup always = {*
-  Scan.succeed (SIMPLE_METHOD' o always_tac) *}
+method_setup always = \<open>
+  Scan.succeed (SIMPLE_METHOD' o always_tac)\<close>
   "for proving invariants"
 
 end