updated Isabelle and deleted mono rules
authorChristian Urban <urbanc@in.tum.de>
Sun, 06 Dec 2009 11:39:34 +0100
changeset 578 070161f1996a
parent 577 8dab8d82f26b
child 581 2da4fb1894d2
child 582 a082e2d138ab
updated Isabelle and deleted mono rules
IntEx2.thy
QuotMain.thy
--- a/IntEx2.thy	Sun Dec 06 11:21:29 2009 +0100
+++ b/IntEx2.thy	Sun Dec 06 11:39:34 2009 +0100
@@ -6,6 +6,7 @@
   ("Tools/int_arith.ML")
 begin
 
+
 fun
   intrel :: "(nat \<times> nat) \<Rightarrow> (nat \<times> nat) \<Rightarrow> bool" (infix "\<approx>" 50)
 where
--- a/QuotMain.thy	Sun Dec 06 11:21:29 2009 +0100
+++ b/QuotMain.thy	Sun Dec 06 11:39:34 2009 +0100
@@ -494,14 +494,6 @@
 
 *)
 
-(* FIXME: they should be in in the new Isabelle *)
-lemma [mono]: 
-  "(\<And>x. P x \<longrightarrow> Q x) \<Longrightarrow> (Ex P) \<longrightarrow> (Ex Q)"
-by blast
-
-lemma [mono]: "P \<longrightarrow> Q \<Longrightarrow> \<not>Q \<longrightarrow> \<not>P"
-by auto
-
 (* FIXME: OPTION_equivp, PAIR_equivp, ... *)
 ML {*
 fun equiv_tac rel_eqvs =
@@ -511,6 +503,8 @@
      rtac @{thm list_equivp}])
 *}
 
+thm ball_reg_eqv
+
 ML {*
 fun ball_reg_eqv_simproc rel_eqvs ss redex =
   let
@@ -610,6 +604,9 @@
   end
 *}
 
+thm ball_reg_eqv_range
+thm bex_reg_eqv_range
+
 ML {*
 fun bex_reg_eqv_range_simproc rel_eqvs ss redex =
   let