Wed, 30 Sep 2009 00:17:06 +0200 added chained_goal, which presents the goal thm as seen by semi-structured methods;
wenzelm [Wed, 30 Sep 2009 00:17:06 +0200] rev 32769
added chained_goal, which presents the goal thm as seen by semi-structured methods;
Tue, 29 Sep 2009 23:19:26 +0200 tuned;
wenzelm [Tue, 29 Sep 2009 23:19:26 +0200] rev 32768
tuned;
Tue, 29 Sep 2009 23:14:57 +0200 removed dead/duplicate code;
wenzelm [Tue, 29 Sep 2009 23:14:57 +0200] rev 32767
removed dead/duplicate code;
Tue, 29 Sep 2009 22:53:07 +0200 aliases for Thomas Sewell;
wenzelm [Tue, 29 Sep 2009 22:53:07 +0200] rev 32766
aliases for Thomas Sewell;
Tue, 29 Sep 2009 22:48:24 +0200 modernized Balanced_Tree;
wenzelm [Tue, 29 Sep 2009 22:48:24 +0200] rev 32765
modernized Balanced_Tree;
Tue, 29 Sep 2009 22:33:27 +0200 replaced meta_iffD2 by existing Drule.equal_elim_rule2;
wenzelm [Tue, 29 Sep 2009 22:33:27 +0200] rev 32764
replaced meta_iffD2 by existing Drule.equal_elim_rule2; replaced SymSymTab by existing Symreltab; more antiquotations; eliminated old-style Library.foldl, Library.foldl_map; tuned;
Tue, 29 Sep 2009 21:36:49 +0200 tuned header;
wenzelm [Tue, 29 Sep 2009 21:36:49 +0200] rev 32763
tuned header;
Tue, 29 Sep 2009 21:36:33 +0200 Thomas Sewell, NICTA: more efficient HOL/record implementation;
wenzelm [Tue, 29 Sep 2009 21:36:33 +0200] rev 32762
Thomas Sewell, NICTA: more efficient HOL/record implementation;
Tue, 29 Sep 2009 21:34:59 +0200 tuned whitespace -- recover basic Isabelle conventions;
wenzelm [Tue, 29 Sep 2009 21:34:59 +0200] rev 32761
tuned whitespace -- recover basic Isabelle conventions;
Tue, 29 Sep 2009 18:14:08 +0200 merged
wenzelm [Tue, 29 Sep 2009 18:14:08 +0200] rev 32760
merged
Tue, 29 Sep 2009 14:26:33 +1000 Merge with isabelle dev changes.
Thomas Sewell <tsewell@nicta.com.au> [Tue, 29 Sep 2009 14:26:33 +1000] rev 32759
Merge with isabelle dev changes.
Tue, 29 Sep 2009 14:25:42 +1000 Replace OldTerm.term_vars with Term.add_vars in named_cterm_instantiate.
Thomas Sewell <tsewell@nicta.com.au> [Tue, 29 Sep 2009 14:25:42 +1000] rev 32758
Replace OldTerm.term_vars with Term.add_vars in named_cterm_instantiate.
Mon, 28 Sep 2009 15:37:19 +1000 Avoid a possible variable name conflict in instantiating a theorem.
Thomas Sewell <tsewell@nicta.com.au> [Mon, 28 Sep 2009 15:37:19 +1000] rev 32757
Avoid a possible variable name conflict in instantiating a theorem. Instantiating a theorem variable with new variables created a possible variable name conflict if a record was defined with a field named 'f', 'x' etc. Using variable indices of 1 avoids the problem.
Mon, 28 Sep 2009 14:16:01 +1000 Fix unescaped expressions breaking latex output in Record.thy
Thomas Sewell <tsewell@nicta.com.au> [Mon, 28 Sep 2009 14:16:01 +1000] rev 32756
Fix unescaped expressions breaking latex output in Record.thy Expressions containing _ and ^ need to be adjusted or antiquoted in text comments for latex compatibility. This is in fact a little annoying, since it makes the comment less readable in both source and HTML form.
Mon, 28 Sep 2009 11:13:11 +1000 Merge record patch with updates from isabelle mainline.
Thomas Sewell <tsewell@nicta.com.au> [Mon, 28 Sep 2009 11:13:11 +1000] rev 32755
Merge record patch with updates from isabelle mainline.
Fri, 25 Sep 2009 19:04:18 +1000 Avoid record-inner constants in polymorphic definitions in Bali
Thomas Sewell <tsewell@nicta.com.au> [Fri, 25 Sep 2009 19:04:18 +1000] rev 32754
Avoid record-inner constants in polymorphic definitions in Bali The Bali package needs to insert a record extension into a type class and define an associated polymorphic constant. There is no elegant way to do this. The existing approach was to insert every record extension into the type class, defining the polymorphic constant at each layer using inner operations created by the record package. Some of those operations have been removed. They can be replaced by use of record_name.extend if necessary, but we can also sidestep this altogether. The simpler approach here is to use defs(overloaded) once to provide a single definition for the composition of all the type constructors, which seems to be permitted. This gets us exactly the fact we need, with the cost that some types that were admitted to the type class have no definition for the constant at all.
Thu, 24 Sep 2009 11:33:05 +1000 Merge with changes from isabelle dev repository.
Thomas Sewell <tsewell@nicta.com.au> [Thu, 24 Sep 2009 11:33:05 +1000] rev 32753
Merge with changes from isabelle dev repository.
Wed, 23 Sep 2009 19:17:48 +1000 Initial response to feedback from Norbert, Makarius on record patch
tsewell@rubicon.NSW.bigpond.net.au [Wed, 23 Sep 2009 19:17:48 +1000] rev 32752
Initial response to feedback from Norbert, Makarius on record patch As Norbert recommended, the IsTuple.thy and istuple_support.ML files have been integrated into Record.thy and record.ML. I haven't merged the structures - record.ML now contains Record and IsTupleSupport. Some of the cosmetic changes Makarius requested have been made, including renaming variables with camel-case and run-together names and removing the tab character from the Author: line. Constants are defined with definition rather than constdefs. The split_ex_prf inner function has been cleaned up.
Tue, 22 Sep 2009 13:52:19 +1000 Branch merge for isabelle mainline updates.
Thomas Sewell <tsewell@nicta.com.au> [Tue, 22 Sep 2009 13:52:19 +1000] rev 32751
Branch merge for isabelle mainline updates.
Thu, 17 Sep 2009 14:17:37 +1000 Branch merge with updates from mainline isabelle.
Thomas Sewell <tsewell@nicta.com.au> [Thu, 17 Sep 2009 14:17:37 +1000] rev 32750
Branch merge with updates from mainline isabelle.
Fri, 11 Sep 2009 20:58:29 +1000 Implement previous fix (don't duplicate ext_def) correctly.
Thomas Sewell <tsewell@nicta.com.au> [Fri, 11 Sep 2009 20:58:29 +1000] rev 32749
Implement previous fix (don't duplicate ext_def) correctly.
Fri, 11 Sep 2009 18:03:30 +1000 There's no particular reason to duplicate the extension
Thomas Sewell <tsewell@nicta.com.au> [Fri, 11 Sep 2009 18:03:30 +1000] rev 32748
There's no particular reason to duplicate the extension constant's definition under the name "ext_def", and it also prevents you having a field called ext.
Fri, 11 Sep 2009 15:57:16 +1000 Merged with mainline changes.
Thomas Sewell <tsewell@nicta.com.au> [Fri, 11 Sep 2009 15:57:16 +1000] rev 32747
Merged with mainline changes.
Fri, 11 Sep 2009 15:56:51 +1000 Adjust some documentation.
Thomas Sewell <tsewell@nicta.com.au> [Fri, 11 Sep 2009 15:56:51 +1000] rev 32746
Adjust some documentation.
Thu, 10 Sep 2009 16:38:18 +1000 Simplification of various aspects of the IsTuple component
Thomas Sewell <tsewell@nicta.com.au> [Thu, 10 Sep 2009 16:38:18 +1000] rev 32745
Simplification of various aspects of the IsTuple component of the new record package. Extensive documentation added in IsTuple.thy - it should now be possible to figure out what's going on from the sources supplied.
Thu, 10 Sep 2009 15:18:43 +1000 Record patch imported and working.
Thomas Sewell <tsewell@nicta.com.au> [Thu, 10 Sep 2009 15:18:43 +1000] rev 32744
Record patch imported and working.
Thu, 27 Aug 2009 00:40:53 +1000 Initial attempt at porting record update to repository Isabelle.
tsewell@rubicon.NSW.bigpond.net.au [Thu, 27 Aug 2009 00:40:53 +1000] rev 32743
Initial attempt at porting record update to repository Isabelle.
Tue, 29 Sep 2009 16:42:29 +0200 Synchronized and Unsynchronized;
wenzelm [Tue, 29 Sep 2009 16:42:29 +0200] rev 32742
Synchronized and Unsynchronized;
Tue, 29 Sep 2009 16:42:02 +0200 hide "ref" by default, to enforce excplicit indication as Unsynchronized;
wenzelm [Tue, 29 Sep 2009 16:42:02 +0200] rev 32741
hide "ref" by default, to enforce excplicit indication as Unsynchronized;
Tue, 29 Sep 2009 16:24:36 +0200 explicit indication of Unsynchronized.ref;
wenzelm [Tue, 29 Sep 2009 16:24:36 +0200] rev 32740
explicit indication of Unsynchronized.ref;
Tue, 29 Sep 2009 14:59:24 +0200 open_unsynchronized for interactive Isar loop;
wenzelm [Tue, 29 Sep 2009 14:59:24 +0200] rev 32739
open_unsynchronized for interactive Isar loop;
Tue, 29 Sep 2009 11:49:22 +0200 explicit indication of Unsynchronized.ref;
wenzelm [Tue, 29 Sep 2009 11:49:22 +0200] rev 32738
explicit indication of Unsynchronized.ref;
Tue, 29 Sep 2009 11:48:32 +0200 Raw ML references as unsynchronized state variables.
wenzelm [Tue, 29 Sep 2009 11:48:32 +0200] rev 32737
Raw ML references as unsynchronized state variables.
Mon, 28 Sep 2009 23:51:13 +0200 Dummy version of state variables -- plain refs for sequential access.
wenzelm [Mon, 28 Sep 2009 23:51:13 +0200] rev 32736
Dummy version of state variables -- plain refs for sequential access.
Mon, 28 Sep 2009 23:19:50 +0200 reactivated at-sml-dev-e;
wenzelm [Mon, 28 Sep 2009 23:19:50 +0200] rev 32735
reactivated at-sml-dev-e;
Mon, 28 Sep 2009 23:13:37 +0200 misc tuning and modernization;
wenzelm [Mon, 28 Sep 2009 23:13:37 +0200] rev 32734
misc tuning and modernization;
Mon, 28 Sep 2009 22:47:34 +0200 moved generic cong_tac from HOL/Tools/datatype_aux.ML to Tools/cong_tac.ML, proper subgoal selection (failure, not exception);
wenzelm [Mon, 28 Sep 2009 22:47:34 +0200] rev 32733
moved generic cong_tac from HOL/Tools/datatype_aux.ML to Tools/cong_tac.ML, proper subgoal selection (failure, not exception);
Mon, 28 Sep 2009 21:35:57 +0200 merged
wenzelm [Mon, 28 Sep 2009 21:35:57 +0200] rev 32732
merged
Mon, 28 Sep 2009 15:25:43 +0200 less auxiliary functions
haftmann [Mon, 28 Sep 2009 15:25:43 +0200] rev 32731
less auxiliary functions
Mon, 28 Sep 2009 14:54:15 +0200 tuned
haftmann [Mon, 28 Sep 2009 14:54:15 +0200] rev 32730
tuned
Mon, 28 Sep 2009 14:48:30 +0200 shared code between rep_datatype and datatype
haftmann [Mon, 28 Sep 2009 14:48:30 +0200] rev 32729
shared code between rep_datatype and datatype
Mon, 28 Sep 2009 10:51:12 +0200 further unification of datatype and rep_datatype
haftmann [Mon, 28 Sep 2009 10:51:12 +0200] rev 32728
further unification of datatype and rep_datatype
Mon, 28 Sep 2009 10:20:21 +0200 avoid compound fields in datatype info record
haftmann [Mon, 28 Sep 2009 10:20:21 +0200] rev 32727
avoid compound fields in datatype info record
Mon, 28 Sep 2009 20:52:05 +0200 fold_body_thms: pass pthm identifier;
wenzelm [Mon, 28 Sep 2009 20:52:05 +0200] rev 32726
fold_body_thms: pass pthm identifier; fold_body_thms: dismiss path-etic attempt to check for cycles (cf. e24acd21e60e) -- could be masked by "seen"; fulfill_proof/thm_proof: check for thm cycles at the substitution point;
Mon, 28 Sep 2009 12:09:55 +0200 tuned internal source structure;
wenzelm [Mon, 28 Sep 2009 12:09:55 +0200] rev 32725
tuned internal source structure;
Mon, 28 Sep 2009 12:09:18 +0200 added fork_deps_pri;
wenzelm [Mon, 28 Sep 2009 12:09:18 +0200] rev 32724
added fork_deps_pri;
Mon, 28 Sep 2009 09:47:32 +0200 merged
haftmann [Mon, 28 Sep 2009 09:47:32 +0200] rev 32723
merged
Mon, 28 Sep 2009 09:47:18 +0200 explicit pointless checkpoint
haftmann [Mon, 28 Sep 2009 09:47:18 +0200] rev 32722
explicit pointless checkpoint
Sun, 27 Sep 2009 20:58:25 +0200 emerging common infrastructure for datatype and rep_datatype
haftmann [Sun, 27 Sep 2009 20:58:25 +0200] rev 32721
emerging common infrastructure for datatype and rep_datatype
Sun, 27 Sep 2009 20:43:47 +0200 streamlined rep_datatype further
haftmann [Sun, 27 Sep 2009 20:43:47 +0200] rev 32720
streamlined rep_datatype further
Sun, 27 Sep 2009 20:34:50 +0200 simplified rep_datatype
haftmann [Sun, 27 Sep 2009 20:34:50 +0200] rev 32719
simplified rep_datatype
Sun, 27 Sep 2009 20:19:56 +0200 more appropriate order of field in dt_info
haftmann [Sun, 27 Sep 2009 20:19:56 +0200] rev 32718
more appropriate order of field in dt_info
Sun, 27 Sep 2009 20:15:45 +0200 re-established reasonable inner outline for module
haftmann [Sun, 27 Sep 2009 20:15:45 +0200] rev 32717
re-established reasonable inner outline for module
Sun, 27 Sep 2009 22:25:13 +0200 merged
wenzelm [Sun, 27 Sep 2009 22:25:13 +0200] rev 32716
merged
Sun, 27 Sep 2009 19:58:24 +0200 adjusted to changes in datatype package
haftmann [Sun, 27 Sep 2009 19:58:24 +0200] rev 32715
adjusted to changes in datatype package
Sun, 27 Sep 2009 10:05:17 +0200 merged
haftmann [Sun, 27 Sep 2009 10:05:17 +0200] rev 32714
merged
Sun, 27 Sep 2009 09:52:25 +0200 dropped dead code
haftmann [Sun, 27 Sep 2009 09:52:25 +0200] rev 32713
dropped dead code
Sun, 27 Sep 2009 09:52:23 +0200 registering split rules and projected induction rules; ML identifiers more close to Isar theorem names
haftmann [Sun, 27 Sep 2009 09:52:23 +0200] rev 32712
registering split rules and projected induction rules; ML identifiers more close to Isar theorem names
Sun, 27 Sep 2009 21:08:13 +0200 fold_body_thms/join_bodies: explicitly check for cyclic theorem references;
wenzelm [Sun, 27 Sep 2009 21:08:13 +0200] rev 32711
fold_body_thms/join_bodies: explicitly check for cyclic theorem references;
Sun, 27 Sep 2009 21:06:43 +0200 tuned;
wenzelm [Sun, 27 Sep 2009 21:06:43 +0200] rev 32710
tuned;
Sun, 27 Sep 2009 19:39:40 +0200 reachable: recovered reverse post-order (lost in 73ad4884441f), which is expected for all_preds/all_succs and required for topological_order;
wenzelm [Sun, 27 Sep 2009 19:39:40 +0200] rev 32709
reachable: recovered reverse post-order (lost in 73ad4884441f), which is expected for all_preds/all_succs and required for topological_order;
Fri, 25 Sep 2009 13:48:27 +0100 merged
paulson [Fri, 25 Sep 2009 13:48:27 +0100] rev 32708
merged
Fri, 25 Sep 2009 13:47:28 +0100 New lemmas involving the real numbers, especially limits and series
paulson [Fri, 25 Sep 2009 13:47:28 +0100] rev 32707
New lemmas involving the real numbers, especially limits and series
Fri, 25 Sep 2009 10:20:03 +0200 NEWS; corrected spelling
haftmann [Fri, 25 Sep 2009 10:20:03 +0200] rev 32706
NEWS; corrected spelling
Fri, 25 Sep 2009 09:50:31 +0200 merged
haftmann [Fri, 25 Sep 2009 09:50:31 +0200] rev 32705
merged
Wed, 23 Sep 2009 16:32:53 +0200 simplified proof
haftmann [Wed, 23 Sep 2009 16:32:53 +0200] rev 32704
simplified proof
Wed, 23 Sep 2009 16:32:53 +0200 removed potentially dangerous rules from pred_set_conv
haftmann [Wed, 23 Sep 2009 16:32:53 +0200] rev 32703
removed potentially dangerous rules from pred_set_conv
Wed, 23 Sep 2009 16:32:53 +0200 explicitly hide empty, inter, union
haftmann [Wed, 23 Sep 2009 16:32:53 +0200] rev 32702
explicitly hide empty, inter, union
Wed, 23 Sep 2009 14:00:43 +0200 merged
haftmann [Wed, 23 Sep 2009 14:00:43 +0200] rev 32701
merged
Wed, 23 Sep 2009 11:34:21 +0200 merged
haftmann [Wed, 23 Sep 2009 11:34:21 +0200] rev 32700
merged
Wed, 23 Sep 2009 08:26:12 +0200 merged
haftmann [Wed, 23 Sep 2009 08:26:12 +0200] rev 32699
merged
Wed, 23 Sep 2009 08:25:51 +0200 inf/sup_absorb are no default simp rules any longer
haftmann [Wed, 23 Sep 2009 08:25:51 +0200] rev 32698
inf/sup_absorb are no default simp rules any longer
Tue, 22 Sep 2009 15:39:46 +0200 merged
haftmann [Tue, 22 Sep 2009 15:39:46 +0200] rev 32697
merged
Mon, 21 Sep 2009 16:02:00 +0200 merged
haftmann [Mon, 21 Sep 2009 16:02:00 +0200] rev 32696
merged
Mon, 21 Sep 2009 15:56:15 +0200 adapted proof
haftmann [Mon, 21 Sep 2009 15:56:15 +0200] rev 32695
adapted proof
Mon, 21 Sep 2009 15:35:24 +0200 merged
haftmann [Mon, 21 Sep 2009 15:35:24 +0200] rev 32694
merged
Mon, 21 Sep 2009 15:35:15 +0200 tuned proofs
haftmann [Mon, 21 Sep 2009 15:35:15 +0200] rev 32693
tuned proofs
Mon, 21 Sep 2009 15:35:14 +0200 tuned header
haftmann [Mon, 21 Sep 2009 15:35:14 +0200] rev 32692
tuned header
Mon, 21 Sep 2009 15:35:14 +0200 added note on simp rules
haftmann [Mon, 21 Sep 2009 15:35:14 +0200] rev 32691
added note on simp rules
Mon, 21 Sep 2009 14:23:12 +0200 merged
haftmann [Mon, 21 Sep 2009 14:23:12 +0200] rev 32690
merged
Mon, 21 Sep 2009 14:23:04 +0200 tuned proof; tuned headers
haftmann [Mon, 21 Sep 2009 14:23:04 +0200] rev 32689
tuned proof; tuned headers
Mon, 21 Sep 2009 12:24:21 +0200 merged
haftmann [Mon, 21 Sep 2009 12:24:21 +0200] rev 32688
merged
Mon, 21 Sep 2009 12:23:52 +0200 tuned proofs; be more cautios wrt. default simp rules
haftmann [Mon, 21 Sep 2009 12:23:52 +0200] rev 32687
tuned proofs; be more cautios wrt. default simp rules
Mon, 21 Sep 2009 11:01:49 +0200 merged
haftmann [Mon, 21 Sep 2009 11:01:49 +0200] rev 32686
merged
Mon, 21 Sep 2009 11:01:39 +0200 tuned proofs
haftmann [Mon, 21 Sep 2009 11:01:39 +0200] rev 32685
tuned proofs
Sat, 19 Sep 2009 07:38:11 +0200 merged
haftmann [Sat, 19 Sep 2009 07:38:11 +0200] rev 32684
merged
Sat, 19 Sep 2009 07:38:03 +0200 inter and union are mere abbreviations for inf and sup
haftmann [Sat, 19 Sep 2009 07:38:03 +0200] rev 32683
inter and union are mere abbreviations for inf and sup
Thu, 24 Sep 2009 19:14:18 +0200 merged
haftmann [Thu, 24 Sep 2009 19:14:18 +0200] rev 32682
merged
Thu, 24 Sep 2009 18:29:29 +0200 lemma relating fold1 and foldl; code_unfold rules for Inf_fin, Sup_fin, Min, Max, Inf, Sup
haftmann [Thu, 24 Sep 2009 18:29:29 +0200] rev 32681
lemma relating fold1 and foldl; code_unfold rules for Inf_fin, Sup_fin, Min, Max, Inf, Sup
Thu, 24 Sep 2009 18:29:29 +0200 subsumed by more general setup in List.thy
haftmann [Thu, 24 Sep 2009 18:29:29 +0200] rev 32680
subsumed by more general setup in List.thy
Thu, 24 Sep 2009 18:29:29 +0200 idempotency case for fold1
haftmann [Thu, 24 Sep 2009 18:29:29 +0200] rev 32679
idempotency case for fold1
Thu, 24 Sep 2009 18:29:28 +0200 added dual for complete lattice
haftmann [Thu, 24 Sep 2009 18:29:28 +0200] rev 32678
added dual for complete lattice
Thu, 24 Sep 2009 17:26:05 +0200 merged
nipkow [Thu, 24 Sep 2009 17:26:05 +0200] rev 32677
merged
Thu, 24 Sep 2009 17:25:42 +0200 record how many "proof"s are solved by s/h
nipkow [Thu, 24 Sep 2009 17:25:42 +0200] rev 32676
record how many "proof"s are solved by s/h
Thu, 24 Sep 2009 15:00:17 +0200 added quotes for filenames;
boehmes [Thu, 24 Sep 2009 15:00:17 +0200] rev 32675
added quotes for filenames; truncated remaining time (no floats supported by ulimit)
Thu, 24 Sep 2009 08:28:27 +0200 merged; adopted to changes from Code_Evaluation in the predicate compiler
bulwahn [Thu, 24 Sep 2009 08:28:27 +0200] rev 32674
merged; adopted to changes from Code_Evaluation in the predicate compiler
(0) -30000 -10000 -3000 -1000 -300 -100 -96 +96 +100 +300 +1000 +3000 +10000 +30000 tip