src/HOL/Algebra/abstract/Ring.thy
changeset 17956 369e2af8ee45
parent 17877 67d5ab1cb0d8
child 20044 92cc2f4c7335
equal deleted inserted replaced
17955:3b34516662c6 17956:369e2af8ee45
   162         ["t + u::'a::ring",
   162         ["t + u::'a::ring",
   163 	 "t - u::'a::ring",
   163 	 "t - u::'a::ring",
   164 	 "t * u::'a::ring",
   164 	 "t * u::'a::ring",
   165 	 "- t::'a::ring"];
   165 	 "- t::'a::ring"];
   166     fun proc sg ss t = 
   166     fun proc sg ss t = 
   167       let val rew = Tactic.prove sg [] []
   167       let val rew = Goal.prove sg [] []
   168             (HOLogic.mk_Trueprop
   168             (HOLogic.mk_Trueprop
   169               (HOLogic.mk_eq (t, Var (("x", Term.maxidx_of_term t + 1), fastype_of t))))
   169               (HOLogic.mk_eq (t, Var (("x", Term.maxidx_of_term t + 1), fastype_of t))))
   170                 (fn _ => simp_tac (Simplifier.inherit_context ss ring_ss) 1)
   170                 (fn _ => simp_tac (Simplifier.inherit_context ss ring_ss) 1)
   171             |> mk_meta_eq;
   171             |> mk_meta_eq;
   172           val (t', u) = Logic.dest_equals (Thm.prop_of rew);
   172           val (t', u) = Logic.dest_equals (Thm.prop_of rew);