hoelzl [Fri, 12 Mar 2010 16:02:42 +0100] rev 35753
merged
himmelma [Tue, 09 Mar 2010 15:42:23 +0100] rev 35752
reset smt_certificates
himmelma [Tue, 09 Mar 2010 15:39:26 +0100] rev 35751
added lemmas
nipkow [Fri, 12 Mar 2010 15:48:37 +0100] rev 35750
merged
nipkow [Fri, 12 Mar 2010 15:48:18 +0100] rev 35749
Added Hoare_Op.thy
hoelzl [Fri, 12 Mar 2010 15:35:41 +0100] rev 35748
Equality of integral and infinite sum.
blanchet [Fri, 12 Mar 2010 12:02:22 +0100] rev 35747
make tests less demanding, to prevent sporadic failures
wenzelm [Sat, 13 Mar 2010 15:12:56 +0100] rev 35746
more antiquotations;
wenzelm [Sat, 13 Mar 2010 15:12:47 +0100] rev 35745
command 'typedef' now works within a local theory context;
wenzelm [Sat, 13 Mar 2010 15:12:17 +0100] rev 35744
removed obsolete HOL 'typedecl';
local theory version of HOL 'typedef';
wenzelm [Sat, 13 Mar 2010 14:44:47 +0100] rev 35743
adapted to localized typedef: handle single global interpretation only;
wenzelm [Sat, 13 Mar 2010 14:43:04 +0100] rev 35742
global typedef;
wenzelm [Sat, 13 Mar 2010 14:42:16 +0100] rev 35741
localized typedef;
Typedef.get_info can yield multiple typedef interpretations, even in a global context;
misc tuning and modernization;
wenzelm [Sat, 13 Mar 2010 14:41:37 +0100] rev 35740
added typedecl_wrt, which affects default sorts of type args;
misc tuning and simplification;
wenzelm [Sat, 13 Mar 2010 14:41:14 +0100] rev 35739
Local_Defs.contract convenience;
wenzelm [Sat, 13 Mar 2010 14:40:36 +0100] rev 35738
added Local_Theory.alias operations (independent of target);
wenzelm [Thu, 11 Mar 2010 23:47:16 +0100] rev 35737
merged
nipkow [Thu, 11 Mar 2010 19:06:03 +0100] rev 35736
merged
nipkow [Thu, 11 Mar 2010 19:05:46 +0100] rev 35735
converted proofs to Isar
haftmann [Thu, 11 Mar 2010 17:52:15 +0100] rev 35734
merged
haftmann [Thu, 11 Mar 2010 17:39:45 +0100] rev 35733
merged
haftmann [Thu, 11 Mar 2010 15:52:35 +0100] rev 35732
tuned prefix of ac rules
haftmann [Thu, 11 Mar 2010 15:52:35 +0100] rev 35731
deleted default simp rule card.insert
haftmann [Thu, 11 Mar 2010 15:52:34 +0100] rev 35730
updated generated certificate
haftmann [Thu, 11 Mar 2010 15:52:34 +0100] rev 35729
replaced card_def by card_eq_setsum
haftmann [Thu, 11 Mar 2010 15:52:33 +0100] rev 35728
NEWS
haftmann [Thu, 11 Mar 2010 14:40:29 +0100] rev 35727
Big_Operators now in Main rather than Plain
haftmann [Thu, 11 Mar 2010 14:39:58 +0100] rev 35726
tuned prefixes of ac interpretations
haftmann [Thu, 11 Mar 2010 14:39:58 +0100] rev 35725
Big_Operators now in Main rather than Plain src/HOL/Wellfounded.thy
haftmann [Thu, 11 Mar 2010 14:38:20 +0100] rev 35724
fixed typo
haftmann [Thu, 11 Mar 2010 14:38:19 +0100] rev 35723
tuned monoid locales and prefix of sublocale interpretations
haftmann [Thu, 11 Mar 2010 14:38:13 +0100] rev 35722
moved cardinality to Finite_Set as far as appropriate; added locales for fold_image
haftmann [Thu, 11 Mar 2010 14:38:09 +0100] rev 35721
fixed typo
haftmann [Wed, 10 Mar 2010 16:53:43 +0100] rev 35720
added locales for monoids
haftmann [Wed, 10 Mar 2010 16:53:27 +0100] rev 35719
split off theory Big_Operators from theory Finite_Set
blanchet [Thu, 11 Mar 2010 17:48:07 +0100] rev 35718
moved some Nitpick code around
wenzelm [Thu, 11 Mar 2010 23:45:41 +0100] rev 35717
more basic Local_Defs.export_cterm;
wenzelm [Thu, 11 Mar 2010 23:07:12 +0100] rev 35716
tuned signature;
wenzelm [Thu, 11 Mar 2010 23:07:02 +0100] rev 35715
tuned;
wenzelm [Thu, 11 Mar 2010 18:52:50 +0100] rev 35714
actually apply morphism to binding;
wenzelm [Thu, 11 Mar 2010 16:56:22 +0100] rev 35713
absolute lib_path relative to ML_HOME -- for improved robustness;
explicit warning if shared library failed to load;
blanchet [Thu, 11 Mar 2010 15:33:45 +0100] rev 35712
added a mechanism to Nitpick to support custom rendering of terms, and used it for multisets
blanchet [Thu, 11 Mar 2010 12:22:11 +0100] rev 35711
added term postprocessor to Nitpick, to provide custom syntax for typedefs
blanchet [Thu, 11 Mar 2010 10:13:24 +0100] rev 35710
made "Manual_Nits" tests more robust
haftmann [Thu, 11 Mar 2010 09:09:51 +0100] rev 35709
merged
haftmann [Thu, 11 Mar 2010 09:09:43 +0100] rev 35708
made smlnj happy
huffman [Wed, 10 Mar 2010 16:06:48 -0800] rev 35707
replace Nat_Int_Bij with Nat_Bijection in ROOT.ML
huffman [Wed, 10 Mar 2010 16:00:51 -0800] rev 35706
remove obsolete theory Nat_Int_Bij
huffman [Wed, 10 Mar 2010 15:58:53 -0800] rev 35705
switch from Nat_Int_Bij to Nat_Bijection
huffman [Wed, 10 Mar 2010 15:57:01 -0800] rev 35704
convert HOL-Probability to use Nat_Bijection library
huffman [Wed, 10 Mar 2010 15:38:33 -0800] rev 35703
convert SET_Protocol to use Nat_Bijection library
huffman [Wed, 10 Mar 2010 15:33:13 -0800] rev 35702
convert TLS to use Nat_Bijection library
huffman [Wed, 10 Mar 2010 15:20:13 -0800] rev 35701
adapt HOLCF to use Nat_Bijection library
huffman [Wed, 10 Mar 2010 14:57:13 -0800] rev 35700
new theory Library/Nat_Bijection.thy
blanchet [Wed, 10 Mar 2010 19:21:59 +0100] rev 35699
improve precision of "card" in Nitpick
blanchet [Wed, 10 Mar 2010 17:46:28 +0100] rev 35698
merged
blanchet [Wed, 10 Mar 2010 16:17:11 +0100] rev 35697
merged
blanchet [Wed, 10 Mar 2010 15:06:40 +0100] rev 35696
show nice error message in Nitpick when "java" is not available
blanchet [Wed, 10 Mar 2010 14:21:01 +0100] rev 35695
fixed soundness bug in Nitpick
hoelzl [Wed, 10 Mar 2010 16:40:20 +0100] rev 35694
merged
hoelzl [Tue, 09 Mar 2010 16:30:43 +0100] rev 35693
Use same order of neq-elimination as in proof search.
hoelzl [Mon, 08 Mar 2010 11:30:55 +0100] rev 35692
Moved theorems in Lebesgue to the right places
haftmann [Wed, 10 Mar 2010 15:29:23 +0100] rev 35691
constdefs is legacy
haftmann [Wed, 10 Mar 2010 15:29:22 +0100] rev 35690
recdef is legacy
haftmann [Wed, 10 Mar 2010 15:29:22 +0100] rev 35689
fixed typo
haftmann [Wed, 10 Mar 2010 15:29:22 +0100] rev 35688
avoid confusion
haftmann [Wed, 10 Mar 2010 15:29:21 +0100] rev 35687
tuned whitespace
haftmann [Wed, 10 Mar 2010 08:04:50 +0100] rev 35686
merged
haftmann [Wed, 10 Mar 2010 08:04:39 +0100] rev 35685
tuned
haftmann [Tue, 09 Mar 2010 21:19:49 +0100] rev 35684
clarified transfer code proper; more natural declaration of return rules
haftmann [Tue, 09 Mar 2010 21:19:48 +0100] rev 35683
misc tuning
wenzelm [Tue, 09 Mar 2010 23:32:49 +0100] rev 35682
Typedecl.typedecl_global;
wenzelm [Tue, 09 Mar 2010 23:32:13 +0100] rev 35681
localized typedecl;
wenzelm [Tue, 09 Mar 2010 23:29:04 +0100] rev 35680
aliases for class/type/const;
tuned;
wenzelm [Tue, 09 Mar 2010 23:27:35 +0100] rev 35679
added Name_Space.alias -- additional accesses for an existing entry;
wenzelm [Tue, 09 Mar 2010 20:23:19 +0100] rev 35678
merged
haftmann [Tue, 09 Mar 2010 18:33:01 +0100] rev 35677
merged
haftmann [Tue, 09 Mar 2010 18:31:37 +0100] rev 35676
data administration using canonical functorial operations
haftmann [Tue, 09 Mar 2010 16:15:19 +0100] rev 35675
tuned data structures; using AList.map_default
haftmann [Tue, 09 Mar 2010 15:47:16 +0100] rev 35674
consistent field names; tuned interface
haftmann [Tue, 09 Mar 2010 15:47:15 +0100] rev 35673
weakend class ring_div; tuned
blanchet [Tue, 09 Mar 2010 16:40:31 +0100] rev 35672
more work on Nitpick's finite sets
blanchet [Tue, 09 Mar 2010 14:18:21 +0100] rev 35671
improved Nitpick's precision for "card" and "setsum" + fix incorrect outcome code w.r.t. "bisim_depth = -1"
wenzelm [Tue, 09 Mar 2010 14:36:41 +0100] rev 35670
ProofContext.read_class/read_type_name_proper;
wenzelm [Tue, 09 Mar 2010 14:35:02 +0100] rev 35669
added ProofContext.tsig_of -- proforma version for local name space only, not logical content;
added ProofContext.read_type_name_proper;
localized ProofContext.read_class/read_arity/cert_arity;
localized ProofContext.class_space/type_space etc.;
wenzelm [Tue, 09 Mar 2010 14:29:47 +0100] rev 35668
simplified Syntax.basic_syntax (again);
separate Syntax.type_ast_trs depending on read_class/read_type;
wenzelm [Tue, 09 Mar 2010 14:55:25 +0100] rev 35667
tuned -- eliminated Sign.intern_sort;
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;
blanchet [Tue, 09 Mar 2010 09:25:23 +0100] rev 35665
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
huffman [Mon, 08 Mar 2010 15:20:40 -0800] rev 35664
merged
huffman [Mon, 08 Mar 2010 14:42:40 -0800] rev 35663
remove unnecessary error handling code
huffman [Mon, 08 Mar 2010 14:12:51 -0800] rev 35662
construct fully typed goal in proof of 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
huffman [Mon, 08 Mar 2010 12:43:44 -0800] rev 35660
remove redundant function arguments
huffman [Mon, 08 Mar 2010 12:36:26 -0800] rev 35659
include take_info within take_induct_info type
huffman [Mon, 08 Mar 2010 12:21:07 -0800] rev 35658
pass take_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
huffman [Mon, 08 Mar 2010 11:48:29 -0800] rev 35656
add type take_induct_info
huffman [Mon, 08 Mar 2010 11:34:53 -0800] rev 35655
generate take_induct lemmas
huffman [Mon, 08 Mar 2010 09:37:03 -0800] rev 35654
move proofs of reach and take lemmas to domain_take_proofs.ML
huffman [Mon, 08 Mar 2010 09:33:05 -0800] rev 35653
move lemmas from Domain.thy to Domain_Aux.thy
huffman [Mon, 08 Mar 2010 08:12:48 -0800] rev 35652
move take-proofs stuff into new theory Domain_Aux.thy
huffman [Mon, 08 Mar 2010 07:37:11 -0800] rev 35651
add type take_info
huffman [Mon, 08 Mar 2010 07:22:30 -0800] rev 35650
add function add_qualified_def
haftmann [Mon, 08 Mar 2010 17:37:09 +0100] rev 35649
merged
haftmann [Mon, 08 Mar 2010 14:41:56 +0100] rev 35648
proper ML interface; further polishing
haftmann [Mon, 08 Mar 2010 13:22:41 +0100] rev 35647
code simplification and tuning
berghofe [Mon, 08 Mar 2010 15:00:34 +0100] rev 35646
Added inducts field to inductive_result.
haftmann [Mon, 08 Mar 2010 09:38:59 +0100] rev 35645
transfer: avoid camel case, more standard coding conventions, misc tuning
haftmann [Mon, 08 Mar 2010 09:38:58 +0100] rev 35644
transfer: avoid camel case
huffman [Sun, 07 Mar 2010 17:33:01 -0800] rev 35643
merged
huffman [Sun, 07 Mar 2010 16:39:31 -0800] rev 35642
generate separate qualified theorem name for each type's reach and take_lemma