Tue, 09 Mar 2010 14:55:25 +0100 tuned -- eliminated Sign.intern_sort;
wenzelm [Tue, 09 Mar 2010 14:55:25 +0100] rev 35667
tuned -- eliminated Sign.intern_sort;
Tue, 09 Mar 2010 14:18:06 +0100 renamed mk_const_def to legacy_const_def, because of slightly odd Sign.intern_term;
wenzelm [Tue, 09 Mar 2010 14:18:06 +0100] rev 35666
renamed mk_const_def to legacy_const_def, because of slightly odd Sign.intern_term;
Tue, 09 Mar 2010 09:25:23 +0100 added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet [Tue, 09 Mar 2010 09:25:23 +0100] rev 35665
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
Mon, 08 Mar 2010 15:20:40 -0800 merged
huffman [Mon, 08 Mar 2010 15:20:40 -0800] rev 35664
merged
Mon, 08 Mar 2010 14:42:40 -0800 remove unnecessary error handling code
huffman [Mon, 08 Mar 2010 14:42:40 -0800] rev 35663
remove unnecessary error handling code
Mon, 08 Mar 2010 14:12:51 -0800 construct fully typed goal in proof of induction rule
huffman [Mon, 08 Mar 2010 14:12:51 -0800] rev 35662
construct fully typed goal in proof of induction rule
Mon, 08 Mar 2010 13:58:00 -0800 don't generate rule foo.finites for non-flat domains; use take_induct rule to prove induction rule
huffman [Mon, 08 Mar 2010 13:58:00 -0800] rev 35661
don't generate rule foo.finites for non-flat domains; use take_induct rule to prove induction rule
Mon, 08 Mar 2010 12:43:44 -0800 remove redundant function arguments
huffman [Mon, 08 Mar 2010 12:43:44 -0800] rev 35660
remove redundant function arguments
Mon, 08 Mar 2010 12:36:26 -0800 include take_info within take_induct_info type
huffman [Mon, 08 Mar 2010 12:36:26 -0800] rev 35659
include take_info within take_induct_info type
Mon, 08 Mar 2010 12:21:07 -0800 pass take_info as an argument to comp_theorems
huffman [Mon, 08 Mar 2010 12:21:07 -0800] rev 35658
pass take_info as an argument to comp_theorems
Mon, 08 Mar 2010 11:58:40 -0800 pass take_induct_info as an argument to comp_theorems
huffman [Mon, 08 Mar 2010 11:58:40 -0800] rev 35657
pass take_induct_info as an argument to comp_theorems
Mon, 08 Mar 2010 11:48:29 -0800 add type take_induct_info
huffman [Mon, 08 Mar 2010 11:48:29 -0800] rev 35656
add type take_induct_info
Mon, 08 Mar 2010 11:34:53 -0800 generate take_induct lemmas
huffman [Mon, 08 Mar 2010 11:34:53 -0800] rev 35655
generate take_induct lemmas
Mon, 08 Mar 2010 09:37:03 -0800 move proofs of reach and take lemmas to domain_take_proofs.ML
huffman [Mon, 08 Mar 2010 09:37:03 -0800] rev 35654
move proofs of reach and take lemmas to domain_take_proofs.ML
Mon, 08 Mar 2010 09:33:05 -0800 move lemmas from Domain.thy to Domain_Aux.thy
huffman [Mon, 08 Mar 2010 09:33:05 -0800] rev 35653
move lemmas from Domain.thy to Domain_Aux.thy
Mon, 08 Mar 2010 08:12:48 -0800 move take-proofs stuff into new theory Domain_Aux.thy
huffman [Mon, 08 Mar 2010 08:12:48 -0800] rev 35652
move take-proofs stuff into new theory Domain_Aux.thy
Mon, 08 Mar 2010 07:37:11 -0800 add type take_info
huffman [Mon, 08 Mar 2010 07:37:11 -0800] rev 35651
add type take_info
Mon, 08 Mar 2010 07:22:30 -0800 add function add_qualified_def
huffman [Mon, 08 Mar 2010 07:22:30 -0800] rev 35650
add function add_qualified_def
Mon, 08 Mar 2010 17:37:09 +0100 merged
haftmann [Mon, 08 Mar 2010 17:37:09 +0100] rev 35649
merged
Mon, 08 Mar 2010 14:41:56 +0100 proper ML interface; further polishing
haftmann [Mon, 08 Mar 2010 14:41:56 +0100] rev 35648
proper ML interface; further polishing
Mon, 08 Mar 2010 13:22:41 +0100 code simplification and tuning
haftmann [Mon, 08 Mar 2010 13:22:41 +0100] rev 35647
code simplification and tuning
Mon, 08 Mar 2010 15:00:34 +0100 Added inducts field to inductive_result.
berghofe [Mon, 08 Mar 2010 15:00:34 +0100] rev 35646
Added inducts field to inductive_result.
Mon, 08 Mar 2010 09:38:59 +0100 transfer: avoid camel case, more standard coding conventions, misc tuning
haftmann [Mon, 08 Mar 2010 09:38:59 +0100] rev 35645
transfer: avoid camel case, more standard coding conventions, misc tuning
Mon, 08 Mar 2010 09:38:58 +0100 transfer: avoid camel case
haftmann [Mon, 08 Mar 2010 09:38:58 +0100] rev 35644
transfer: avoid camel case
Sun, 07 Mar 2010 17:33:01 -0800 merged
huffman [Sun, 07 Mar 2010 17:33:01 -0800] rev 35643
merged
Sun, 07 Mar 2010 16:39:31 -0800 generate separate qualified theorem name for each type's reach and take_lemma
huffman [Sun, 07 Mar 2010 16:39:31 -0800] rev 35642
generate separate qualified theorem name for each type's reach and take_lemma
Sun, 07 Mar 2010 16:12:01 -0800 add simp rule LAM_strict
huffman [Sun, 07 Mar 2010 16:12:01 -0800] rev 35641
add simp rule LAM_strict
Sun, 07 Mar 2010 13:34:53 -0800 fix bug that occurred with 'domain_isomorphism foo = foo * tr * tr'
huffman [Sun, 07 Mar 2010 13:34:53 -0800] rev 35640
fix bug that occurred with 'domain_isomorphism foo = foo * tr * tr'
Sun, 07 Mar 2010 22:36:36 +0100 merged
haftmann [Sun, 07 Mar 2010 22:36:36 +0100] rev 35639
merged
Sun, 07 Mar 2010 08:46:12 +0100 dropped dead code; adhere more closely to standard coding conventions
haftmann [Sun, 07 Mar 2010 08:46:12 +0100] rev 35638
dropped dead code; adhere more closely to standard coding conventions
Sun, 07 Mar 2010 10:03:16 -0800 merged
huffman [Sun, 07 Mar 2010 10:03:16 -0800] rev 35637
merged
Sun, 07 Mar 2010 09:57:30 -0800 arith tactic uses 'priority' instead of 'warning' to print messages
huffman [Sun, 07 Mar 2010 09:57:30 -0800] rev 35636
arith tactic uses 'priority' instead of 'warning' to print messages
Sun, 07 Mar 2010 09:21:16 -0800 add simp rules about Ints, Nats
huffman [Sun, 07 Mar 2010 09:21:16 -0800] rev 35635
add simp rules about Ints, Nats
Sun, 07 Mar 2010 08:40:38 -0800 add more simp rules for Ints
huffman [Sun, 07 Mar 2010 08:40:38 -0800] rev 35634
add more simp rules for Ints
Sun, 07 Mar 2010 07:42:46 -0800 add lemmas Nats_cases and Nats_induct
huffman [Sun, 07 Mar 2010 07:42:46 -0800] rev 35633
add lemmas Nats_cases and Nats_induct
Sun, 07 Mar 2010 07:29:34 -0800 generalize some lemmas, and remove a few unnecessary ones
huffman [Sun, 07 Mar 2010 07:29:34 -0800] rev 35632
generalize some lemmas, and remove a few unnecessary ones
Sat, 06 Mar 2010 18:24:30 -0800 generalize some lemmas from class linordered_ring_strict to linordered_ring
huffman [Sat, 06 Mar 2010 18:24:30 -0800] rev 35631
generalize some lemmas from class linordered_ring_strict to linordered_ring
Sat, 06 Mar 2010 16:02:22 -0800 add case_names attribute to casedist and ind rules
huffman [Sat, 06 Mar 2010 16:02:22 -0800] rev 35630
add case_names attribute to casedist and ind rules
Sat, 06 Mar 2010 08:08:30 -0800 add some lemmas about complete lattices
huffman [Sat, 06 Mar 2010 08:08:30 -0800] rev 35629
add some lemmas about complete lattices
Sun, 07 Mar 2010 15:51:29 +0100 Digesting strings according to SHA-1.
wenzelm [Sun, 07 Mar 2010 15:51:29 +0100] rev 35628
Digesting strings according to SHA-1.
Sun, 07 Mar 2010 15:49:49 +0100 proper int wrapping for Word32;
wenzelm [Sun, 07 Mar 2010 15:49:49 +0100] rev 35627
proper int wrapping for Word32;
Sun, 07 Mar 2010 12:47:02 +0100 separate structure Typedecl;
wenzelm [Sun, 07 Mar 2010 12:47:02 +0100] rev 35626
separate structure Typedecl;
Sun, 07 Mar 2010 12:19:47 +0100 modernized structure Object_Logic;
wenzelm [Sun, 07 Mar 2010 12:19:47 +0100] rev 35625
modernized structure Object_Logic;
Sun, 07 Mar 2010 11:57:16 +0100 modernized structure Local_Defs;
wenzelm [Sun, 07 Mar 2010 11:57:16 +0100] rev 35624
modernized structure Local_Defs;
Sat, 06 Mar 2010 19:17:59 +0000 merged
paulson [Sat, 06 Mar 2010 19:17:59 +0000] rev 35623
merged
Sat, 06 Mar 2010 17:21:59 +0000 merged
paulson [Sat, 06 Mar 2010 17:21:59 +0000] rev 35622
merged
Sat, 06 Mar 2010 17:19:29 +0000 simplified
paulson [Sat, 06 Mar 2010 17:19:29 +0000] rev 35621
simplified
Sat, 06 Mar 2010 20:16:31 +0100 merged
haftmann [Sat, 06 Mar 2010 20:16:31 +0100] rev 35620
merged
Sat, 06 Mar 2010 15:31:31 +0100 lemma restrict_complement_singleton_eq
haftmann [Sat, 06 Mar 2010 15:31:31 +0100] rev 35619
lemma restrict_complement_singleton_eq
Sat, 06 Mar 2010 15:31:30 +0100 some lemma refinements
haftmann [Sat, 06 Mar 2010 15:31:30 +0100] rev 35618
some lemma refinements
Sat, 06 Mar 2010 15:31:30 +0100 added Table.thy
haftmann [Sat, 06 Mar 2010 15:31:30 +0100] rev 35617
added Table.thy
Sat, 06 Mar 2010 17:53:04 +0100 provide ProofContext.def_type depending on "pattern" mode;
wenzelm [Sat, 06 Mar 2010 17:53:04 +0100] rev 35616
provide ProofContext.def_type depending on "pattern" mode;
Sat, 06 Mar 2010 17:32:45 +0100 record_type_tr': more robust strip_fields (printed types are not necessarily well-formed, e.g. in Syntax.pretty_arity);
wenzelm [Sat, 06 Mar 2010 17:32:45 +0100] rev 35615
record_type_tr': more robust strip_fields (printed types are not necessarily well-formed, e.g. in Syntax.pretty_arity);
Sat, 06 Mar 2010 16:13:22 +0100 record_type_abbr_tr': removed obsolete workaround for decode_type, which now retains syntactic categories of variables vs. constructors (authentic syntax);
wenzelm [Sat, 06 Mar 2010 16:13:22 +0100] rev 35614
record_type_abbr_tr': removed obsolete workaround for decode_type, which now retains syntactic categories of variables vs. constructors (authentic syntax);
Sat, 06 Mar 2010 15:39:16 +0100 eliminated Args.bang_facts (legacy feature);
wenzelm [Sat, 06 Mar 2010 15:39:16 +0100] rev 35613
eliminated Args.bang_facts (legacy feature);
Sat, 06 Mar 2010 15:34:29 +0100 eliminated old-style prems;
wenzelm [Sat, 06 Mar 2010 15:34:29 +0100] rev 35612
eliminated old-style prems; tuned proofs;
Sat, 06 Mar 2010 14:35:06 +0100 removed unused term_lift_inst_rule (superceded by Subgoal.FOCUS etc.);
wenzelm [Sat, 06 Mar 2010 14:35:06 +0100] rev 35611
removed unused term_lift_inst_rule (superceded by Subgoal.FOCUS etc.);
Sat, 06 Mar 2010 14:28:31 +0100 Some notes on platform support of Isabelle.
wenzelm [Sat, 06 Mar 2010 14:28:31 +0100] rev 35610
Some notes on platform support of Isabelle.
Sat, 06 Mar 2010 11:21:09 +0100 "private" map_of_map lemma
haftmann [Sat, 06 Mar 2010 11:21:09 +0100] rev 35609
"private" map_of_map lemma
Sat, 06 Mar 2010 09:58:33 +0100 added insort_insert
haftmann [Sat, 06 Mar 2010 09:58:33 +0100] rev 35608
added insort_insert
(0) -30000 -10000 -3000 -1000 -300 -100 -60 +60 +100 +300 +1000 +3000 +10000 +30000 tip