Calculation.thy: Setup transitivity rules for calculational proofs.
authorwenzelm
Fri, 04 Jun 1999 19:57:31 +0200
changeset 6779 2912aff958bd
parent 6778 2f66eea8a025
child 6780 769cea1985e4
Calculation.thy: Setup transitivity rules for calculational proofs.
src/HOL/Calculation.thy
src/HOL/IsaMakefile
src/HOL/Main.thy
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/Calculation.thy	Fri Jun 04 19:57:31 1999 +0200
@@ -0,0 +1,23 @@
+(*  Title:      HOL/Calculation.thy
+    ID:         $Id$
+    Author:     Markus Wenzel, TU Muenchen
+
+Setup transitivity rules for calculational proofs.
+*)
+
+theory Calculation = Int:
+
+
+theorems[trans] = HOL.trans			(*  =  =  =  *)
+theorems[trans] = HOL.ssubst                    (*  =  *  *  *)
+theorems[trans] = HOL.subst[COMP swap_prems_rl]	(*  *  =  *  *)
+
+theorems[trans] = Ord.order_trans		(*  <= <= <= *)
+theorems[trans] = Ord.order_less_trans		(*  <  <  <  *)
+theorems[trans] = Ord.order_le_less_trans	(*  <= <  <  *)
+theorems[trans] = Ord.order_less_le_trans	(*  <  <= <  *)
+
+theorems[trans] = Divides.dvd_trans		(* dvd dvd dvd *)
+
+
+end
--- a/src/HOL/IsaMakefile	Fri Jun 04 19:55:41 1999 +0200
+++ b/src/HOL/IsaMakefile	Fri Jun 04 19:57:31 1999 +0200
@@ -43,24 +43,24 @@
   $(SRC)/TFL/thms.sig $(SRC)/TFL/thms.sml $(SRC)/TFL/thry.sig \
   $(SRC)/TFL/thry.sml $(SRC)/TFL/usyntax.sig $(SRC)/TFL/usyntax.sml \
   $(SRC)/TFL/utils.sig $(SRC)/TFL/utils.sml Arith.ML Arith.thy \
-  Datatype.thy Divides.ML Divides.thy Finite.ML Finite.thy Fun.ML \
-  Fun.thy Gfp.ML Gfp.thy HOL.ML HOL.thy Inductive.thy Integ/Bin.ML \
-  Integ/Bin.thy Integ/Equiv.ML Integ/Equiv.thy Integ/IntDef.ML \
-  Integ/IntDef.thy Integ/Int.ML Integ/Int.thy Integ/simproc.ML Lfp.ML \
-  Lfp.thy List.ML List.thy Main.thy Map.ML Map.thy Nat.ML Nat.thy \
-  NatDef.ML NatDef.thy Option.ML Option.thy Ord.ML Ord.thy Power.ML \
-  Power.thy Prod.ML Prod.thy ROOT.ML Recdef.thy Record.thy RelPow.ML \
-  RelPow.thy Relation.ML Relation.thy Set.ML Set.thy Sexp.ML Sexp.thy \
-  String.thy Sum.ML Sum.thy Tools/datatype_aux.ML \
-  Tools/datatype_abs_proofs.ML Tools/datatype_package.ML \
-  Tools/datatype_prop.ML Tools/datatype_rep_proofs.ML \
-  Tools/induct_method.ML Tools/inductive_package.ML \
-  Tools/primrec_package.ML Tools/recdef_package.ML \
-  Tools/record_package.ML Tools/typedef_package.ML Trancl.ML \
-  Trancl.thy Univ.ML Univ.thy Vimage.ML Vimage.thy WF.ML WF.thy \
-  WF_Rel.ML WF_Rel.thy cladata.ML equalities.ML equalities.thy \
-  hologic.ML mono.ML mono.thy simpdata.ML subset.ML subset.thy \
-  thy_syntax.ML
+  Calculation.thy Datatype.thy Divides.ML Divides.thy Finite.ML \
+  Finite.thy Fun.ML Fun.thy Gfp.ML Gfp.thy HOL.ML HOL.thy \
+  Inductive.thy Integ/Bin.ML Integ/Bin.thy Integ/Equiv.ML \
+  Integ/Equiv.thy Integ/IntDef.ML Integ/IntDef.thy Integ/Int.ML \
+  Integ/Int.thy Integ/simproc.ML Lfp.ML Lfp.thy List.ML List.thy \
+  Main.thy Map.ML Map.thy Nat.ML Nat.thy NatDef.ML NatDef.thy \
+  Option.ML Option.thy Ord.ML Ord.thy Power.ML Power.thy Prod.ML \
+  Prod.thy ROOT.ML Recdef.thy Record.thy RelPow.ML RelPow.thy \
+  Relation.ML Relation.thy Set.ML Set.thy Sexp.ML Sexp.thy String.thy \
+  Sum.ML Sum.thy Tools/datatype_aux.ML Tools/datatype_abs_proofs.ML \
+  Tools/datatype_package.ML Tools/datatype_prop.ML \
+  Tools/datatype_rep_proofs.ML Tools/induct_method.ML \
+  Tools/inductive_package.ML Tools/primrec_package.ML \
+  Tools/recdef_package.ML Tools/record_package.ML \
+  Tools/typedef_package.ML Trancl.ML Trancl.thy Univ.ML Univ.thy \
+  Vimage.ML Vimage.thy WF.ML WF.thy WF_Rel.ML WF_Rel.thy cladata.ML \
+  equalities.ML equalities.thy hologic.ML mono.ML mono.thy simpdata.ML \
+  subset.ML subset.thy thy_syntax.ML
 	@$(ISATOOL) usedir -b $(OUT)/Pure HOL
 
 
--- a/src/HOL/Main.thy	Fri Jun 04 19:55:41 1999 +0200
+++ b/src/HOL/Main.thy	Fri Jun 04 19:57:31 1999 +0200
@@ -1,4 +1,4 @@
 
 (*theory Main includes everything*)
 
-Main = Bin + Map + Recdef + Record + RelPow + Sexp + String
+Main = Bin + Map + Recdef + Record + RelPow + Sexp + String + Calculation