Quot/QuotMain.thy
changeset 873 f14e41e9b08f
parent 870 2a19e0a37131
child 896 4e0b89d886ac
--- a/Quot/QuotMain.thy	Thu Jan 14 12:14:35 2010 +0100
+++ b/Quot/QuotMain.thy	Thu Jan 14 12:17:39 2010 +0100
@@ -95,6 +95,7 @@
 section {* ML setup *}
 
 (* Auxiliary data for the quotient package *)
+
 use "quotient_info.ML"
 
 declare [[map "fun" = (fun_map, fun_rel)]]
@@ -147,30 +148,6 @@
 use "quotient_tacs.ML"
 
 
-(* Atomize infrastructure *)
-(* FIXME/TODO: is this really needed? *)
-(*
-lemma atomize_eqv[atomize]:
-  shows "(Trueprop A \<equiv> Trueprop B) \<equiv> (A \<equiv> B)"
-proof
-  assume "A \<equiv> B"
-  then show "Trueprop A \<equiv> Trueprop B" by unfold
-next
-  assume *: "Trueprop A \<equiv> Trueprop B"
-  have "A = B"
-  proof (cases A)
-    case True
-    have "A" by fact
-    then show "A = B" using * by simp
-  next
-    case False
-    have "\<not>A" by fact
-    then show "A = B" using * by auto
-  qed
-  then show "A \<equiv> B" by (rule eq_reflection)
-qed
-*)
-
 section {* Methods / Interface *}
 
 ML {*