Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-10000
-3000
-1000
-480
+480
+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.
class package and codegen refinements
2006-07-21, by haftmann
added give_names and alphanum
2006-07-21, by haftmann
Some cases in "case ... of ..." expressions may now
2006-07-21, by berghofe
- Added new "undefined" constant
2006-07-21, by berghofe
removed Variable.monomorphic;
2006-07-20, by wenzelm
comments fixed, member function renamed
2006-07-20, by webertj
Change to algebra method.
2006-07-19, by ballarin
Reimplemented algebra method; now controlled by attribute.
2006-07-19, by ballarin
Strict dfs traversal of imported and registered identifiers.
2006-07-19, by ballarin
added map_default, internal restructuring
2006-07-19, by haftmann
export is_tid;
2006-07-19, by wenzelm
thm_of_proof: improved generation of variables;
2006-07-19, by wenzelm
Sign.infer_types: Name.context;
2006-07-19, by wenzelm
reorganize declarations (more efficient);
2006-07-19, by wenzelm
Name.context for used'';
2006-07-19, by wenzelm
added variant_frees;
2006-07-19, by wenzelm
tuned;
2006-07-19, by wenzelm
export make_context, is_declared;
2006-07-19, by wenzelm
prove: Variable.declare_internal (more efficient);
2006-07-19, by wenzelm
add_local: simplified interface, all frees are known'';
2006-07-19, by wenzelm
Sign.infer_types: Name.context;
2006-07-19, by wenzelm
renamed Variable.rename_wrt to Variable.variant_frees;
2006-07-19, by wenzelm
Fixed the bugs introduced by the last commit! Output is now *identical* to that
2006-07-19, by paulson
MiniSat proof trace format changed; MiniSat is now expected to produce a proof also for "trivial" problems
2006-07-19, by webertj
thm_of_proof: tuned Name operations;
2006-07-18, by wenzelm
print_statement: tuned Variable operations;
2006-07-18, by wenzelm
added newly_fixed, focus;
2006-07-18, by wenzelm
added declare_term_names;
2006-07-18, by wenzelm
fold_proof_terms: canonical arguments;
2006-07-18, by wenzelm
Term.declare_term_names;
2006-07-18, by wenzelm
Started implementing uniqueness proof for recursion
2006-07-18, by berghofe
typo (theorerms) fixed
2006-07-18, by webertj
typo (theorerms) fixed
2006-07-18, by webertj
AList.join now with 'DUP' exception
2006-07-18, by haftmann
added Table.map_default
2006-07-18, by haftmann
removed obsolete ML files;
2006-07-18, by wenzelm
replaced butlast by Library.split_last;
2006-07-17, by wenzelm
replaced butlast by Library.split_last;
2006-07-17, by wenzelm
butlast removed (use fst o split_last instead)
2006-07-17, by webertj
support for MiniSat proof traces added
2006-07-17, by webertj
support for MiniSat proof traces added
2006-07-17, by webertj
has_consts renamed to has_conn, now actually parses the first-order formula
2006-07-16, by paulson
function butlast added
2006-07-15, by webertj
Replaced a-lists by tables to improve efficiency
2006-07-15, by paulson
Pass user lemmas' names to ResHolClause.tptp_write_file and dfg_write_file.
2006-07-15, by mengj
Only include combinators if required by goals and user specified lemmas.
2006-07-15, by mengj
Term.term_lpo takes order on terms rather than strings as argument.
2006-07-14, by ballarin
keep/transaction: unified execution model (with debugging etc.);
2006-07-14, by wenzelm
trivial whitespace changes
2006-07-14, by webertj
simp method: depth_limit;
2006-07-14, by wenzelm
"conjecture" must be lower case
2006-07-13, by paulson
tuned insert_list;
2006-07-13, by wenzelm
Name.context already declares empty names;
2006-07-13, by wenzelm
strip_abs_eta: proper use of Name.context;
2006-07-13, by wenzelm
do not export make_context;
2006-07-13, by wenzelm
removed colon from sym category;
2006-07-13, by wenzelm
fix to refl_clause_aux: added occurs check
2006-07-13, by paulson
* Isar: ":" (colon) is no longer a symbolic identifier character;
2006-07-12, by wenzelm
removed duplicate of Tactic.make_elim_preserve;
2006-07-12, by wenzelm
removed obsolete adhoc_freeze_vars (may use Variable.import_terms instead);
2006-07-12, by wenzelm
exported make_elim_preserve;
2006-07-12, by wenzelm
prove_conv: Variable.import_terms instead of Term.addhoc_freeze_vars;
2006-07-12, by wenzelm
simplified prove_conv;
2006-07-12, by wenzelm
removed ':' from category of symbolic identifier chars;
2006-07-12, by wenzelm
query/bang_colon: separate tokens;
2006-07-12, by wenzelm
purged website sources
2006-07-12, by haftmann
added strip_abs_eta
2006-07-12, by haftmann
added chop_prefix
2006-07-12, by haftmann
class_of_param instead of class_of
2006-07-12, by haftmann
adaptions in class_package
2006-07-12, by haftmann
adaptions in codegen
2006-07-12, by haftmann
variants: special treatment of empty name;
2006-07-12, by wenzelm
avoid reference to internal skolem;
2006-07-11, by wenzelm
separate names filed (covers fixes/defaults);
2006-07-11, by wenzelm
adapted Name.defaults_of;
2006-07-11, by wenzelm
removed obsolete xless;
2006-07-11, by wenzelm
clean: no special treatment of empty name;
2006-07-11, by wenzelm
removed obsolete xless;
2006-07-11, by wenzelm
replaced mk_listT by HOLogic.listT; trivial whitespace/comment changes
2006-07-11, by webertj
uniform treatment of num/xnum;
2006-07-11, by wenzelm
replaced read_radixint by read_intinf;
2006-07-11, by wenzelm
removed str_to_int in favour of general Syntax.read_xnum;
2006-07-11, by wenzelm
num/xnum: bin or hex;
2006-07-11, by wenzelm
Name.internal;
2006-07-11, by wenzelm
tuned;
2006-07-11, by wenzelm
* Pure: structure Name;
2006-07-11, by wenzelm
Names of basic logical entities (variables etc.).
2006-07-11, by wenzelm
replaced Term.variant(list) by Name.variant(_list);
2006-07-11, by wenzelm
Name.internal;
2006-07-11, by wenzelm
adapted to more efficient Name/Variable implementation;
2006-07-11, by wenzelm
replaced Term.variant(list) by Name.variant(_list);
2006-07-11, by wenzelm
maintain Name.context for fixes/defaults;
2006-07-11, by wenzelm
removed obsolete mem_ix;
2006-07-11, by wenzelm
removed obsolete ins_ix, mem_ix, ins_term, mem_term;
2006-07-11, by wenzelm
Name.dest_skolem;
2006-07-11, by wenzelm
Name.bound;
2006-07-11, by wenzelm
replaced Term.variant(list) by Name.variant(_list);
2006-07-11, by wenzelm
replaced Term.variant(list) by Name.variant(_list);
2006-07-11, by wenzelm
replaced Term.variant(list) by Name.variant(_list);
2006-07-11, by wenzelm
Name.invent_list;
2006-07-11, by wenzelm
added name.ML;
2006-07-11, by wenzelm
Name.is_bound;
2006-07-11, by wenzelm
removed obsolete mem_term;
2006-07-11, by wenzelm
Name.internal;
2006-07-11, by wenzelm
replaced Term.variant(list) by Name.variant(_list);
2006-07-11, by wenzelm
let_simproc: activate Variable.import;
2006-07-11, by wenzelm
Witness theorems of interpretations now transfered to current theory.
2006-07-11, by ballarin
New function transfer_witness lifting Thm.transfer to witnesses.
2006-07-11, by ballarin
hex and binary numerals (contributed by Rafal Kolanski)
2006-07-11, by kleing
minor optimization wrt. certifying terms
2006-07-10, by webertj
tuned;
2006-07-08, by wenzelm
tuned;
2006-07-08, by wenzelm
updated;
2006-07-08, by wenzelm
tuned interface;
2006-07-08, by wenzelm
tuned interface;
2006-07-08, by wenzelm
removed dead code;
2006-07-08, by wenzelm
Element.prove_witness: context;
2006-07-08, by wenzelm
prove_witness: context;
2006-07-08, by wenzelm
tuned exception handling;
2006-07-08, by wenzelm
prove/prove_multi: context;
2006-07-08, by wenzelm
simprocs: no theory argument -- use simpset context instead;
2006-07-08, by wenzelm
distinct simproc/simpset: proper context;
2006-07-08, by wenzelm
presburger_ss: proper context;
2006-07-08, by wenzelm
presburger_ss: proper context;
2006-07-08, by wenzelm
tuned;
2006-07-08, by wenzelm
avoid Force_tac, which uses a different context;
2006-07-08, by wenzelm
Goal.prove: context;
2006-07-08, by wenzelm
tactic/method simpset: maintain proper context;
2006-07-08, by wenzelm
Goal.prove_global;
2006-07-08, by wenzelm
Goal.prove_global;
2006-07-08, by wenzelm
simprocs: no theory argument -- use simpset context instead;
2006-07-08, by wenzelm
simprocs: no theory argument -- use simpset context instead;
2006-07-08, by wenzelm
updated;
2006-07-08, by wenzelm
updated Goal.prove, Goal.prove_global;
2006-07-08, by wenzelm
added some bits on variables;
2006-07-08, by wenzelm
* Pure: structure Variable provides operations for proper treatment of fixed/schematic variables;
2006-07-08, by wenzelm
"solver" reference added to make the SAT solver configurable
2006-07-07, by webertj
Some tidying.
2006-07-07, by paulson
Fixed erroneous check-in.
2006-07-07, by ballarin
made evaluation_conv and normalization_conv visible.
2006-07-07, by nipkow
Internal restructuring: identify no longer computes syntax.
2006-07-07, by ballarin
Modified comment.
2006-07-07, by ballarin
added support for MiniSat 1.14
2006-07-07, by webertj
removed obsolete locale view;
2006-07-06, by wenzelm
apply_text: support Method.Source_i;
2006-07-06, by wenzelm
added method_i and Source_i;
2006-07-06, by wenzelm
thm parsers: include Args.internal_fact;
2006-07-06, by wenzelm
add/del_simps: warning for inactive simpset (no context);
2006-07-06, by wenzelm
updated;
2006-07-06, by wenzelm
Local variables;
2006-07-06, by wenzelm
Isar.context ();
2006-07-06, by wenzelm
tuned;
2006-07-06, by wenzelm
added Isar.context;
2006-07-06, by wenzelm
some tidying; fixed the output of theorem names
2006-07-06, by paulson
def_export: Drule.generalize;
2006-07-06, by wenzelm
matchers: fall back on plain first_order_matchers, not pattern;
2006-07-06, by wenzelm
make sure $DISTPREFIX exists before calling makedist
2006-07-05, by kleing
removed the "tagging" feature
2006-07-05, by paulson
made the conversion of elimination rules more robust
2006-07-05, by paulson
Literals aren't sorted any more.
2006-07-05, by mengj
Literals aren't sorted any more. Output overloaded constants' type var instantiations.
2006-07-05, by mengj
fixed let-simproc
2006-07-05, by schirmer
Isar: 'print_facts' prints all local facts;
2006-07-04, by wenzelm
print_lthms: include unnamed facts from index;
2006-07-04, by wenzelm
added content;
2006-07-04, by wenzelm
added props selector;
2006-07-04, by wenzelm
print_facts: all facts;
2006-07-04, by wenzelm
add_abbrevs/polymorphic: Variable.exportT_terms avoids over-generalization;
2006-07-04, by wenzelm
instantiate_tfrees: Thm.generalize;
2006-07-04, by wenzelm
removed parrot comment;
2006-07-04, by wenzelm
Proof by guessing.
2006-07-04, by wenzelm
guess: proper context for polymorphic parameters;
2006-07-04, by wenzelm
polymorphic: always generalize wrt. used_types;
2006-07-04, by wenzelm
varifyT: no longer pervasive;
2006-07-04, by wenzelm
added generalize/instantiate_option;
2006-07-04, by wenzelm
added map_proof_terms_option;
2006-07-04, by wenzelm
added generalize;
2006-07-04, by wenzelm
Thm.varifyT;
2006-07-04, by wenzelm
added ex/Guess.thy;
2006-07-04, by wenzelm
skip_proofs: do not skip proofs of schematic goals (warning);
2006-07-04, by wenzelm
added schematic_goal;
2006-07-04, by wenzelm
added 'unfolding';
2006-07-04, by wenzelm
added simplification rules to the fresh_guess tactic
2006-07-04, by urbanc
made calc_atm stronger by including some relative
2006-07-04, by urbanc
Locales no longer generate views. The following functions have changed
2006-07-04, by ballarin
added 'definition', 'unfolding', 'done';
2006-07-04, by wenzelm
tuned;
2006-07-04, by wenzelm
added 'value';
2006-07-04, by wenzelm
- put declarations inside a structure (NominalPermeq)
2006-07-04, by berghofe
- nominal_permeq.ML is now loaded before nominal_package.ML
2006-07-04, by berghofe
Implemented proofs of equivariance and finite support
2006-07-04, by berghofe
Method intro_locales replaced by intro_locales and unfold_locales.
2006-07-04, by ballarin
updated
2006-07-04, by urbanc
Typo.
2006-07-04, by ballarin
Minor new lemmas.
2006-07-04, by ballarin
replaced respects2 by congruent2 because of type problem
2006-07-03, by nipkow
replaced translation by abbreviation
2006-07-03, by nipkow
obtain_export: Thm.generalize;
2006-07-03, by wenzelm
project_algebra: norm_sort;
2006-07-03, by wenzelm
comments fixed, minor optimization wrt. certifying terms
2006-07-03, by webertj
fix to subst in order to allow subst when head of a term is a bound variable.
2006-07-03, by dixon
CNF tactic invocations moved into comments
2006-07-03, by webertj
comment added
2006-07-03, by webertj
added more infrastructure for the recursion combinator
2006-07-02, by urbanc
normal_form to lemma test
2006-06-30, by nipkow
normalization uses refl now
2006-06-30, by nipkow
Removed some incorrect axioms.
2006-06-30, by mengj
fixed stale theory bug
2006-06-30, by haftmann
slight refinements
2006-06-30, by haftmann
refinement in instance command
2006-06-30, by haftmann
small change in class_package
2006-06-30, by haftmann
added the "th" field to datatype Clause
2006-06-29, by paulson
fixed the "factor" method
2006-06-29, by paulson
new function norm_term
2006-06-29, by nipkow
new method "normalization"
2006-06-29, by nipkow
use -f in cp to overwrite read-only files (e.g. .svn in document/)
2006-06-29, by kleing
world map now transparent
2006-06-28, by webertj
improvements in Classpackage
2006-06-28, by haftmann
reduced code, better instance command
2006-06-28, by haftmann
slight improvements in code generation
2006-06-28, by haftmann
added lookup function for parameters
2006-06-28, by haftmann
disjunctive wellfoundedness
2006-06-28, by paulson
class package refinements, slight code generation refinements
2006-06-27, by haftmann
added class projection
2006-06-27, by haftmann
slight improvement
2006-06-27, by haftmann
replaced subgraph by project
2006-06-27, by haftmann
fix/fixes: tuned type constraints;
2006-06-24, by wenzelm
minor tuning of definitions/proofs;
2006-06-24, by wenzelm
fixed translations for _MapUpd: CONST;
2006-06-24, by wenzelm
beautification
2006-06-23, by nipkow
added webmaster
2006-06-23, by haftmann
Introduction of Ramsey's theorem
2006-06-23, by paulson
Removed debugging code.
2006-06-22, by ballarin
Improved handling of defines imported in duplicate.
2006-06-22, by ballarin
new standard dir structure
2006-06-22, by kleing
world map updated
2006-06-21, by webertj
world map updated
2006-06-21, by webertj
Removed (term_of o cterm_of)-Hack, Added error message for unknown definition at "termination"-command
2006-06-21, by krauss
fixed bug resolving Haskell names
2006-06-21, by haftmann
fixed error bug
2006-06-21, by haftmann
renamed thy data
2006-06-21, by haftmann
Added split_cong rule
2006-06-21, by krauss
hyps better than prems
2006-06-21, by haftmann
fixed sml/nj value restriction problem
2006-06-20, by haftmann
Restructured locales with predicates: import is now an interpretation.
2006-06-20, by ballarin
Fixed another variable order bug...
2006-06-20, by krauss
switched to open locales for classes
2006-06-20, by haftmann
switched to open locales for classes
2006-06-20, by haftmann
refrain from reforming TFL -- back to previous revision;
2006-06-19, by wenzelm
added declare_thm, thm_context;
2006-06-19, by wenzelm
eliminated freeze/varify in favour of Variable.import/export/trade;
2006-06-19, by wenzelm
world map updated
2006-06-19, by webertj
world map updated
2006-06-19, by webertj
Fixed name clash.
2006-06-19, by krauss
world map updated
2006-06-19, by webertj
matchers: try pattern_matchers only *after* general matching (The
2006-06-19, by wenzelm
ProofContext.exports: simultaneous facts;
2006-06-17, by wenzelm
moved internal/skolem to term.ML;
2006-06-17, by wenzelm
mutual_rule: proper context;
2006-06-17, by wenzelm
export: simultaneous facts, refer to Variable.export;
2006-06-17, by wenzelm
ProofContext.exports: simultaneous facts;
2006-06-17, by wenzelm
Variable.importT_inst;
2006-06-17, by wenzelm
standard: simultaneous facts;
2006-06-17, by wenzelm
added singleton;
2006-06-17, by wenzelm
major reworking of export functionality -- based on Term/Thm.generalize;
2006-06-17, by wenzelm
added generalize rule;
2006-06-17, by wenzelm
added exists_subtype;
2006-06-17, by wenzelm
added generalize rule;
2006-06-17, by wenzelm
Term.skolem;
2006-06-17, by wenzelm
Term.internal;
2006-06-17, by wenzelm
ProofContext.export: singleton;
2006-06-17, by wenzelm
RuleCases.mutual_rule: ctxt;
2006-06-17, by wenzelm
RuleCases.mutual_rule: ctxt;
2006-06-17, by wenzelm
added interface for making term contexts.
2006-06-17, by dixon
fixed symlink bug
2006-06-16, by haftmann
ProofContext: moved variable operations to struct Variable;
2006-06-15, by wenzelm
Fixed type/term variables and polymorphic term abbreviations.
2006-06-15, by wenzelm
added variable.ML;
2006-06-15, by wenzelm
ProofContext: moved variable operations to struct Variable;
2006-06-15, by wenzelm
*** empty log message ***
2006-06-15, by nipkow
*** empty log message ***
2006-06-15, by nipkow
the "all_theorems" option and some fixes
2006-06-15, by paulson
the enumerate operator
2006-06-15, by paulson
Jia Meng added to world map
2006-06-14, by webertj
keyword update
2006-06-14, by haftmann
slight adaption for code generator
2006-06-14, by haftmann
slight adaptions for code generator
2006-06-14, by haftmann
slight adaptions
2006-06-14, by haftmann
slight refinements for code generator
2006-06-14, by haftmann
added hook for case const defs
2006-06-14, by haftmann
added codegen_simtype
2006-06-14, by haftmann
improvements in code generator
2006-06-14, by haftmann
avoid global Drule.unvarify;
2006-06-13, by wenzelm
tuned interfaces;
2006-06-13, by wenzelm
added hyps_of;
2006-06-13, by wenzelm
added equiv;
2006-06-13, by wenzelm
(un)varify: tuned exceptions;
2006-06-13, by wenzelm
removed weak_eq_thm;
2006-06-13, by wenzelm
Drule.equiv_thm supercedes Drule.weak_eq_thm;
2006-06-13, by wenzelm
tuned;
2006-06-13, by wenzelm
avoid unqualified exception names;
2006-06-13, by wenzelm
ProjectRule now context dependent;
2006-06-13, by wenzelm
use Drule.unvarify instead of obsolete Drule.freeze_all;
2006-06-13, by wenzelm
corrected w.r.t. search order for subst.
2006-06-13, by dixon
Corrected search order for zippers.
2006-06-13, by dixon
new results
2006-06-13, by paulson
removal of the obsolete "infinite_nonempty"
2006-06-13, by paulson
tuned;
2006-06-12, by wenzelm
added declare_typ;
2006-06-12, by wenzelm
tuned;
2006-06-12, by wenzelm
tuned interfaces;
2006-06-12, by wenzelm
added matchers, matches_list;
2006-06-12, by wenzelm
removed matches_seq -- didn't quite work;
2006-06-12, by wenzelm
Unify.matches_list;
2006-06-12, by wenzelm
tuned Seq/Envir/Unify interfaces;
2006-06-12, by wenzelm
fixed subst step;
2006-06-12, by wenzelm
avoid accidental binding of ?Jmp;
2006-06-12, by wenzelm
added lemma fresh_unit to Nominal.thy
2006-06-12, by urbanc
Added fresh_guess_tac.
2006-06-12, by berghofe
Removed comments around declaration of fresh_guess method.
2006-06-12, by berghofe
Added "evaluation" method.
2006-06-12, by berghofe
updated keywords
2006-06-12, by haftmann
made smlnj happy;
2006-06-12, by wenzelm
fixed smlnj incompat.
2006-06-12, by haftmann
Completely rewrote code for defining graph of recursion combinator.
2006-06-12, by berghofe
fixed subst step;
2006-06-11, by wenzelm
actually invoke result elements;
2006-06-11, by wenzelm
improved treatment of TERM TYPE syntax;
2006-06-11, by wenzelm
added import -- fixes schematic variables;
2006-06-11, by wenzelm
fixes: include mixfix syntax;
2006-06-11, by wenzelm
added for_fixes;
2006-06-11, by wenzelm
fixes: include mixfix syntax;
2006-06-11, by wenzelm
added satisfy_ctxt;
2006-06-11, by wenzelm
outer_params: Syntax.dest_internal;
2006-06-11, by wenzelm
avoid unqualified exception;
2006-06-11, by wenzelm
added quoting via back quotes
2006-06-11, by nipkow
updated IsaMakefiles for new location of IsaPlanner.
2006-06-11, by dixon
removed IsaPlanner - these are now in Provers.
2006-06-11, by dixon
removed IsaPlannner things from Pure. Moved to Provers.
2006-06-11, by dixon
moved to new location in Provers.
2006-06-11, by dixon
added updated version of IsaPlanner and substitution.
2006-06-11, by dixon
unique_names no longer set to false (thanks to improved naming
2006-06-09, by berghofe
- Changed naming scheme: names of "internal" constructors now have
2006-06-09, by berghofe
nbe -> NormalForm
2006-06-09, by nipkow
CVS: ----------------------------------------------------------------------
2006-06-09, by webertj
renamed command
2006-06-09, by nipkow
renamed file
2006-06-09, by nipkow
Removed "code del" declarations again.
2006-06-08, by berghofe
fixed owner bug
2006-06-08, by haftmann
less_equal -> less_eq (someone had screwd up here)
2006-06-08, by nipkow
Splitting order changed.
2006-06-08, by chaieb
added John's example
2006-06-08, by nipkow
replaced REPEAT by REPOEAT_DETERM
2006-06-08, by nipkow
gmake vs. make
2006-06-08, by haftmann
removed obsolete ML files;
2006-06-07, by wenzelm
removed obsolete ML files;
2006-06-07, by wenzelm
removed obsolete ML files;
2006-06-07, by wenzelm
adding case theorems for code generator
2006-06-07, by haftmann
slight code generator cleanup
2006-06-07, by haftmann
removed 'primitive definitions' added (non)strict generation, minor fixes
2006-06-07, by haftmann
fixed typo
2006-06-07, by haftmann
* Theory syntax: some popular names (e.g. "class", "if") are now keywords.
2006-06-07, by wenzelm
Schematic invocation of locale expression in proof context.
2006-06-07, by wenzelm
added invoke.ML;
2006-06-07, by wenzelm
added locale_insts;
2006-06-07, by wenzelm
renamed Type.(un)varifyT to Logic.(un)varifyT;
2006-06-07, by wenzelm
added 'if' and 'for' keywords;
2006-06-07, by wenzelm
added facts_of;
2006-06-07, by wenzelm
added Tools/invoke.ML;
2006-06-07, by wenzelm
renamed Type.(un)varifyT to Logic.(un)varifyT;
2006-06-07, by wenzelm
do not open Logic;
2006-06-07, by wenzelm
tuned;
2006-06-07, by wenzelm
removed obsolete ML files;
2006-06-07, by wenzelm
removed obsolete ML files;
2006-06-07, by wenzelm
removed obsolete ML files;
2006-06-07, by wenzelm
removed Toplevel.debug;
2006-06-06, by wenzelm
added zip_options;
2006-06-06, by wenzelm
tuned;
2006-06-06, by wenzelm
updated;
2006-06-06, by wenzelm
quoted "if";
2006-06-06, by wenzelm
added type inference at the end of normalization
2006-06-06, by nipkow
revised nbe command and examples
2006-06-06, by nipkow
new lemmas concerning finite cardinalities
2006-06-06, by paulson
quoted "if";
2006-06-06, by wenzelm
refined code generation
2006-06-06, by haftmann
added arbitray setup for codegen 2
2006-06-06, by haftmann
small fix
2006-06-06, by haftmann
deleted legacy
2006-06-06, by haftmann
improved code lemmas
2006-06-06, by haftmann
fixed typo
2006-06-06, by haftmann
bugfixes
2006-06-06, by haftmann
HOL/Tools/function_package: Applies CodeGen attributes again, where possible.
2006-06-06, by krauss
Improved parameter management of locales.
2006-06-06, by ballarin
HOL/Tools/function_package: imporoved handling of guards, added an example
2006-06-06, by krauss
HOL/Tools/function_package: More cleanup
2006-06-06, by krauss
export read/cert_expr;
2006-06-05, by wenzelm
guess: more careful about local polymorphism;
2006-06-05, by wenzelm
assm_tac: try rule termI;
2006-06-05, by wenzelm
added params_of, prems_of;
2006-06-05, by wenzelm
added matches_seq (left-to-right matching, intermediate beta-normalization);
2006-06-05, by wenzelm
support embedded terms;
2006-06-05, by wenzelm
allow non-trivial schematic goals (via embedded term vars);
2006-06-05, by wenzelm
HOL/Tools/fundef_package: Cleanup
2006-06-05, by krauss
added some further lemmas that deal with permutations and set-operators
2006-06-05, by urbanc
added the lemma perm_diff
2006-06-05, by urbanc
HOL/Tools/function_package: Added support for mutual recursive definitions.
2006-06-05, by krauss
Added [simp]-lemmas "in_inv_image" and "in_lex_prod" in the spirit of "in_measure".
2006-06-05, by krauss
ATP/res_clasimpset.ML has been merged into res_atp.ML.
2006-06-04, by mengj
Functions of Tools/ATP/res_clasimpset.ML are now in Tools/res_atp.ML. res_clasimpset.ML is not used anymore.
2006-06-04, by mengj
generalized wfI
2006-06-03, by paulson
misc cleanup;
2006-06-02, by wenzelm
removed obsolete ML files;
2006-06-02, by wenzelm
tuned;
2006-06-02, by wenzelm
tuned;
2006-06-02, by wenzelm
removed obsolete ML files;
2006-06-02, by wenzelm
merge: always normalize (and check!) reductions;
2006-06-02, by wenzelm
removed legacy ML scripts
2006-06-01, by huffman
tuned;
2006-06-01, by wenzelm
removed obsolete ML files;
2006-06-01, by wenzelm
lemmas strip;
2006-06-01, by wenzelm
removed obsolete ML files;
2006-06-01, by wenzelm
added some installation notes for the nominal package
2006-06-01, by urbanc
Tiny code cleanup
2006-06-01, by paulson
added an example suggested by D. Wang on the PoplMark-mailing list;
2006-06-01, by urbanc
added the hack "reset NameSpace.unique_names" to Nominal.thy
2006-06-01, by urbanc
tuned type print-translations
2006-05-30, by schirmer
proper meta definition;
2006-05-29, by wenzelm
fixed bug in type print translations
2006-05-29, by schirmer
tuned;
2006-05-29, by wenzelm
warnings to debug outputs
2006-05-29, by paulson
warnings to debug outputs; default translation to const-typed
2006-05-29, by paulson
Giving the "--silent" switch to E, to produce less output
2006-05-29, by paulson
fixing a variable-clash bug in rule_by_tactic
2006-05-29, by paulson
removed legacy ML scripts;
2006-05-28, by wenzelm
removed legacy ML scripts;
2006-05-28, by wenzelm
removed legacy ML scripts;
2006-05-27, by wenzelm
removed legacy ML scripts;
2006-05-27, by wenzelm
removed legacy ML scripts;
2006-05-27, by wenzelm
tuned;
2006-05-27, by wenzelm
tuned;
2006-05-27, by wenzelm
complete_split_rule: all Vars;
2006-05-27, by wenzelm
unfold/refold: LocalDefs.meta_rewrite_rule;
2006-05-27, by wenzelm
removed unused extern_thm;
2006-05-26, by wenzelm
activate Defines: fix frees;
2006-05-26, by wenzelm
pretty: do not exterm thm names;
2006-05-26, by wenzelm
forall_intr_list: do not ignore errors;
2006-05-26, by wenzelm
separate checks for acyclic/wellformed;
2006-05-26, by wenzelm
freeze_spec: gensym;
2006-05-26, by wenzelm
tuned;
2006-05-25, by wenzelm
axiomatization java_lang;
2006-05-25, by wenzelm
Changed the DFG format's functions' declaration procedure.
2006-05-25, by mengj
Fixed a bug.
2006-05-25, by mengj
A new "spass" method.
2006-05-25, by mengj
Added in settings used by "spass" method.
2006-05-25, by mengj
Added in SPASS oracle.
2006-05-25, by mengj
HOL problems now have DFG output format.
2006-05-25, by mengj
Changed input interface of dfg_write_file.
2006-05-25, by mengj
Added support for DFG format, used by SPASS.
2006-05-25, by mengj
Helper files in DFG format.
2006-05-25, by mengj
add_datatype_axm: finalize specified consts;
2006-05-24, by wenzelm
tuned;
2006-05-24, by wenzelm
tuned;
2006-05-24, by wenzelm
made smlnj happy;
2006-05-24, by wenzelm
wellformed: be less ambitious about structural containment;
2006-05-24, by wenzelm
Pure: update on overloaded defs;
2006-05-24, by wenzelm
Extended strong induction rule with additional
2006-05-24, by berghofe
add theorem cfcomp_strict
2006-05-24, by huffman
added add_deps, which actually records dependencies of consts (unlike add_finals);
2006-05-24, by wenzelm
tuned;
2006-05-24, by wenzelm
axiomatize class: Theory.add_deps;
2006-05-24, by wenzelm
simplified info/get_info;
2006-05-24, by wenzelm
simplified TypedefPackage.get_info;
2006-05-24, by wenzelm
made smlnj happy;
2006-05-23, by wenzelm
pretty_full_theory: tuned output of definitions;
2006-05-23, by wenzelm
export plain_args;
2006-05-23, by wenzelm
Defs.specifications_of: lhs/rhs now use typargs;
2006-05-22, by wenzelm
removed unchecked'';
2006-05-22, by wenzelm
pretty_full_theory: defs;
2006-05-22, by wenzelm
specifications_of: lhs/rhs represented as typargs;
2006-05-22, by wenzelm
export raw_unifys, could_unifys;
2006-05-22, by wenzelm
less
more
|
(0)
-10000
-3000
-1000
-480
+480
+1000
+3000
+10000
+30000
tip