src/HOL/Rat.thy
changeset 55143 04448228381d
parent 54863 82acc20ded73
child 55974 c835a9379026
--- a/src/HOL/Rat.thy	Sat Jan 25 21:52:04 2014 +0100
+++ b/src/HOL/Rat.thy	Sat Jan 25 22:06:07 2014 +0100
@@ -622,8 +622,8 @@
     (* not needed because x < (y::int) can be rewritten as x + 1 <= y: of_int_less_iff RS iffD2 *)
   #> Lin_Arith.add_simps [@{thm neg_less_iff_less},
       @{thm True_implies_equals},
-      read_instantiate @{context} [(("a", 0), "(numeral ?v)")] @{thm distrib_left},
-      read_instantiate @{context} [(("a", 0), "(- numeral ?v)")] @{thm distrib_left},
+      @{thm distrib_left [where a = "numeral v" for v]},
+      @{thm distrib_left [where a = "- numeral v" for v]},
       @{thm divide_1}, @{thm divide_zero_left},
       @{thm times_divide_eq_right}, @{thm times_divide_eq_left},
       @{thm minus_divide_left} RS sym, @{thm minus_divide_right} RS sym,