added atomize_eq;
authorwenzelm
Fri, 10 Nov 2000 19:00:51 +0100
changeset 10430 d3f780c3af0c
parent 10429 8820f787e61e
child 10431 bb67f704d631
added atomize_eq;
src/FOL/FOL.thy
--- a/src/FOL/FOL.thy	Fri Nov 10 19:00:22 2000 +0100
+++ b/src/FOL/FOL.thy	Fri Nov 10 19:00:51 2000 +0100
@@ -25,7 +25,7 @@
 
 use "FOL_lemmas1.ML"
 
-lemma all_eq: "(!!x. P(x)) == Trueprop (ALL x. P(x))"
+lemma atomize_all: "(!!x. P(x)) == Trueprop (ALL x. P(x))"
 proof (rule equal_intr_rule)
   assume "!!x. P(x)"
   show "ALL x. P(x)" by (rule allI)
@@ -34,7 +34,7 @@
   thus "!!x. P(x)" by (rule allE)
 qed
 
-lemma imp_eq: "(A ==> B) == Trueprop (A --> B)"
+lemma atomize_imp: "(A ==> B) == Trueprop (A --> B)"
 proof (rule equal_intr_rule)
   assume r: "A ==> B"
   show "A --> B" by (rule impI) (rule r)
@@ -43,7 +43,17 @@
   thus B by (rule mp)
 qed
 
-lemmas atomize = all_eq imp_eq
+lemma atomize_eq: "(x == y) == Trueprop (x = y)"
+proof (rule equal_intr_rule)
+  assume "x == y"
+  show "x = y" by (unfold prems) (rule refl)
+next
+  assume "x = y"
+  thus "x == y" by (rule eq_reflection)
+qed
+
+lemmas atomize = atomize_all atomize_imp
+lemmas atomize' = atomize atomize_eq
 
 use "cladata.ML"
 setup Cla.setup