src/HOL/ex/unsolved.ML
changeset 1465 5d7a7e439cec
parent 969 b051e2fc2e34
child 1586 d91296e4deb3
equal deleted inserted replaced
1464:a608f83e3421 1465:5d7a7e439cec
     1 (*  Title: 	HOL/ex/unsolved
     1 (*  Title:      HOL/ex/unsolved
     2     ID:         $Id$
     2     ID:         $Id$
     3     Author: 	Lawrence C Paulson, Cambridge University Computer Laboratory
     3     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     4     Copyright   1992  University of Cambridge
     4     Copyright   1992  University of Cambridge
     5 
     5 
     6 Problems that currently defeat the MESON procedure as well as best_tac
     6 Problems that currently defeat the MESON procedure as well as best_tac
     7 *)
     7 *)
     8 
     8 
    12 \                                       (Q(x',y) | ~Q(y,z') | S(x',x'))";
    12 \                                       (Q(x',y) | ~Q(y,z') | S(x',x'))";
    13 
    13 
    14 
    14 
    15 writeln"Problem 47  Schubert's Steamroller";
    15 writeln"Problem 47  Schubert's Steamroller";
    16 goal HOL.thy
    16 goal HOL.thy
    17     "(! x. P1(x) --> P0(x)) & (? x.P1(x)) &	\
    17     "(! x. P1(x) --> P0(x)) & (? x.P1(x)) &     \
    18 \    (! x. P2(x) --> P0(x)) & (? x.P2(x)) &	\
    18 \    (! x. P2(x) --> P0(x)) & (? x.P2(x)) &     \
    19 \    (! x. P3(x) --> P0(x)) & (? x.P3(x)) &	\
    19 \    (! x. P3(x) --> P0(x)) & (? x.P3(x)) &     \
    20 \    (! x. P4(x) --> P0(x)) & (? x.P4(x)) &	\
    20 \    (! x. P4(x) --> P0(x)) & (? x.P4(x)) &     \
    21 \    (! x. P5(x) --> P0(x)) & (? x.P5(x)) &	\
    21 \    (! x. P5(x) --> P0(x)) & (? x.P5(x)) &     \
    22 \    (! x. Q1(x) --> Q0(x)) & (? x.Q1(x)) &	\
    22 \    (! x. Q1(x) --> Q0(x)) & (? x.Q1(x)) &     \
    23 \    (! x. P0(x) --> ((! y.Q0(y)-->R(x,y)) | 	\
    23 \    (! x. P0(x) --> ((! y.Q0(y)-->R(x,y)) |    \
    24 \		      (! y.P0(y) & S(y,x) & 	\
    24 \                     (! y.P0(y) & S(y,x) &     \
    25 \		           (? z.Q0(z)&R(y,z)) --> R(x,y)))) &	\
    25 \                          (? z.Q0(z)&R(y,z)) --> R(x,y)))) &   \
    26 \    (! x y. P3(y) & (P5(x)|P4(x)) --> S(x,y)) &	\
    26 \    (! x y. P3(y) & (P5(x)|P4(x)) --> S(x,y)) &        \
    27 \    (! x y. P3(x) & P2(y) --> S(x,y)) &	\
    27 \    (! x y. P3(x) & P2(y) --> S(x,y)) &        \
    28 \    (! x y. P2(x) & P1(y) --> S(x,y)) &	\
    28 \    (! x y. P2(x) & P1(y) --> S(x,y)) &        \
    29 \    (! x y. P1(x) & (P2(y)|Q1(y)) --> ~R(x,y)) &	\
    29 \    (! x y. P1(x) & (P2(y)|Q1(y)) --> ~R(x,y)) &       \
    30 \    (! x y. P3(x) & P4(y) --> R(x,y)) &	\
    30 \    (! x y. P3(x) & P4(y) --> R(x,y)) &        \
    31 \    (! x y. P3(x) & P5(y) --> ~R(x,y)) &	\
    31 \    (! x y. P3(x) & P5(y) --> ~R(x,y)) &       \
    32 \    (! x. (P4(x)|P5(x)) --> (? y.Q0(y) & R(x,y)))	\
    32 \    (! x. (P4(x)|P5(x)) --> (? y.Q0(y) & R(x,y)))      \
    33 \    --> (? x y. P0(x) & P0(y) & (? z. Q1(z) & R(y,z) & R(x,y)))";
    33 \    --> (? x y. P0(x) & P0(y) & (? z. Q1(z) & R(y,z) & R(x,y)))";
    34 
    34 
    35 
    35 
    36 writeln"Problem 55";
    36 writeln"Problem 55";
    37 
    37