src/HOL/Hyperreal/HLog.ML
changeset 14370 b0064703967b
parent 14334 6137d24eef79
child 14371 c78c7da09519
equal deleted inserted replaced
14369:c50188fe6366 14370:b0064703967b
   112 by (blast_tac (claset() addIs [powhr_less_cancel,powhr_less_mono]) 1);
   112 by (blast_tac (claset() addIs [powhr_less_cancel,powhr_less_mono]) 1);
   113 qed "powhr_less_cancel_iff";
   113 qed "powhr_less_cancel_iff";
   114 Addsimps [powhr_less_cancel_iff];
   114 Addsimps [powhr_less_cancel_iff];
   115 
   115 
   116 Goal "1 < x ==> (x powhr a <= x powhr b) = (a <= b)";
   116 Goal "1 < x ==> (x powhr a <= x powhr b) = (a <= b)";
   117 by (auto_tac (claset(),simpset() addsimps [hypreal_le_def]));
   117 by (auto_tac (claset(),simpset() addsimps [linorder_not_less RS sym]));
   118 qed "powhr_le_cancel_iff";
   118 qed "powhr_le_cancel_iff";
   119 Addsimps [powhr_le_cancel_iff];
   119 Addsimps [powhr_le_cancel_iff];
   120 
   120 
   121 Goalw [hlog_def]
   121 Goalw [hlog_def]
   122      "hlog (Abs_hypreal(hyprel `` {X})) (Abs_hypreal(hyprel `` {Y})) = \
   122      "hlog (Abs_hypreal(hyprel `` {X})) (Abs_hypreal(hyprel `` {Y})) = \
   244 by (ALLGOALS(Ultra_tac));
   244 by (ALLGOALS(Ultra_tac));
   245 qed "hlog_less_cancel_iff";
   245 qed "hlog_less_cancel_iff";
   246 Addsimps [hlog_less_cancel_iff];
   246 Addsimps [hlog_less_cancel_iff];
   247 
   247 
   248 Goal "[| 1 < a; 0 < x; 0 < y |] ==> (hlog a x <= hlog a y) = (x <= y)";
   248 Goal "[| 1 < a; 0 < x; 0 < y |] ==> (hlog a x <= hlog a y) = (x <= y)";
   249 by (auto_tac (claset(),simpset() addsimps [hypreal_le_def]));
   249 by (auto_tac (claset(),simpset() addsimps [linorder_not_less RS sym]));
   250 qed "hlog_le_cancel_iff";
   250 qed "hlog_le_cancel_iff";
   251 Addsimps [hlog_le_cancel_iff];
   251 Addsimps [hlog_le_cancel_iff];
   252 
   252 
   253 (* should be in NSA.ML *)
   253 (* should be in NSA.ML *)
   254 goalw HLog.thy [epsilon_def] "0 <= epsilon";
   254 goalw HLog.thy [epsilon_def] "0 <= epsilon";