Sat, 21 Jan 2006 23:02:28 +0100 removed duplicate type_solver (cf. Tools/typechk.ML);
wenzelm [Sat, 21 Jan 2006 23:02:28 +0100] rev 18735
removed duplicate type_solver (cf. Tools/typechk.ML);
Sat, 21 Jan 2006 23:02:27 +0100 simplified type attribute;
wenzelm [Sat, 21 Jan 2006 23:02:27 +0100] rev 18734
simplified type attribute; removed rule/declaration (cf. thm.ML); removed obsolete theory/proof/generic/common; removed obsolete global/local/context_attribute(_i); added attribute(_i); renamed attribute to internal;
Sat, 21 Jan 2006 23:02:25 +0100 simplified type attribute;
wenzelm [Sat, 21 Jan 2006 23:02:25 +0100] rev 18733
simplified type attribute; added rule/declaration_attribute (from drule.ML); added theory/proof_attributes; removed apply(s)_attributes;
Sat, 21 Jan 2006 23:02:24 +0100 simplified type attribute;
wenzelm [Sat, 21 Jan 2006 23:02:24 +0100] rev 18732
simplified type attribute; moved rule/declaration_attribute to thm.ML;
Sat, 21 Jan 2006 23:02:23 +0100 rename map_theory/proof to theory/proof_map;
wenzelm [Sat, 21 Jan 2006 23:02:23 +0100] rev 18731
rename map_theory/proof to theory/proof_map; added separate map_theory/proof;
Sat, 21 Jan 2006 23:02:21 +0100 tuned proofs;
wenzelm [Sat, 21 Jan 2006 23:02:21 +0100] rev 18730
tuned proofs;
Sat, 21 Jan 2006 23:02:20 +0100 simplified type attribute;
wenzelm [Sat, 21 Jan 2006 23:02:20 +0100] rev 18729
simplified type attribute; tuned;
Sat, 21 Jan 2006 23:02:14 +0100 simplified type attribute;
wenzelm [Sat, 21 Jan 2006 23:02:14 +0100] rev 18728
simplified type attribute;
Fri, 20 Jan 2006 04:53:59 +0100 type information is now also printed.
mengj [Fri, 20 Jan 2006 04:53:59 +0100] rev 18727
type information is now also printed.
Fri, 20 Jan 2006 04:50:01 +0100 added some debugging code.
mengj [Fri, 20 Jan 2006 04:50:01 +0100] rev 18726
added some debugging code.
Fri, 20 Jan 2006 04:35:23 +0100 fixed a bug
mengj [Fri, 20 Jan 2006 04:35:23 +0100] rev 18725
fixed a bug
Thu, 19 Jan 2006 21:22:30 +0100 quote "atom";
wenzelm [Thu, 19 Jan 2006 21:22:30 +0100] rev 18724
quote "atom";
Thu, 19 Jan 2006 21:22:29 +0100 updated;
wenzelm [Thu, 19 Jan 2006 21:22:29 +0100] rev 18723
updated;
Thu, 19 Jan 2006 21:22:27 +0100 * ML/Isar: theory setup has type (theory -> theory);
wenzelm [Thu, 19 Jan 2006 21:22:27 +0100] rev 18722
* ML/Isar: theory setup has type (theory -> theory);
Thu, 19 Jan 2006 21:22:26 +0100 use/use_thy: Output.toplevel_errors;
wenzelm [Thu, 19 Jan 2006 21:22:26 +0100] rev 18721
use/use_thy: Output.toplevel_errors;
Thu, 19 Jan 2006 21:22:25 +0100 added basic syntax;
wenzelm [Thu, 19 Jan 2006 21:22:25 +0100] rev 18720
added basic syntax; removed pure syntax;
Thu, 19 Jan 2006 21:22:24 +0100 moved pure syntax to Syntax/syntax.ML and pure_thy.ML;
wenzelm [Thu, 19 Jan 2006 21:22:24 +0100] rev 18719
moved pure syntax to Syntax/syntax.ML and pure_thy.ML;
Thu, 19 Jan 2006 21:22:23 +0100 keep: disable Output.toplevel_errors;
wenzelm [Thu, 19 Jan 2006 21:22:23 +0100] rev 18718
keep: disable Output.toplevel_errors; program: Output.ML_errors;
Thu, 19 Jan 2006 21:22:22 +0100 run_thy: removed Output.toplevel_errors;
wenzelm [Thu, 19 Jan 2006 21:22:22 +0100] rev 18717
run_thy: removed Output.toplevel_errors;
Thu, 19 Jan 2006 21:22:21 +0100 added ML_errors;
wenzelm [Thu, 19 Jan 2006 21:22:21 +0100] rev 18716
added ML_errors;
Thu, 19 Jan 2006 21:22:20 +0100 use: Output.ML_errors;
wenzelm [Thu, 19 Jan 2006 21:22:20 +0100] rev 18715
use: Output.ML_errors;
Thu, 19 Jan 2006 21:22:19 +0100 Syntax.basic_syn;
wenzelm [Thu, 19 Jan 2006 21:22:19 +0100] rev 18714
Syntax.basic_syn;
Thu, 19 Jan 2006 21:22:18 +0100 setup: theory -> theory;
wenzelm [Thu, 19 Jan 2006 21:22:18 +0100] rev 18713
setup: theory -> theory; added syntax (from Syntax/mixfix.ML); added HTML output syntax for _lambda;
Thu, 19 Jan 2006 21:22:17 +0100 tuned setmp;
wenzelm [Thu, 19 Jan 2006 21:22:17 +0100] rev 18712
tuned setmp;
Thu, 19 Jan 2006 21:22:16 +0100 setup: theory -> theory;
wenzelm [Thu, 19 Jan 2006 21:22:16 +0100] rev 18711
setup: theory -> theory; use_output: Output.ML_errors;
Thu, 19 Jan 2006 21:22:15 +0100 tuned comments;
wenzelm [Thu, 19 Jan 2006 21:22:15 +0100] rev 18710
tuned comments;
Thu, 19 Jan 2006 21:22:14 +0100 setup: theory -> theory;
wenzelm [Thu, 19 Jan 2006 21:22:14 +0100] rev 18709
setup: theory -> theory; Syntax.appl(C)_syntax;
Thu, 19 Jan 2006 21:22:08 +0100 setup: theory -> theory;
wenzelm [Thu, 19 Jan 2006 21:22:08 +0100] rev 18708
setup: theory -> theory;
Thu, 19 Jan 2006 15:45:10 +0100 Use generic Simplifier.simp_add attribute instead
berghofe [Thu, 19 Jan 2006 15:45:10 +0100] rev 18707
Use generic Simplifier.simp_add attribute instead of Simplifier.simp_add_global.
Thu, 19 Jan 2006 14:59:55 +0100 Re-inserted consts_code declaration accidentally deleted
berghofe [Thu, 19 Jan 2006 14:59:55 +0100] rev 18706
Re-inserted consts_code declaration accidentally deleted during last commit.
Thu, 19 Jan 2006 10:22:13 +0100 strengthened some lemmas; simplified some proofs
paulson [Thu, 19 Jan 2006 10:22:13 +0100] rev 18705
strengthened some lemmas; simplified some proofs
Wed, 18 Jan 2006 11:55:50 +0100 substantial improvement in serialization handling
haftmann [Wed, 18 Jan 2006 11:55:50 +0100] rev 18704
substantial improvement in serialization handling
Wed, 18 Jan 2006 02:48:58 +0100 fixed one proof that broke because of the changes
urbanc [Wed, 18 Jan 2006 02:48:58 +0100] rev 18703
fixed one proof that broke because of the changes Markus did on the rules ex1I
Tue, 17 Jan 2006 16:36:57 +0100 substantial improvements in code generator
haftmann [Tue, 17 Jan 2006 16:36:57 +0100] rev 18702
substantial improvements in code generator
Tue, 17 Jan 2006 10:26:50 +0100 these hacks are no longer needed
paulson [Tue, 17 Jan 2006 10:26:50 +0100] rev 18701
these hacks are no longer needed
Tue, 17 Jan 2006 10:26:36 +0100 improved SPASS support
paulson [Tue, 17 Jan 2006 10:26:36 +0100] rev 18700
improved SPASS support
Mon, 16 Jan 2006 21:55:17 +0100 case_result: drop_schematic, i.e. be permissive about illegal binds;
wenzelm [Mon, 16 Jan 2006 21:55:17 +0100] rev 18699
case_result: drop_schematic, i.e. be permissive about illegal binds;
Mon, 16 Jan 2006 21:55:15 +0100 put_facts: do not pretend local thms were named;
wenzelm [Mon, 16 Jan 2006 21:55:15 +0100] rev 18698
put_facts: do not pretend local thms were named;
Mon, 16 Jan 2006 21:55:14 +0100 declare the1_equality [elim?];
wenzelm [Mon, 16 Jan 2006 21:55:14 +0100] rev 18697
declare the1_equality [elim?];
Sun, 15 Jan 2006 20:04:05 +0100 tuned;
wenzelm [Sun, 15 Jan 2006 20:04:05 +0100] rev 18696
tuned;
Sun, 15 Jan 2006 20:00:59 +0100 tuned;
wenzelm [Sun, 15 Jan 2006 20:00:59 +0100] rev 18695
tuned;
Sun, 15 Jan 2006 19:58:57 +0100 * Classical: optional weight for attributes;
wenzelm [Sun, 15 Jan 2006 19:58:57 +0100] rev 18694
* Classical: optional weight for attributes; * HOL: prefer ex1I over ex_ex1I in single-step reasoning;
Sun, 15 Jan 2006 19:58:56 +0100 guess: used fixed inferred_type of vars;
wenzelm [Sun, 15 Jan 2006 19:58:56 +0100] rev 18693
guess: used fixed inferred_type of vars;
Sun, 15 Jan 2006 19:58:55 +0100 export add_args;
wenzelm [Sun, 15 Jan 2006 19:58:55 +0100] rev 18692
export add_args; tuned;
Sun, 15 Jan 2006 19:58:54 +0100 attributes: optional weight;
wenzelm [Sun, 15 Jan 2006 19:58:54 +0100] rev 18691
attributes: optional weight; tuned;
Sun, 15 Jan 2006 19:58:53 +0100 classical attributes: optional weight;
wenzelm [Sun, 15 Jan 2006 19:58:53 +0100] rev 18690
classical attributes: optional weight;
Sun, 15 Jan 2006 19:58:51 +0100 prefer ex1I over ex_ex1I in single-step reasoning;
wenzelm [Sun, 15 Jan 2006 19:58:51 +0100] rev 18689
prefer ex1I over ex_ex1I in single-step reasoning;
Sat, 14 Jan 2006 22:25:34 +0100 generic attributes;
wenzelm [Sat, 14 Jan 2006 22:25:34 +0100] rev 18688
generic attributes;
Sat, 14 Jan 2006 17:20:51 +0100 tuned;
wenzelm [Sat, 14 Jan 2006 17:20:51 +0100] rev 18687
tuned;
Sat, 14 Jan 2006 17:15:24 +0100 * ML/Isar: simplified treatment of user-level errors;
wenzelm [Sat, 14 Jan 2006 17:15:24 +0100] rev 18686
* ML/Isar: simplified treatment of user-level errors;
Sat, 14 Jan 2006 17:14:18 +0100 sane ERROR vs. TOPLEVEL_ERROR handling;
wenzelm [Sat, 14 Jan 2006 17:14:18 +0100] rev 18685
sane ERROR vs. TOPLEVEL_ERROR handling; added program;
Sat, 14 Jan 2006 17:14:17 +0100 added Isar.toplevel;
wenzelm [Sat, 14 Jan 2006 17:14:17 +0100] rev 18684
added Isar.toplevel;
Sat, 14 Jan 2006 17:14:16 +0100 Output.error_msg;
wenzelm [Sat, 14 Jan 2006 17:14:16 +0100] rev 18683
Output.error_msg;
Sat, 14 Jan 2006 17:14:15 +0100 removed special ERROR handling stuff (transform_error etc.);
wenzelm [Sat, 14 Jan 2006 17:14:15 +0100] rev 18682
removed special ERROR handling stuff (transform_error etc.); moved plain ERROR/error to library.ML; added toplevel_errors, exception TOPLEVEL_ERROR; error_msg, panic, info, debug no longer pervasive;
Sat, 14 Jan 2006 17:14:14 +0100 added exception ERROR, error, cat_error, sys_error, assert, deny, assert_all;
wenzelm [Sat, 14 Jan 2006 17:14:14 +0100] rev 18681
added exception ERROR, error, cat_error, sys_error, assert, deny, assert_all; added transform_failure; added prefix;
Sat, 14 Jan 2006 17:14:13 +0100 Output.debug;
wenzelm [Sat, 14 Jan 2006 17:14:13 +0100] rev 18680
Output.debug;
Sat, 14 Jan 2006 17:14:11 +0100 generated code: raise Match instead of ERROR;
wenzelm [Sat, 14 Jan 2006 17:14:11 +0100] rev 18679
generated code: raise Match instead of ERROR;
Sat, 14 Jan 2006 17:14:06 +0100 sane ERROR handling;
wenzelm [Sat, 14 Jan 2006 17:14:06 +0100] rev 18678
sane ERROR handling;
Fri, 13 Jan 2006 17:39:41 +0100 blacklist experiments
paulson [Fri, 13 Jan 2006 17:39:41 +0100] rev 18677
blacklist experiments
Fri, 13 Jan 2006 17:39:19 +0100 more readable divide ops
paulson [Fri, 13 Jan 2006 17:39:19 +0100] rev 18676
more readable divide ops
Fri, 13 Jan 2006 17:39:03 +0100 more practical time limit
paulson [Fri, 13 Jan 2006 17:39:03 +0100] rev 18675
more practical time limit
Fri, 13 Jan 2006 14:43:09 +0100 *** empty log message ***
nipkow [Fri, 13 Jan 2006 14:43:09 +0100] rev 18674
*** empty log message ***
Fri, 13 Jan 2006 01:13:17 +0100 mixfix: added Structure;
wenzelm [Fri, 13 Jan 2006 01:13:17 +0100] rev 18673
mixfix: added Structure;
Fri, 13 Jan 2006 01:13:16 +0100 uniform handling of fixes: read/cert_vars, add_fixes(_i), body flag;
wenzelm [Fri, 13 Jan 2006 01:13:16 +0100] rev 18672
uniform handling of fixes: read/cert_vars, add_fixes(_i), body flag; mixfix: added Structure; renamed type exporter to export; removed obsolete sign_of; tuned signature; tuned;
Fri, 13 Jan 2006 01:13:15 +0100 uniform handling of fixes;
wenzelm [Fri, 13 Jan 2006 01:13:15 +0100] rev 18671
uniform handling of fixes; mixfix: added Structure; tuned;
Fri, 13 Jan 2006 01:13:11 +0100 uniform handling of fixes;
wenzelm [Fri, 13 Jan 2006 01:13:11 +0100] rev 18670
uniform handling of fixes;
Fri, 13 Jan 2006 01:13:08 +0100 uniform handling of fixes;
wenzelm [Fri, 13 Jan 2006 01:13:08 +0100] rev 18669
uniform handling of fixes; mixfix: added Structure;
Fri, 13 Jan 2006 01:13:06 +0100 uniform handling of fixes;
wenzelm [Fri, 13 Jan 2006 01:13:06 +0100] rev 18668
uniform handling of fixes; tuned;
Fri, 13 Jan 2006 01:13:05 +0100 tuned;
wenzelm [Fri, 13 Jan 2006 01:13:05 +0100] rev 18667
tuned;
Fri, 13 Jan 2006 01:13:03 +0100 generic_setup: optional argument, defaults to Context.setup();
wenzelm [Fri, 13 Jan 2006 01:13:03 +0100] rev 18666
generic_setup: optional argument, defaults to Context.setup();
Fri, 13 Jan 2006 01:13:02 +0100 added map_theory, map_proof;
wenzelm [Fri, 13 Jan 2006 01:13:02 +0100] rev 18665
added map_theory, map_proof;
Fri, 13 Jan 2006 01:13:00 +0100 removed obsolete sign_of;
wenzelm [Fri, 13 Jan 2006 01:13:00 +0100] rev 18664
removed obsolete sign_of;
Fri, 13 Jan 2006 01:12:59 +0100 implicit setup, which admits exception_trace;
wenzelm [Fri, 13 Jan 2006 01:12:59 +0100] rev 18663
implicit setup, which admits exception_trace;
Fri, 13 Jan 2006 01:12:58 +0100 ProofContext.def_export;
wenzelm [Fri, 13 Jan 2006 01:12:58 +0100] rev 18662
ProofContext.def_export;
Wed, 11 Jan 2006 18:46:31 +0100 updated to new induction principle
urbanc [Wed, 11 Jan 2006 18:46:31 +0100] rev 18661
updated to new induction principle
Wed, 11 Jan 2006 18:39:19 +0100 cahges to use the new induction-principle (now proved in
urbanc [Wed, 11 Jan 2006 18:39:19 +0100] rev 18660
cahges to use the new induction-principle (now proved in full glory)
Wed, 11 Jan 2006 18:38:32 +0100 changes to make use of the new induction principle proved by
urbanc [Wed, 11 Jan 2006 18:38:32 +0100] rev 18659
changes to make use of the new induction principle proved by Stefan horay (hooraayyy)
Wed, 11 Jan 2006 18:21:23 +0100 Implemented proof of (strong) induction rule.
berghofe [Wed, 11 Jan 2006 18:21:23 +0100] rev 18658
Implemented proof of (strong) induction rule.
Wed, 11 Jan 2006 18:20:59 +0100 Added theorem at_finite_select.
berghofe [Wed, 11 Jan 2006 18:20:59 +0100] rev 18657
Added theorem at_finite_select.
Wed, 11 Jan 2006 17:12:30 +0100 added lemmas perm_empty, perm_insert to do with
urbanc [Wed, 11 Jan 2006 17:12:30 +0100] rev 18656
added lemmas perm_empty, perm_insert to do with permutations on sets
Wed, 11 Jan 2006 17:10:11 +0100 merged the silly lemmas into the eqvt proof of subtype
urbanc [Wed, 11 Jan 2006 17:10:11 +0100] rev 18655
merged the silly lemmas into the eqvt proof of subtype
Wed, 11 Jan 2006 17:07:57 +0100 tuned proofs
urbanc [Wed, 11 Jan 2006 17:07:57 +0100] rev 18654
tuned proofs
Wed, 11 Jan 2006 14:00:11 +0100 tuned the eqvt-proof
urbanc [Wed, 11 Jan 2006 14:00:11 +0100] rev 18653
tuned the eqvt-proof
Wed, 11 Jan 2006 12:21:01 +0100 rolled back the last addition since these lemmas were already
urbanc [Wed, 11 Jan 2006 12:21:01 +0100] rev 18652
rolled back the last addition since these lemmas were already in the simpset.
Wed, 11 Jan 2006 12:14:25 +0100 added the thms-collection "pt_id" (collection of all pt_<ak>1 lemmas)
urbanc [Wed, 11 Jan 2006 12:14:25 +0100] rev 18651
added the thms-collection "pt_id" (collection of all pt_<ak>1 lemmas)
Wed, 11 Jan 2006 12:11:53 +0100 tuned
urbanc [Wed, 11 Jan 2006 12:11:53 +0100] rev 18650
tuned
Wed, 11 Jan 2006 11:00:26 +0100 tidied, and added missing thm divide_less_eq_1_neg
paulson [Wed, 11 Jan 2006 11:00:26 +0100] rev 18649
tidied, and added missing thm divide_less_eq_1_neg
Wed, 11 Jan 2006 10:59:55 +0100 tidied, and giving theorems names
paulson [Wed, 11 Jan 2006 10:59:55 +0100] rev 18648
tidied, and giving theorems names
Wed, 11 Jan 2006 03:10:04 +0100 add transitivity rules
huffman [Wed, 11 Jan 2006 03:10:04 +0100] rev 18647
add transitivity rules
Wed, 11 Jan 2006 00:11:05 +0100 tuned;
wenzelm [Wed, 11 Jan 2006 00:11:05 +0100] rev 18646
tuned;
Wed, 11 Jan 2006 00:11:02 +0100 updated;
wenzelm [Wed, 11 Jan 2006 00:11:02 +0100] rev 18645
updated;
Tue, 10 Jan 2006 19:36:59 +0100 tuned;
wenzelm [Tue, 10 Jan 2006 19:36:59 +0100] rev 18644
tuned;
Tue, 10 Jan 2006 19:34:04 +0100 generic attributes;
wenzelm [Tue, 10 Jan 2006 19:34:04 +0100] rev 18643
generic attributes;
Tue, 10 Jan 2006 19:33:42 +0100 * ML: generic context, data, attributes;
wenzelm [Tue, 10 Jan 2006 19:33:42 +0100] rev 18642
* ML: generic context, data, attributes;
Tue, 10 Jan 2006 19:33:41 +0100 added context_of -- generic context;
wenzelm [Tue, 10 Jan 2006 19:33:41 +0100] rev 18641
added context_of -- generic context;
Tue, 10 Jan 2006 19:33:39 +0100 generic attributes;
wenzelm [Tue, 10 Jan 2006 19:33:39 +0100] rev 18640
generic attributes; tuned;
Tue, 10 Jan 2006 19:33:38 +0100 print rules: generic context;
wenzelm [Tue, 10 Jan 2006 19:33:38 +0100] rev 18639
print rules: generic context;
Tue, 10 Jan 2006 19:33:37 +0100 Specification.pretty_consts ctxt;
wenzelm [Tue, 10 Jan 2006 19:33:37 +0100] rev 18638
Specification.pretty_consts ctxt;
Tue, 10 Jan 2006 19:33:36 +0100 generic data and attributes;
wenzelm [Tue, 10 Jan 2006 19:33:36 +0100] rev 18637
generic data and attributes; tuned;
Tue, 10 Jan 2006 19:33:35 +0100 added rule, declaration;
wenzelm [Tue, 10 Jan 2006 19:33:35 +0100] rev 18636
added rule, declaration; support generic attributes: theory, context, generic, common, generic_attribute(_i); added generic syntax; basic attributes now generic; tuned;
Tue, 10 Jan 2006 19:33:34 +0100 added generic syntax;
wenzelm [Tue, 10 Jan 2006 19:33:34 +0100] rev 18635
added generic syntax; mk_attribute: generic;
Tue, 10 Jan 2006 19:33:33 +0100 tuned dependencies;
wenzelm [Tue, 10 Jan 2006 19:33:33 +0100] rev 18634
tuned dependencies;
Tue, 10 Jan 2006 19:33:32 +0100 added declaration_attribute;
wenzelm [Tue, 10 Jan 2006 19:33:32 +0100] rev 18633
added declaration_attribute;
Tue, 10 Jan 2006 19:33:31 +0100 support for generic contexts with data;
wenzelm [Tue, 10 Jan 2006 19:33:31 +0100] rev 18632
support for generic contexts with data;
Tue, 10 Jan 2006 19:33:30 +0100 fix_tac: no warning;
wenzelm [Tue, 10 Jan 2006 19:33:30 +0100] rev 18631
fix_tac: no warning;
Tue, 10 Jan 2006 19:33:29 +0100 generic attributes;
wenzelm [Tue, 10 Jan 2006 19:33:29 +0100] rev 18630
generic attributes; added low-level modifiers from Pure/context_rules.ML;
Tue, 10 Jan 2006 19:33:27 +0100 Attrib.rule;
wenzelm [Tue, 10 Jan 2006 19:33:27 +0100] rev 18629
Attrib.rule;
Tue, 10 Jan 2006 15:23:31 +0100 tuned
urbanc [Tue, 10 Jan 2006 15:23:31 +0100] rev 18628
tuned
Tue, 10 Jan 2006 02:32:10 +0100 added the lemmas supp_char and supp_string
urbanc [Tue, 10 Jan 2006 02:32:10 +0100] rev 18627
added the lemmas supp_char and supp_string
Mon, 09 Jan 2006 15:55:15 +0100 added some lemmas to the collection "abs_fresh"
urbanc [Mon, 09 Jan 2006 15:55:15 +0100] rev 18626
added some lemmas to the collection "abs_fresh" the lemmas are of the form finite (supp x) ==> (b # [a].x) = (b=a \/ b # x) previously only lemmas of the form (b # [a].x) = (b=a \/ b # x) with the type-constraint that x is finitely supported were included.
Mon, 09 Jan 2006 13:29:08 +0100 _E suffix for compatibility with AddIffs
paulson [Mon, 09 Jan 2006 13:29:08 +0100] rev 18625
_E suffix for compatibility with AddIffs
Mon, 09 Jan 2006 13:28:34 +0100 tidied
paulson [Mon, 09 Jan 2006 13:28:34 +0100] rev 18624
tidied
Mon, 09 Jan 2006 13:28:06 +0100 simplified the special-case simprules
paulson [Mon, 09 Jan 2006 13:28:06 +0100] rev 18623
simplified the special-case simprules
Mon, 09 Jan 2006 13:27:44 +0100 theorems need names
paulson [Mon, 09 Jan 2006 13:27:44 +0100] rev 18622
theorems need names
Mon, 09 Jan 2006 00:05:10 +0100 commented the transitivity and narrowing proof
urbanc [Mon, 09 Jan 2006 00:05:10 +0100] rev 18621
commented the transitivity and narrowing proof
Sat, 07 Jan 2006 23:28:01 +0100 Theory specifications --- with type-inference, but no internal polymorphism.
wenzelm [Sat, 07 Jan 2006 23:28:01 +0100] rev 18620
Theory specifications --- with type-inference, but no internal polymorphism.
Sat, 07 Jan 2006 23:28:00 +0100 added infer_type, declared_type;
wenzelm [Sat, 07 Jan 2006 23:28:00 +0100] rev 18619
added infer_type, declared_type;
Sat, 07 Jan 2006 23:27:59 +0100 added param, spec, named_spec;
wenzelm [Sat, 07 Jan 2006 23:27:59 +0100] rev 18618
added param, spec, named_spec;
Sat, 07 Jan 2006 23:27:58 +0100 added init;
wenzelm [Sat, 07 Jan 2006 23:27:58 +0100] rev 18617
added init; tuned signature;
Sat, 07 Jan 2006 23:27:56 +0100 added 'axiomatization';
wenzelm [Sat, 07 Jan 2006 23:27:56 +0100] rev 18616
added 'axiomatization';
(0) -10000 -3000 -1000 -120 +120 +1000 +3000 +10000 +30000 tip