author | paulson |
Wed, 28 Jun 2000 10:54:21 +0200 | |
changeset 9169 | 85a47aa21f74 |
parent 5068 | fb28eaa07e01 |
child 9245 | 428385c4bc50 |
permissions | -rw-r--r-- |
2644 | 1 |
(* Title: HOLCF/Porder0.ML |
2 |
ID: $Id$ |
|
3 |
Author: Oscar Slotosch |
|
4 |
Copyright 1997 Technische Universitaet Muenchen |
|
5 |
||
6 |
derive the characteristic axioms for the characteristic constants *) |
|
7 |
||
8 |
open Porder0; |
|
9 |
||
2841
c2508f4ab739
Added "discrete" CPOs and modified IMP to use those rather than "lift"
nipkow
parents:
2644
diff
changeset
|
10 |
AddIffs [refl_less]; |
c2508f4ab739
Added "discrete" CPOs and modified IMP to use those rather than "lift"
nipkow
parents:
2644
diff
changeset
|
11 |
|
2644 | 12 |
(* ------------------------------------------------------------------------ *) |
13 |
(* minimal fixes least element *) |
|
14 |
(* ------------------------------------------------------------------------ *) |
|
3842 | 15 |
bind_thm("minimal2UU",allI RS (prove_goal thy "!x::'a::po. uu<<x==>uu=(@u.!y. u<<y)" |
2644 | 16 |
(fn prems => |
17 |
[ |
|
18 |
(cut_facts_tac prems 1), |
|
19 |
(rtac antisym_less 1), |
|
20 |
(etac spec 1), |
|
21 |
(res_inst_tac [("a","uu")] selectI2 1), |
|
22 |
(atac 1), |
|
23 |
(etac spec 1) |
|
24 |
]))); |
|
3026
7a5611f66b72
moved antisym_less_inverse,box_less from Porder.ML to Porder0.ML
slotosch
parents:
2841
diff
changeset
|
25 |
|
7a5611f66b72
moved antisym_less_inverse,box_less from Porder.ML to Porder0.ML
slotosch
parents:
2841
diff
changeset
|
26 |
(* ------------------------------------------------------------------------ *) |
7a5611f66b72
moved antisym_less_inverse,box_less from Porder.ML to Porder0.ML
slotosch
parents:
2841
diff
changeset
|
27 |
(* the reverse law of anti--symmetrie of << *) |
7a5611f66b72
moved antisym_less_inverse,box_less from Porder.ML to Porder0.ML
slotosch
parents:
2841
diff
changeset
|
28 |
(* ------------------------------------------------------------------------ *) |
7a5611f66b72
moved antisym_less_inverse,box_less from Porder.ML to Porder0.ML
slotosch
parents:
2841
diff
changeset
|
29 |
|
9169 | 30 |
Goal "(x::'a::po)=y ==> x << y & y << x"; |
31 |
by (rtac conjI 1); |
|
32 |
by ((rtac subst 1) THEN (rtac refl_less 2) THEN (atac 1)); |
|
33 |
by ((rtac subst 1) THEN (rtac refl_less 2) THEN (etac sym 1)); |
|
34 |
qed "antisym_less_inverse"; |
|
3026
7a5611f66b72
moved antisym_less_inverse,box_less from Porder.ML to Porder0.ML
slotosch
parents:
2841
diff
changeset
|
35 |
|
7a5611f66b72
moved antisym_less_inverse,box_less from Porder.ML to Porder0.ML
slotosch
parents:
2841
diff
changeset
|
36 |
|
9169 | 37 |
Goal "[| (a::'a::po) << b; c << a; b << d|] ==> c << d"; |
38 |
by (etac trans_less 1); |
|
39 |
by (etac trans_less 1); |
|
40 |
by (atac 1); |
|
41 |
qed "box_less"; |
|
3026
7a5611f66b72
moved antisym_less_inverse,box_less from Porder.ML to Porder0.ML
slotosch
parents:
2841
diff
changeset
|
42 |
|
5068 | 43 |
Goal "((x::'a::po)=y) = (x << y & y << x)"; |
4423 | 44 |
by (fast_tac (HOL_cs addSEs [antisym_less_inverse] addSIs [antisym_less]) 1); |
3460 | 45 |
qed "po_eq_conv"; |