Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip
Find changesets by keywords (author, files, the commit message), revision number or hash, or
revset expression
.
The revision graph only works with JavaScript-enabled browsers.
replaced 'ML' by diagnostic 'ML_command';
2008-03-29, by wenzelm
updated generated file;
2008-03-29, by wenzelm
simplified PureThy.store_thm;
2008-03-29, by wenzelm
replaced 'ML_setup' by 'ML';
2008-03-29, by wenzelm
* Eliminated destructive theorem database.
2008-03-29, by wenzelm
eliminated quiete_mode ref (not really needed);
2008-03-29, by wenzelm
eliminated quiete_mode ref (turned into proper argument);
2008-03-29, by wenzelm
eliminated quiete_mode ref (unused);
2008-03-29, by wenzelm
eliminated quiet_mode ref of some packages (avoid CRITICAL setmp!);
2008-03-29, by wenzelm
added forget_structure;
2008-03-28, by wenzelm
eval_wrapper: non-critical version via unique Isabelle structure, proper forget_structure;
2008-03-28, by wenzelm
ml_tactic: non-critical version via proof data and thread data;
2008-03-28, by wenzelm
NAMED_CRITICAL;
2008-03-28, by wenzelm
unfold_locales now part of default tactic
2008-03-28, by haftmann
import Main explicitly
2008-03-28, by haftmann
dropped now superfluous ad-hoc adaption
2008-03-28, by haftmann
not depends on Main any longer
2008-03-28, by haftmann
accomodated to sledgehammer theory dependency requirement
2008-03-28, by haftmann
only invoke interpret
2008-03-28, by haftmann
updated generated file;
2008-03-28, by wenzelm
Context.>> : operate on Context.generic;
2008-03-28, by wenzelm
avoid rebinding of existing facts;
2008-03-28, by wenzelm
some styling
2008-03-28, by haftmann
some styling
2008-03-28, by haftmann
some styling
2008-03-28, by haftmann
tuned proofs
2008-03-28, by urbanc
tuned;
2008-03-28, by wenzelm
updated dependencies;
2008-03-28, by wenzelm
reorganized signature of ML_Context;
2008-03-28, by wenzelm
remove commented text
2008-03-27, by huffman
avoid ambiguity of State.state vs. JVMType.state;
2008-03-27, by wenzelm
declare cont_lemmas_ext as simp rules individually
2008-03-27, by huffman
avoid amiguity of Continuity.chain vs. Porder.chain;
2008-03-27, by wenzelm
avoid amiguity of State.state vs. JVMType.state;
2008-03-27, by wenzelm
changed wrong assignement in signature sections
2008-03-27, by haftmann
clarified character serializations
2008-03-27, by haftmann
added Enum
2008-03-27, by haftmann
circumventing merge problem
2008-03-27, by haftmann
explicit case names for rule list_induct2
2008-03-27, by haftmann
instance for functions, explicit characters
2008-03-27, by haftmann
lemmas about map_of (zip _ _)
2008-03-27, by haftmann
restructuring; explicit case names for rule list_induct2
2008-03-27, by haftmann
no "attach UNIV" any more
2008-03-27, by haftmann
tuned comments;
2008-03-27, by wenzelm
tuned comments;
2008-03-27, by wenzelm
fixed theory imports;
2008-03-27, by wenzelm
tuned appendix;
2008-03-27, by wenzelm
removed obsolete appl_syntax, applC_syntax;
2008-03-27, by wenzelm
eliminated delayed theory setup
2008-03-27, by wenzelm
Command 'setup': discontinued implicit version.
2008-03-27, by wenzelm
eliminated theory ProtoPure;
2008-03-27, by wenzelm
renamed ML_Context.the_context to ML_Context.the_global_context;
2008-03-27, by wenzelm
added process_file;
2008-03-27, by wenzelm
eliminated theory ProtoPure;
2008-03-27, by wenzelm
moved old the_context here;
2008-03-27, by wenzelm
eliminated theory ProtoPure;
2008-03-27, by wenzelm
implicit setup of emerging theory Pure;
2008-03-27, by wenzelm
reduced to theory body (cf. OuterSyntax.process_file);
2008-03-27, by wenzelm
renamed ML_Context.the_context to ML_Context.the_global_context;
2008-03-27, by wenzelm
eliminated theory ProtoPure;
2008-03-27, by wenzelm
removed Display.raw_string_of_XXX (use regular Sign.string_of_XXX);
2008-03-27, by wenzelm
HOL (and FOL): renamed variables in rules imp_elim and swap;
2008-03-27, by wenzelm
nonfix >>;
2008-03-27, by wenzelm
make preorder locale into a superclass of class po
2008-03-27, by huffman
removed obsolete Thy/thm_database.ML (cf. ML/ml_context.ML);
2008-03-26, by wenzelm
removed legacy ML bindings;
2008-03-26, by wenzelm
rule swap: renamed Pa to P;
2008-03-26, by wenzelm
added store_thms etc. (formerly in Thy/thm_database.ML);
2008-03-26, by wenzelm
adapted to Context.thread_data interface;
2008-03-26, by wenzelm
moved bind_thm(s) to ML/ml_context.ML;
2008-03-26, by wenzelm
added thread data (formerly global ref in ML/ml_context.ML);
2008-03-26, by wenzelm
pass imp_elim (instead of mp) and swap explicitly -- avoids store_thm;
2008-03-26, by wenzelm
pass imp_elim, swap to classical prover;
2008-03-26, by wenzelm
updated generated file;
2008-03-26, by wenzelm
renamed ML_Context.>> to Context.>> (again);
2008-03-26, by wenzelm
converted legacy ML scripts;
2008-03-26, by wenzelm
rename class bifinite_cpo to profinite; generalize powerdomains from bifinite to profinite
2008-03-26, by huffman
fix spelling errors
2008-03-26, by huffman
removed obsolete pass, save;
2008-03-26, by wenzelm
use_thy: removed obsolete ML_Context.save;
2008-03-26, by wenzelm
removed obsolete use_thy (cf. isar_syn.ML);
2008-03-26, by wenzelm
use poly-cvs as name
2008-03-26, by kleing
Functor NamedThmsFun: data is available to the user as dynamic fact;
2008-03-25, by wenzelm
update_context: always store as "Nominal.eqvts";
2008-03-25, by wenzelm
added command 'ML_val' (presently just a clone of 'ML');
2008-03-25, by wenzelm
removed redundant axiomatizations of XXX_infinite (fact already proven);
2008-03-25, by wenzelm
add dynamic fact binding;
2008-03-25, by wenzelm
added 'ML_val' command (diagnostic);
2008-03-25, by wenzelm
get fact: do not compare names;
2008-03-25, by wenzelm
*** empty log message ***
2008-03-25, by wenzelm
support dynamic facts;
2008-03-25, by wenzelm
setup for dynamic "prems" (legacy);
2008-03-25, by wenzelm
more antiquotations;
2008-03-25, by wenzelm
moved multithreaded "profile" to multithreading_polyml.ML;
2008-03-25, by wenzelm
use polyml_old_compiler5.ML;
2008-03-25, by wenzelm
removed
2008-03-25, by haftmann
removed obsolete use_legacy_bindings;
2008-03-24, by wenzelm
ML runtime compilation: pass position, tuned signature;
2008-03-24, by wenzelm
ML runtime compilation: pass position, tuned signature;
2008-03-24, by wenzelm
removed junk;
2008-03-24, by wenzelm
Runtime compilation -- for old version of PolyML.compilerEx (version 5.0, 5.1).
2008-03-24, by wenzelm
Runtime compilation -- for old version of PolyML.compiler (version 4.x).
2008-03-24, by wenzelm
Compatibility wrapper for Poly/ML 5.1.
2008-03-24, by wenzelm
removed pointer_eq from polyml_common.ML (structure Address no longer available after 5.1);
2008-03-24, by wenzelm
updated use_text/file for 5.2;
2008-03-24, by wenzelm
moved use_text/file to polyml_old_compiler5.ML;
2008-03-24, by wenzelm
removed pointer_eq from polyml_common.ML (structure Address no longer available after 5.1);
2008-03-24, by wenzelm
added ML-Systems/polyml-5.1.ML, ML-Systems/polyml_old_compiler4.ML, ML-Systems/polyml_old_compiler5.ML;
2008-03-24, by wenzelm
back to feeder -- Isabelle ML setup no longer evaluates command line;
2008-03-24, by wenzelm
simplified thm_antiq;
2008-03-24, by wenzelm
removed unused print_properties, print_position;
2008-03-24, by wenzelm
replaced obsolete /usr/proj by /home;
2008-03-24, by wenzelm
replaced obsolete /usr/proj by /home;
2008-03-24, by wenzelm
remote CVSROOT: default to atbroy100 instead of sunbroy2;
2008-03-24, by wenzelm
tuned settings for target platforms;
2008-03-24, by wenzelm
thm_antiq: produce error at runtime, not compile time;
2008-03-20, by wenzelm
get_thms etc.: improved reporting of source position;
2008-03-20, by wenzelm
added pos_of_ref;
2008-03-20, by wenzelm
fixed proof;
2008-03-20, by wenzelm
Equivariance prover now uses permutation simprocs as well.
2008-03-20, by berghofe
less
more
|
(0)
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip