diff -r a80d8ec6c998 -r 3dda49e08b9d src/FOL/ex/Propositional_Int.thy --- a/src/FOL/ex/Propositional_Int.thy Fri Jan 04 21:49:06 2019 +0100 +++ b/src/FOL/ex/Propositional_Int.thy Fri Jan 04 23:22:53 2019 +0100 @@ -12,94 +12,94 @@ text \commutative laws of \\\ and \\\\ lemma \P \ Q \ Q \ P\ - by (tactic "IntPr.fast_tac @{context} 1") + by (tactic "IntPr.fast_tac \<^context> 1") lemma \P \ Q \ Q \ P\ - by (tactic "IntPr.fast_tac @{context} 1") + by (tactic "IntPr.fast_tac \<^context> 1") text \associative laws of \\\ and \\\\ lemma \(P \ Q) \ R \ P \ (Q \ R)\ - by (tactic "IntPr.fast_tac @{context} 1") + by (tactic "IntPr.fast_tac \<^context> 1") lemma \(P \ Q) \ R \ P \ (Q \ R)\ - by (tactic "IntPr.fast_tac @{context} 1") + by (tactic "IntPr.fast_tac \<^context> 1") text \distributive laws of \\\ and \\\\ lemma \(P \ Q) \ R \ (P \ R) \ (Q \ R)\ - by (tactic "IntPr.fast_tac @{context} 1") + by (tactic "IntPr.fast_tac \<^context> 1") lemma \(P \ R) \ (Q \ R) \ (P \ Q) \ R\ - by (tactic "IntPr.fast_tac @{context} 1") + by (tactic "IntPr.fast_tac \<^context> 1") lemma \(P \ Q) \ R \ (P \ R) \ (Q \ R)\ - by (tactic "IntPr.fast_tac @{context} 1") + by (tactic "IntPr.fast_tac \<^context> 1") lemma \(P \ R) \ (Q \ R) \ (P \ Q) \ R\ - by (tactic "IntPr.fast_tac @{context} 1") + by (tactic "IntPr.fast_tac \<^context> 1") text \Laws involving implication\ lemma \(P \ R) \ (Q \ R) \ (P \ Q \ R)\ - by (tactic "IntPr.fast_tac @{context} 1") + by (tactic "IntPr.fast_tac \<^context> 1") lemma \(P \ Q \ R) \ (P \ (Q \ R))\ - by (tactic "IntPr.fast_tac @{context} 1") + by (tactic "IntPr.fast_tac \<^context> 1") lemma \((P \ R) \ R) \ ((Q \ R) \ R) \ (P \ Q \ R) \ R\ - by (tactic "IntPr.fast_tac @{context} 1") + by (tactic "IntPr.fast_tac \<^context> 1") lemma \\ (P \ R) \ \ (Q \ R) \ \ (P \ Q \ R)\ - by (tactic "IntPr.fast_tac @{context} 1") + by (tactic "IntPr.fast_tac \<^context> 1") lemma \(P \ Q \ R) \ (P \ Q) \ (P \ R)\ - by (tactic "IntPr.fast_tac @{context} 1") + by (tactic "IntPr.fast_tac \<^context> 1") text \Propositions-as-types\ \ \The combinator K\ lemma \P \ (Q \ P)\ - by (tactic "IntPr.fast_tac @{context} 1") + by (tactic "IntPr.fast_tac \<^context> 1") \ \The combinator S\ lemma \(P \ Q \ R) \ (P \ Q) \ (P \ R)\ - by (tactic "IntPr.fast_tac @{context} 1") + by (tactic "IntPr.fast_tac \<^context> 1") \ \Converse is classical\ lemma \(P \ Q) \ (P \ R) \ (P \ Q \ R)\ - by (tactic "IntPr.fast_tac @{context} 1") + by (tactic "IntPr.fast_tac \<^context> 1") lemma \(P \ Q) \ (\ Q \ \ P)\ - by (tactic "IntPr.fast_tac @{context} 1") + by (tactic "IntPr.fast_tac \<^context> 1") text \Schwichtenberg's examples (via T. Nipkow)\ lemma stab_imp: \(((Q \ R) \ R) \ Q) \ (((P \ Q) \ R) \ R) \ P \ Q\ - by (tactic "IntPr.fast_tac @{context} 1") + by (tactic "IntPr.fast_tac \<^context> 1") lemma stab_to_peirce: \(((P \ R) \ R) \ P) \ (((Q \ R) \ R) \ Q) \ ((P \ Q) \ P) \ P\ - by (tactic "IntPr.fast_tac @{context} 1") + by (tactic "IntPr.fast_tac \<^context> 1") lemma peirce_imp1: \(((Q \ R) \ Q) \ Q) \ (((P \ Q) \ R) \ P \ Q) \ P \ Q\ - by (tactic "IntPr.fast_tac @{context} 1") + by (tactic "IntPr.fast_tac \<^context> 1") lemma peirce_imp2: \(((P \ R) \ P) \ P) \ ((P \ Q \ R) \ P) \ P\ - by (tactic "IntPr.fast_tac @{context} 1") + by (tactic "IntPr.fast_tac \<^context> 1") lemma mints: \((((P \ Q) \ P) \ P) \ Q) \ Q\ - by (tactic "IntPr.fast_tac @{context} 1") + by (tactic "IntPr.fast_tac \<^context> 1") lemma mints_solovev: \(P \ (Q \ R) \ Q) \ ((P \ Q) \ R) \ R\ - by (tactic "IntPr.fast_tac @{context} 1") + by (tactic "IntPr.fast_tac \<^context> 1") lemma tatsuta: \(((P7 \ P1) \ P10) \ P4 \ P5) @@ -107,7 +107,7 @@ \ (P1 \ P8) \ P6 \ P7 \ (((P3 \ P2) \ P9) \ P4) \ (P1 \ P3) \ (((P6 \ P1) \ P2) \ P9) \ P5\ - by (tactic "IntPr.fast_tac @{context} 1") + by (tactic "IntPr.fast_tac \<^context> 1") lemma tatsuta1: \(((P8 \ P2) \ P9) \ P3 \ P10) @@ -115,6 +115,6 @@ \ (((P6 \ P1) \ P2) \ P9) \ (((P7 \ P1) \ P10) \ P4 \ P5) \ (P1 \ P3) \ (P1 \ P8) \ P6 \ P7 \ P5\ - by (tactic "IntPr.fast_tac @{context} 1") + by (tactic "IntPr.fast_tac \<^context> 1") end