added some ~= rules;
authorwenzelm
Tue, 21 Sep 1999 17:28:33 +0200
changeset 7561 ff8dbd0589aa
parent 7560 19c3be2d285c
child 7562 8519d5019309
added some ~= rules;
src/HOL/Calculation.thy
--- a/src/HOL/Calculation.thy	Tue Sep 21 17:28:02 1999 +0200
+++ b/src/HOL/Calculation.thy	Tue Sep 21 17:28:33 1999 +0200
@@ -17,6 +17,12 @@
 
 theorems [trans] = dvd_trans;                               (* dvd dvd dvd *)
 
+theorem [trans]: "[| x ~= y; (x::'a::order) <= y |] ==> x < y";     (*  ~=  <=  < *)
+  by (simp! add: order_less_le);
+
+theorem [trans]: "[| (x::'a::order) <= y; x ~= y |] ==> x < y";     (*  <=  ~=  < *)
+  by (simp! add: order_less_le);
+
 theorem [trans]: "[| (x::'a::order) < y; y < x |] ==> P";   (*  <  >  P  *)
   by (rule order_less_asym);