src/FOLP/ex/Intuitionistic.thy
changeset 62020 5d208fd2507d
parent 61337 4645502c3c64
child 67443 3abf6a722518
equal deleted inserted replaced
62019:9de1eb745aeb 62020:5d208fd2507d
   136 schematic_goal "?p : ~~((P-->Q) | (Q-->P))"
   136 schematic_goal "?p : ~~((P-->Q) | (Q-->P))"
   137   by (tactic \<open>IntPr.fast_tac @{context} 1\<close>)
   137   by (tactic \<open>IntPr.fast_tac @{context} 1\<close>)
   138 
   138 
   139 text "Problem ~~17"
   139 text "Problem ~~17"
   140 schematic_goal "?p : ~~(((P & (Q-->R))-->S) <-> ((~P | Q | S) & (~P | ~R | S)))"
   140 schematic_goal "?p : ~~(((P & (Q-->R))-->S) <-> ((~P | Q | S) & (~P | ~R | S)))"
   141   by (tactic \<open>IntPr.fast_tac @{context} 1\<close>)  -- slow
   141   by (tactic \<open>IntPr.fast_tac @{context} 1\<close>)  \<comment> slow
   142 
   142 
   143 
   143 
   144 subsection \<open>Examples with quantifiers\<close>
   144 subsection \<open>Examples with quantifiers\<close>
   145 
   145 
   146 text "The converse is classical in the following implications..."
   146 text "The converse is classical in the following implications..."
   259 text "Problem 32"
   259 text "Problem 32"
   260 schematic_goal "?p : (ALL x. P(x) & (Q(x)|R(x))-->S(x)) &  
   260 schematic_goal "?p : (ALL x. P(x) & (Q(x)|R(x))-->S(x)) &  
   261         (ALL x. S(x) & R(x) --> L(x)) &  
   261         (ALL x. S(x) & R(x) --> L(x)) &  
   262         (ALL x. M(x) --> R(x))   
   262         (ALL x. M(x) --> R(x))   
   263     --> (ALL x. P(x) & M(x) --> L(x))"
   263     --> (ALL x. P(x) & M(x) --> L(x))"
   264   by (tactic "IntPr.best_tac @{context} 1") -- slow
   264   by (tactic "IntPr.best_tac @{context} 1") \<comment> slow
   265 
   265 
   266 text "Problem 39"
   266 text "Problem 39"
   267 schematic_goal "?p : ~ (EX x. ALL y. F(y,x) <-> ~F(y,y))"
   267 schematic_goal "?p : ~ (EX x. ALL y. F(y,x) <-> ~F(y,y))"
   268   by (tactic "IntPr.best_tac @{context} 1")
   268   by (tactic "IntPr.best_tac @{context} 1")
   269 
   269 
   270 text "Problem 40.  AMENDED"
   270 text "Problem 40.  AMENDED"
   271 schematic_goal "?p : (EX y. ALL x. F(x,y) <-> F(x,x)) -->   
   271 schematic_goal "?p : (EX y. ALL x. F(x,y) <-> F(x,x)) -->   
   272               ~(ALL x. EX y. ALL z. F(z,y) <-> ~ F(z,x))"
   272               ~(ALL x. EX y. ALL z. F(z,y) <-> ~ F(z,x))"
   273   by (tactic "IntPr.best_tac @{context} 1") -- slow
   273   by (tactic "IntPr.best_tac @{context} 1") \<comment> slow
   274 
   274 
   275 text "Problem 44"
   275 text "Problem 44"
   276 schematic_goal "?p : (ALL x. f(x) -->                                    
   276 schematic_goal "?p : (ALL x. f(x) -->                                    
   277               (EX y. g(y) & h(x,y) & (EX y. g(y) & ~ h(x,y))))  &        
   277               (EX y. g(y) & h(x,y) & (EX y. g(y) & ~ h(x,y))))  &        
   278               (EX x. j(x) & (ALL y. g(y) --> h(x,y)))                    
   278               (EX x. j(x) & (ALL y. g(y) --> h(x,y)))                    
   285 
   285 
   286 text "Problem 51"
   286 text "Problem 51"
   287 schematic_goal
   287 schematic_goal
   288     "?p : (EX z w. ALL x y. P(x,y) <->  (x=z & y=w)) -->   
   288     "?p : (EX z w. ALL x y. P(x,y) <->  (x=z & y=w)) -->   
   289      (EX z. ALL x. EX w. (ALL y. P(x,y) <-> y=w) <-> x=z)"
   289      (EX z. ALL x. EX w. (ALL y. P(x,y) <-> y=w) <-> x=z)"
   290   by (tactic "IntPr.best_tac @{context} 1") -- \<open>60 seconds\<close>
   290   by (tactic "IntPr.best_tac @{context} 1") \<comment> \<open>60 seconds\<close>
   291 
   291 
   292 text "Problem 56"
   292 text "Problem 56"
   293 schematic_goal "?p : (ALL x. (EX y. P(y) & x=f(y)) --> P(x)) <-> (ALL x. P(x) --> P(f(x)))"
   293 schematic_goal "?p : (ALL x. (EX y. P(y) & x=f(y)) --> P(x)) <-> (ALL x. P(x) --> P(f(x)))"
   294   by (tactic "IntPr.best_tac @{context} 1")
   294   by (tactic "IntPr.best_tac @{context} 1")
   295 
   295