webertj [Tue, 01 Dec 2009 22:29:46 +0000] rev 33937
read_dimacs_cnf_file can now read DIMACS files that contain successive
white-space characters.
kleing [Sun, 29 Nov 2009 12:56:30 +1100] rev 33936
Expand nested abbreviations before applying dummy patterns.
berghofe [Fri, 27 Nov 2009 16:26:23 +0100] rev 33935
Removed eq_to_mono2, added not_mono.
berghofe [Fri, 27 Nov 2009 16:26:04 +0100] rev 33934
Streamlined setup for monotonicity rules (no longer requires classical rules).
berghofe [Fri, 27 Nov 2009 16:24:31 +0100] rev 33933
Simplified treatment of monotonicity rules.
wenzelm [Thu, 03 Dec 2009 19:31:55 +0100] rev 33932
removed obsolete test tags;
wenzelm [Thu, 03 Dec 2009 19:30:42 +0100] rev 33931
Added tag Isabelle2009-1 for changeset 6a973bd43949
wenzelm [Wed, 02 Dec 2009 12:04:07 +0100] rev 33930
slightly less ambitious settings, to avoid potential out-of-memory problem;
wenzelm [Mon, 30 Nov 2009 23:55:19 +0100] rev 33929
even higher proof-shell-quit-timeout -- saving main HOL takes 20s on a *fast* machine;
wenzelm [Mon, 30 Nov 2009 17:13:19 +0100] rev 33928
updated date;
wenzelm [Mon, 30 Nov 2009 17:13:12 +0100] rev 33927
more robust treatment of spaces in directory names;
bulwahn [Mon, 30 Nov 2009 08:44:08 +0100] rev 33926
adding subsection about the predicate compiler to the code generator tutorial
wenzelm [Sun, 29 Nov 2009 20:23:03 +0100] rev 33925
Added tag isa2009-1-test for changeset e1c262952b02
wenzelm [Sun, 29 Nov 2009 20:20:22 +0100] rev 33924
updated date;
kleing [Sun, 29 Nov 2009 12:56:30 +1100] rev 33923
Expand nested abbreviations before applying dummy patterns.
wenzelm [Sun, 29 Nov 2009 17:44:44 +0100] rev 33922
raised proof-shell-quit-timeout to accomodate bulky write-back images;
wenzelm [Sun, 29 Nov 2009 17:34:41 +0100] rev 33921
deactivated default for E_HOME, SPASS_HOME -- now configured as components;
deactivated default for VAMPIRE_HOME -- superceded by remote_vampire;
wenzelm [Sun, 29 Nov 2009 17:23:39 +0100] rev 33920
double check file permissions of write-back image -- more robust for root or administrator on Cygwin;
wenzelm [Sun, 29 Nov 2009 17:14:24 +0100] rev 33919
tuned message;
wenzelm [Sun, 29 Nov 2009 17:13:27 +0100] rev 33918
added HOLCF image;
wenzelm [Sat, 28 Nov 2009 22:28:15 +0100] rev 33917
workaround for strange compiler crash of Poly/ML 5.0 and 5.1 at this point http://isabelle.in.tum.de/repos/isabelle/file/a2fc533175ff/src/HOL/Tools/Nitpick/nitpick_nut.ML#l997
wenzelm [Sat, 28 Nov 2009 20:03:07 +0100] rev 33916
updated generated files;
wenzelm [Sat, 28 Nov 2009 18:17:10 +0100] rev 33915
proper quoting of array expansion -- allow spaces in components;
wenzelm [Sat, 28 Nov 2009 17:59:02 +0100] rev 33914
added "sos";
added subgoal focus;
wenzelm [Sat, 28 Nov 2009 16:16:17 +0100] rev 33913
PG version 3.7.1.1;
wenzelm [Sat, 28 Nov 2009 15:54:25 +0100] rev 33912
allow spaces within PROOFGENERAL_EMACS;
wenzelm [Sat, 28 Nov 2009 15:53:10 +0100] rev 33911
allow spaces within command-line arguments;
wenzelm [Fri, 27 Nov 2009 23:08:26 +0100] rev 33910
proper quotes;
wenzelm [Fri, 27 Nov 2009 22:38:22 +0100] rev 33909
more abstract handling of repository name;
wenzelm [Fri, 27 Nov 2009 00:59:01 +0100] rev 33908
more menu entries -- backport from PG 4.0 branch;
wenzelm [Fri, 27 Nov 2009 00:11:56 +0100] rev 33907
re-package Isabelle distribution with add-on components;
Philipp Meyer [Thu, 26 Nov 2009 20:07:02 +0100] rev 33906
fixed csdp output parser
wenzelm [Thu, 26 Nov 2009 15:28:42 +0100] rev 33905
additional menu entries;
wenzelm [Thu, 26 Nov 2009 15:03:31 +0100] rev 33904
Added tag isa2009-1-test for changeset 14ff44e21bec
wenzelm [Thu, 26 Nov 2009 14:54:56 +0100] rev 33903
adhoc delay after font installation -- increases chance that Emacs will actually see them;
wenzelm [Thu, 26 Nov 2009 14:42:52 +0100] rev 33902
implicit font installation for Mac OS;
wenzelm [Thu, 26 Nov 2009 12:55:24 +0100] rev 33901
modernized interface script for PG 3.7.1 -- backport from PG 4.0 branch;
wenzelm [Thu, 26 Nov 2009 12:13:43 +0100] rev 33900
patch for the infamous antiquotation font-lock problem of Proof General 3.7.1 with GNU Emacs, cf. http://proofgeneral.inf.ed.ac.uk/trac/ticket/236
wenzelm [Wed, 25 Nov 2009 15:30:03 +0100] rev 33899
refer to isabelle-release branch;
wenzelm [Wed, 25 Nov 2009 15:21:41 +0100] rev 33898
include HOL-SMT keywords;
wenzelm [Wed, 25 Nov 2009 15:04:20 +0100] rev 33897
tuned affiliation;
boehmes [Wed, 25 Nov 2009 12:31:43 +0100] rev 33896
extended list of HOL-Boogie contributors
boehmes [Wed, 25 Nov 2009 12:30:54 +0100] rev 33895
only add nat/int conversion rules if necessary
boehmes [Wed, 25 Nov 2009 12:29:37 +0100] rev 33894
more generic explosion of options (also accept newlines, etc.)
boehmes [Wed, 25 Nov 2009 12:28:29 +0100] rev 33893
respect "unique" attribute: generate distinctness axioms
blanchet [Tue, 24 Nov 2009 18:36:18 +0100] rev 33892
fixed arity of some empty relations in Nitpick's Kodkod generator;
these previously resulted in Kodkod arity errors (similar to type errors for other logics)
blanchet [Tue, 24 Nov 2009 18:35:21 +0100] rev 33891
fix soundness bug in "uncurry" option of Nitpick
wenzelm [Tue, 24 Nov 2009 17:54:33 +0100] rev 33890
Added tag isa2009-1-test for changeset 4328de748fb2
wenzelm [Tue, 24 Nov 2009 17:19:33 +0100] rev 33889
some rearangement of load order to keep preferences adjacent -- slightly fragile;
blanchet [Tue, 24 Nov 2009 16:11:50 +0100] rev 33888
use correct Isabelle version name in README file
blanchet [Tue, 24 Nov 2009 16:07:31 +0100] rev 33887
remove version number from Nitpick manual
blanchet [Tue, 24 Nov 2009 15:22:00 +0100] rev 33886
fix soundness bug in Nitpick's Kodkod generator for the relational composition case
blanchet [Tue, 24 Nov 2009 13:57:25 +0100] rev 33885
merged
blanchet [Tue, 24 Nov 2009 13:55:14 +0100] rev 33884
generate clearer atom names in Nitpick for types that end with a digit;
requested by a user
wenzelm [Tue, 24 Nov 2009 13:54:29 +0100] rev 33883
Added tag isa2009-1-test for changeset 9db7854eafc7
blanchet [Tue, 24 Nov 2009 13:22:18 +0100] rev 33882
fix soundness bug in Nitpick's handling of negative literals (e.g., -1::rat)
haftmann [Tue, 24 Nov 2009 12:29:08 +0100] rev 33881
consisten upper/lower case
blanchet [Tue, 24 Nov 2009 10:33:21 +0100] rev 33880
merge
blanchet [Tue, 24 Nov 2009 10:33:02 +0100] rev 33879
fixed soundness bug / type error in handling of unpolarized (co)inductive predicates in Nitpick
blanchet [Tue, 24 Nov 2009 10:31:01 +0100] rev 33878
removed "nitpick_def" attributes from (r)trancl(p), since "Nitpick.thy" overrides these
blanchet [Mon, 23 Nov 2009 18:29:00 +0100] rev 33877
fix Nitpick soundness bug related to "finite (UNIV::'a set)" where "'a" is constrained by a sort to be infinite
blanchet [Mon, 23 Nov 2009 17:59:22 +0100] rev 33876
fixed soundness bug in Nitpick's handling of typedefs
wenzelm [Mon, 23 Nov 2009 22:59:48 +0100] rev 33875
multiplatform polyml.tar.gz;
wenzelm [Mon, 23 Nov 2009 22:47:41 +0100] rev 33874
updated keywords;
wenzelm [Mon, 23 Nov 2009 22:47:08 +0100] rev 33873
more tuning for release;
wenzelm [Mon, 23 Nov 2009 22:35:54 +0100] rev 33872
added command 'ProofGeneral.pr' for PG 4.0;
bulwahn [Mon, 23 Nov 2009 21:56:07 +0100] rev 33871
merged
bulwahn [Mon, 23 Nov 2009 19:42:52 +0100] rev 33870
improving the setup for the tabled transitive closure thanks to usage of Andreas Lochbihler
wenzelm [Mon, 23 Nov 2009 21:24:15 +0100] rev 33869
updated for release;
ballarin [Mon, 23 Nov 2009 21:04:00 +0100] rev 33868
Generated files.
ballarin [Mon, 23 Nov 2009 21:03:49 +0100] rev 33867
Typos in documenation.
haftmann [Mon, 23 Nov 2009 19:03:16 +0100] rev 33866
ANNOUNCE
blanchet [Mon, 23 Nov 2009 17:27:43 +0100] rev 33865
merge
blanchet [Mon, 23 Nov 2009 17:26:32 +0100] rev 33864
fix Nitpick soundness bugs related to integration (in particular, "code_numeral")
blanchet [Mon, 23 Nov 2009 14:34:05 +0100] rev 33863
generate arguments of relational composition in the right order in Nitpick
haftmann [Mon, 23 Nov 2009 16:24:28 +0100] rev 33862
CONTRIBUTORS
haftmann [Mon, 23 Nov 2009 16:15:39 +0100] rev 33861
merged
haftmann [Mon, 23 Nov 2009 16:15:18 +0100] rev 33860
tuned NEWS
krauss [Mon, 23 Nov 2009 15:11:21 +0100] rev 33859
do not add host suffix -- it is appended by test framework
krauss [Mon, 23 Nov 2009 15:06:38 +0100] rev 33858
documented size_change in isar-ref manual
krauss [Mon, 23 Nov 2009 15:06:37 +0100] rev 33857
clarified; checked
krauss [Mon, 23 Nov 2009 15:06:34 +0100] rev 33856
mentioned method size_change in function tutorial
krauss [Mon, 23 Nov 2009 15:05:59 +0100] rev 33855
eliminated dead code and some unused bindings, reported by polyml
blanchet [Mon, 23 Nov 2009 13:45:16 +0100] rev 33854
fixed a Kodkod generation exception in Nitpick, reported by a Karlsruhe user
blanchet [Mon, 23 Nov 2009 13:24:32 +0100] rev 33853
fixed soundness bug in Nitpick that occurred because unrolled predicate iterators were considered to be a "precise" type
blanchet [Mon, 23 Nov 2009 13:23:39 +0100] rev 33852
improved annotated type of equality in Nitpick's monotonicity check, based on a discovery by Alex
blanchet [Mon, 23 Nov 2009 13:22:40 +0100] rev 33851
fixed error in Nitpick's "star_linear_preds" optimization, which resulted in an ill-typed term;
reported by Stefan
wenzelm [Sun, 22 Nov 2009 22:10:31 +0100] rev 33850
merged
haftmann [Sun, 22 Nov 2009 17:02:46 +0100] rev 33849
more uniform view on various number theory refinement steps
ballarin [Sun, 22 Nov 2009 15:42:48 +0100] rev 33848
Merged.
ballarin [Sun, 22 Nov 2009 15:37:49 +0100] rev 33847
Generated latex code.
ballarin [Sun, 22 Nov 2009 15:37:14 +0100] rev 33846
Updated locale documentation.
wenzelm [Sun, 22 Nov 2009 22:04:51 +0100] rev 33845
made SML/NJ happy;
wenzelm [Sun, 22 Nov 2009 14:59:27 +0100] rev 33844
remove presently unused Isabelle application;
wenzelm [Sun, 22 Nov 2009 14:49:36 +0100] rev 33843
more NEWS, more tuning for release;
wenzelm [Sun, 22 Nov 2009 14:13:18 +0100] rev 33842
misc tuning and updates for official release;
wenzelm [Sat, 21 Nov 2009 20:44:16 +0100] rev 33841
tuned;
wenzelm [Sat, 21 Nov 2009 20:41:29 +0100] rev 33840
updated keywords;
ballarin [Sat, 21 Nov 2009 18:33:55 +0100] rev 33839
Use less whitespace in documentation.
ballarin [Sat, 21 Nov 2009 18:25:53 +0100] rev 33838
Publication details and minor correction of the text.
ballarin [Sat, 21 Nov 2009 17:39:54 +0100] rev 33837
Removed obsolete comment.
ballarin [Sat, 21 Nov 2009 17:37:07 +0100] rev 33836
Merged.
ballarin [Sat, 21 Nov 2009 17:35:55 +0100] rev 33835
More tests for locale interpretation.
wenzelm [Sat, 21 Nov 2009 17:01:44 +0100] rev 33834
adapted local theory operations -- eliminated odd kind;
wenzelm [Sat, 21 Nov 2009 16:07:58 +0100] rev 33833
minimal Poly/ML startup script;
wenzelm [Sat, 21 Nov 2009 15:49:29 +0100] rev 33832
explicitly mark some legacy freeze operations;
wenzelm [Sat, 21 Nov 2009 14:03:36 +0100] rev 33831
minimal test of current repository version;
wenzelm [Sat, 21 Nov 2009 14:02:55 +0100] rev 33830
slightly longer log tail;
kleing [Sat, 21 Nov 2009 17:04:03 +1100] rev 33829
add explicit platform check to wwwfind tool
explicit platform check to avoid calling external programs with strange parameters
kleing [Sat, 21 Nov 2009 16:56:53 +1100] rev 33828
adjusted help text
kleing [Sat, 21 Nov 2009 11:47:38 +1100] rev 33827
wwwfind support currently for Linux only
huffman [Fri, 20 Nov 2009 15:29:56 -0800] rev 33826
make repdef work without (open) option
huffman [Fri, 20 Nov 2009 14:35:55 -0800] rev 33825
NEWS: HOLCF changes since the last release
wenzelm [Fri, 20 Nov 2009 17:56:06 +0100] rev 33824
removed hard tabs from text (not pattern);
wenzelm [Fri, 20 Nov 2009 16:08:14 +0100] rev 33823
standardized headers;
wenzelm [Fri, 20 Nov 2009 15:48:36 +0100] rev 33822
provide standard isabelle make targets;
slightly more accurate dependencies;
wenzelm [Fri, 20 Nov 2009 15:34:11 +0100] rev 33821
merged
wenzelm [Fri, 20 Nov 2009 15:33:10 +0100] rev 33820
load ML directly into theory Code_Generator (quickcheck also requires this);
kleing [Fri, 20 Nov 2009 22:38:41 +1100] rev 33819
made script executable
kleing [Fri, 20 Nov 2009 22:28:39 +1100] rev 33818
added NEWS item for wwwfind
kleing [Fri, 20 Nov 2009 18:36:44 +1100] rev 33817
WWW_Find component: find_theorems via web browser
wenzelm [Fri, 20 Nov 2009 10:40:30 +0100] rev 33816
merged
nipkow [Fri, 20 Nov 2009 09:22:14 +0100] rev 33815
merged
nipkow [Fri, 20 Nov 2009 09:21:59 +0100] rev 33814
Rene tuned proof
huffman [Fri, 20 Nov 2009 00:06:04 -0800] rev 33813
example theory for new domain package
huffman [Thu, 19 Nov 2009 23:15:24 -0800] rev 33812
thy_decl outer syntax for repdef
huffman [Thu, 19 Nov 2009 22:30:14 -0800] rev 33811
merged
huffman [Thu, 19 Nov 2009 22:28:36 -0800] rev 33810
nicer warning message for indirect-recursive domain definitions
huffman [Thu, 19 Nov 2009 22:25:11 -0800] rev 33809
store map_ID thms in theory data; automate proofs of reach lemmas
huffman [Thu, 19 Nov 2009 21:44:37 -0800] rev 33808
add map_ID lemmas
huffman [Thu, 19 Nov 2009 21:06:22 -0800] rev 33807
domain_isomorphism package defines combined copy function
nipkow [Fri, 20 Nov 2009 07:24:21 +0100] rev 33806
merged
nipkow [Fri, 20 Nov 2009 07:24:08 +0100] rev 33805
added Rene Thiemann's normalize function
nipkow [Fri, 20 Nov 2009 07:23:36 +0100] rev 33804
added lemma
huffman [Thu, 19 Nov 2009 20:09:56 -0800] rev 33803
merged
huffman [Thu, 19 Nov 2009 17:53:22 -0800] rev 33802
domain_isomorphism package defines copy functions
huffman [Thu, 19 Nov 2009 16:50:25 -0800] rev 33801
copy_of_dtyp uses map table from theory data
huffman [Thu, 19 Nov 2009 16:48:40 -0800] rev 33800
Domain.thy imports Representable.thy
huffman [Thu, 19 Nov 2009 16:47:18 -0800] rev 33799
fix definitions of copy combinators
huffman [Thu, 19 Nov 2009 15:41:52 -0800] rev 33798
clean up indentation; add 'definitional' option flag
huffman [Thu, 19 Nov 2009 15:31:19 -0800] rev 33797
rename generated abs_iso, rep_iso lemmas
huffman [Thu, 19 Nov 2009 13:23:58 -0800] rev 33796
clean up indentation
huffman [Thu, 19 Nov 2009 12:38:25 -0800] rev 33795
add dependency on domain_isomorphism.ML
huffman [Thu, 19 Nov 2009 12:38:02 -0800] rev 33794
set up domain_isomorphism package in Representable.thy
huffman [Thu, 19 Nov 2009 12:31:55 -0800] rev 33793
automate proofs of map_ID theorems
huffman [Thu, 19 Nov 2009 12:05:49 -0800] rev 33792
change Theory.requires
huffman [Thu, 19 Nov 2009 11:54:23 -0800] rev 33791
use theory data for REP_simps and isodefl_rules
huffman [Thu, 19 Nov 2009 11:13:34 -0800] rev 33790
replace defl_tab and map_tab with theory data
huffman [Thu, 19 Nov 2009 10:45:34 -0800] rev 33789
separate conjuncts of isodefl theorem
huffman [Thu, 19 Nov 2009 10:27:29 -0800] rev 33788
automate isodefl proof
huffman [Thu, 19 Nov 2009 10:26:53 -0800] rev 33787
change example to use recursion with continuous function space
huffman [Thu, 19 Nov 2009 10:25:17 -0800] rev 33786
add lemma isodefl_cprod
huffman [Thu, 19 Nov 2009 09:04:58 -0800] rev 33785
automate definition of map functions; remove unused code
huffman [Thu, 19 Nov 2009 08:22:00 -0800] rev 33784
change naming convention for deflation combinators
huffman [Thu, 19 Nov 2009 08:08:57 -0800] rev 33783
add new makefile dependencies
huffman [Thu, 19 Nov 2009 08:00:42 -0800] rev 33782
prove isomorphism and isodefl rules
huffman [Thu, 19 Nov 2009 07:09:04 -0800] rev 33781
avoid using csplit; define copy functions exactly like the current domain package
huffman [Thu, 19 Nov 2009 06:01:02 -0800] rev 33780
merged
huffman [Wed, 18 Nov 2009 16:57:58 -0800] rev 33779
remove one_typ and tr_typ; add abs/rep lemmas
huffman [Wed, 18 Nov 2009 16:14:28 -0800] rev 33778
automate definition of rep/abs functions
huffman [Wed, 18 Nov 2009 15:54:47 -0800] rev 33777
get rid of numbers on thy variables
huffman [Wed, 18 Nov 2009 15:51:35 -0800] rev 33776
automate proofs of REP equations
huffman [Wed, 18 Nov 2009 15:01:00 -0800] rev 33775
cleaned up; factored out fixed-point definition code
huffman [Wed, 18 Nov 2009 12:41:43 -0800] rev 33774
automate solution of domain equations
Christian Urban <urbanc@in.tum.de> [Fri, 20 Nov 2009 00:54:20 +0100] rev 33773
removed fixme - quick-and-dirty flag is appropriate
Christian Urban <urbanc@in.tum.de> [Fri, 20 Nov 2009 00:20:32 +0100] rev 33772
use of thm-antiquotation
berghofe [Thu, 19 Nov 2009 16:07:53 +0100] rev 33771
Added new counterexample generator SML_inductive for goals involving
inductive predicates.
berghofe [Thu, 19 Nov 2009 16:04:31 +0100] rev 33770
Added infrastructure for embedding random data generators into code generated
for inductive predicates.
wenzelm [Thu, 19 Nov 2009 19:42:54 +0100] rev 33769
unused_thms: show only results from 'theorem(s)' package (via old-style kinds);
misc tuning -- slightly less hermetic names;
wenzelm [Thu, 19 Nov 2009 17:29:39 +0100] rev 33768
future_result: purge flexflex pairs, which should normally be trivial anyway -- prevent Thm.future_result from complaining about tpairs;
wenzelm [Thu, 19 Nov 2009 17:26:28 +0100] rev 33767
toplevel pretty printer for Synchronized.var;
wenzelm [Thu, 19 Nov 2009 14:46:33 +0100] rev 33766
adapted Local_Theory.define -- eliminated odd thm kind;
wenzelm [Thu, 19 Nov 2009 14:45:56 +0100] rev 33765
Specification.definition: Thm.definitionK marks exactly the high-level end-user result;
wenzelm [Thu, 19 Nov 2009 14:44:22 +0100] rev 33764
Local_Theory.define: eliminated slightly odd kind argument -- such low-level definitions should be hardly ever exposed to end-users anyway;
wenzelm [Thu, 19 Nov 2009 13:00:16 +0100] rev 33763
merged
paulson [Thu, 19 Nov 2009 11:19:25 +0000] rev 33762
merged
paulson [Thu, 19 Nov 2009 10:58:36 +0000] rev 33761
Minor correction
wenzelm [Thu, 19 Nov 2009 12:59:32 +0100] rev 33760
some attempts to improve termination of isatest;
hoelzl [Thu, 19 Nov 2009 11:57:30 +0100] rev 33759
Added the contributions of Robert Himmelmann to CONTRIBUTIONS and NEWS
hoelzl [Thu, 19 Nov 2009 11:51:37 +0100] rev 33758
Renamed vector_less_eq_def to the more usual name vector_le_def.
bulwahn [Thu, 19 Nov 2009 10:49:43 +0100] rev 33757
merged
bulwahn [Thu, 19 Nov 2009 08:25:57 +0100] rev 33756
replacing Predicate_Compile_Preproc_Const_Defs by more general Spec_Rules
bulwahn [Thu, 19 Nov 2009 08:25:54 +0100] rev 33755
concealing internal definitions of primrec specifications
bulwahn [Thu, 19 Nov 2009 08:25:53 +0100] rev 33754
adding derived constant Predicate.holds to Predicate theory; adopting the predicate compiler
bulwahn [Thu, 19 Nov 2009 08:25:51 +0100] rev 33753
changing the proof procedure for parameters; adding a testcase for negation and parameters; adopting print_tac to the latest function print_tac' in the predicate compiler
bulwahn [Thu, 19 Nov 2009 08:25:47 +0100] rev 33752
adopting proposed_modes; adding a new dimension of complexity for nicer error messages; tuned
krauss [Thu, 19 Nov 2009 10:33:20 +0100] rev 33751
check if equations are present for all functions to avoid low-level exception later
nipkow [Thu, 19 Nov 2009 08:19:57 +0100] rev 33750
anti_sym -> antisym
boehmes [Wed, 18 Nov 2009 14:00:08 +0100] rev 33749
optionally trace theorems used in proof reconstruction
boehmes [Wed, 18 Nov 2009 09:34:53 +0100] rev 33748
added arithmetic example using div and mod
blanchet [Tue, 17 Nov 2009 23:47:57 +0100] rev 33747
bump up Nitpick's axiom/definition unfolding limits, because some real-world problems (e.g. from Boogie) ran into the previous limits;
the limits are there to prevent infinite recursion; they can be set arbitrarily high without much harm
blanchet [Tue, 17 Nov 2009 22:51:00 +0100] rev 33746
merged
blanchet [Tue, 17 Nov 2009 22:20:51 +0100] rev 33745
comment out debugging code in Nitpick
blanchet [Tue, 17 Nov 2009 19:47:27 +0100] rev 33744
fixed bug in Nitpick's handling of "The" and "Eps" when the return type is a "bool"
blanchet [Tue, 17 Nov 2009 19:12:10 +0100] rev 33743
made "NitpickHOL.normalized_rhs_of" more robust in the face of locale definitions
blanchet [Tue, 17 Nov 2009 19:08:02 +0100] rev 33742
removed "debug := true" that shouldn't have been submitted in the first place
hoelzl [Tue, 17 Nov 2009 18:52:30 +0100] rev 33741
Added derivation and Brouwer's fixpoint theorem in Multivariate Analysis (translated by Robert Himmelmann from HOL-light)
blanchet [Tue, 17 Nov 2009 18:25:05 +0100] rev 33740
merged
blanchet [Tue, 17 Nov 2009 18:24:43 +0100] rev 33739
run Nitpick examples if Kodkodi is available
wenzelm [Tue, 17 Nov 2009 15:55:30 +0100] rev 33738
merged
blanchet [Tue, 17 Nov 2009 14:10:31 +0100] rev 33737
fixed "expect" of Nitpick examples to reflect latest changes in Nitpick
blanchet [Tue, 17 Nov 2009 13:51:56 +0100] rev 33736
merged
blanchet [Tue, 17 Nov 2009 13:51:16 +0100] rev 33735
use SAT solver that's available everywhere for this example
blanchet [Tue, 17 Nov 2009 13:50:46 +0100] rev 33734
invoke Kodkodi from Nitpick using new $KODKOD/bin/kodkodi script;
this requires downloading Kodkodi 1.2.4, or writing a "kodkodi" script that invokes "java de.tum.in.isabelle.Kodkodi.Kodkodi $@"
blanchet [Tue, 17 Nov 2009 10:58:37 +0100] rev 33733
merged
blanchet [Mon, 16 Nov 2009 11:03:08 +0100] rev 33732
added constraint for Eq^- in Nitpick's implementation of the monotonicity calculus
blanchet [Mon, 16 Nov 2009 10:24:28 +0100] rev 33731
change the order in which Nitpick tries SAT solvers;
so that the binary JNIs come further down the list and can
easily be overridden
webertj [Tue, 17 Nov 2009 11:10:22 +0000] rev 33730
Fixed splitting of div and mod on integers (split theorem differed from implementation).
webertj [Tue, 17 Nov 2009 10:18:51 +0000] rev 33729
merged
webertj [Tue, 17 Nov 2009 10:17:53 +0000] rev 33728
Fixed splitting of div and mod on integers (split theorem differed from implementation).
wenzelm [Tue, 17 Nov 2009 15:53:35 +0100] rev 33727
init_theory: Runtime.controlled_execution for proper exception trace etc.;
wenzelm [Tue, 17 Nov 2009 14:51:57 +0100] rev 33726
eliminated slightly odd name space grouping -- now managed by Isar toplevel;
wenzelm [Tue, 17 Nov 2009 14:51:32 +0100] rev 33725
implicit name space grouping for theory/local_theory transactions;
wenzelm [Tue, 17 Nov 2009 14:50:55 +0100] rev 33724
uniform new_group/reset_group;
tuned signature;
wenzelm [Tue, 17 Nov 2009 14:48:21 +0100] rev 33723
eliminated dead code;
wenzelm [Mon, 16 Nov 2009 21:57:16 +0100] rev 33722
generalized procs for rewrite_proof: allow skeleton;
fulfill_norm_proof: always normalize result here, no re-normalization after filling;
wenzelm [Mon, 16 Nov 2009 21:56:32 +0100] rev 33721
member/cons: slightly more correct treatment of multi-index, notably empty one;
wenzelm [Mon, 16 Nov 2009 20:23:02 +0100] rev 33720
merged
webertj [Mon, 16 Nov 2009 18:33:12 +0000] rev 33719
Fixed a typo in a comment.
webertj [Mon, 16 Nov 2009 17:22:10 +0000] rev 33718
Fixed a typo in a comment.
paulson [Mon, 16 Nov 2009 14:32:35 +0000] rev 33717
merged
paulson [Mon, 16 Nov 2009 14:32:12 +0000] rev 33716
A few more lemmas from Jeremy
hoelzl [Mon, 16 Nov 2009 15:03:23 +0100] rev 33715
removed hassize predicate
hoelzl [Mon, 16 Nov 2009 15:06:34 +0100] rev 33714
Added new lemmas to Euclidean Space by Robert Himmelmann
wenzelm [Mon, 16 Nov 2009 13:53:31 +0100] rev 33713
eliminated obsolete thm position stuff;
wenzelm [Mon, 16 Nov 2009 13:53:02 +0100] rev 33712
tuned signature;
wenzelm [Mon, 16 Nov 2009 13:49:21 +0100] rev 33711
guard future proofs by Goal.future_enabled;
boehmes [Mon, 16 Nov 2009 12:09:59 +0100] rev 33710
further explosion of HOL-Boogie verification conditions
haftmann [Mon, 16 Nov 2009 11:14:43 +0100] rev 33709
merged
haftmann [Mon, 16 Nov 2009 10:16:40 +0100] rev 33708
proper purge
haftmann [Mon, 16 Nov 2009 11:03:14 +0100] rev 33707
dropped obsolete documentation; updated generated sources
blanchet [Mon, 16 Nov 2009 10:03:58 +0100] rev 33706
merged
blanchet [Fri, 13 Nov 2009 15:59:53 +0100] rev 33705
removed a few global names in Nitpick (styp, nat_less, pairf)
wenzelm [Sun, 15 Nov 2009 21:58:40 +0100] rev 33704
add_expand_thm: explicit indication of is_def instead of fragile heuristic, tuned signature;
explicit extraction_expand vs. extraction_expand_def attribute;
wenzelm [Sun, 15 Nov 2009 20:57:42 +0100] rev 33703
axiomatization: declare Spec_Rules, direct result;
wenzelm [Sun, 15 Nov 2009 20:56:34 +0100] rev 33702
use simultaneous Morphics.fact;
wenzelm [Sun, 15 Nov 2009 20:39:22 +0100] rev 33701
primitive defs: clarified def (axiom name) vs. description;
wenzelm [Sun, 15 Nov 2009 19:45:05 +0100] rev 33700
eliminated obsolete thm position tags;
wenzelm [Sun, 15 Nov 2009 19:44:29 +0100] rev 33699
permissive AList.merge -- most likely setup for theory data (beware of spurious AList.DUP);
wenzelm [Sun, 15 Nov 2009 19:44:16 +0100] rev 33698
provide actual Nitpick_HOL.extended_context;