--- a/src/HOL/Groebner_Basis.thy Fri May 07 15:05:52 2010 +0200
+++ b/src/HOL/Groebner_Basis.thy Fri May 07 16:12:25 2010 +0200
@@ -7,7 +7,7 @@
theory Groebner_Basis
imports Semiring_Normalization
uses
- ("Tools/Groebner_Basis/groebner.ML")
+ ("Tools/groebner.ML")
begin
subsection {* Groebner Bases *}
@@ -40,7 +40,7 @@
setup Algebra_Simplification.setup
-use "Tools/Groebner_Basis/groebner.ML"
+use "Tools/groebner.ML"
method_setup algebra = Groebner.algebra_method
"solve polynomial equations over (semi)rings and ideal membership problems using Groebner bases"