src/HOL/SMT_Examples/SMT_Tests.thy
changeset 57168 af95a414136a
parent 57165 7b1bf424ec5f
child 57214 c4986877deea
--- a/src/HOL/SMT_Examples/SMT_Tests.thy	Tue Jun 03 14:38:41 2014 +0200
+++ b/src/HOL/SMT_Examples/SMT_Tests.thy	Tue Jun 03 16:02:41 2014 +0200
@@ -174,13 +174,11 @@
 
 lemma
   "a \<noteq> b \<and> a \<noteq> c \<and> b \<noteq> c \<and> (\<forall>x y. f x = f y \<longrightarrow> y = x) \<longrightarrow> f a \<noteq> f b"
-  using [[smt2_oracle=true]] (* FIXME: disable refine_inj_axiom in Z3 *)
   by smt2
 
 lemma
   "(\<forall>x y z. f x y = f x z \<longrightarrow> y = z) \<and> b \<noteq> c \<longrightarrow> f a b \<noteq> f a c"
   "(\<forall>x y z. f x y = f z y \<longrightarrow> x = z) \<and> a \<noteq> d \<longrightarrow> f a b \<noteq> f d b"
-  using [[smt2_oracle=true]] (* FIXME: disable refine_inj_axiom in Z3 *)
   by smt2+