diff -r a80d8ec6c998 -r 3dda49e08b9d src/HOL/Groebner_Basis.thy --- a/src/HOL/Groebner_Basis.thy Fri Jan 04 21:49:06 2019 +0100 +++ b/src/HOL/Groebner_Basis.thy Fri Jan 04 23:22:53 2019 +0100 @@ -10,9 +10,9 @@ subsection \Groebner Bases\ -lemmas bool_simps = simp_thms(1-34) \ \FIXME move to @{theory HOL.HOL}\ +lemmas bool_simps = simp_thms(1-34) \ \FIXME move to \<^theory>\HOL.HOL\\ -lemma nnf_simps: \ \FIXME shadows fact binding in @{theory HOL.HOL}\ +lemma nnf_simps: \ \FIXME shadows fact binding in \<^theory>\HOL.HOL\\ "(\(P \ Q)) = (\P \ \Q)" "(\(P \ Q)) = (\P \ \Q)" "(P \ Q) = (\P \ Q)" "(P = Q) = ((P \ Q) \ (\P \ \ Q))" "(\ \(P)) = P"