changeset 31173 | bbe9e29b9672 |
parent 31172 | 74d72ba262fb |
parent 31166 | a90fe83f58ea |
child 31299 | 0c5baf034d0e |
--- a/src/HOL/HOL.thy Sat May 16 15:23:52 2009 +0200 +++ b/src/HOL/HOL.thy Sat May 16 15:24:35 2009 +0200 @@ -1050,8 +1050,7 @@ "(P | False) = P" "(False | P) = P" "(P | P) = P" "(P | (P | Q)) = (P | Q)" and "(ALL x. P) = P" "(EX x. P) = P" "EX x. x=t" "EX x. t=x" - -- {* needed for the one-point-rule quantifier simplification procs *} - -- {* essential for termination!! *} and + and "!!P. (EX x. x=t & P(x)) = P(t)" "!!P. (EX x. t=x & P(x)) = P(t)" "!!P. (ALL x. x=t --> P(x)) = P(t)"