src/HOL/Groebner_Basis.thy
changeset 35410 1ea89d2a1bd4
parent 35216 7641e8d831d2
child 36305 dbe99291eb3c
--- a/src/HOL/Groebner_Basis.thy	Sun Feb 28 22:30:51 2010 +0100
+++ b/src/HOL/Groebner_Basis.thy	Sun Feb 28 23:51:31 2010 +0100
@@ -510,7 +510,7 @@
     let
       val z = instantiate_cterm ([(zT,T)],[]) zr
       val eq = instantiate_cterm ([(eqT,T)],[]) geq
-      val th = Simplifier.rewrite (ss addsimps simp_thms)
+      val th = Simplifier.rewrite (ss addsimps @{thms simp_thms})
            (Thm.capply @{cterm "Trueprop"} (Thm.capply @{cterm "Not"}
                   (Thm.capply (Thm.capply eq t) z)))
     in equal_elim (symmetric th) TrueI
@@ -640,7 +640,7 @@
 
 val comp_conv = (Simplifier.rewrite
 (HOL_basic_ss addsimps @{thms "Groebner_Basis.comp_arith"}
-              addsimps ths addsimps simp_thms
+              addsimps ths addsimps @{thms simp_thms}
               addsimprocs Numeral_Simprocs.field_cancel_numeral_factors
                addsimprocs [add_frac_frac_simproc, add_frac_num_simproc,
                             ord_frac_simproc]