QuotMain.thy
changeset 219 329111e1c4ba
parent 218 df05cd030d2f
parent 217 9cc87d02190a
child 221 f219011a5e3c
--- a/QuotMain.thy	Wed Oct 28 15:25:11 2009 +0100
+++ b/QuotMain.thy	Wed Oct 28 15:25:36 2009 +0100
@@ -400,7 +400,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
 *}