more accurate keywords;
authorwenzelm
Fri, 07 Nov 2014 15:19:30 +0100
changeset 58925 1b655309617c
parent 58924 b48bbd380d59
child 58926 baf5a3c28f0c
more accurate keywords;
src/HOL/Groebner_Basis.thy
src/HOL/Presburger.thy
--- a/src/HOL/Groebner_Basis.thy	Thu Nov 06 16:10:33 2014 +0100
+++ b/src/HOL/Groebner_Basis.thy	Fri Nov 07 15:19:30 2014 +0100
@@ -6,7 +6,6 @@
 
 theory Groebner_Basis
 imports Semiring_Normalization Parity
-keywords "try0" :: diag
 begin
 
 subsection {* Groebner Bases *}
--- a/src/HOL/Presburger.thy	Thu Nov 06 16:10:33 2014 +0100
+++ b/src/HOL/Presburger.thy	Fri Nov 07 15:19:30 2014 +0100
@@ -6,6 +6,7 @@
 
 theory Presburger
 imports Groebner_Basis Set_Interval
+keywords "try0" :: diag
 begin
 
 ML_file "Tools/Qelim/qelim.ML"