author | wenzelm |
Fri, 23 Jul 1999 16:50:55 +0200 | |
changeset 7067 | 601f930d3739 |
parent 6945 | eeeef70c8fe3 |
child 7202 | 6fcaf006cc40 |
permissions | -rw-r--r-- |
6779
2912aff958bd
Calculation.thy: Setup transitivity rules for calculational proofs.
wenzelm
parents:
diff
changeset
|
1 |
(* Title: HOL/Calculation.thy |
2912aff958bd
Calculation.thy: Setup transitivity rules for calculational proofs.
wenzelm
parents:
diff
changeset
|
2 |
ID: $Id$ |
2912aff958bd
Calculation.thy: Setup transitivity rules for calculational proofs.
wenzelm
parents:
diff
changeset
|
3 |
Author: Markus Wenzel, TU Muenchen |
2912aff958bd
Calculation.thy: Setup transitivity rules for calculational proofs.
wenzelm
parents:
diff
changeset
|
4 |
|
6873 | 5 |
Setup transitivity rules for calculational proofs. Note that in the |
6 |
list below later rules have priority. |
|
6779
2912aff958bd
Calculation.thy: Setup transitivity rules for calculational proofs.
wenzelm
parents:
diff
changeset
|
7 |
*) |
2912aff958bd
Calculation.thy: Setup transitivity rules for calculational proofs.
wenzelm
parents:
diff
changeset
|
8 |
|
6862 | 9 |
theory Calculation = Int:; |
6779
2912aff958bd
Calculation.thy: Setup transitivity rules for calculational proofs.
wenzelm
parents:
diff
changeset
|
10 |
|
6945 | 11 |
|
6873 | 12 |
theorems [trans] = HOL.ssubst; (* = x x *) |
13 |
theorems [trans] = HOL.subst[COMP swap_prems_rl]; (* x = x *) |
|
14 |
||
15 |
theorems [trans] = Divides.dvd_trans; (* dvd dvd dvd *) |
|
16 |
||
6862 | 17 |
theorems [trans] = Ord.order_less_trans; (* < < < *) |
18 |
theorems [trans] = Ord.order_le_less_trans; (* <= < < *) |
|
19 |
theorems [trans] = Ord.order_less_le_trans; (* < <= < *) |
|
6873 | 20 |
theorems [trans] = Ord.order_trans; (* <= <= <= *) |
21 |
theorems [trans] = Ord.order_antisym; (* <= <= = *) |
|
6862 | 22 |
|
6863 | 23 |
theorem [trans]: "[| x <= y; y = z |] ==> x <= z"; (* <= = <= *) |
6873 | 24 |
by (rule HOL.subst); |
6779
2912aff958bd
Calculation.thy: Setup transitivity rules for calculational proofs.
wenzelm
parents:
diff
changeset
|
25 |
|
6863 | 26 |
theorem [trans]: "[| x = y; y <= z |] ==> x <= z"; (* = <= <= *) |
6873 | 27 |
by (rule HOL.ssubst); |
6862 | 28 |
|
6863 | 29 |
theorem [trans]: "[| x < y; y = z |] ==> x < z"; (* < = < *) |
6873 | 30 |
by (rule HOL.subst); |
6779
2912aff958bd
Calculation.thy: Setup transitivity rules for calculational proofs.
wenzelm
parents:
diff
changeset
|
31 |
|
6863 | 32 |
theorem [trans]: "[| x = y; y < z |] ==> x < z"; (* = < < *) |
6873 | 33 |
by (rule HOL.ssubst); |
6779
2912aff958bd
Calculation.thy: Setup transitivity rules for calculational proofs.
wenzelm
parents:
diff
changeset
|
34 |
|
6945 | 35 |
theorems [trans] = HOL.trans (* = = = *) |
36 |
||
6779
2912aff958bd
Calculation.thy: Setup transitivity rules for calculational proofs.
wenzelm
parents:
diff
changeset
|
37 |
|
6862 | 38 |
end; |