Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-10000
-3000
-1000
-240
+240
+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.
renamed def to define;
2007-10-13, by wenzelm
(un)overload: full rewrite;
2007-10-13, by wenzelm
add_abbrevs: unvarify result;
2007-10-13, by wenzelm
replaced obsolete Theory.add_finals_i by Theory.add_deps;
2007-10-13, by wenzelm
Theory.specify_const: added deps argument;
2007-10-13, by wenzelm
renamed LocalTheory.def to LocalTheory.define;
2007-10-13, by wenzelm
typo in comment fixed
2007-10-12, by webertj
significant code overhaul, bugfix for inductive data types
2007-10-12, by webertj
added generic provide_file;
2007-10-12, by wenzelm
pass explicit target record -- more informative peek operation;
2007-10-12, by wenzelm
more informative TheoryTarget.peek operation;
2007-10-12, by wenzelm
fork_mixfix: explicit bool argument;
2007-10-12, by wenzelm
eval_term: moved actual evaluation out of CRITICAL section;
2007-10-12, by wenzelm
preventing eta-redexes in theorems from causing failure
2007-10-12, by paulson
trying to make it run faster
2007-10-12, by paulson
calling the correct interface
2007-10-12, by paulson
replaced syntax/translations by abbreviation;
2007-10-12, by wenzelm
updated
2007-10-12, by haftmann
dropped local_syntax
2007-10-12, by haftmann
tuned
2007-10-12, by haftmann
(intermediate quickfix)
2007-10-12, by haftmann
removed
2007-10-12, by haftmann
added
2007-10-12, by haftmann
metis calls
2007-10-12, by paulson
updated
2007-10-12, by haftmann
moved class power to theory Power
2007-10-12, by haftmann
refined; moved class power to theory Power
2007-10-12, by haftmann
consolidated naming conventions for code generator theories
2007-10-12, by haftmann
class div inherits from class times
2007-10-12, by haftmann
code_include replaces code_moduleprolog
2007-10-12, by haftmann
added subclass command
2007-10-12, by haftmann
enabled Refute_Examples again;
2007-10-11, by wenzelm
local_axioms: impose hyps stemming from local consts as well
2007-10-11, by wenzelm
disabled Refute_Examples temporarily;
2007-10-11, by wenzelm
local_theory: incorporated consts into axioms;
2007-10-11, by wenzelm
removed unused/impure quiet_mode;
2007-10-11, by wenzelm
added export_cterm;
2007-10-11, by wenzelm
local_theory: incorporated consts into axioms;
2007-10-11, by wenzelm
replaced Term.equiv_types by Type.similar_types;
2007-10-11, by wenzelm
replaced Term.equiv_types by Type.similar_types;
2007-10-11, by wenzelm
dest/cert_def: replaced Pretty.pp by explicit Proof.context;
2007-10-11, by wenzelm
added elim_implies (more convenient argument order);
2007-10-11, by wenzelm
removed obsolete flip;
2007-10-11, by wenzelm
moved Drule.unvarify to Thm.unvarify (cf. more_thm.ML);
2007-10-11, by wenzelm
replaced (flip Thm.implies_elim) by Thm.elim_implies;
2007-10-11, by wenzelm
moved Drule.unvarify to Thm.unvarify (cf. more_thm.ML);
2007-10-11, by wenzelm
usedir: added HOL_USEDIR_OPTIONS;
2007-10-11, by wenzelm
reconstruction bug fix
2007-10-11, by paulson
tuned;
2007-10-11, by wenzelm
replaced Sign.add_consts_i by Sign.declare_const;
2007-10-11, by wenzelm
replaced Sign.add_consts_authentic by Sign.declare_const;
2007-10-11, by wenzelm
renamed Syntax.XXX_mode to Syntax.mode_XXX;
2007-10-11, by wenzelm
removed obsolete AxClass.params_of_class;
2007-10-11, by wenzelm
replaced Sign.add_consts_authentic by Sign.declare_const;
2007-10-11, by wenzelm
load axclass.ML before Isar;
2007-10-11, by wenzelm
added specify_const;
2007-10-11, by wenzelm
removed obsolete simple_def;
2007-10-11, by wenzelm
moved define_class_params to Isar/class.ML;
2007-10-11, by wenzelm
load axclass.ML before Isar;
2007-10-11, by wenzelm
Theory.specify_const;
2007-10-11, by wenzelm
moved ProofContext.pp to Syntax.pp;
2007-10-11, by wenzelm
renamed Syntax.XXX_mode to Syntax.mode_XXX;
2007-10-11, by wenzelm
replaced Sign.add_consts_authentic by Sign.declare_const;
2007-10-11, by wenzelm
rationalized redundant code
2007-10-11, by paulson
usage: HOL_USEDIR_OPTIONS;
2007-10-11, by wenzelm
failure messages
2007-10-11, by paulson
'notation': allow structmixfix;
2007-10-11, by wenzelm
update_modesyntax: may delete 'structure' notation as well;
2007-10-11, by wenzelm
'notation': allow 'structure' as well;
2007-10-11, by wenzelm
removed redundant strip_vars/abs_eqn, use improved Drule.abs_def instead;
2007-10-10, by wenzelm
replaced add_modesyntax by general update_modesyntax (add or del);
2007-10-10, by wenzelm
added 'no_notation';
2007-10-10, by wenzelm
generalized notation interface (add or del);
2007-10-10, by wenzelm
tuned;
2007-10-10, by wenzelm
improved abs_def: only abstract over outermost (unique) Vars;
2007-10-10, by wenzelm
proper latex antiquotations instead of adhoc escapes;
2007-10-10, by wenzelm
updated;
2007-10-10, by wenzelm
added no_notation;
2007-10-10, by wenzelm
removed dead code
2007-10-10, by paulson
more metis proofs
2007-10-10, by paulson
Prepare proper interface of interpretation_i, interpret_i.
2007-10-10, by ballarin
getting rid of type typ_var
2007-10-10, by paulson
tuned;
2007-10-09, by wenzelm
class: print result is for locale;
2007-10-09, by wenzelm
context-based treatment of generalization; also handling TFrees in axiom clauses
2007-10-09, by paulson
TheoryTarget.init_cmd;
2007-10-09, by wenzelm
removed LocalTheory.defs/target_morphism operations;
2007-10-09, by wenzelm
renamed AxClass.get_definition to AxClass.get_info (again);
2007-10-09, by wenzelm
removed LocalTheory.defs/target_morphism operations;
2007-10-09, by wenzelm
AxClass.axiomatize and Specification: renamed XXX_i to XXX, and XXX to XXX_cmd;
2007-10-09, by wenzelm
removed LocalTheory.defs/target_morphism operations;
2007-10-09, by wenzelm
renamed AxClass.get_definition to AxClass.get_info (again);
2007-10-09, by wenzelm
renamed AxClass.get_definition to AxClass.get_info (again);
2007-10-09, by wenzelm
renamed AxClass.get_definition to AxClass.get_info (again);
2007-10-09, by wenzelm
Specification: renamed XXX_i to XXX, and XXX to XXX_cmd;
2007-10-09, by wenzelm
AxClass.axiomatize: renamed XXX_i to XXX, and XXX to XXX_cmd;
2007-10-09, by wenzelm
removed LocalTheory.defs, use plain LocalTheory.def;
2007-10-09, by wenzelm
tuned;
2007-10-09, by wenzelm
generic Syntax.pretty/string_of operations;
2007-10-09, by wenzelm
generic Syntax.pretty/string_of operations;
2007-10-09, by wenzelm
generic Syntax.pretty/string_of operations;
2007-10-09, by wenzelm
generic Syntax.pretty/string_of operations;
2007-10-09, by wenzelm
updated keywords
2007-10-08, by haftmann
moved translation kernel to CodeThingol
2007-10-08, by haftmann
tuned
2007-10-08, by haftmann
simplified evaluation
2007-10-08, by haftmann
integrated FixedPoint into Inductive
2007-10-08, by haftmann
added proper subclass concept; improved class target
2007-10-08, by haftmann
fixed bug in grobner_ideal
2007-10-08, by chaieb
tuned generated comment;
2007-10-08, by wenzelm
primitive add_def: strip sorts in axiom;
2007-10-08, by wenzelm
avoid polymorphic equality;
2007-10-08, by wenzelm
maintain typargs for abbrevs as well;
2007-10-08, by wenzelm
Codegen.is_instance: raw match, ignore sort constraints;
2007-10-08, by wenzelm
Codegen.is_instance: raw match, ignore sort constraints;
2007-10-08, by wenzelm
turned keywords invariant/freshness_context into reserved indentifiers;
2007-10-08, by wenzelm
tuned generated comment;
2007-10-08, by wenzelm
updated;
2007-10-08, by wenzelm
moved HOL-Nominal keywords into default collection (isar-keywords.el);
2007-10-08, by wenzelm
list_codegen and char_codegen now call invoke_tycodegen to ensure
2007-10-08, by berghofe
added first version of user-space type system for class target
2007-10-08, by haftmann
clarified
2007-10-08, by haftmann
Isar-fied many proofs
2007-10-08, by urbanc
changed VC-Compatible to VC_Compatible
2007-10-08, by urbanc
changed file name
2007-10-08, by urbanc
added the two new examples from Nominal to the build process
2007-10-08, by urbanc
added two new example files
2007-10-08, by urbanc
modernized specifications;
2007-10-07, by wenzelm
modernized specifications;
2007-10-07, by wenzelm
replaced some 'translations' by 'abbreviation';
2007-10-07, by wenzelm
* Basic Isabelle mode for jEdit.
2007-10-07, by wenzelm
tuned generated comment;
2007-10-07, by wenzelm
tuned;
2007-10-07, by wenzelm
Basic Isabelle mode for jEdit -- http://www.jedit.org/
2007-10-07, by wenzelm
isabelle mode for jEdit;
2007-10-07, by wenzelm
added target tool specification;
2007-10-07, by wenzelm
added target tool specification;
2007-10-07, by wenzelm
emacs vs. jedit;
2007-10-07, by wenzelm
some updates;
2007-10-06, by wenzelm
removed obsolete write_keywords;
2007-10-06, by wenzelm
Dummy session with outer syntax keyword initialization.
2007-10-06, by wenzelm
added Pure-ProofGeneral target (dummy session with outer syntax keyword initialization);
2007-10-06, by wenzelm
tuned;
2007-10-06, by wenzelm
use isatool keywords -- generate from logs instead of session images;
2007-10-06, by wenzelm
removed duplicate target;
2007-10-06, by wenzelm
updated;
2007-10-06, by wenzelm
generate outer syntax keyword files from session logs;
2007-10-06, by wenzelm
export init_outer_syntax;
2007-10-06, by wenzelm
tuned;
2007-10-06, by wenzelm
report on keyword/command declarations;
2007-10-06, by wenzelm
tuned;
2007-10-06, by wenzelm
added keyword_decl, command_decl;
2007-10-06, by wenzelm
added class_expr;
2007-10-06, by wenzelm
simplified interfaces for outer syntax;
2007-10-06, by wenzelm
simplified interfaces for outer syntax;
2007-10-06, by wenzelm
updated;
2007-10-06, by wenzelm
(co)induct: polymorhic taking'';
2007-10-05, by wenzelm
added burrow_options;
2007-10-05, by wenzelm
tuned proofs (via polymorphic taking'');
2007-10-05, by wenzelm
export get_consumes;
2007-10-05, by wenzelm
tuned Induct interface: prefer pred'' over set'';
2007-10-05, by wenzelm
coinduct: instantiation refers to suffix of main prop (major premise or conclusion);
2007-10-05, by wenzelm
tuned induct etc.;
2007-10-05, by wenzelm
execute/system: non-critical;
2007-10-05, by wenzelm
subtract: minor performance tuning;
2007-10-05, by wenzelm
cover only .gz files;
2007-10-05, by wenzelm
metis method: used theorems
2007-10-05, by paulson
filtering out some package theorems
2007-10-05, by paulson
added lemmas
2007-10-05, by nipkow
single-threaded profiling;
2007-10-04, by wenzelm
tuned;
2007-10-04, by wenzelm
Name.uu, Name.aT;
2007-10-04, by wenzelm
added uu, aT;
2007-10-04, by wenzelm
replaced literal 'a by Name.aT;
2007-10-04, by wenzelm
replaced AxClass.param_tyvarname by Name.aT;
2007-10-04, by wenzelm
added nth_drop
2007-10-04, by haftmann
tuned datatype_codegen setup
2007-10-04, by haftmann
certificates for code generator case expressions
2007-10-04, by haftmann
added illustrative diagnostics
2007-10-04, by haftmann
clarified declarations in class ord
2007-10-04, by haftmann
concept for exceptions
2007-10-04, by haftmann
clarified name suffix
2007-10-04, by haftmann
step towards proper purge operation
2007-10-04, by haftmann
put declarations first
2007-10-04, by haftmann
clarified terminology
2007-10-04, by haftmann
intermediate cleanup
2007-10-04, by haftmann
clarified relationship of code generator conversions and evaluations
2007-10-04, by haftmann
abs_conv/forall_conv: proper context (avoid gensym);
2007-10-04, by wenzelm
load variable.ML before conv.ML;
2007-10-04, by wenzelm
Conv.forall_conv: proper context;
2007-10-04, by wenzelm
cover AFP logs as well, using "afp" pseudo-platform;
2007-10-04, by wenzelm
moved Pure/Isar/induct_attrib.ML and Provers/induct_method.ML to Tools/induct.ML;
2007-10-04, by wenzelm
avoid gensym;
2007-10-04, by wenzelm
updated Sign.add_abbrev;
2007-10-04, by wenzelm
combinator translation
2007-10-04, by paulson
avoid unnamed infixes;
2007-10-03, by wenzelm
avoid unnamed infixes;
2007-10-03, by wenzelm
avoid unnamed infixes;
2007-10-03, by wenzelm
modernized specifications;
2007-10-03, by wenzelm
mark inductive results as internal;
2007-10-03, by wenzelm
skolem_cache: ignore internal theorems -- major speedup;
2007-10-03, by wenzelm
major speedup by avoiding metis;
2007-10-03, by wenzelm
modernized definitions;
2007-10-03, by wenzelm
added add_defs_new, which strips sorts for axioms (presently inactive);
2007-10-02, by wenzelm
removed unused add_defss;
2007-10-02, by wenzelm
tuned internal inductive interface;
2007-10-02, by wenzelm
tuned internal interfaces: flags record, added kind for results;
2007-10-02, by wenzelm
inductive: mark internal theorems as Thm.internalK;
2007-10-02, by wenzelm
tuned;
2007-10-02, by wenzelm
export tsig_of;
2007-10-02, by wenzelm
clarified role of class relations
2007-10-02, by haftmann
ignore mutual recursive modules
2007-10-02, by haftmann
integer compatibility: added wrapper for structure Time;
2007-10-01, by wenzelm
fixed use_text;
2007-10-01, by wenzelm
downgraded IntInf with divMod;
2007-10-01, by wenzelm
added auto-quickcheck-time-limit;
2007-10-01, by wenzelm
auto_quickcheck: pervasive options, turned time_limit into plain int, simplified exception handling;
2007-10-01, by wenzelm
added auto_quickcheck feature;
2007-10-01, by wenzelm
Norbert Schirmer: record improvements;
2007-10-01, by wenzelm
preliminary material for Isabelle2007;
2007-10-01, by wenzelm
misc tuning and update;
2007-10-01, by wenzelm
misc tuning and update;
2007-10-01, by wenzelm
misc tuning and update;
2007-10-01, by wenzelm
updated year to 2007;
2007-10-01, by wenzelm
tuned;
2007-10-01, by wenzelm
added some lemmas
2007-10-01, by haftmann
print_state_context: local theory context, not proof context;
2007-10-01, by wenzelm
ContextPosition.put_ctxt;
2007-10-01, by wenzelm
NameSelection: more interval checks;
2007-10-01, by wenzelm
tuned message;
2007-10-01, by wenzelm
turned into generic context data;
2007-10-01, by wenzelm
ML_setup for bind_thms;
2007-10-01, by wenzelm
Simplified interface for printing of interpretations.
2007-10-01, by ballarin
unfold_locales workaround
2007-10-01, by ballarin
Theory/context data restructured; simplified interface for printing of interpretations.
2007-10-01, by ballarin
fixed dir in single-logic test
2007-10-01, by isatest
llabs/sko: removed Name.internal;
2007-09-30, by wenzelm
avoid unnamed infixes;
2007-09-30, by wenzelm
avoid internal names;
2007-09-30, by wenzelm
switch notification email back on
2007-09-30, by isatest
less
more
|
(0)
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
+30000
tip