# HG changeset patch # User wenzelm # Date 1428357253 -7200 # Node ID 6a3098313acf480486a4a1a162cb759e7a7ef085 # Parent bafba7916d5e82add61fda6721dc10ad22d77a44 tuned; diff -r bafba7916d5e -r 6a3098313acf src/FOL/FOL.thy --- a/src/FOL/FOL.thy Mon Apr 06 23:24:45 2015 +0200 +++ b/src/FOL/FOL.thy Mon Apr 06 23:54:13 2015 +0200 @@ -387,21 +387,21 @@ context begin -restricted definition "induct_forall(P) == \x. P(x)" -restricted definition "induct_implies(A, B) == A \ B" -restricted definition "induct_equal(x, y) == x = y" -restricted definition "induct_conj(A, B) == A \ B" +restricted definition "induct_forall(P) \ \x. P(x)" +restricted definition "induct_implies(A, B) \ A \ B" +restricted definition "induct_equal(x, y) \ x = y" +restricted definition "induct_conj(A, B) \ A \ B" -lemma induct_forall_eq: "(!!x. P(x)) == Trueprop(induct_forall(\x. P(x)))" +lemma induct_forall_eq: "(\x. P(x)) \ Trueprop(induct_forall(\x. P(x)))" unfolding atomize_all induct_forall_def . -lemma induct_implies_eq: "(A ==> B) == Trueprop(induct_implies(A, B))" +lemma induct_implies_eq: "(A \ B) \ Trueprop(induct_implies(A, B))" unfolding atomize_imp induct_implies_def . -lemma induct_equal_eq: "(x == y) == Trueprop(induct_equal(x, y))" +lemma induct_equal_eq: "(x \ y) \ Trueprop(induct_equal(x, y))" unfolding atomize_eq induct_equal_def . -lemma induct_conj_eq: "(A &&& B) == Trueprop(induct_conj(A, B))" +lemma induct_conj_eq: "(A &&& B) \ Trueprop(induct_conj(A, B))" unfolding atomize_conj induct_conj_def . lemmas induct_atomize = induct_forall_eq induct_implies_eq induct_equal_eq induct_conj_eq