| author | wenzelm | 
| Mon, 29 Dec 2008 18:27:33 +0100 | |
| changeset 29200 | 787ba47201c7 | 
| parent 28856 | 5e009a80fe6d | 
| child 29606 | fedb8be05f24 | 
| permissions | -rw-r--r-- | 
| 15803 | 1 | (* Title: Pure/Pure.thy | 
| 2 | ID: $Id$ | |
| 18466 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 3 | *) | 
| 15803 | 4 | |
| 26435 | 5 | section {* Further content for the Pure theory *}
 | 
| 20627 | 6 | |
| 18466 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 7 | subsection {* Meta-level connectives in assumptions *}
 | 
| 15803 | 8 | |
| 9 | lemma meta_mp: | |
| 18019 | 10 | assumes "PROP P ==> PROP Q" and "PROP P" | 
| 15803 | 11 | shows "PROP Q" | 
| 18019 | 12 | by (rule `PROP P ==> PROP Q` [OF `PROP P`]) | 
| 15803 | 13 | |
| 23432 | 14 | lemmas meta_impE = meta_mp [elim_format] | 
| 15 | ||
| 15803 | 16 | lemma meta_spec: | 
| 26958 | 17 | assumes "!!x. PROP P x" | 
| 18 | shows "PROP P x" | |
| 19 | by (rule `!!x. PROP P x`) | |
| 15803 | 20 | |
| 21 | lemmas meta_allE = meta_spec [elim_format] | |
| 22 | ||
| 26570 | 23 | lemma swap_params: | 
| 26958 | 24 | "(!!x y. PROP P x y) == (!!y x. PROP P x y)" .. | 
| 26570 | 25 | |
| 18466 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 26 | |
| 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 27 | subsection {* Meta-level conjunction *}
 | 
| 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 28 | |
| 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 29 | lemma all_conjunction: | 
| 28856 
5e009a80fe6d
Pure syntax: more coherent treatment of aprop, permanent TERM and &&&;
 wenzelm parents: 
28699diff
changeset | 30 | "(!!x. PROP A x &&& PROP B x) == ((!!x. PROP A x) &&& (!!x. PROP B x))" | 
| 18466 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 31 | proof | 
| 28856 
5e009a80fe6d
Pure syntax: more coherent treatment of aprop, permanent TERM and &&&;
 wenzelm parents: 
28699diff
changeset | 32 | assume conj: "!!x. PROP A x &&& PROP B x" | 
| 
5e009a80fe6d
Pure syntax: more coherent treatment of aprop, permanent TERM and &&&;
 wenzelm parents: 
28699diff
changeset | 33 | show "(!!x. PROP A x) &&& (!!x. PROP B x)" | 
| 19121 | 34 | proof - | 
| 18466 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 35 | fix x | 
| 26958 | 36 | from conj show "PROP A x" by (rule conjunctionD1) | 
| 37 | from conj show "PROP B x" by (rule conjunctionD2) | |
| 18466 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 38 | qed | 
| 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 39 | next | 
| 28856 
5e009a80fe6d
Pure syntax: more coherent treatment of aprop, permanent TERM and &&&;
 wenzelm parents: 
28699diff
changeset | 40 | assume conj: "(!!x. PROP A x) &&& (!!x. PROP B x)" | 
| 18466 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 41 | fix x | 
| 28856 
5e009a80fe6d
Pure syntax: more coherent treatment of aprop, permanent TERM and &&&;
 wenzelm parents: 
28699diff
changeset | 42 | show "PROP A x &&& PROP B x" | 
| 19121 | 43 | proof - | 
| 26958 | 44 | show "PROP A x" by (rule conj [THEN conjunctionD1, rule_format]) | 
| 45 | show "PROP B x" by (rule conj [THEN conjunctionD2, rule_format]) | |
| 18466 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 46 | qed | 
| 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 47 | qed | 
| 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 48 | |
| 19121 | 49 | lemma imp_conjunction: | 
| 28856 
5e009a80fe6d
Pure syntax: more coherent treatment of aprop, permanent TERM and &&&;
 wenzelm parents: 
28699diff
changeset | 50 | "(PROP A ==> PROP B &&& PROP C) == (PROP A ==> PROP B) &&& (PROP A ==> PROP C)" | 
| 18836 | 51 | proof | 
| 28856 
5e009a80fe6d
Pure syntax: more coherent treatment of aprop, permanent TERM and &&&;
 wenzelm parents: 
28699diff
changeset | 52 | assume conj: "PROP A ==> PROP B &&& PROP C" | 
| 
5e009a80fe6d
Pure syntax: more coherent treatment of aprop, permanent TERM and &&&;
 wenzelm parents: 
28699diff
changeset | 53 | show "(PROP A ==> PROP B) &&& (PROP A ==> PROP C)" | 
| 19121 | 54 | proof - | 
| 18466 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 55 | assume "PROP A" | 
| 19121 | 56 | from conj [OF `PROP A`] show "PROP B" by (rule conjunctionD1) | 
| 57 | from conj [OF `PROP A`] show "PROP C" by (rule conjunctionD2) | |
| 18466 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 58 | qed | 
| 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 59 | next | 
| 28856 
5e009a80fe6d
Pure syntax: more coherent treatment of aprop, permanent TERM and &&&;
 wenzelm parents: 
28699diff
changeset | 60 | assume conj: "(PROP A ==> PROP B) &&& (PROP A ==> PROP C)" | 
| 18466 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 61 | assume "PROP A" | 
| 28856 
5e009a80fe6d
Pure syntax: more coherent treatment of aprop, permanent TERM and &&&;
 wenzelm parents: 
28699diff
changeset | 62 | show "PROP B &&& PROP C" | 
| 19121 | 63 | proof - | 
| 64 | from `PROP A` show "PROP B" by (rule conj [THEN conjunctionD1]) | |
| 65 | from `PROP A` show "PROP C" by (rule conj [THEN conjunctionD2]) | |
| 18466 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 66 | qed | 
| 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 67 | qed | 
| 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 68 | |
| 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 69 | lemma conjunction_imp: | 
| 28856 
5e009a80fe6d
Pure syntax: more coherent treatment of aprop, permanent TERM and &&&;
 wenzelm parents: 
28699diff
changeset | 70 | "(PROP A &&& PROP B ==> PROP C) == (PROP A ==> PROP B ==> PROP C)" | 
| 18466 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 71 | proof | 
| 28856 
5e009a80fe6d
Pure syntax: more coherent treatment of aprop, permanent TERM and &&&;
 wenzelm parents: 
28699diff
changeset | 72 | assume r: "PROP A &&& PROP B ==> PROP C" | 
| 22933 | 73 | assume ab: "PROP A" "PROP B" | 
| 74 | show "PROP C" | |
| 75 | proof (rule r) | |
| 28856 
5e009a80fe6d
Pure syntax: more coherent treatment of aprop, permanent TERM and &&&;
 wenzelm parents: 
28699diff
changeset | 76 | from ab show "PROP A &&& PROP B" . | 
| 22933 | 77 | qed | 
| 18466 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 78 | next | 
| 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 79 | assume r: "PROP A ==> PROP B ==> PROP C" | 
| 28856 
5e009a80fe6d
Pure syntax: more coherent treatment of aprop, permanent TERM and &&&;
 wenzelm parents: 
28699diff
changeset | 80 | assume conj: "PROP A &&& PROP B" | 
| 18466 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 81 | show "PROP C" | 
| 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 82 | proof (rule r) | 
| 19121 | 83 | from conj show "PROP A" by (rule conjunctionD1) | 
| 84 | from conj show "PROP B" by (rule conjunctionD2) | |
| 18466 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 85 | qed | 
| 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 86 | qed | 
| 
389a6f9c31f4
added locale meta_conjunction_syntax and various conjunction rules;
 wenzelm parents: 
18019diff
changeset | 87 |