eliminated odd dislocation of keyword declaration and implementation (leftover from 318cd8ac1817)
--- a/src/HOL/Groebner_Basis.thy Sat Feb 15 21:11:29 2014 +0100
+++ b/src/HOL/Groebner_Basis.thy Sun Feb 16 13:56:48 2014 +0100
@@ -6,6 +6,7 @@
theory Groebner_Basis
imports Semiring_Normalization
+keywords "try0" :: diag
begin
subsection {* Groebner Bases *}
--- a/src/HOL/Metis.thy Sat Feb 15 21:11:29 2014 +0100
+++ b/src/HOL/Metis.thy Sun Feb 16 13:56:48 2014 +0100
@@ -8,7 +8,6 @@
theory Metis
imports ATP
-keywords "try0" :: diag
begin
ML_file "~~/src/Tools/Metis/metis.ML"