author | isatest |
Sat, 26 Oct 2002 13:05:27 +0200 | |
changeset 13680 | a6ce43a59d4a |
parent 12030 | 46d57d0290a2 |
child 14981 | e73f8140af78 |
permissions | -rw-r--r-- |
2644 | 1 |
(* Title: HOLCF/Porder0.ML |
2 |
ID: $Id$ |
|
3 |
Author: Oscar Slotosch |
|
12030 | 4 |
License: GPL (GNU GENERAL PUBLIC LICENSE) |
2644 | 5 |
|
12030 | 6 |
derive the characteristic axioms for the characteristic constants |
9245 | 7 |
*) |
2644 | 8 |
|
2841
c2508f4ab739
Added "discrete" CPOs and modified IMP to use those rather than "lift"
nipkow
parents:
2644
diff
changeset
|
9 |
AddIffs [refl_less]; |
c2508f4ab739
Added "discrete" CPOs and modified IMP to use those rather than "lift"
nipkow
parents:
2644
diff
changeset
|
10 |
|
2644 | 11 |
(* ------------------------------------------------------------------------ *) |
12 |
(* minimal fixes least element *) |
|
13 |
(* ------------------------------------------------------------------------ *) |
|
9245 | 14 |
Goal "!x::'a::po. uu<<x ==> uu=(@u.!y. u<<y)"; |
9969 | 15 |
by (blast_tac (claset() addIs [someI2,antisym_less]) 1); |
9245 | 16 |
bind_thm ("minimal2UU", allI RS result()); |
3026
7a5611f66b72
moved antisym_less_inverse,box_less from Porder.ML to Porder0.ML
slotosch
parents:
2841
diff
changeset
|
17 |
|
7a5611f66b72
moved antisym_less_inverse,box_less from Porder.ML to Porder0.ML
slotosch
parents:
2841
diff
changeset
|
18 |
(* ------------------------------------------------------------------------ *) |
7a5611f66b72
moved antisym_less_inverse,box_less from Porder.ML to Porder0.ML
slotosch
parents:
2841
diff
changeset
|
19 |
(* 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
|
20 |
(* ------------------------------------------------------------------------ *) |
7a5611f66b72
moved antisym_less_inverse,box_less from Porder.ML to Porder0.ML
slotosch
parents:
2841
diff
changeset
|
21 |
|
9169 | 22 |
Goal "(x::'a::po)=y ==> x << y & y << x"; |
9248
e1dee89de037
massive tidy-up: goal -> Goal, remove use of prems, etc.
paulson
parents:
9245
diff
changeset
|
23 |
by (Blast_tac 1); |
9169 | 24 |
qed "antisym_less_inverse"; |
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 |
|
9169 | 27 |
Goal "[| (a::'a::po) << b; c << a; b << d|] ==> c << d"; |
28 |
by (etac trans_less 1); |
|
29 |
by (etac trans_less 1); |
|
30 |
by (atac 1); |
|
31 |
qed "box_less"; |
|
3026
7a5611f66b72
moved antisym_less_inverse,box_less from Porder.ML to Porder0.ML
slotosch
parents:
2841
diff
changeset
|
32 |
|
5068 | 33 |
Goal "((x::'a::po)=y) = (x << y & y << x)"; |
4423 | 34 |
by (fast_tac (HOL_cs addSEs [antisym_less_inverse] addSIs [antisym_less]) 1); |
3460 | 35 |
qed "po_eq_conv"; |