Tue, 04 May 2010 14:10:42 +0200 merged
berghofe [Tue, 04 May 2010 14:10:42 +0200] rev 36644
merged
Tue, 04 May 2010 14:11:28 +0200 Turned Sem into an inductive definition.
berghofe [Tue, 04 May 2010 14:11:28 +0200] rev 36643
Turned Sem into an inductive definition.
Tue, 04 May 2010 12:29:22 +0200 Corrected handling of "for" parameters.
berghofe [Tue, 04 May 2010 12:29:22 +0200] rev 36642
Corrected handling of "for" parameters.
Tue, 04 May 2010 12:26:46 +0200 induct_true_def and induct_false_def are already contained in induct_rulify_fallback.
berghofe [Tue, 04 May 2010 12:26:46 +0200] rev 36641
induct_true_def and induct_false_def are already contained in induct_rulify_fallback.
Tue, 04 May 2010 11:00:17 +0200 added lemma about irreflexivity of pointer inequality in Imperative_HOL
bulwahn [Tue, 04 May 2010 11:00:17 +0200] rev 36640
added lemma about irreflexivity of pointer inequality in Imperative_HOL
Tue, 04 May 2010 11:00:16 +0200 added function ffilter and some lemmas from Finite_Set to the FSet theory
bulwahn [Tue, 04 May 2010 11:00:16 +0200] rev 36639
added function ffilter and some lemmas from Finite_Set to the FSet theory
Tue, 04 May 2010 10:49:46 +0200 merged
haftmann [Tue, 04 May 2010 10:49:46 +0200] rev 36638
merged
Tue, 04 May 2010 10:02:43 +0200 avoid if on rhs of default simp rules
haftmann [Tue, 04 May 2010 10:02:43 +0200] rev 36637
avoid if on rhs of default simp rules
Tue, 04 May 2010 09:25:38 +0200 avoid exception Empty on malformed goal
krauss [Tue, 04 May 2010 09:25:38 +0200] rev 36636
avoid exception Empty on malformed goal
Tue, 04 May 2010 08:55:43 +0200 locale predicates of classes carry a mandatory "class" prefix
haftmann [Tue, 04 May 2010 08:55:43 +0200] rev 36635
locale predicates of classes carry a mandatory "class" prefix
Tue, 04 May 2010 08:55:39 +0200 a ring_div is a ring_1_no_zero_divisors
haftmann [Tue, 04 May 2010 08:55:39 +0200] rev 36634
a ring_div is a ring_1_no_zero_divisors
Tue, 04 May 2010 08:55:34 +0200 NEWS
haftmann [Tue, 04 May 2010 08:55:34 +0200] rev 36633
NEWS
Mon, 03 May 2010 10:28:19 -0700 merged
huffman [Mon, 03 May 2010 10:28:19 -0700] rev 36632
merged
Sat, 01 May 2010 16:13:24 -0700 merged
huffman [Sat, 01 May 2010 16:13:24 -0700] rev 36631
merged
Sat, 01 May 2010 11:46:47 -0700 complete_lattice instance for net type
huffman [Sat, 01 May 2010 11:46:47 -0700] rev 36630
complete_lattice instance for net type
Sat, 01 May 2010 09:43:40 -0700 swap ordering on nets, so x <= y means 'x is finer than y'
huffman [Sat, 01 May 2010 09:43:40 -0700] rev 36629
swap ordering on nets, so x <= y means 'x is finer than y'
Sat, 01 May 2010 07:53:42 -0700 fixrec no longer uses global simpset internally to prove equations
huffman [Sat, 01 May 2010 07:53:42 -0700] rev 36628
fixrec no longer uses global simpset internally to prove equations
Sat, 01 May 2010 07:35:22 -0700 move setsum lemmas to Product_plus.thy
huffman [Sat, 01 May 2010 07:35:22 -0700] rev 36627
move setsum lemmas to Product_plus.thy
Fri, 30 Apr 2010 13:51:17 -0700 remove duplicate lemmas
huffman [Fri, 30 Apr 2010 13:51:17 -0700] rev 36626
remove duplicate lemmas
Fri, 30 Apr 2010 13:31:32 -0700 add lemmas about convergent
huffman [Fri, 30 Apr 2010 13:31:32 -0700] rev 36625
add lemmas about convergent
Mon, 03 May 2010 14:35:10 +0200 Cleanup information theory
hoelzl [Mon, 03 May 2010 14:35:10 +0200] rev 36624
Cleanup information theory
Mon, 03 May 2010 14:35:10 +0200 Moved Convex theory to library.
hoelzl [Mon, 03 May 2010 14:35:10 +0200] rev 36623
Moved Convex theory to library.
Tue, 20 Apr 2010 17:58:34 +0200 Generalize swap_inj_on; add simps for Times; add Ex_list_of_length, log_inj; Added missing locale edges for linordered semiring with 1.
hoelzl [Tue, 20 Apr 2010 17:58:34 +0200] rev 36622
Generalize swap_inj_on; add simps for Times; add Ex_list_of_length, log_inj; Added missing locale edges for linordered semiring with 1.
Tue, 04 May 2010 14:38:59 +0200 proof terms for strip_shyps, based on the version by krauss/schropp with some notable differences:
wenzelm [Tue, 04 May 2010 14:38:59 +0200] rev 36621
proof terms for strip_shyps, based on the version by krauss/schropp with some notable differences: * present type variables are only compared wrt. first component (the atomic type), not the duplicated sort; * extra sorts are grounded towards fixed 'a, potentially with different sorts (the original version with Name.names could cause name clashes with other present variables, too, but this should not be a problem); * deriv_rule_unconditional ensures that proof terms are always maintained independently of the "proofs" flag -- this improves robustness and preserves basic PThm proofs required for extraction attributes, e.g. in theory HOL/Extraction;
Tue, 04 May 2010 12:30:15 +0200 simplified/unified fundamental operations on types/terms/proofterms -- prefer Same.operation over "option" variant;
wenzelm [Tue, 04 May 2010 12:30:15 +0200] rev 36620
simplified/unified fundamental operations on types/terms/proofterms -- prefer Same.operation over "option" variant;
Tue, 04 May 2010 11:02:50 +0200 renamed Proofterm.freezeT to Proofterm.legacy_freezeT (cf. 88756a5a92fc);
wenzelm [Tue, 04 May 2010 11:02:50 +0200] rev 36619
renamed Proofterm.freezeT to Proofterm.legacy_freezeT (cf. 88756a5a92fc);
Tue, 04 May 2010 10:52:43 +0200 specification goal: eliminated redundant Thm.legacy_freezeT -- the goal is properly declared and should always produce fixed types in the result;
wenzelm [Tue, 04 May 2010 10:52:43 +0200] rev 36618
specification goal: eliminated redundant Thm.legacy_freezeT -- the goal is properly declared and should always produce fixed types in the result; specification result: replaced Thm.legacy_freezeT by Thm.unvarify_global -- the final result appears to be a closed term that is globally exported;
Mon, 03 May 2010 22:00:06 +0200 UNDISCH/DISJ_CASESL: eliminated slightly odd Thm.legacy_freezeT -- these rules appear to be applied to thms with fixed types only;
wenzelm [Mon, 03 May 2010 22:00:06 +0200] rev 36617
UNDISCH/DISJ_CASESL: eliminated slightly odd Thm.legacy_freezeT -- these rules appear to be applied to thms with fixed types only;
Mon, 03 May 2010 20:53:49 +0200 replaced Thm.legacy_freezeT by Thm.unvarify_global -- these facts stem from closed definitions, i.e. there are no term Vars;
wenzelm [Mon, 03 May 2010 20:53:49 +0200] rev 36616
replaced Thm.legacy_freezeT by Thm.unvarify_global -- these facts stem from closed definitions, i.e. there are no term Vars;
Mon, 03 May 2010 20:13:36 +0200 renamed Thm.freezeT to Thm.legacy_freezeT -- it is based on Type.legacy_freeze;
wenzelm [Mon, 03 May 2010 20:13:36 +0200] rev 36615
renamed Thm.freezeT to Thm.legacy_freezeT -- it is based on Type.legacy_freeze;
Mon, 03 May 2010 16:26:47 +0200 minor tuning of Thm.strip_shyps -- no longer pervasive;
wenzelm [Mon, 03 May 2010 16:26:47 +0200] rev 36614
minor tuning of Thm.strip_shyps -- no longer pervasive;
Mon, 03 May 2010 15:34:55 +0200 simplified primitive Thm.future: more direct theory check, do not hardwire strip_shyps here;
wenzelm [Mon, 03 May 2010 15:34:55 +0200] rev 36613
simplified primitive Thm.future: more direct theory check, do not hardwire strip_shyps here;
Mon, 03 May 2010 14:38:18 +0200 old NEWS on global operations;
wenzelm [Mon, 03 May 2010 14:38:18 +0200] rev 36612
old NEWS on global operations;
Mon, 03 May 2010 14:31:33 +0200 ProofContext.init_global;
wenzelm [Mon, 03 May 2010 14:31:33 +0200] rev 36611
ProofContext.init_global;
Mon, 03 May 2010 14:25:56 +0200 renamed ProofContext.init to ProofContext.init_global to emphasize that this is not the real thing;
wenzelm [Mon, 03 May 2010 14:25:56 +0200] rev 36610
renamed ProofContext.init to ProofContext.init_global to emphasize that this is not the real thing;
Mon, 03 May 2010 07:59:51 +0200 merged
haftmann [Mon, 03 May 2010 07:59:51 +0200] rev 36609
merged
Fri, 30 Apr 2010 18:34:51 +0200 do not generate code per default -- touches file of parent session
haftmann [Fri, 30 Apr 2010 18:34:51 +0200] rev 36608
do not generate code per default -- touches file of parent session
Sat, 01 May 2010 21:29:03 +0200 made sml/nj happy about Sledgehammer and Nitpick (cf. 6f11c9b1fb3e, 3c2438efe224)
krauss [Sat, 01 May 2010 21:29:03 +0200] rev 36607
made sml/nj happy about Sledgehammer and Nitpick (cf. 6f11c9b1fb3e, 3c2438efe224)
Sat, 01 May 2010 20:49:39 +0200 Backed out changeset 6f11c9b1fb3e (breaks compilation of HOL image)
krauss [Sat, 01 May 2010 20:49:39 +0200] rev 36606
Backed out changeset 6f11c9b1fb3e (breaks compilation of HOL image)
Sat, 01 May 2010 10:37:31 +0200 now if this doesn't make SML/NJ happy, nothing will
blanchet [Sat, 01 May 2010 10:37:31 +0200] rev 36605
now if this doesn't make SML/NJ happy, nothing will
Sat, 01 May 2010 00:23:57 +0200 more stats;
wenzelm [Sat, 01 May 2010 00:23:57 +0200] rev 36604
more stats;
Fri, 30 Apr 2010 23:53:37 +0200 renamed Variable.thm_context to Variable.global_thm_context to emphasize that this is not the real thing;
wenzelm [Fri, 30 Apr 2010 23:53:37 +0200] rev 36603
renamed Variable.thm_context to Variable.global_thm_context to emphasize that this is not the real thing;
Fri, 30 Apr 2010 23:43:09 +0200 slightly more standard induct_simp_add/del attributes;
wenzelm [Fri, 30 Apr 2010 23:43:09 +0200] rev 36602
slightly more standard induct_simp_add/del attributes; provide explicit context for internal addsimps;
Fri, 30 Apr 2010 23:40:14 +0200 map_css: explicitly provide a temporary context, which might be required for mksimps, mkcongs etc.;
wenzelm [Fri, 30 Apr 2010 23:40:14 +0200] rev 36601
map_css: explicitly provide a temporary context, which might be required for mksimps, mkcongs etc.;
Fri, 30 Apr 2010 23:33:42 +0200 export Simplifier.with_context;
wenzelm [Fri, 30 Apr 2010 23:33:42 +0200] rev 36600
export Simplifier.with_context;
Fri, 30 Apr 2010 21:10:57 +0200 removed some old comments;
wenzelm [Fri, 30 Apr 2010 21:10:57 +0200] rev 36599
removed some old comments;
Fri, 30 Apr 2010 09:54:04 -0700 merged
huffman [Fri, 30 Apr 2010 09:54:04 -0700] rev 36598
merged
Fri, 30 Apr 2010 08:47:07 -0700 merged
huffman [Fri, 30 Apr 2010 08:47:07 -0700] rev 36597
merged
Thu, 29 Apr 2010 15:24:22 -0700 generalize lemma adjoint_unique; simplify some proofs
huffman [Thu, 29 Apr 2010 15:24:22 -0700] rev 36596
generalize lemma adjoint_unique; simplify some proofs
Thu, 29 Apr 2010 14:32:24 -0700 fix latex url
huffman [Thu, 29 Apr 2010 14:32:24 -0700] rev 36595
fix latex url
Thu, 29 Apr 2010 11:42:34 -0700 merged
huffman [Thu, 29 Apr 2010 11:42:34 -0700] rev 36594
merged
Thu, 29 Apr 2010 11:41:04 -0700 define linear algebra concepts using scaleR instead of (op *s); generalized many lemmas, though a few theorems that used to work on type int^'n are a bit less general
huffman [Thu, 29 Apr 2010 11:41:04 -0700] rev 36593
define linear algebra concepts using scaleR instead of (op *s); generalized many lemmas, though a few theorems that used to work on type int^'n are a bit less general
Thu, 29 Apr 2010 09:29:47 -0700 remove unused function vector_power, unused lemma one_plus_of_nat_neq_0
huffman [Thu, 29 Apr 2010 09:29:47 -0700] rev 36592
remove unused function vector_power, unused lemma one_plus_of_nat_neq_0
Thu, 29 Apr 2010 09:17:25 -0700 move class instantiations from Euclidean_Space.thy to Finite_Cartesian_Product.thy
huffman [Thu, 29 Apr 2010 09:17:25 -0700] rev 36591
move class instantiations from Euclidean_Space.thy to Finite_Cartesian_Product.thy
Thu, 29 Apr 2010 07:22:01 -0700 remove redundant constants pastecart, fstcart, sndcart; users should prefer Pair, fst, snd instead
huffman [Thu, 29 Apr 2010 07:22:01 -0700] rev 36590
remove redundant constants pastecart, fstcart, sndcart; users should prefer Pair, fst, snd instead
Wed, 28 Apr 2010 23:08:31 -0700 generalize LIMSEQ_vector to tendsto_vector
huffman [Wed, 28 Apr 2010 23:08:31 -0700] rev 36589
generalize LIMSEQ_vector to tendsto_vector
Wed, 28 Apr 2010 22:36:45 -0700 generalize orthogonal_clauses
huffman [Wed, 28 Apr 2010 22:36:45 -0700] rev 36588
generalize orthogonal_clauses
Wed, 28 Apr 2010 22:20:59 -0700 remove redundant lemma vector_dist_norm
huffman [Wed, 28 Apr 2010 22:20:59 -0700] rev 36587
remove redundant lemma vector_dist_norm
Wed, 28 Apr 2010 22:02:55 -0700 remove redundant lemma norm_0
huffman [Wed, 28 Apr 2010 22:02:55 -0700] rev 36586
remove redundant lemma norm_0
Wed, 28 Apr 2010 21:39:14 -0700 generalize some euclidean space lemmas
huffman [Wed, 28 Apr 2010 21:39:14 -0700] rev 36585
generalize some euclidean space lemmas
Wed, 28 Apr 2010 17:48:59 -0700 prove lemma openin_subopen without using choice
huffman [Wed, 28 Apr 2010 17:48:59 -0700] rev 36584
prove lemma openin_subopen without using choice
Wed, 28 Apr 2010 16:11:07 -0700 move path-related stuff into new theory file
huffman [Wed, 28 Apr 2010 16:11:07 -0700] rev 36583
move path-related stuff into new theory file
Wed, 28 Apr 2010 15:07:03 -0700 add new Multivariate_Analysis files to IsaMakefile
huffman [Wed, 28 Apr 2010 15:07:03 -0700] rev 36582
add new Multivariate_Analysis files to IsaMakefile
Wed, 28 Apr 2010 15:05:45 -0700 move operator norm stuff to new theory file
huffman [Wed, 28 Apr 2010 15:05:45 -0700] rev 36581
move operator norm stuff to new theory file
Fri, 30 Apr 2010 18:29:04 +0200 eliminated spurious sledgehammer invocation;
wenzelm [Fri, 30 Apr 2010 18:29:04 +0200] rev 36580
eliminated spurious sledgehammer invocation;
Fri, 30 Apr 2010 18:12:41 +0200 merged
wenzelm [Fri, 30 Apr 2010 18:12:41 +0200] rev 36579
merged
Fri, 30 Apr 2010 17:53:49 +0200 merged
haftmann [Fri, 30 Apr 2010 17:53:49 +0200] rev 36578
merged
Fri, 30 Apr 2010 14:23:00 +0200 merged
haftmann [Fri, 30 Apr 2010 14:23:00 +0200] rev 36577
merged
Fri, 30 Apr 2010 14:20:55 +0200 enclose case expression in brackets
haftmann [Fri, 30 Apr 2010 14:20:55 +0200] rev 36576
enclose case expression in brackets
Fri, 30 Apr 2010 14:58:21 +0200 catch the right exception
blanchet [Fri, 30 Apr 2010 14:58:21 +0200] rev 36575
catch the right exception
Fri, 30 Apr 2010 14:52:49 +0200 eliminate trivial case splits from Isar proofs
blanchet [Fri, 30 Apr 2010 14:52:49 +0200] rev 36574
eliminate trivial case splits from Isar proofs
Fri, 30 Apr 2010 14:52:06 +0200 remove debugging code
blanchet [Fri, 30 Apr 2010 14:52:06 +0200] rev 36573
remove debugging code
Fri, 30 Apr 2010 14:00:47 +0200 merged
blanchet [Fri, 30 Apr 2010 14:00:47 +0200] rev 36572
merged
Fri, 30 Apr 2010 14:00:09 +0200 minor improvements
blanchet [Fri, 30 Apr 2010 14:00:09 +0200] rev 36571
minor improvements
Fri, 30 Apr 2010 13:58:35 +0200 identify axioms/conjectures more reliably in ATP proofs (an empty dependency list doesn't always indicate an axiom or conjecture!)
blanchet [Fri, 30 Apr 2010 13:58:35 +0200] rev 36570
identify axioms/conjectures more reliably in ATP proofs (an empty dependency list doesn't always indicate an axiom or conjecture!)
Fri, 30 Apr 2010 09:36:45 +0200 added "no_atp" for theorems that are automatically used or included by Sledgehammer when appropriate (about combinators and fequal)
blanchet [Fri, 30 Apr 2010 09:36:45 +0200] rev 36569
added "no_atp" for theorems that are automatically used or included by Sledgehammer when appropriate (about combinators and fequal)
Thu, 29 Apr 2010 19:08:02 +0200 in "overlord" mode: ignore problem prefix specified in the .thy file
blanchet [Thu, 29 Apr 2010 19:08:02 +0200] rev 36568
in "overlord" mode: ignore problem prefix specified in the .thy file
Thu, 29 Apr 2010 19:07:36 +0200 uncomment code
blanchet [Thu, 29 Apr 2010 19:07:36 +0200] rev 36567
uncomment code
Thu, 29 Apr 2010 19:02:04 +0200 redid some Sledgehammer/Metis proofs
blanchet [Thu, 29 Apr 2010 19:02:04 +0200] rev 36566
redid some Sledgehammer/Metis proofs
Thu, 29 Apr 2010 18:24:52 +0200 fix more "undeclared symbol" errors related to SPASS's DFG format
blanchet [Thu, 29 Apr 2010 18:24:52 +0200] rev 36565
fix more "undeclared symbol" errors related to SPASS's DFG format
Thu, 29 Apr 2010 17:45:39 +0200 be more discriminate: some one-line Isar proofs are silly
blanchet [Thu, 29 Apr 2010 17:45:39 +0200] rev 36564
be more discriminate: some one-line Isar proofs are silly
Thu, 29 Apr 2010 17:39:46 +0200 one-step Isar proofs are not always pointless
blanchet [Thu, 29 Apr 2010 17:39:46 +0200] rev 36563
one-step Isar proofs are not always pointless
Thu, 29 Apr 2010 17:31:08 +0200 the SPASS output syntax is more general than I thought -- such a pity that there's no documentation
blanchet [Thu, 29 Apr 2010 17:31:08 +0200] rev 36562
the SPASS output syntax is more general than I thought -- such a pity that there's no documentation
Thu, 29 Apr 2010 13:41:51 +0200 redo more Metis/Sledgehammer example
blanchet [Thu, 29 Apr 2010 13:41:51 +0200] rev 36561
redo more Metis/Sledgehammer example
Thu, 29 Apr 2010 12:21:20 +0200 fixed definition of "bad frees" so that it actually works
blanchet [Thu, 29 Apr 2010 12:21:20 +0200] rev 36560
fixed definition of "bad frees" so that it actually works
Thu, 29 Apr 2010 11:38:23 +0200 don't remove last line of proof
blanchet [Thu, 29 Apr 2010 11:38:23 +0200] rev 36559
don't remove last line of proof
Thu, 29 Apr 2010 11:22:24 +0200 handle previously unknown SPASS syntaxes in Sledgehammer's proof reconstruction
blanchet [Thu, 29 Apr 2010 11:22:24 +0200] rev 36558
handle previously unknown SPASS syntaxes in Sledgehammer's proof reconstruction
Thu, 29 Apr 2010 10:55:59 +0200 make SML/NJ happy, take 2
blanchet [Thu, 29 Apr 2010 10:55:59 +0200] rev 36557
make SML/NJ happy, take 2
Thu, 29 Apr 2010 10:25:26 +0200 use readable names in "debug" mode for type vars + don't pipe facts using "using" but rather give them directly to metis (works better with type variables)
blanchet [Thu, 29 Apr 2010 10:25:26 +0200] rev 36556
use readable names in "debug" mode for type vars + don't pipe facts using "using" but rather give them directly to metis (works better with type variables)
Thu, 29 Apr 2010 01:17:14 +0200 expand combinators in Isar proofs constructed by Sledgehammer;
blanchet [Thu, 29 Apr 2010 01:17:14 +0200] rev 36555
expand combinators in Isar proofs constructed by Sledgehammer; this requires shuffling around a couple of functions previously defined in Refute
Thu, 29 Apr 2010 01:11:06 +0200 more neg_clausify proofs that get replaced by direct proofs
blanchet [Thu, 29 Apr 2010 01:11:06 +0200] rev 36554
more neg_clausify proofs that get replaced by direct proofs
Wed, 28 Apr 2010 22:36:39 +0200 redo some of the metis proofs
blanchet [Wed, 28 Apr 2010 22:36:39 +0200] rev 36553
redo some of the metis proofs
Wed, 28 Apr 2010 22:00:48 +0200 back to Vampire 9 -- Vampire 11 sometimes outputs really weird proofs
blanchet [Wed, 28 Apr 2010 22:00:48 +0200] rev 36552
back to Vampire 9 -- Vampire 11 sometimes outputs really weird proofs
Wed, 28 Apr 2010 21:59:29 +0200 improve unskolemization
blanchet [Wed, 28 Apr 2010 21:59:29 +0200] rev 36551
improve unskolemization
Wed, 28 Apr 2010 18:11:11 +0200 make sure short theorem names are preferred to composite ones in Sledgehammer;
blanchet [Wed, 28 Apr 2010 18:11:11 +0200] rev 36550
make sure short theorem names are preferred to composite ones in Sledgehammer; this code used to work at some point
Wed, 28 Apr 2010 17:56:07 +0200 properly extract SPASS proof
blanchet [Wed, 28 Apr 2010 17:56:07 +0200] rev 36549
properly extract SPASS proof
Wed, 28 Apr 2010 17:47:30 +0200 try out Vampire 11 and parse its output correctly;
blanchet [Wed, 28 Apr 2010 17:47:30 +0200] rev 36548
try out Vampire 11 and parse its output correctly; will revert to Vampire 9 if 11 doesn't perform as well
Fri, 30 Apr 2010 13:47:39 +0200 return updated info record after termination proof
krauss [Fri, 30 Apr 2010 13:47:39 +0200] rev 36547
return updated info record after termination proof
Fri, 30 Apr 2010 18:06:29 +0200 proper context for rule_by_tactic;
wenzelm [Fri, 30 Apr 2010 18:06:29 +0200] rev 36546
proper context for rule_by_tactic;
Fri, 30 Apr 2010 17:18:29 +0200 conditional warnings: explicitly observe context visibility flag, not just accidental presence of a context;
wenzelm [Fri, 30 Apr 2010 17:18:29 +0200] rev 36545
conditional warnings: explicitly observe context visibility flag, not just accidental presence of a context; map_ss: explicitly provide a temporary context, which might be required for mksimps, mkcongs etc.;
Thu, 29 Apr 2010 23:55:43 +0200 hgweb style: show author in filelog; full description in annotate hover
krauss [Thu, 29 Apr 2010 23:55:43 +0200] rev 36544
hgweb style: show author in filelog; full description in annotate hover
Thu, 29 Apr 2010 22:56:32 +0200 proper context for mksimps etc. -- via simpset of the running Simplifier;
wenzelm [Thu, 29 Apr 2010 22:56:32 +0200] rev 36543
proper context for mksimps etc. -- via simpset of the running Simplifier;
Thu, 29 Apr 2010 22:08:57 +0200 read_const: disallow internal names as usual in visible Isar text;
wenzelm [Thu, 29 Apr 2010 22:08:57 +0200] rev 36542
read_const: disallow internal names as usual in visible Isar text;
Thu, 29 Apr 2010 21:05:54 +0200 more explicit treatment of context, although not fully localized;
wenzelm [Thu, 29 Apr 2010 21:05:54 +0200] rev 36541
more explicit treatment of context, although not fully localized;
Thu, 29 Apr 2010 20:00:26 +0200 removed some Emacs junk;
wenzelm [Thu, 29 Apr 2010 20:00:26 +0200] rev 36540
removed some Emacs junk;
Thu, 29 Apr 2010 18:41:38 +0200 merged
haftmann [Thu, 29 Apr 2010 18:41:38 +0200] rev 36539
merged
Thu, 29 Apr 2010 15:22:16 +0200 make random engine persistent using code_reflect
haftmann [Thu, 29 Apr 2010 15:22:16 +0200] rev 36538
make random engine persistent using code_reflect
Thu, 29 Apr 2010 15:00:43 +0200 repaired subtle misunderstanding: statement names are only passed for name resolution
haftmann [Thu, 29 Apr 2010 15:00:43 +0200] rev 36537
repaired subtle misunderstanding: statement names are only passed for name resolution
Thu, 29 Apr 2010 15:00:43 +0200 fixed underscore typo
haftmann [Thu, 29 Apr 2010 15:00:43 +0200] rev 36536
fixed underscore typo
Thu, 29 Apr 2010 15:00:42 +0200 more coherent naming with ML serializer
haftmann [Thu, 29 Apr 2010 15:00:42 +0200] rev 36535
more coherent naming with ML serializer
Thu, 29 Apr 2010 15:00:42 +0200 dropped code_datatype antiquotation
haftmann [Thu, 29 Apr 2010 15:00:42 +0200] rev 36534
dropped code_datatype antiquotation
Thu, 29 Apr 2010 15:00:41 +0200 dropped unnecessary ML code
haftmann [Thu, 29 Apr 2010 15:00:41 +0200] rev 36533
dropped unnecessary ML code
Thu, 29 Apr 2010 15:00:41 +0200 avoid popular infixes
haftmann [Thu, 29 Apr 2010 15:00:41 +0200] rev 36532
avoid popular infixes
Thu, 29 Apr 2010 15:00:40 +0200 code_reflect: specify module name directly after keyword
haftmann [Thu, 29 Apr 2010 15:00:40 +0200] rev 36531
code_reflect: specify module name directly after keyword
Thu, 29 Apr 2010 15:00:39 +0200 NEWS: code_reflect
haftmann [Thu, 29 Apr 2010 15:00:39 +0200] rev 36530
NEWS: code_reflect
Thu, 29 Apr 2010 10:35:09 +0200 merged
haftmann [Thu, 29 Apr 2010 10:35:09 +0200] rev 36529
merged
Wed, 28 Apr 2010 21:41:06 +0200 updated generated file
haftmann [Wed, 28 Apr 2010 21:41:06 +0200] rev 36528
updated generated file
Wed, 28 Apr 2010 21:41:05 +0200 modernized structure name
haftmann [Wed, 28 Apr 2010 21:41:05 +0200] rev 36527
modernized structure name
Wed, 28 Apr 2010 21:41:05 +0200 use code_reflect
haftmann [Wed, 28 Apr 2010 21:41:05 +0200] rev 36526
use code_reflect
Thu, 29 Apr 2010 17:50:11 +0200 merged
wenzelm [Thu, 29 Apr 2010 17:50:11 +0200] rev 36525
merged
(0) -30000 -10000 -3000 -1000 -120 +120 +1000 +3000 +10000 +30000 tip