Tue, 07 Dec 2010 17:23:14 +0100 eliminated some hard tabulators (deprecated);
wenzelm [Tue, 07 Dec 2010 17:23:14 +0100] rev 41067
eliminated some hard tabulators (deprecated);
Tue, 07 Dec 2010 16:27:07 +0100 pass constant arguments to the built-in check function, cf. d2b1fc1b8e19
blanchet [Tue, 07 Dec 2010 16:27:07 +0100] rev 41066
pass constant arguments to the built-in check function, cf. d2b1fc1b8e19
Tue, 07 Dec 2010 15:55:35 +0100 merged
boehmes [Tue, 07 Dec 2010 15:55:35 +0100] rev 41065
merged
Tue, 07 Dec 2010 15:44:38 +0100 updated SMT certificates
boehmes [Tue, 07 Dec 2010 15:44:38 +0100] rev 41064
updated SMT certificates
Tue, 07 Dec 2010 15:01:42 +0100 reduced unnecessary complexity; improved documentation; tuned
boehmes [Tue, 07 Dec 2010 15:01:42 +0100] rev 41063
reduced unnecessary complexity; improved documentation; tuned
Tue, 07 Dec 2010 15:01:37 +0100 tuned
boehmes [Tue, 07 Dec 2010 15:01:37 +0100] rev 41062
tuned
Tue, 07 Dec 2010 14:54:31 +0100 centralized handling of built-in types and constants for bitvectors
boehmes [Tue, 07 Dec 2010 14:54:31 +0100] rev 41061
centralized handling of built-in types and constants for bitvectors
Tue, 07 Dec 2010 14:53:44 +0100 moved smt_word.ML into the directory of the Word library
boehmes [Tue, 07 Dec 2010 14:53:44 +0100] rev 41060
moved smt_word.ML into the directory of the Word library
Tue, 07 Dec 2010 14:53:12 +0100 centralized handling of built-in types and constants;
boehmes [Tue, 07 Dec 2010 14:53:12 +0100] rev 41059
centralized handling of built-in types and constants; also store types and constants which are rewritten during preprocessing; interfaces are identified by classes (supporting inheritance, at least on the level of built-in symbols); removed term_eq in favor of type replacements: term-level occurrences of type bool are replaced by type term_bool (only for the translation)
Mon, 06 Dec 2010 16:54:22 +0100 more aggressive unfolding of unknowns in Z3 models
boehmes [Mon, 06 Dec 2010 16:54:22 +0100] rev 41058
more aggressive unfolding of unknowns in Z3 models
Mon, 06 Dec 2010 15:38:02 +0100 tuned
boehmes [Mon, 06 Dec 2010 15:38:02 +0100] rev 41057
tuned
Tue, 07 Dec 2010 13:33:28 +0100 adding a definition for refl_on which is friendly for quickcheck and nitpick
bulwahn [Tue, 07 Dec 2010 13:33:28 +0100] rev 41056
adding a definition for refl_on which is friendly for quickcheck and nitpick
Tue, 07 Dec 2010 12:10:13 +0100 merged
blanchet [Tue, 07 Dec 2010 12:10:13 +0100] rev 41055
merged
Tue, 07 Dec 2010 11:56:56 +0100 simplify monotonicity code after killing "fin_fun" optimization
blanchet [Tue, 07 Dec 2010 11:56:56 +0100] rev 41054
simplify monotonicity code after killing "fin_fun" optimization
Tue, 07 Dec 2010 11:56:56 +0100 updated Nitpick's documentation w.r.t. finitization
blanchet [Tue, 07 Dec 2010 11:56:56 +0100] rev 41053
updated Nitpick's documentation w.r.t. finitization
Tue, 07 Dec 2010 11:56:53 +0100 remove the "fin_fun" optimization in Nitpick -- it was always a hack and didn't help much
blanchet [Tue, 07 Dec 2010 11:56:53 +0100] rev 41052
remove the "fin_fun" optimization in Nitpick -- it was always a hack and didn't help much
Tue, 07 Dec 2010 11:56:01 +0100 give the inner timeout mechanism a chance, since it gives more precise information to the user
blanchet [Tue, 07 Dec 2010 11:56:01 +0100] rev 41051
give the inner timeout mechanism a chance, since it gives more precise information to the user
Tue, 07 Dec 2010 11:56:01 +0100 updated monotonicity calculus w.r.t. set products
blanchet [Tue, 07 Dec 2010 11:56:01 +0100] rev 41050
updated monotonicity calculus w.r.t. set products
Tue, 07 Dec 2010 11:56:01 +0100 removed needless optimization for image -- there might be cases that benefit from it but there are others where it is clearly evil
blanchet [Tue, 07 Dec 2010 11:56:01 +0100] rev 41049
removed needless optimization for image -- there might be cases that benefit from it but there are others where it is clearly evil
Tue, 07 Dec 2010 11:56:01 +0100 added a hint when the user obviously just forgot a colon after the lemma's name
blanchet [Tue, 07 Dec 2010 11:56:01 +0100] rev 41048
added a hint when the user obviously just forgot a colon after the lemma's name
Tue, 07 Dec 2010 11:56:01 +0100 simplified special handling of set products
blanchet [Tue, 07 Dec 2010 11:56:01 +0100] rev 41047
simplified special handling of set products
Tue, 07 Dec 2010 11:56:01 +0100 fix special handling of set products
blanchet [Tue, 07 Dec 2010 11:56:01 +0100] rev 41046
fix special handling of set products
Tue, 07 Dec 2010 11:56:01 +0100 use heuristic to determine whether to keep or drop an existing "let" -- and drop all higher-order lets
blanchet [Tue, 07 Dec 2010 11:56:01 +0100] rev 41045
use heuristic to determine whether to keep or drop an existing "let" -- and drop all higher-order lets
Tue, 07 Dec 2010 11:50:16 +0100 merged
bulwahn [Tue, 07 Dec 2010 11:50:16 +0100] rev 41044
merged
Tue, 07 Dec 2010 10:03:43 +0100 testing smartly in two dimensions (cardinality and size) in quickcheck
bulwahn [Tue, 07 Dec 2010 10:03:43 +0100] rev 41043
testing smartly in two dimensions (cardinality and size) in quickcheck
Tue, 07 Dec 2010 09:58:56 +0100 load "try" after "Metis" and move "Async_Manager" back to Sledgehammer
blanchet [Tue, 07 Dec 2010 09:58:56 +0100] rev 41042
load "try" after "Metis" and move "Async_Manager" back to Sledgehammer
Tue, 07 Dec 2010 09:58:52 +0100 make SML/NJ happy
blanchet [Tue, 07 Dec 2010 09:58:52 +0100] rev 41041
make SML/NJ happy
Tue, 07 Dec 2010 09:52:07 +0100 merge
blanchet [Tue, 07 Dec 2010 09:52:07 +0100] rev 41040
merge
Mon, 06 Dec 2010 14:47:58 +0100 show strings as "s_1" etc. rather than "l_1" etc.
blanchet [Mon, 06 Dec 2010 14:47:58 +0100] rev 41039
show strings as "s_1" etc. rather than "l_1" etc.
Mon, 06 Dec 2010 14:47:58 +0100 quiet Metis in "try"
blanchet [Mon, 06 Dec 2010 14:47:58 +0100] rev 41038
quiet Metis in "try"
Tue, 07 Dec 2010 09:36:12 +0100 removed experimental equality checking of closures; acknowledge underapproximation of equality in function name
haftmann [Tue, 07 Dec 2010 09:36:12 +0100] rev 41037
removed experimental equality checking of closures; acknowledge underapproximation of equality in function name
Mon, 06 Dec 2010 14:17:35 -0800 add set-union-like syntax for powerdomain bind operators
huffman [Mon, 06 Dec 2010 14:17:35 -0800] rev 41036
add set-union-like syntax for powerdomain bind operators
Mon, 06 Dec 2010 13:43:05 -0800 merged
huffman [Mon, 06 Dec 2010 13:43:05 -0800] rev 41035
merged
Mon, 06 Dec 2010 13:34:05 -0800 instance unit :: domain
huffman [Mon, 06 Dec 2010 13:34:05 -0800] rev 41034
instance unit :: domain
Mon, 06 Dec 2010 12:53:06 -0800 simplify ideal completion proofs
huffman [Mon, 06 Dec 2010 12:53:06 -0800] rev 41033
simplify ideal completion proofs
Mon, 06 Dec 2010 11:44:30 -0800 remove unused lemmas
huffman [Mon, 06 Dec 2010 11:44:30 -0800] rev 41032
remove unused lemmas
Mon, 06 Dec 2010 11:22:42 -0800 remove lemma cont_cfun;
huffman [Mon, 06 Dec 2010 11:22:42 -0800] rev 41031
remove lemma cont_cfun; rename thelub_cfun to lub_cfun
Mon, 06 Dec 2010 10:08:33 -0800 rename lub_fun -> is_lub_fun, thelub_fun -> lub_fun
huffman [Mon, 06 Dec 2010 10:08:33 -0800] rev 41030
rename lub_fun -> is_lub_fun, thelub_fun -> lub_fun
Mon, 06 Dec 2010 08:59:58 -0800 pcpodef no longer generates _defined lemmas, use _bottom_iff lemmas instead
huffman [Mon, 06 Dec 2010 08:59:58 -0800] rev 41029
pcpodef no longer generates _defined lemmas, use _bottom_iff lemmas instead
Mon, 06 Dec 2010 08:43:52 -0800 cpodef no longer generates lemma is_lub_foo, since it is redundant with lub_foo
huffman [Mon, 06 Dec 2010 08:43:52 -0800] rev 41028
cpodef no longer generates lemma is_lub_foo, since it is redundant with lub_foo
Mon, 06 Dec 2010 08:30:00 -0800 add lemmas lub_APP, lub_LAM
huffman [Mon, 06 Dec 2010 08:30:00 -0800] rev 41027
add lemmas lub_APP, lub_LAM
Mon, 06 Dec 2010 19:54:56 +0100 folding on arbitrary Lebesgue integrable functions
hoelzl [Mon, 06 Dec 2010 19:54:56 +0100] rev 41026
folding on arbitrary Lebesgue integrable functions
Mon, 06 Dec 2010 19:54:53 +0100 fixed spelling errors
hoelzl [Mon, 06 Dec 2010 19:54:53 +0100] rev 41025
fixed spelling errors
Mon, 06 Dec 2010 19:54:48 +0100 move coercions to appropriate places
hoelzl [Mon, 06 Dec 2010 19:54:48 +0100] rev 41024
move coercions to appropriate places
Fri, 03 Dec 2010 15:25:14 +0100 it is known as the extended reals, not the infinite reals
hoelzl [Fri, 03 Dec 2010 15:25:14 +0100] rev 41023
it is known as the extended reals, not the infinite reals
Mon, 06 Dec 2010 19:18:02 +0100 moved coercion decl. for int
nipkow [Mon, 06 Dec 2010 19:18:02 +0100] rev 41022
moved coercion decl. for int
Mon, 06 Dec 2010 17:33:25 +0100 adapting copied bash code in mutabelle script
bulwahn [Mon, 06 Dec 2010 17:33:25 +0100] rev 41021
adapting copied bash code in mutabelle script
Mon, 06 Dec 2010 16:37:15 +0100 more correct NEWS;
wenzelm [Mon, 06 Dec 2010 16:37:15 +0100] rev 41020
more correct NEWS;
Mon, 06 Dec 2010 16:18:56 +0100 merged
wenzelm [Mon, 06 Dec 2010 16:18:56 +0100] rev 41019
merged
Mon, 06 Dec 2010 13:46:45 +0100 fix monotonicity type of None
blanchet [Mon, 06 Dec 2010 13:46:45 +0100] rev 41018
fix monotonicity type of None
Mon, 06 Dec 2010 13:36:28 +0100 compile
blanchet [Mon, 06 Dec 2010 13:36:28 +0100] rev 41017
compile
Mon, 06 Dec 2010 13:33:09 +0100 introduced hack to exploit the symmetry of equality in monotonicity calculus
blanchet [Mon, 06 Dec 2010 13:33:09 +0100] rev 41016
introduced hack to exploit the symmetry of equality in monotonicity calculus
Mon, 06 Dec 2010 13:33:09 +0100 cleanup example
blanchet [Mon, 06 Dec 2010 13:33:09 +0100] rev 41015
cleanup example
Mon, 06 Dec 2010 13:33:09 +0100 add more flexibility to the monotonicity calculus: instead of hardcoding F-arrows, also allow G-arrows, simulating applications of the Sub rule
blanchet [Mon, 06 Dec 2010 13:33:09 +0100] rev 41014
add more flexibility to the monotonicity calculus: instead of hardcoding F-arrows, also allow G-arrows, simulating applications of the Sub rule
Mon, 06 Dec 2010 13:33:09 +0100 fixed bug in monotonicity solution display, whereby the polarity of literals was ignored
blanchet [Mon, 06 Dec 2010 13:33:09 +0100] rev 41013
fixed bug in monotonicity solution display, whereby the polarity of literals was ignored
Mon, 06 Dec 2010 13:33:09 +0100 improve precision of forall in constancy part of the monotonicity calculus
blanchet [Mon, 06 Dec 2010 13:33:09 +0100] rev 41012
improve precision of forall in constancy part of the monotonicity calculus
Mon, 06 Dec 2010 13:33:09 +0100 added some missing well-annotatedness constraints to monotonicity calculus
blanchet [Mon, 06 Dec 2010 13:33:09 +0100] rev 41011
added some missing well-annotatedness constraints to monotonicity calculus
Mon, 06 Dec 2010 13:33:09 +0100 more work on the monotonicity evaluation driver
blanchet [Mon, 06 Dec 2010 13:33:09 +0100] rev 41010
more work on the monotonicity evaluation driver
Mon, 06 Dec 2010 13:33:09 +0100 improve precision of finite functions in monotonicity calculus
blanchet [Mon, 06 Dec 2010 13:33:09 +0100] rev 41009
improve precision of finite functions in monotonicity calculus
Mon, 06 Dec 2010 13:33:09 +0100 added ML code for testing entire theories for monotonicity
blanchet [Mon, 06 Dec 2010 13:33:09 +0100] rev 41008
added ML code for testing entire theories for monotonicity
Mon, 06 Dec 2010 13:33:09 +0100 use ML SAT solvers up to a certain time limit, then switch to faster solvers with a timeout -- this becomes necessary with the new, more powerful monotonicity calculus
blanchet [Mon, 06 Dec 2010 13:33:09 +0100] rev 41007
use ML SAT solvers up to a certain time limit, then switch to faster solvers with a timeout -- this becomes necessary with the new, more powerful monotonicity calculus
Mon, 06 Dec 2010 13:33:09 +0100 added examples to exercise new monotonicity code
blanchet [Mon, 06 Dec 2010 13:33:09 +0100] rev 41006
added examples to exercise new monotonicity code
Mon, 06 Dec 2010 13:33:09 +0100 fixed quantifier handling of new monotonicity calculus
blanchet [Mon, 06 Dec 2010 13:33:09 +0100] rev 41005
fixed quantifier handling of new monotonicity calculus
Mon, 06 Dec 2010 13:33:09 +0100 tune parentheses and indentation
blanchet [Mon, 06 Dec 2010 13:33:09 +0100] rev 41004
tune parentheses and indentation
Mon, 06 Dec 2010 13:33:09 +0100 proper handling of frames for connectives in monotonicity calculus
blanchet [Mon, 06 Dec 2010 13:33:09 +0100] rev 41003
proper handling of frames for connectives in monotonicity calculus
Mon, 06 Dec 2010 13:33:09 +0100 tune indentation
blanchet [Mon, 06 Dec 2010 13:33:09 +0100] rev 41002
tune indentation
Mon, 06 Dec 2010 13:33:09 +0100 removed old baggage from monotonicity calculus -- the "calculus" option didn't really work anyway because of on-the-fly simplifications
blanchet [Mon, 06 Dec 2010 13:33:09 +0100] rev 41001
removed old baggage from monotonicity calculus -- the "calculus" option didn't really work anyway because of on-the-fly simplifications
Mon, 06 Dec 2010 13:33:05 +0100 implemented All rules from new monotonicity calculus
blanchet [Mon, 06 Dec 2010 13:33:05 +0100] rev 41000
implemented All rules from new monotonicity calculus
Mon, 06 Dec 2010 13:30:57 +0100 fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet [Mon, 06 Dec 2010 13:30:57 +0100] rev 40999
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
Mon, 06 Dec 2010 13:30:38 +0100 started implementing the new monotonicity rules for application
blanchet [Mon, 06 Dec 2010 13:30:38 +0100] rev 40998
started implementing the new monotonicity rules for application
Mon, 06 Dec 2010 13:30:36 +0100 implemented connectives in new monotonicity calculus
blanchet [Mon, 06 Dec 2010 13:30:36 +0100] rev 40997
implemented connectives in new monotonicity calculus
Mon, 06 Dec 2010 13:29:23 +0100 added "Neq" operator to monotonicity inference module
blanchet [Mon, 06 Dec 2010 13:29:23 +0100] rev 40996
added "Neq" operator to monotonicity inference module
Mon, 06 Dec 2010 13:26:27 +0100 started implementing connectives in new monotonicity calculus
blanchet [Mon, 06 Dec 2010 13:26:27 +0100] rev 40995
started implementing connectives in new monotonicity calculus
Mon, 06 Dec 2010 13:26:23 +0100 more work on frames in the new monotonicity calculus
blanchet [Mon, 06 Dec 2010 13:26:23 +0100] rev 40994
more work on frames in the new monotonicity calculus
Mon, 06 Dec 2010 13:18:25 +0100 support 3 monotonicity calculi in one and fix soundness bug
blanchet [Mon, 06 Dec 2010 13:18:25 +0100] rev 40993
support 3 monotonicity calculi in one and fix soundness bug
Mon, 06 Dec 2010 13:18:25 +0100 tuning
blanchet [Mon, 06 Dec 2010 13:18:25 +0100] rev 40992
tuning
Mon, 06 Dec 2010 13:18:25 +0100 proper handling of assignment disjunctions vs. conjunctions
blanchet [Mon, 06 Dec 2010 13:18:25 +0100] rev 40991
proper handling of assignment disjunctions vs. conjunctions
Mon, 06 Dec 2010 13:18:25 +0100 adapt monotonicity code to four annotation types
blanchet [Mon, 06 Dec 2010 13:18:25 +0100] rev 40990
adapt monotonicity code to four annotation types
Mon, 06 Dec 2010 13:18:25 +0100 more monotonicity tuning
blanchet [Mon, 06 Dec 2010 13:18:25 +0100] rev 40989
more monotonicity tuning
Mon, 06 Dec 2010 13:18:25 +0100 tuning
blanchet [Mon, 06 Dec 2010 13:18:25 +0100] rev 40988
tuning
Mon, 06 Dec 2010 13:18:25 +0100 added frame component to Gamma in monotonicity calculus
blanchet [Mon, 06 Dec 2010 13:18:25 +0100] rev 40987
added frame component to Gamma in monotonicity calculus
Mon, 06 Dec 2010 13:18:25 +0100 use boolean pair to encode annotation, which may now take four values
blanchet [Mon, 06 Dec 2010 13:18:25 +0100] rev 40986
use boolean pair to encode annotation, which may now take four values
Mon, 06 Dec 2010 13:18:25 +0100 started generalizing monotonicity code to accommodate new calculus
blanchet [Mon, 06 Dec 2010 13:18:25 +0100] rev 40985
started generalizing monotonicity code to accommodate new calculus
Mon, 06 Dec 2010 13:17:26 +0100 merged
blanchet [Mon, 06 Dec 2010 13:17:26 +0100] rev 40984
merged
Mon, 06 Dec 2010 11:41:24 +0100 handle "max_relevant" uniformly
blanchet [Mon, 06 Dec 2010 11:41:24 +0100] rev 40983
handle "max_relevant" uniformly
Mon, 06 Dec 2010 11:26:17 +0100 honor the default max relevant facts setting from the SMT solvers in Sledgehammer
blanchet [Mon, 06 Dec 2010 11:26:17 +0100] rev 40982
honor the default max relevant facts setting from the SMT solvers in Sledgehammer
Mon, 06 Dec 2010 11:25:21 +0100 have SMT solvers report the number of facts that they should have by default in Sledgehammer -- the information might not seem to belong there but it also belongs nowhere else, for how is Sledgehammer to know how different solvers deal with hundreds of facts?
blanchet [Mon, 06 Dec 2010 11:25:21 +0100] rev 40981
have SMT solvers report the number of facts that they should have by default in Sledgehammer -- the information might not seem to belong there but it also belongs nowhere else, for how is Sledgehammer to know how different solvers deal with hundreds of facts?
Mon, 06 Dec 2010 10:32:39 +0100 return all facts for CVC3 and Yices, since there is no proof parsing / unsat core extraction
blanchet [Mon, 06 Dec 2010 10:32:39 +0100] rev 40980
return all facts for CVC3 and Yices, since there is no proof parsing / unsat core extraction
Mon, 06 Dec 2010 10:31:29 +0100 trust SMT filter's timeout -- nested timeouts seem to be at the origin of spontaneous Interrupt exceptions in some cases
blanchet [Mon, 06 Dec 2010 10:31:29 +0100] rev 40979
trust SMT filter's timeout -- nested timeouts seem to be at the origin of spontaneous Interrupt exceptions in some cases
Mon, 06 Dec 2010 10:23:31 +0100 reraise interrupt exceptions
blanchet [Mon, 06 Dec 2010 10:23:31 +0100] rev 40978
reraise interrupt exceptions
Mon, 06 Dec 2010 09:54:58 +0100 [mq]: sledge_binary_minimizer
blanchet [Mon, 06 Dec 2010 09:54:58 +0100] rev 40977
[mq]: sledge_binary_minimizer
Mon, 06 Dec 2010 10:52:48 +0100 correcting usage documentation in mirabelle tool
bulwahn [Mon, 06 Dec 2010 10:52:48 +0100] rev 40976
correcting usage documentation in mirabelle tool
Mon, 06 Dec 2010 10:52:46 +0100 adding mutabelle as a component and an isabelle tool to be used in regression testing
bulwahn [Mon, 06 Dec 2010 10:52:46 +0100] rev 40975
adding mutabelle as a component and an isabelle tool to be used in regression testing
Mon, 06 Dec 2010 10:52:45 +0100 commenting out sledgehammer_mtd in Mutabelle
bulwahn [Mon, 06 Dec 2010 10:52:45 +0100] rev 40974
commenting out sledgehammer_mtd in Mutabelle
Mon, 06 Dec 2010 10:52:45 +0100 removing declaration in quickcheck to really enable exhaustive testing
bulwahn [Mon, 06 Dec 2010 10:52:45 +0100] rev 40973
removing declaration in quickcheck to really enable exhaustive testing
Mon, 06 Dec 2010 10:52:44 +0100 adding timeout to try invocation in mutabelle
bulwahn [Mon, 06 Dec 2010 10:52:44 +0100] rev 40972
adding timeout to try invocation in mutabelle
Mon, 06 Dec 2010 10:52:43 +0100 adding filtering, sytactic welltyping, and sledgehammer method in mutabelle
bulwahn [Mon, 06 Dec 2010 10:52:43 +0100] rev 40971
adding filtering, sytactic welltyping, and sledgehammer method in mutabelle
Mon, 06 Dec 2010 09:34:57 +0100 replace `type_mapper` by the more adequate `type_lifting`
haftmann [Mon, 06 Dec 2010 09:34:57 +0100] rev 40970
replace `type_mapper` by the more adequate `type_lifting`
Mon, 06 Dec 2010 09:25:05 +0100 moved bootstrap of type_lifting to Fun
haftmann [Mon, 06 Dec 2010 09:25:05 +0100] rev 40969
moved bootstrap of type_lifting to Fun
Mon, 06 Dec 2010 09:19:10 +0100 replace `type_mapper` by the more adequate `type_lifting`
haftmann [Mon, 06 Dec 2010 09:19:10 +0100] rev 40968
replace `type_mapper` by the more adequate `type_lifting`
Mon, 06 Dec 2010 14:45:29 +0100 avoid explicit encoding -- acknowledge UTF-8 as global default and Isabelle/jEdit preference of UTF-8-Isabelle;
wenzelm [Mon, 06 Dec 2010 14:45:29 +0100] rev 40967
avoid explicit encoding -- acknowledge UTF-8 as global default and Isabelle/jEdit preference of UTF-8-Isabelle;
Sun, 05 Dec 2010 15:23:33 +0100 IsabelleText font: include Cyrillic, Hebrew, Arabic from DejaVu Sans 2.32;
wenzelm [Sun, 05 Dec 2010 15:23:33 +0100] rev 40966
IsabelleText font: include Cyrillic, Hebrew, Arabic from DejaVu Sans 2.32;
Sun, 05 Dec 2010 14:02:16 +0100 command 'notepad' replaces former 'example_proof';
wenzelm [Sun, 05 Dec 2010 14:02:16 +0100] rev 40965
command 'notepad' replaces former 'example_proof';
Sun, 05 Dec 2010 13:42:58 +0100 prefer 'notepad' over 'example_proof';
wenzelm [Sun, 05 Dec 2010 13:42:58 +0100] rev 40964
prefer 'notepad' over 'example_proof';
Sun, 05 Dec 2010 08:34:02 +0100 merged
haftmann [Sun, 05 Dec 2010 08:34:02 +0100] rev 40963
merged
Sat, 04 Dec 2010 21:53:00 +0100 more intimate definition of fold_list / fold_once in terms of fold
haftmann [Sat, 04 Dec 2010 21:53:00 +0100] rev 40962
more intimate definition of fold_list / fold_once in terms of fold
Sat, 04 Dec 2010 21:26:33 +0100 canonical fold signature
haftmann [Sat, 04 Dec 2010 21:26:33 +0100] rev 40961
canonical fold signature
Sat, 04 Dec 2010 21:26:55 +0100 formal notepad without any result;
wenzelm [Sat, 04 Dec 2010 21:26:55 +0100] rev 40960
formal notepad without any result;
Sat, 04 Dec 2010 18:41:12 +0100 added Syntax.default_root;
wenzelm [Sat, 04 Dec 2010 18:41:12 +0100] rev 40959
added Syntax.default_root; simplified Syntax.parse operations; clarified treatment of syntax root for translation rules -- refrain from logical_type replacement; tuned error message;
Sat, 04 Dec 2010 15:14:28 +0100 eliminated obsolete Token.Malformed -- subsumed by Token.Error;
wenzelm [Sat, 04 Dec 2010 15:14:28 +0100] rev 40958
eliminated obsolete Token.Malformed -- subsumed by Token.Error;
Sat, 04 Dec 2010 14:59:25 +0100 tuned @{datatype} using Syntax.pretty_priority (NB: postfix type application yields Syntax.max_pri, so arguments in prefix application require higher priority);
wenzelm [Sat, 04 Dec 2010 14:59:25 +0100] rev 40957
tuned @{datatype} using Syntax.pretty_priority (NB: postfix type application yields Syntax.max_pri, so arguments in prefix application require higher priority);
Sat, 04 Dec 2010 14:57:04 +0100 added Syntax.pretty_priority;
wenzelm [Sat, 04 Dec 2010 14:57:04 +0100] rev 40956
added Syntax.pretty_priority;
Fri, 03 Dec 2010 22:40:26 +0100 merged
haftmann [Fri, 03 Dec 2010 22:40:26 +0100] rev 40955
merged
Fri, 03 Dec 2010 14:46:58 +0100 conventional point-free characterization of rsp_fold
haftmann [Fri, 03 Dec 2010 14:46:58 +0100] rev 40954
conventional point-free characterization of rsp_fold
Fri, 03 Dec 2010 14:39:15 +0100 replaced memb by existing List.member
haftmann [Fri, 03 Dec 2010 14:39:15 +0100] rev 40953
replaced memb by existing List.member
Fri, 03 Dec 2010 14:22:24 +0100 explicit type constraint;
haftmann [Fri, 03 Dec 2010 14:22:24 +0100] rev 40952
explicit type constraint; streamlined notation
Fri, 03 Dec 2010 22:39:34 +0100 tuned proposition
haftmann [Fri, 03 Dec 2010 22:39:34 +0100] rev 40951
tuned proposition
Fri, 03 Dec 2010 22:34:20 +0100 lemma multiset_of_rev
haftmann [Fri, 03 Dec 2010 22:34:20 +0100] rev 40950
lemma multiset_of_rev
Fri, 03 Dec 2010 22:34:20 +0100 lemmas fold_remove1_split and fold_multiset_equiv
haftmann [Fri, 03 Dec 2010 22:34:20 +0100] rev 40949
lemmas fold_remove1_split and fold_multiset_equiv
Fri, 03 Dec 2010 22:08:14 +0100 minor tuning for release;
wenzelm [Fri, 03 Dec 2010 22:08:14 +0100] rev 40948
minor tuning for release;
Fri, 03 Dec 2010 21:34:54 +0100 source files are always encoded as UTF-8;
wenzelm [Fri, 03 Dec 2010 21:34:54 +0100] rev 40947
source files are always encoded as UTF-8;
Fri, 03 Dec 2010 21:30:41 +0100 eliminated fragile HTML.with_charset -- always use utf-8;
wenzelm [Fri, 03 Dec 2010 21:30:41 +0100] rev 40946
eliminated fragile HTML.with_charset -- always use utf-8;
Fri, 03 Dec 2010 20:38:58 +0100 recoded latin1 as utf8;
wenzelm [Fri, 03 Dec 2010 20:38:58 +0100] rev 40945
recoded latin1 as utf8; use textcomp for some text symbols where it appears appropriate;
Fri, 03 Dec 2010 20:26:57 +0100 removed old generated stuff;
wenzelm [Fri, 03 Dec 2010 20:26:57 +0100] rev 40944
removed old generated stuff; removed DOS line endings;
Fri, 03 Dec 2010 20:02:57 +0100 comment;
wenzelm [Fri, 03 Dec 2010 20:02:57 +0100] rev 40943
comment;
Fri, 03 Dec 2010 18:29:49 +0100 update documentation
blanchet [Fri, 03 Dec 2010 18:29:49 +0100] rev 40942
update documentation
Fri, 03 Dec 2010 18:29:14 +0100 replace "smt" prover with specific SMT solvers, e.g. "z3" -- whatever the SMT module gives us
blanchet [Fri, 03 Dec 2010 18:29:14 +0100] rev 40941
replace "smt" prover with specific SMT solvers, e.g. "z3" -- whatever the SMT module gives us
Fri, 03 Dec 2010 18:27:21 +0100 export more information about available SMT solvers
blanchet [Fri, 03 Dec 2010 18:27:21 +0100] rev 40940
export more information about available SMT solvers
(0) -30000 -10000 -3000 -1000 -128 +128 +1000 +3000 +10000 +30000 tip