QuotMain.thy
changeset 217 9cc87d02190a
parent 214 a66f81c264aa
child 219 329111e1c4ba
--- a/QuotMain.thy	Wed Oct 28 12:22:06 2009 +0100
+++ b/QuotMain.thy	Wed Oct 28 14:59:24 2009 +0100
@@ -355,7 +355,7 @@
   val thm' = forall_intr_vars thm
   val thm'' = ObjectLogic.atomize (cprop_of thm')
 in
-  Thm.freezeT (Simplifier.rewrite_rule [thm''] thm')
+  Thm.freezeT @{thm Pure.equal_elim_rule1} OF [thm'', thm']
 end
 *}