Wed, 30 Sep 2009 08:21:53 +0200 haftmann tuned whitespace
Wed, 30 Sep 2009 00:57:28 +0200 wenzelm replaced chained_goal by slightly more appropriate flat_goal;
Wed, 30 Sep 2009 00:27:19 +0200 wenzelm made SML/NJ happy;
Wed, 30 Sep 2009 00:17:06 +0200 wenzelm added chained_goal, which presents the goal thm as seen by semi-structured methods;
Tue, 29 Sep 2009 23:19:26 +0200 wenzelm tuned;
Tue, 29 Sep 2009 23:14:57 +0200 wenzelm removed dead/duplicate code;
Tue, 29 Sep 2009 22:53:07 +0200 wenzelm aliases for Thomas Sewell;
Tue, 29 Sep 2009 22:48:24 +0200 wenzelm modernized Balanced_Tree;
Tue, 29 Sep 2009 22:33:27 +0200 wenzelm replaced meta_iffD2 by existing Drule.equal_elim_rule2;
Tue, 29 Sep 2009 21:36:49 +0200 wenzelm tuned header;
Tue, 29 Sep 2009 21:36:33 +0200 wenzelm Thomas Sewell, NICTA: more efficient HOL/record implementation;
Tue, 29 Sep 2009 21:34:59 +0200 wenzelm tuned whitespace -- recover basic Isabelle conventions;
Tue, 29 Sep 2009 18:14:08 +0200 wenzelm merged
Tue, 29 Sep 2009 14:26:33 +1000 Thomas Sewell Merge with isabelle dev changes.
Tue, 29 Sep 2009 14:25:42 +1000 Thomas Sewell Replace OldTerm.term_vars with Term.add_vars in named_cterm_instantiate.
Mon, 28 Sep 2009 15:37:19 +1000 Thomas Sewell Avoid a possible variable name conflict in instantiating a theorem.
Mon, 28 Sep 2009 14:16:01 +1000 Thomas Sewell Fix unescaped expressions breaking latex output in Record.thy
Mon, 28 Sep 2009 11:13:11 +1000 Thomas Sewell Merge record patch with updates from isabelle mainline.
Fri, 25 Sep 2009 19:04:18 +1000 Thomas Sewell Avoid record-inner constants in polymorphic definitions in Bali
Thu, 24 Sep 2009 11:33:05 +1000 Thomas Sewell Merge with changes from isabelle dev repository.
Wed, 23 Sep 2009 19:17:48 +1000 tsewell Initial response to feedback from Norbert, Makarius on record patch
Tue, 22 Sep 2009 13:52:19 +1000 Thomas Sewell Branch merge for isabelle mainline updates.
Thu, 17 Sep 2009 14:17:37 +1000 Thomas Sewell Branch merge with updates from mainline isabelle.
Fri, 11 Sep 2009 20:58:29 +1000 Thomas Sewell Implement previous fix (don't duplicate ext_def) correctly.
Fri, 11 Sep 2009 18:03:30 +1000 Thomas Sewell There's no particular reason to duplicate the extension
Fri, 11 Sep 2009 15:57:16 +1000 Thomas Sewell Merged with mainline changes.
Fri, 11 Sep 2009 15:56:51 +1000 Thomas Sewell Adjust some documentation.
Thu, 10 Sep 2009 16:38:18 +1000 Thomas Sewell Simplification of various aspects of the IsTuple component
Thu, 10 Sep 2009 15:18:43 +1000 Thomas Sewell Record patch imported and working.
Thu, 27 Aug 2009 00:40:53 +1000 tsewell Initial attempt at porting record update to repository Isabelle.
Tue, 29 Sep 2009 16:42:29 +0200 wenzelm Synchronized and Unsynchronized;
Tue, 29 Sep 2009 16:42:02 +0200 wenzelm hide "ref" by default, to enforce excplicit indication as Unsynchronized;
Tue, 29 Sep 2009 16:24:36 +0200 wenzelm explicit indication of Unsynchronized.ref;
Tue, 29 Sep 2009 14:59:24 +0200 wenzelm open_unsynchronized for interactive Isar loop;
Tue, 29 Sep 2009 11:49:22 +0200 wenzelm explicit indication of Unsynchronized.ref;
Tue, 29 Sep 2009 11:48:32 +0200 wenzelm Raw ML references as unsynchronized state variables.
Mon, 28 Sep 2009 23:51:13 +0200 wenzelm Dummy version of state variables -- plain refs for sequential access.
Mon, 28 Sep 2009 23:19:50 +0200 wenzelm reactivated at-sml-dev-e;
Mon, 28 Sep 2009 23:13:37 +0200 wenzelm misc tuning and modernization;
Mon, 28 Sep 2009 22:47:34 +0200 wenzelm 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 wenzelm merged
Mon, 28 Sep 2009 15:25:43 +0200 haftmann less auxiliary functions
Mon, 28 Sep 2009 14:54:15 +0200 haftmann tuned
Mon, 28 Sep 2009 14:48:30 +0200 haftmann shared code between rep_datatype and datatype
Mon, 28 Sep 2009 10:51:12 +0200 haftmann further unification of datatype and rep_datatype
Mon, 28 Sep 2009 10:20:21 +0200 haftmann avoid compound fields in datatype info record
Mon, 28 Sep 2009 20:52:05 +0200 wenzelm fold_body_thms: pass pthm identifier;
Mon, 28 Sep 2009 12:09:55 +0200 wenzelm tuned internal source structure;
Mon, 28 Sep 2009 12:09:18 +0200 wenzelm added fork_deps_pri;
Mon, 28 Sep 2009 09:47:32 +0200 haftmann merged
Mon, 28 Sep 2009 09:47:18 +0200 haftmann explicit pointless checkpoint
Sun, 27 Sep 2009 20:58:25 +0200 haftmann emerging common infrastructure for datatype and rep_datatype
Sun, 27 Sep 2009 20:43:47 +0200 haftmann streamlined rep_datatype further
Sun, 27 Sep 2009 20:34:50 +0200 haftmann simplified rep_datatype
Sun, 27 Sep 2009 20:19:56 +0200 haftmann more appropriate order of field in dt_info
Sun, 27 Sep 2009 20:15:45 +0200 haftmann re-established reasonable inner outline for module
Sun, 27 Sep 2009 22:25:13 +0200 wenzelm merged
Sun, 27 Sep 2009 19:58:24 +0200 haftmann adjusted to changes in datatype package
Sun, 27 Sep 2009 10:05:17 +0200 haftmann merged
Sun, 27 Sep 2009 09:52:25 +0200 haftmann dropped dead code
Sun, 27 Sep 2009 09:52:23 +0200 haftmann registering split rules and projected induction rules; ML identifiers more close to Isar theorem names
Sun, 27 Sep 2009 21:08:13 +0200 wenzelm fold_body_thms/join_bodies: explicitly check for cyclic theorem references;
Sun, 27 Sep 2009 21:06:43 +0200 wenzelm tuned;
Sun, 27 Sep 2009 19:39:40 +0200 wenzelm 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 paulson merged
Fri, 25 Sep 2009 13:47:28 +0100 paulson New lemmas involving the real numbers, especially limits and series
Fri, 25 Sep 2009 10:20:03 +0200 haftmann NEWS; corrected spelling
Fri, 25 Sep 2009 09:50:31 +0200 haftmann merged
Wed, 23 Sep 2009 16:32:53 +0200 haftmann simplified proof
Wed, 23 Sep 2009 16:32:53 +0200 haftmann removed potentially dangerous rules from pred_set_conv
Wed, 23 Sep 2009 16:32:53 +0200 haftmann explicitly hide empty, inter, union
Wed, 23 Sep 2009 14:00:43 +0200 haftmann merged
Wed, 23 Sep 2009 11:34:21 +0200 haftmann merged
Wed, 23 Sep 2009 08:26:12 +0200 haftmann merged
Wed, 23 Sep 2009 08:25:51 +0200 haftmann inf/sup_absorb are no default simp rules any longer
Tue, 22 Sep 2009 15:39:46 +0200 haftmann merged
Mon, 21 Sep 2009 16:02:00 +0200 haftmann merged
Mon, 21 Sep 2009 15:56:15 +0200 haftmann adapted proof
Mon, 21 Sep 2009 15:35:24 +0200 haftmann merged
Mon, 21 Sep 2009 15:35:15 +0200 haftmann tuned proofs
Mon, 21 Sep 2009 15:35:14 +0200 haftmann tuned header
Mon, 21 Sep 2009 15:35:14 +0200 haftmann added note on simp rules
Mon, 21 Sep 2009 14:23:12 +0200 haftmann merged
Mon, 21 Sep 2009 14:23:04 +0200 haftmann tuned proof; tuned headers
Mon, 21 Sep 2009 12:24:21 +0200 haftmann merged
Mon, 21 Sep 2009 12:23:52 +0200 haftmann tuned proofs; be more cautios wrt. default simp rules
Mon, 21 Sep 2009 11:01:49 +0200 haftmann merged
Mon, 21 Sep 2009 11:01:39 +0200 haftmann tuned proofs
Sat, 19 Sep 2009 07:38:11 +0200 haftmann merged
Sat, 19 Sep 2009 07:38:03 +0200 haftmann inter and union are mere abbreviations for inf and sup
Thu, 24 Sep 2009 19:14:18 +0200 haftmann merged
Thu, 24 Sep 2009 18:29:29 +0200 haftmann 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 haftmann subsumed by more general setup in List.thy
Thu, 24 Sep 2009 18:29:29 +0200 haftmann idempotency case for fold1
Thu, 24 Sep 2009 18:29:28 +0200 haftmann added dual for complete lattice
Thu, 24 Sep 2009 17:26:05 +0200 nipkow merged
Thu, 24 Sep 2009 17:25:42 +0200 nipkow record how many "proof"s are solved by s/h
Thu, 24 Sep 2009 15:00:17 +0200 boehmes added quotes for filenames;
Thu, 24 Sep 2009 08:28:27 +0200 bulwahn merged; adopted to changes from Code_Evaluation in the predicate compiler
Wed, 23 Sep 2009 16:20:13 +0200 bulwahn replaced sorry by oops; removed old debug functions in predicate compiler
Wed, 23 Sep 2009 16:20:13 +0200 bulwahn added first version of quickcheck based on the predicate compiler; added a few quickcheck examples
Wed, 23 Sep 2009 16:20:12 +0200 bulwahn adapted configuration for DatatypeCase.make_case
Wed, 23 Sep 2009 16:20:12 +0200 bulwahn added a new example for the predicate compiler
Wed, 23 Sep 2009 16:20:12 +0200 bulwahn added context free grammar example; removed dead code; adapted to work without quick and dirty mode; fixed typo
Wed, 23 Sep 2009 16:20:12 +0200 bulwahn added first prototype of the extended predicate compiler
Wed, 23 Sep 2009 16:20:12 +0200 bulwahn moved predicate compiler to Tools
Wed, 23 Sep 2009 16:20:12 +0200 bulwahn removed generation of strange tuple modes in predicate compiler
Wed, 23 Sep 2009 16:20:12 +0200 bulwahn extending predicate compiler and proof procedure to support tuples; testing predicate wirh HOL-MicroJava semantics
Wed, 23 Sep 2009 16:20:12 +0200 bulwahn modified predicate compiler further to support tuples
Wed, 23 Sep 2009 16:20:12 +0200 bulwahn changed preprocessing due to problems with LightweightJava; added transfer of thereoms; changed the type of mode to support tuples in the predicate compiler
Wed, 23 Sep 2009 16:20:12 +0200 bulwahn handling of definitions
Wed, 23 Sep 2009 16:20:12 +0200 bulwahn experimenting to add some useful interface for definitions
Wed, 23 Sep 2009 16:20:12 +0200 bulwahn added predicate compile preprocessing structure for definitional thms -- probably is replaced by hooking the theorem command differently
Wed, 23 Sep 2009 16:20:12 +0200 bulwahn modified handling of side conditions in proof procedure of predicate compiler
Wed, 23 Sep 2009 15:25:25 +0200 haftmann merged
Wed, 23 Sep 2009 14:00:12 +0200 haftmann Code_Eval(uation)
Wed, 23 Sep 2009 13:48:16 +0200 blanchet merged
Wed, 23 Sep 2009 13:47:08 +0200 blanchet Added "nitpick_const_simp" tags to lazy list theories.
Wed, 23 Sep 2009 13:48:35 +0200 krauss atbroy101 is long dead, use atbroy99; comment out broken SML test invocation
Wed, 23 Sep 2009 13:42:53 +0200 haftmann merged
(0) -30000 -10000 -3000 -1000 -120 +120 +1000 +3000 +10000 +30000 tip