src/Sequents/Washing.thy
changeset 26480 544cef16045b
parent 21426 87ac12bed1ab
child 35762 af3ff2ba4c54
--- a/src/Sequents/Washing.thy	Sat Mar 29 19:13:58 2008 +0100
+++ b/src/Sequents/Washing.thy	Sat Mar 29 19:14:00 2008 +0100
@@ -35,10 +35,10 @@
 
 (* "activate" definitions for use in proof *)
 
-ML_setup {* bind_thms ("changeI", [thm "context1"] RL ([thm "change"] RLN (2,[thm "cut"]))) *}
-ML_setup {* bind_thms ("load1I", [thm "context1"] RL ([thm "load1"] RLN (2,[thm "cut"]))) *}
-ML_setup {* bind_thms ("washI", [thm "context1"] RL ([thm "wash"] RLN (2,[thm "cut"]))) *}
-ML_setup {* bind_thms ("dryI", [thm "context1"] RL ([thm "dry"] RLN (2,[thm "cut"]))) *}
+ML {* bind_thms ("changeI", [thm "context1"] RL ([thm "change"] RLN (2,[thm "cut"]))) *}
+ML {* bind_thms ("load1I", [thm "context1"] RL ([thm "load1"] RLN (2,[thm "cut"]))) *}
+ML {* bind_thms ("washI", [thm "context1"] RL ([thm "wash"] RLN (2,[thm "cut"]))) *}
+ML {* bind_thms ("dryI", [thm "context1"] RL ([thm "dry"] RLN (2,[thm "cut"]))) *}
 
 (* a load of dirty clothes and two dollars gives you clean clothes *)