author | nipkow |
Fri, 27 Nov 1998 16:54:59 +0100 | |
changeset 5982 | aeb97860d352 |
parent 5147 | 825877190618 |
child 6141 | a6922171b396 |
permissions | -rw-r--r-- |
1461 | 1 |
(* Title: ZF/ex/CoUnit.ML |
365 | 2 |
ID: $Id$ |
1461 | 3 |
Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
515 | 4 |
Copyright 1994 University of Cambridge |
365 | 5 |
|
6 |
Trivial codatatype definitions, one of which goes wrong! |
|
7 |
||
515 | 8 |
See discussion in |
9 |
L C Paulson. A Concrete Final Coalgebra Theorem for ZF Set Theory. |
|
10 |
Report 334, Cambridge University Computer Laboratory. 1994. |
|
365 | 11 |
*) |
12 |
||
515 | 13 |
open CoUnit; |
365 | 14 |
|
15 |
(*USELESS because folding on Con(?xa) == ?xa fails*) |
|
515 | 16 |
val ConE = counit.mk_cases counit.con_defs "Con(x) : counit"; |
365 | 17 |
|
18 |
(*Proving freeness results*) |
|
515 | 19 |
val Con_iff = counit.mk_free "Con(x)=Con(y) <-> x=y"; |
365 | 20 |
|
21 |
(*Should be a singleton, not everything!*) |
|
5068 | 22 |
Goal "counit = quniv(0)"; |
515 | 23 |
by (rtac (counit.dom_subset RS equalityI) 1); |
365 | 24 |
by (rtac subsetI 1); |
515 | 25 |
by (etac counit.coinduct 1); |
365 | 26 |
by (rtac subset_refl 1); |
515 | 27 |
by (rewrite_goals_tac counit.con_defs); |
2469 | 28 |
by (Fast_tac 1); |
782
200a16083201
added bind_thm for theorems defined by "standard ..."
clasohm
parents:
760
diff
changeset
|
29 |
qed "counit_eq_univ"; |
365 | 30 |
|
31 |
||
32 |
(*A similar example, but the constructor is non-degenerate and it works! |
|
33 |
The resulting set is a singleton. |
|
34 |
*) |
|
35 |
||
515 | 36 |
val Con2E = counit2.mk_cases counit2.con_defs "Con2(x,y) : counit2"; |
365 | 37 |
|
38 |
(*Proving freeness results*) |
|
515 | 39 |
val Con2_iff = counit2.mk_free "Con2(x,y)=Con2(x',y') <-> x=x' & y=y'"; |
365 | 40 |
|
5068 | 41 |
Goalw counit2.con_defs "bnd_mono(univ(0), %x. Con2(x,x))"; |
365 | 42 |
by (rtac bnd_monoI 1); |
43 |
by (REPEAT (ares_tac [subset_refl, QPair_subset_univ, QPair_mono] 1)); |
|
782
200a16083201
added bind_thm for theorems defined by "standard ..."
clasohm
parents:
760
diff
changeset
|
44 |
qed "Con2_bnd_mono"; |
365 | 45 |
|
5068 | 46 |
Goal "lfp(univ(0), %x. Con2(x,x)) : counit2"; |
515 | 47 |
by (rtac (singletonI RS counit2.coinduct) 1); |
365 | 48 |
by (rtac (qunivI RS singleton_subsetI) 1); |
49 |
by (rtac ([lfp_subset, empty_subsetI RS univ_mono] MRS subset_trans) 1); |
|
4091 | 50 |
by (fast_tac (claset() addSIs [Con2_bnd_mono RS lfp_Tarski]) 1); |
760 | 51 |
qed "lfp_Con2_in_counit2"; |
365 | 52 |
|
53 |
(*Lemma for proving finality. Borrowed from ex/llist_eq.ML!*) |
|
5147
825877190618
More tidying and removal of "\!\!... from Goal commands
paulson
parents:
5137
diff
changeset
|
54 |
Goal "Ord(i) ==> ALL x y. x: counit2 & y: counit2 --> x Int Vset(i) <= y"; |
365 | 55 |
by (etac trans_induct 1); |
56 |
by (safe_tac subset_cs); |
|
515 | 57 |
by (etac counit2.elim 1); |
58 |
by (etac counit2.elim 1); |
|
59 |
by (rewrite_goals_tac counit2.con_defs); |
|
2469 | 60 |
by (fast_tac (subset_cs |
61 |
addSIs [QPair_Int_Vset_subset_UN RS subset_trans, QPair_mono] |
|
62 |
addSEs [Ord_in_Ord, Pair_inject]) 1); |
|
782
200a16083201
added bind_thm for theorems defined by "standard ..."
clasohm
parents:
760
diff
changeset
|
63 |
qed "counit2_Int_Vset_subset_lemma"; |
365 | 64 |
|
65 |
val counit2_Int_Vset_subset = standard |
|
1461 | 66 |
(counit2_Int_Vset_subset_lemma RS spec RS spec RS mp); |
365 | 67 |
|
5137 | 68 |
Goal "[| x: counit2; y: counit2 |] ==> x=y"; |
365 | 69 |
by (rtac equalityI 1); |
70 |
by (REPEAT (ares_tac [conjI, counit2_Int_Vset_subset RS Int_Vset_subset] 1)); |
|
782
200a16083201
added bind_thm for theorems defined by "standard ..."
clasohm
parents:
760
diff
changeset
|
71 |
qed "counit2_implies_equal"; |
365 | 72 |
|
5068 | 73 |
Goal "counit2 = {lfp(univ(0), %x. Con2(x,x))}"; |
365 | 74 |
by (rtac equalityI 1); |
75 |
by (rtac (lfp_Con2_in_counit2 RS singleton_subsetI) 2); |
|
76 |
by (rtac subsetI 1); |
|
77 |
by (dtac (lfp_Con2_in_counit2 RS counit2_implies_equal) 1); |
|
78 |
by (etac subst 1); |
|
79 |
by (rtac singletonI 1); |
|
782
200a16083201
added bind_thm for theorems defined by "standard ..."
clasohm
parents:
760
diff
changeset
|
80 |
qed "counit2_eq_univ"; |