diff -r 304a47739407 -r 04ce6bb14d85 src/HOL/MetisExamples/Message.thy --- a/src/HOL/MetisExamples/Message.thy Thu Sep 24 19:14:18 2009 +0200 +++ b/src/HOL/MetisExamples/Message.thy Fri Sep 25 09:50:31 2009 +0200 @@ -1,5 +1,4 @@ (* Title: HOL/MetisTest/Message.thy - ID: $Id$ Author: Lawrence C Paulson, Cambridge University Computer Laboratory Testing the metis method @@ -711,17 +710,17 @@ proof (neg_clausify) assume 0: "analz (synth H) \ analz H \ synth H" have 1: "\X1 X3. sup (analz (sup X3 X1)) (synth X3) = analz (sup (synth X3) X1)" - by (metis analz_synth_Un sup_set_eq sup_set_eq sup_set_eq) + by (metis analz_synth_Un) have 2: "sup (analz H) (synth H) \ analz (synth H)" - by (metis 0 sup_set_eq) + by (metis 0) have 3: "\X1 X3. sup (synth X3) (analz (sup X3 X1)) = analz (sup (synth X3) X1)" - by (metis 1 Un_commute sup_set_eq sup_set_eq) + by (metis 1 Un_commute) have 4: "\X3. sup (synth X3) (analz X3) = analz (sup (synth X3) {})" - by (metis 3 Un_empty_right sup_set_eq) + by (metis 3 Un_empty_right) have 5: "\X3. sup (synth X3) (analz X3) = analz (synth X3)" - by (metis 4 Un_empty_right sup_set_eq) + by (metis 4 Un_empty_right) have 6: "\X3. sup (analz X3) (synth X3) = analz (synth X3)" - by (metis 5 Un_commute sup_set_eq sup_set_eq) + by (metis 5 Un_commute) show "False" by (metis 2 6) qed