src/HOL/Hyperreal/Lim.ML
changeset 14294 f4d806fd72ce
parent 14293 22542982bffd
child 14299 0b5c0b0a3eba
equal deleted inserted replaced
14293:22542982bffd 14294:f4d806fd72ce
   130 by (REPEAT(dres_inst_tac [("x","xa")] spec 2) 
   130 by (REPEAT(dres_inst_tac [("x","xa")] spec 2) 
   131     THEN step_tac (claset() addSEs [order_less_trans]) 2);
   131     THEN step_tac (claset() addSEs [order_less_trans]) 2);
   132 by (REPEAT(dres_inst_tac [("x","xa")] spec 3) 
   132 by (REPEAT(dres_inst_tac [("x","xa")] spec 3) 
   133     THEN step_tac (claset() addSEs [order_less_trans]) 3);
   133     THEN step_tac (claset() addSEs [order_less_trans]) 3);
   134 by (ALLGOALS(res_inst_tac [("t","r")] (real_mult_1 RS subst)));
   134 by (ALLGOALS(res_inst_tac [("t","r")] (real_mult_1 RS subst)));
   135 by (ALLGOALS(rtac abs_mult_less2));
   135 by (ALLGOALS(rtac abs_mult_less));
   136 by Auto_tac;
   136 by Auto_tac;
   137 qed "LIM_mult_zero";
   137 qed "LIM_mult_zero";
   138 
   138 
   139 Goalw [LIM_def] "(%x. x) -- a --> a";
   139 Goalw [LIM_def] "(%x. x) -- a --> a";
   140 by Auto_tac;
   140 by Auto_tac;
  1663 by (dres_inst_tac [("x","s")] spec 1);
  1663 by (dres_inst_tac [("x","s")] spec 1);
  1664 by (Clarify_tac 1);
  1664 by (Clarify_tac 1);
  1665 by (cut_inst_tac [("x","f x"),("y","y")] linorder_less_linear 1);
  1665 by (cut_inst_tac [("x","f x"),("y","y")] linorder_less_linear 1);
  1666 by Safe_tac;
  1666 by Safe_tac;
  1667 by (dres_inst_tac [("x","ba - x")] spec 1);
  1667 by (dres_inst_tac [("x","ba - x")] spec 1);
  1668 by (ALLGOALS (asm_full_simp_tac (simpset() addsimps [abs_iff])));
  1668 by (ALLGOALS (asm_full_simp_tac (simpset() addsimps [thm"abs_if"])));
  1669 by (dres_inst_tac [("x","aa - x")] spec 1);
  1669 by (dres_inst_tac [("x","aa - x")] spec 1);
  1670 by (case_tac "x \\<le> aa" 1);
  1670 by (case_tac "x \\<le> aa" 1);
  1671 by (ALLGOALS Asm_full_simp_tac);
  1671 by (ALLGOALS Asm_full_simp_tac);
  1672 by (dres_inst_tac [("z","x"),("w","aa")] real_le_anti_sym 1);
  1672 by (dres_inst_tac [("z","x"),("w","aa")] real_le_anti_sym 1);
  1673 by (assume_tac 1 THEN Asm_full_simp_tac 1);
  1673 by (assume_tac 1 THEN Asm_full_simp_tac 1);