traytel [Wed, 24 Apr 2013 12:15:06 +0200] rev 51753
took out workaround for bug fixed in 5af40820948b
traytel [Wed, 24 Apr 2013 11:36:11 +0200] rev 51752
merged
traytel [Wed, 24 Apr 2013 11:06:53 +0200] rev 51751
slightly more aggressive syntax translation for printing case expressions
haftmann [Wed, 24 Apr 2013 11:32:54 +0200] rev 51750
avoid odd reinit after sublocale declaration
nipkow [Wed, 24 Apr 2013 10:23:47 +0200] rev 51749
moved defs into locale to reduce unnecessary polymorphism; tuned
haftmann [Tue, 23 Apr 2013 19:40:33 +0200] rev 51748
dropped dead code
haftmann [Tue, 23 Apr 2013 19:31:24 +0200] rev 51747
documentation and NEWS
blanchet [Tue, 23 Apr 2013 17:46:12 +0200] rev 51746
avoid accidental specialization of the types in the "map" property of codatatypes
blanchet [Tue, 23 Apr 2013 17:15:44 +0200] rev 51745
simplify "Inl () = Inr ()" as well (not entirely clear why this is necessary)
blanchet [Tue, 23 Apr 2013 17:13:14 +0200] rev 51744
more examples
blanchet [Tue, 23 Apr 2013 16:49:14 +0200] rev 51743
tuning
blanchet [Tue, 23 Apr 2013 16:41:59 +0200] rev 51742
fix bugs in expand tactic w.r.t. datatypes with "needless" discriminators (e.g. lists with is_Nil instead of ~= Nil)
blanchet [Tue, 23 Apr 2013 16:30:30 +0200] rev 51741
tuning
blanchet [Tue, 23 Apr 2013 16:30:29 +0200] rev 51740
tuned_comment
traytel [Tue, 23 Apr 2013 11:43:09 +0200] rev 51739
(co)rec is (just as the (un)fold) the unique morphism;
haftmann [Tue, 23 Apr 2013 11:14:51 +0200] rev 51738
tuned: unnamed contexts, interpretation and sublocale in locale target;
corrected slip in List.thy: setsum requires commmutativity
haftmann [Tue, 23 Apr 2013 11:14:50 +0200] rev 51737
target-sensitive user-level commands interpretation and sublocale
haftmann [Tue, 23 Apr 2013 11:14:50 +0200] rev 51736
ML interfaces for various kinds of interpretation
haftmann [Tue, 23 Apr 2013 11:14:50 +0200] rev 51735
brittleness stamping for local theories
haftmann [Tue, 23 Apr 2013 11:14:50 +0200] rev 51734
tuned
immler [Mon, 22 Apr 2013 18:39:12 +0200] rev 51733
removed type constraints
hoelzl [Mon, 22 Apr 2013 16:36:02 +0200] rev 51732
NEWS
haftmann [Sun, 21 Apr 2013 20:08:13 +0200] rev 51731
more sharing
haftmann [Sun, 21 Apr 2013 16:29:40 +0200] rev 51730
interpretation: distinguish theories and proofs by explicit parameter rather than generic context;
formal initialisation of theory target during interpretation;
prefer Local_Theory.notes_kind to register mixin equations during interpretation;
more uniformity between note_eqns_register and note_eqns_dependency
haftmann [Sun, 21 Apr 2013 10:41:18 +0200] rev 51729
dropped unusued identifier
haftmann [Sun, 21 Apr 2013 10:41:18 +0200] rev 51728
avoid odd bifurcation with Attrib.local_notes vs. Locale.add_thmss -- n.b. note_eqns_dependency operates in a specific locale target
haftmann [Sun, 21 Apr 2013 10:41:18 +0200] rev 51727
tuned for uniformity
haftmann [Sun, 21 Apr 2013 10:41:18 +0200] rev 51726
reflection as official HOL tool
haftmann [Sun, 21 Apr 2013 10:41:18 +0200] rev 51725
follow Isabelle spacing praxis more thoroughly
haftmann [Sun, 21 Apr 2013 10:41:18 +0200] rev 51724
honour FIXMEs as far as feasible at the moment
haftmann [Sun, 21 Apr 2013 10:41:18 +0200] rev 51723
combined reify_data.ML into reflection.ML;
attempt to establish a more accessible and more consistent terminology;
more ML code in ML file rather than setup theory;
ML slightly tuned wrt. Isabelle coding conventions
nipkow [Sat, 20 Apr 2013 20:57:49 +0200] rev 51722
proved termination for fun-based AI
nipkow [Sat, 20 Apr 2013 19:30:04 +0200] rev 51721
tuned
nipkow [Fri, 19 Apr 2013 12:04:57 +0200] rev 51720
tuned
wenzelm [Thu, 18 Apr 2013 21:31:24 +0200] rev 51719
merged
wenzelm [Thu, 18 Apr 2013 21:10:12 +0200] rev 51718
tuned signature;
wenzelm [Thu, 18 Apr 2013 17:07:01 +0200] rev 51717
simplifier uses proper Proof.context instead of historic type simpset;
nipkow [Thu, 18 Apr 2013 20:18:50 +0200] rev 51716
merged
nipkow [Thu, 18 Apr 2013 20:18:37 +0200] rev 51715
avoided map_of in def of fun_rep (but still needed for efficient code)
haftmann [Thu, 18 Apr 2013 18:57:02 +0200] rev 51714
spelling
haftmann [Thu, 18 Apr 2013 18:55:23 +0200] rev 51713
spelling
nipkow [Wed, 17 Apr 2013 21:23:35 +0200] rev 51712
tuned
nipkow [Wed, 17 Apr 2013 21:11:01 +0200] rev 51711
complete revision: finally got rid of annoying L-predicate
nipkow [Wed, 17 Apr 2013 20:53:26 +0200] rev 51710
moved leastness lemma
wenzelm [Tue, 16 Apr 2013 17:54:14 +0200] rev 51709
proper prolog command-line instead of hashbang, which might switch to invalid executable and thus fail (notably on lxbroy2);
speculative update for yap (untested);
hoelzl [Mon, 15 Apr 2013 22:51:55 +0200] rev 51708
use automatic type coerctions in Sqrt example
wenzelm [Mon, 15 Apr 2013 12:03:16 +0200] rev 51707
make SML/NJ happy;
blanchet [Mon, 15 Apr 2013 10:41:03 +0200] rev 51706
not all Nitpick 'constructors' are injective -- careful
kleing [Sun, 14 Apr 2013 21:54:45 +1000] rev 51705
added another definition snipped
wenzelm [Fri, 12 Apr 2013 17:56:51 +0200] rev 51704
actually fail on prolog errors -- such as swipl startup failure due to missing shared libraries -- assuming it normally produces clean return code 0;
wenzelm [Fri, 12 Apr 2013 17:21:51 +0200] rev 51703
modifiers for classical wrappers operate on Proof.context instead of claset;
wenzelm [Fri, 12 Apr 2013 17:02:55 +0200] rev 51702
removed historic comments;
wenzelm [Fri, 12 Apr 2013 15:30:38 +0200] rev 51701
tuned exceptions -- avoid composing error messages in low-level situations;
wenzelm [Fri, 12 Apr 2013 14:54:14 +0200] rev 51700
tuned signature;
tuned comments;
wenzelm [Fri, 12 Apr 2013 12:20:51 +0200] rev 51699
proper identifiers -- avoid crash of case translations;
nipkow [Fri, 12 Apr 2013 08:27:43 +0200] rev 51698
reduced duplication
traytel [Thu, 11 Apr 2013 16:58:54 +0200] rev 51697
do not add case translation syntax in rep_datatype compatibility mode
traytel [Thu, 11 Apr 2013 16:39:01 +0200] rev 51696
run type inference on input to wrap_data
traytel [Thu, 11 Apr 2013 16:03:11 +0200] rev 51695
installed case translations in BNF package
nipkow [Thu, 11 Apr 2013 15:10:22 +0200] rev 51694
tuned