src/HOLCF/IOA/NTP/Impl.thy
changeset 24327 a207114007c6
parent 19741 f65265d71426
child 25113 008c964dd47f
--- a/src/HOLCF/IOA/NTP/Impl.thy	Sat Aug 18 17:42:38 2007 +0200
+++ b/src/HOLCF/IOA/NTP/Impl.thy	Sat Aug 18 17:42:39 2007 +0200
@@ -357,11 +357,9 @@
 
 text {* rebind them *}
 
-ML_setup {*
-bind_thm ("inv1", rewrite_rule [thm "Impl.inv1_def"] (thm "inv1" RS thm "invariantE"));
-bind_thm ("inv2", rewrite_rule [thm "Impl.inv2_def"] (thm "inv2" RS thm "invariantE"));
-bind_thm ("inv3", rewrite_rule [thm "Impl.inv3_def"] (thm "inv3" RS thm "invariantE"));
-bind_thm ("inv4", rewrite_rule [thm "Impl.inv4_def"] (thm "inv4" RS thm "invariantE"));
-*}
+lemmas inv1 = inv1 [THEN invariantE, unfolded inv1_def]
+  and inv2 = inv2 [THEN invariantE, unfolded inv2_def]
+  and inv3 = inv3 [THEN invariantE, unfolded inv3_def]
+  and inv4 = inv4 [THEN invariantE, unfolded inv4_def]
 
 end