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.
simplified AxClass interfaces;
2006-03-11, by wenzelm
added axclass_instance_XXX (from axclass.ML);
2006-03-11, by wenzelm
*** empty log message ***
2006-03-11, by wenzelm
added read_class, read/cert_classrel/arity (from axclass.ML);
2006-03-11, by wenzelm
moved read_class, read/cert_classrel/arity to sign.ML;
2006-03-11, by wenzelm
use axclass.ML earlier (in Isar/ROOT.ML);
2006-03-11, by wenzelm
nbe: no_document;
2006-03-11, by wenzelm
tuned;
2006-03-10, by wenzelm
exporting reapAll and killChild
2006-03-10, by paulson
text delimiter fixed
2006-03-10, by webertj
comment delimiter fixed
2006-03-10, by webertj
clauses now use (meta-)hyps instead of (meta-)implications; significant speedup
2006-03-10, by webertj
fix for document preparation
2006-03-10, by haftmann
Added Library/AssocList.thy
2006-03-10, by schirmer
renamed HOL + - * etc. to HOL.plus HOL.minus HOL.times etc.
2006-03-10, by haftmann
Changed some warnings to debug messages
2006-03-10, by paulson
Frequency analysis of constants (with types).
2006-03-10, by paulson
Shortened the exception messages from assume.
2006-03-10, by mengj
METAHYPS catches THM assume exception and prints out the terms containing schematic vars.
2006-03-10, by mengj
added many simple lemmas
2006-03-10, by huffman
Added more functions to the signature and tidied up some functions.
2006-03-09, by mengj
tuned;
2006-03-08, by wenzelm
tuned some proofs
2006-03-08, by urbanc
select_goals: split original conjunctions;
2006-03-08, by wenzelm
method: goal restriction defaults to [1];
2006-03-08, by wenzelm
infer_derivs: avoid allocating empty MinProof;
2006-03-08, by wenzelm
tuned;
2006-03-08, by wenzelm
Isar/method: goal restriction;
2006-03-08, by wenzelm
constdecl: always allow 'where';
2006-03-08, by wenzelm
deleted some proofs "on comment"
2006-03-08, by urbanc
tuned some proofs
2006-03-08, by urbanc
tuned some of the proofs about fresh_fun
2006-03-08, by urbanc
first running version of type classes
2006-03-08, by haftmann
first running version of type classes
2006-03-08, by haftmann
first running version of type classes
2006-03-08, by haftmann
Frequency strategy. Revised indentation, etc.
2006-03-08, by paulson
*** empty log message ***
2006-03-08, by nipkow
added ROOT.ML
2006-03-07, by obua
Indentation
2006-03-07, by paulson
Tidying and restructuring.
2006-03-07, by paulson
Tidying and tracing. Handling exn CLAUSE so that errors don't reach top-level.
2006-03-07, by paulson
Tidying. clausify_rules_pairs_abs now returns clauses in the same order as before.
2006-03-07, by paulson
Tidying. New invoke_atp_ml for top-level debugging. Flag to force FOL mode.
2006-03-07, by paulson
Tidying, and getting rid of SELECT_GOAL (as it does something different now)
2006-03-07, by paulson
Added HOL-ZF to Isabelle.
2006-03-07, by obua
substantial improvement in codegen iml
2006-03-07, by haftmann
Function get_clasimp_atp_lemmas gets all lemmas from claset, simpet and atpset.
2006-03-07, by mengj
relevance_filter takes input axioms as Term.term.
2006-03-07, by mengj
Proof reconstruction now only takes names of theorems as input.
2006-03-07, by mengj
Added tptp_write_file to write all necessary ATP input clauses to one file.
2006-03-07, by mengj
tptp_write_file now takes goals and axioms as Term.term and writes them to a file.
2006-03-07, by mengj
Added functions to retrieve local and global atpset rules.
2006-03-07, by mengj
Moved the settings for ATP time limit to res_atp.ML
2006-03-07, by mengj
Merged res_atp_setup.ML into res_atp.ML.
2006-03-07, by mengj
When ATP methods call ATPs, all input clauses from one subgoal are written to one file.
2006-03-07, by mengj
Merged res_atp_setup.ML into res_atp.ML.
2006-03-07, by mengj
SELECT_GOAL: fixed trivial case;
2006-03-05, by wenzelm
fixed a typo in a comment
2006-03-05, by webertj
tuned;
2006-03-04, by wenzelm
method: SelectGoals;
2006-03-04, by wenzelm
method: syntax for SelectGoals;
2006-03-04, by wenzelm
text: added SelectGoals;
2006-03-04, by wenzelm
tuned conj_curry;
2006-03-04, by wenzelm
added extract, retrofit;
2006-03-04, by wenzelm
added mk_conjunction;
2006-03-04, by wenzelm
method: restriction to first n sub-goals;
2006-03-04, by wenzelm
minor changes
2006-03-03, by nipkow
more examples
2006-03-03, by nipkow
changed and retracted change of location of code lemmas.
2006-03-03, by nipkow
ignore repeated vars on lhs, cleanup
2006-03-03, by nipkow
improvements for nbe
2006-03-03, by haftmann
reformatting
2006-03-02, by paulson
subset_refl now included using the atp attribute
2006-03-02, by paulson
moved the "use" directive
2006-03-02, by paulson
fixed the bugs itroduced by the previous commit
2006-03-02, by urbanc
made some small changes to generate nicer latex-output
2006-03-02, by urbanc
split the files
2006-03-02, by urbanc
Added in a signature.
2006-03-02, by mengj
fixed a problem where a permutation is not analysed
2006-03-01, by urbanc
streamlined the proof
2006-03-01, by urbanc
refined representation of codegen intermediate language
2006-03-01, by haftmann
some small tunings
2006-03-01, by urbanc
added fresh_fun_eqvt theorem to the theorem collection
2006-03-01, by urbanc
added initialisation-code for finite_guess
2006-03-01, by urbanc
made some small tunings in the decision-procedure
2006-03-01, by urbanc
Added setup for "atpset" (a rule set for ATPs).
2006-03-01, by mengj
Added file Tools/res_atpset.ML.
2006-03-01, by mengj
Merged HOL and FOL clauses and combined some functions.
2006-03-01, by mengj
A new file that sets up rules set used by ATPs. Rules are added to and removed from the set using "atp" attribute.
2006-03-01, by mengj
some minor tuning on the proofs
2006-03-01, by urbanc
initial commit (especially 2nd half needs to be cleaned up)
2006-02-28, by urbanc
removal of theory blacklist
2006-02-28, by paulson
new order for arity clauses
2006-02-28, by paulson
fixed but in freeze_spec
2006-02-28, by paulson
splitting up METAHYPS into smaller functions
2006-02-28, by paulson
typos
2006-02-28, by paulson
added a finite_guess tactic, which solves
2006-02-27, by urbanc
class package and codegen refinements
2006-02-27, by haftmann
added nbe
2006-02-27, by haftmann
added temp. nbe test
2006-02-27, by nipkow
added nbe, updated neb_*
2006-02-27, by nipkow
added nbe
2006-02-27, by nipkow
Typo.
2006-02-27, by ballarin
added support for arbitrary atoms in the simproc
2006-02-27, by urbanc
put_thms: do_index;
2006-02-26, by wenzelm
rewrite_goals_rule_aux: actually use prems if present;
2006-02-26, by wenzelm
add_local: do_index;
2006-02-26, by wenzelm
replaced the lemma at_two by at_different;
2006-02-26, by urbanc
improved the decision-procedure for permutations;
2006-02-26, by urbanc
improved codegen bootstrap
2006-02-25, by haftmann
change in codegen syntax
2006-02-25, by haftmann
some refinements
2006-02-25, by haftmann
added more detailed data to consts
2006-02-25, by haftmann
Reverted to old interface of AxClass.add_inst_arity(_i)
2006-02-24, by berghofe
Adapted to Florian's recent changes to the AxClass package.
2006-02-24, by berghofe
added lemmas
2006-02-23, by urbanc
make SML/NJ happy;
2006-02-23, by wenzelm
Default type level is T_FULL now.
2006-02-23, by mengj
eprover removes tmp files too.
2006-02-23, by mengj
vampire/eprover methods can now be applied repeatedly until they fail.
2006-02-23, by mengj
removed obsolete meta_conjunction_tr';
2006-02-22, by wenzelm
rew: handle conjunctionI/D1/D2;
2006-02-22, by wenzelm
simplified Pure conjunction, based on actual const;
2006-02-22, by wenzelm
removed rename_indexes_wrt;
2006-02-22, by wenzelm
renamed class_axms to class_intros;
2006-02-22, by wenzelm
tuned proofs;
2006-02-22, by wenzelm
simplified Pure conjunction;
2006-02-22, by wenzelm
not_equal: replaced syntax translation by abbreviation;
2006-02-22, by wenzelm
abandoned merge_alists' in favour of generic AList.merge
2006-02-22, by haftmann
added Tools/nbe, fixes
2006-02-21, by nipkow
added Tools/nbe
2006-02-21, by nipkow
New normalization-by-evaluation package
2006-02-21, by nipkow
distinct (op =);
2006-02-21, by wenzelm
fixed
2006-02-20, by kleing
Inclusion of subset_refl in ATP calls
2006-02-20, by paulson
Fix variable-naming bug (?) by removing a needless recursive call
2006-02-20, by paulson
slight code generator serialization improvements
2006-02-20, by haftmann
moved intro_classes from AxClass to ClassPackage
2006-02-20, by haftmann
fixed document
2006-02-19, by kleing
* denumerability of rationals by Benjamin Porter, based on NatPair (by Stefan Richter)
2006-02-19, by kleing
added a few lemmas to do with permutation-equivalence for the
2006-02-19, by urbanc
* added Library/ASeries (sum of arithmetic series with instantiation to nat and int)
2006-02-19, by kleing
use minimal imports
2006-02-19, by huffman
use qualified name for return
2006-02-19, by huffman
dest_def: tuned error msg;
2006-02-18, by wenzelm
const constraints: provide TFrees instead of TVars,
2006-02-17, by wenzelm
checkpoint/copy_node: reset body context;
2006-02-17, by wenzelm
global_qeds: transfer body context;
2006-02-17, by wenzelm
add_const_constraint(_i): demand TFrees instead of TVars, optional type (i.e. may delete constraints);
2006-02-17, by wenzelm
constrain: assert const declaration, optional type (i.e. may delete constraints);
2006-02-17, by wenzelm
removed Import/lazy_scan.ML;
2006-02-17, by wenzelm
hyperlinks in the PDF work now
2006-02-17, by paulson
replaced Symbol.explode by explode
2006-02-17, by obua
updated mailing list archive link
2006-02-17, by haftmann
use monomorphic sequences / scanners
2006-02-17, by obua
make maybe into a real type constructor; remove monad syntax
2006-02-17, by huffman
use VectorScannerSeq instead of ListScannerSeq in xml.ML
2006-02-16, by obua
removed lazy_scan
2006-02-16, by obua
improved scanning
2006-02-16, by obua
tuned;
2006-02-16, by wenzelm
Abstract Natural Numbers with polymorphic recursion.
2006-02-16, by wenzelm
new-style definitions/abbreviations;
2006-02-16, by wenzelm
added ex/Abstract_NAT.thy;
2006-02-16, by wenzelm
tuned;
2006-02-16, by wenzelm
tuned;
2006-02-16, by wenzelm
removed silly stuff
2006-02-16, by haftmann
* Isar/locales: new derived specification elements 'definition', 'abbreviation', 'axiomatization';
2006-02-16, by wenzelm
added abbreviation(_i);
2006-02-16, by wenzelm
added put_thms_internal: local_naming, no fact index;
2006-02-16, by wenzelm
added put_thms_internal;
2006-02-16, by wenzelm
added abbrev element;
2006-02-16, by wenzelm
added 'abbreviation';
2006-02-16, by wenzelm
added premsN;
2006-02-16, by wenzelm
Proof.put_thms_internal;
2006-02-16, by wenzelm
removed pointless replace;
2006-02-16, by wenzelm
tuned;
2006-02-16, by wenzelm
dest_def: actually return beta-eta contracted equation;
2006-02-16, by wenzelm
derived specifications: definition, abbreviation, axiomatization;
2006-02-16, by wenzelm
updated;
2006-02-16, by wenzelm
cache improvements
2006-02-16, by obua
variable counter is now also cached
2006-02-16, by obua
adapted to kernel changes
2006-02-16, by obua
tuned subst_bound(s);
2006-02-16, by wenzelm
fixed bugs, added caching
2006-02-15, by obua
added cases_node;
2006-02-15, by wenzelm
replaced qualified_force_prefix to sticky_prefix;
2006-02-15, by wenzelm
removed distinct, renamed gen_distinct to distinct;
2006-02-15, by wenzelm
check_text: Toplevel.node option;
2006-02-15, by wenzelm
init/exit no longer change the theory (no naming);
2006-02-15, by wenzelm
evaluate antiquotes depending on Toplevel.node option;
2006-02-15, by wenzelm
simplified presentation commands;
2006-02-15, by wenzelm
sane version of distinct_subgoals_tac, based on composition with Drule.distinct_prems_rl;
2006-02-15, by wenzelm
removed qualified_force_prefix;
2006-02-15, by wenzelm
replaced qualified_force_prefix to sticky_prefix;
2006-02-15, by wenzelm
chop is no longer pervasive;
2006-02-15, by wenzelm
rewrite_cterm: Thm.adjust_maxidx prevents unnecessary increments on rules;
2006-02-15, by wenzelm
added distinct_prems_rl;
2006-02-15, by wenzelm
specifications_of: avoid partiality;
2006-02-15, by wenzelm
counter example: avoid vacuous trace;
2006-02-15, by wenzelm
cannot use section before setup;
2006-02-15, by wenzelm
used Tactic.distinct_subgoals_tac;
2006-02-15, by wenzelm
removed distinct, renamed gen_distinct to distinct;
2006-02-15, by wenzelm
added lemma pt_perm_compose'
2006-02-15, by urbanc
got rid of superfluous linorder_neqE-instance for int.
2006-02-15, by nipkow
typo in a comment fixed
2006-02-15, by webertj
exported some interfaces useful for other code generator approaches
2006-02-15, by haftmann
some fixes
2006-02-15, by haftmann
exported specifications_of
2006-02-15, by haftmann
added theory of executable rational numbers
2006-02-14, by haftmann
improved handling of iml abstractions
2006-02-14, by haftmann
fixed tracing
2006-02-14, by paulson
Adapted to Context.generic syntax.
2006-02-13, by berghofe
Fixed a bug of type unification.
2006-02-13, by mengj
* ML/Pure/General: improved join interface for tables;
2006-02-12, by wenzelm
consts: maintain thy version for efficient transfer;
2006-02-12, by wenzelm
tuned;
2006-02-12, by wenzelm
export exception SAME (for join);
2006-02-12, by wenzelm
low-level tuning of merge: maintain identity of accesses;
2006-02-12, by wenzelm
share exception UNDEF with Table;
2006-02-12, by wenzelm
structure Datatab: private copy avoids potential conflict of table exceptions;
2006-02-12, by wenzelm
added eq_consts;
2006-02-12, by wenzelm
minor tuning of proofs, notably induct;
2006-02-12, by wenzelm
simplified TableFun.join;
2006-02-12, by wenzelm
\usepackage{amssymb};
2006-02-12, by wenzelm
* include generalised MVT in HyperReal (contributed by Benjamin Porter)
2006-02-12, by kleing
* moved ThreeDivides from Isar_examples to better suited HOL/ex
2006-02-12, by kleing
divisibility by 3 theorem, contributed by Benjamin Porter,
2006-02-12, by kleing
replaced mixfix_conflict by mixfix_content;
2006-02-11, by wenzelm
added map_theory;
2006-02-11, by wenzelm
added abbreviations: activated by init, no expressions yet;
2006-02-11, by wenzelm
added restore;
2006-02-11, by wenzelm
tuned mixfixes, mixfix_conflict;
2006-02-11, by wenzelm
removed custom_accesses;
2006-02-11, by wenzelm
added variant_name;
2006-02-11, by wenzelm
removed custom_accesses;
2006-02-11, by wenzelm
tuned;
2006-02-11, by wenzelm
added chop (sane version of splitAt);
2006-02-11, by wenzelm
Changed some code due to changes in reduce_axiomsN.ML.
2006-02-11, by mengj
Added another filter strategy.
2006-02-11, by mengj
improved code generator devarification
2006-02-10, by haftmann
statement: improved error msg;
2006-02-10, by wenzelm
* ML/Pure: generic Args/Attrib syntax everywhere;
2006-02-10, by wenzelm
moved fixedN to lexicon.ML;
2006-02-10, by wenzelm
added mfix_delims;
2006-02-10, by wenzelm
added mixfix_conflict;
2006-02-10, by wenzelm
added fixedN, constN;
2006-02-10, by wenzelm
tuned comment;
2006-02-10, by wenzelm
tuned comment;
2006-02-10, by wenzelm
syntax: Context.generic;
2006-02-10, by wenzelm
Context.generic is canonical state of parsers;
2006-02-10, by wenzelm
Local syntax depending on theory syntax.
2006-02-10, by wenzelm
decode: observe Syntax.constN;
2006-02-10, by wenzelm
removed obsolete add_typ/term_classes/tycons;
2006-02-10, by wenzelm
tuned extern_term, pretty_term';
2006-02-10, by wenzelm
removed set quick_and_dirty and ThmDeps.enable -- no effect here;
2006-02-10, by wenzelm
abbrevs: store in reverted orientation;
2006-02-10, by wenzelm
use proof_general.ML: setmp quick_and_dirty captures default value;
2006-02-10, by wenzelm
added Isar/local_syntax.ML;
2006-02-10, by wenzelm
tuned;
2006-02-10, by wenzelm
Args/Attrib syntax: Context.generic;
2006-02-10, by wenzelm
simplified polyml example;
2006-02-10, by wenzelm
tidying
2006-02-09, by paulson
blacklist tweaks
2006-02-09, by paulson
names for simprules
2006-02-09, by paulson
removed redundant lemmas
2006-02-09, by huffman
no longer need All_equiv lemmas
2006-02-09, by huffman
map_type_tvar/tfree: map_atyps;
2006-02-08, by wenzelm
tuned;
2006-02-08, by wenzelm
*** empty log message ***
2006-02-08, by nipkow
made "dvd" on numbers executable by simp.
2006-02-08, by nipkow
introduced gen_distinct in place of distinct
2006-02-08, by haftmann
fixed the most silly bug conceivable in map_atyps
2006-02-08, by haftmann
lambda: base name of Const;
2006-02-07, by wenzelm
adapted Sign.infer_types;
2006-02-07, by wenzelm
has_duplicates;
2006-02-07, by wenzelm
adapted Sign.infer_types;
2006-02-07, by wenzelm
added local consts component;
2006-02-07, by wenzelm
Library.is_equal;
2006-02-07, by wenzelm
removed obsolete sign_of_cterm;
2006-02-07, by wenzelm
adapted Sign.infer_types(_simult), Sign.certify_term/prop;
2006-02-07, by wenzelm
export consts_of;
2006-02-07, by wenzelm
removed eq-polymorphic duplicates;
2006-02-07, by wenzelm
renamed space to space_of;
2006-02-07, by wenzelm
renamed gen_duplicates to duplicates;
2006-02-07, by wenzelm
slight improvements in code generation
2006-02-07, by haftmann
updated;
2006-02-06, by wenzelm
Logic.combound;
2006-02-06, by wenzelm
adapted Consts.dest;
2006-02-06, by wenzelm
Sign.cert_def;
2006-02-06, by wenzelm
added bound_vars;
2006-02-06, by wenzelm
TableFun: renamed xxx_multi to xxx_list;
2006-02-06, by wenzelm
Envir.(beta_)eta_contract;
2006-02-06, by wenzelm
added local_theory, with optional locale xname;
2006-02-06, by wenzelm
type local_theory;
2006-02-06, by wenzelm
norm_term: Sign.const_expansion, Envir.expand_atom;
2006-02-06, by wenzelm
TableFun: renamed xxx_multi to xxx_list;
2006-02-06, by wenzelm
type local_theory = Proof.context;
2006-02-06, by wenzelm
cert_def: use Logic.dest_def;
2006-02-06, by wenzelm
Toplevel.local_theory;
2006-02-06, by wenzelm
LocalDefs.cert_def;
2006-02-06, by wenzelm
eq_prop: Envir.beta_eta_contract;
2006-02-06, by wenzelm
renamed xxx_multi to xxx_list;
2006-02-06, by wenzelm
moved combound, rlist_abs to logic.ML;
2006-02-06, by wenzelm
union_tpairs: Library.merge;
2006-02-06, by wenzelm
moved no_vars to sign.ML;
2006-02-06, by wenzelm
lambda: abstract over any const;
2006-02-06, by wenzelm
added add_abbrevs(_i);
2006-02-06, by wenzelm
moved (beta_)eta_contract to envir.ML;
2006-02-06, by wenzelm
tuned;
2006-02-06, by wenzelm
added generic dest_def (mostly from theory.ML);
2006-02-06, by wenzelm
added (beta_)eta_contract (from pattern.ML);
2006-02-06, by wenzelm
print_theory: const abbreviations;
2006-02-06, by wenzelm
added abbreviations;
2006-02-06, by wenzelm
load envir.ML and logic.ML early;
2006-02-06, by wenzelm
Logic.rlist_abs;
2006-02-06, by wenzelm
Logic.const_of_class/class_of_const;
2006-02-06, by wenzelm
TableFun: renamed xxx_multi to xxx_list;
2006-02-06, by wenzelm
replaced Symtab.merge_multi by local merge_rules;
2006-02-06, by wenzelm
Envir.(beta_)eta_contract;
2006-02-06, by wenzelm
subsituted gen_duplicates / has_duplicates for duplicates whenever appropriate
2006-02-06, by haftmann
added strip_abs
2006-02-06, by haftmann
clarified semantics of merge
2006-02-06, by haftmann
speedup: use simproc for AC rules
2006-02-04, by huffman
UU_reorient_simproc no longer rewrites UU = numeral
2006-02-04, by huffman
removed obsolete gen_ins/mem;
2006-02-03, by wenzelm
removed add/del_rules;
2006-02-03, by wenzelm
canonical member/insert/merge;
2006-02-03, by wenzelm
removal of case analysis clauses
2006-02-03, by paulson
fix
2006-02-03, by haftmann
minor improvements
2006-02-03, by haftmann
refined signature of locale module
2006-02-03, by haftmann
no toplevel 'thy' anymore
2006-02-03, by haftmann
fix in codegen
2006-02-03, by haftmann
do not open structure;
2006-02-02, by wenzelm
reimplemented using Equiv_Relations.thy
2006-02-02, by huffman
improvement in devarifications
2006-02-02, by haftmann
alternative syntax for instances
2006-02-02, by haftmann
tuned;
2006-02-02, by wenzelm
consumes: negative argument relative to total number of prems;
2006-02-02, by wenzelm
added refine_insert;
2006-02-02, by wenzelm
Proof.refine_insert;
2006-02-02, by wenzelm
always use Attrib.src;
2006-02-02, by wenzelm
more generic type for map_specs/facts;
2006-02-02, by wenzelm
'obtains' element;
2006-02-02, by wenzelm
'obtain': optional case name;
2006-02-02, by wenzelm
index elements;
2006-02-02, by wenzelm
* Isar: 'obtains' element;
2006-02-02, by wenzelm
tuned msg;
2006-02-02, by wenzelm
theorem(_in_locale): Element.statement, Obtain.statement;
2006-02-02, by wenzelm
added parname;
2006-02-02, by wenzelm
obtain(_i): optional name for 'that';
2006-02-02, by wenzelm
tuned comments;
2006-02-02, by wenzelm
moved (general_)statement to outer_parse.ML;
2006-02-02, by wenzelm
added concluding statements: Shows/Obtains;
2006-02-02, by wenzelm
moved specific map_typ/term to sign.ML;
2006-02-02, by wenzelm
added specific map_typ/term (from term.ML);
2006-02-02, by wenzelm
Exporting recdef's hints for use by new recdef package
2006-02-02, by krauss
*_asms_of fixed.
2006-02-02, by ballarin
add 64bit atbroy98 platform
2006-02-02, by kleing
updated;
2006-02-01, by wenzelm
Added "evaluation" method and oracle.
2006-02-01, by berghofe
new and updated protocol proofs by Giamp Bella
2006-02-01, by paulson
substantial cleanup and simplifications
2006-02-01, by haftmann
name clarifications
2006-02-01, by haftmann
added map_entry_yield
2006-02-01, by haftmann
- renamed some lemmas (some had names coming from ancient
2006-02-01, by urbanc
added all constructors from PhD
2006-02-01, by urbanc
axiomatization: retrict parameters to occurrences in specs;
2006-01-31, by wenzelm
improved comments;
2006-01-31, by wenzelm
tuned LocalDefs.unfold;
2006-01-31, by wenzelm
(un)fold: removed '(raw)' option;
2006-01-31, by wenzelm
added consts_retricted;
2006-01-31, by wenzelm
(un)fold: no raw flag;
2006-01-31, by wenzelm
tuned;
2006-01-31, by wenzelm
tuned LocalTheory.pretty_consts;
2006-01-31, by wenzelm
(un)folded: removed '(raw)' option;
2006-01-31, by wenzelm
lambda: abstract over TYPE argument, too;
2006-01-31, by wenzelm
tuned comments;
2006-01-31, by wenzelm
removal of ResClause.num_of_clauses and other simplifications
2006-01-31, by paulson
working SPASS support; much tidying
2006-01-31, by paulson
added serialization for arbitrary
2006-01-31, by haftmann
minor change to CodegenPackage interface
2006-01-31, by haftmann
minor cleanups
2006-01-31, by haftmann
more coherent lookup extraction functions
2006-01-31, by haftmann
reorganization of code to support DFG otuput
2006-01-31, by paulson
* Pure: 'advanced' translation functions use Context.generic instead of just theory;
2006-01-31, by wenzelm
declare defn rules;
2006-01-31, by wenzelm
all styles now reset to defaults first, i.e. the document may switch styles back and forth;
2006-01-31, by wenzelm
export meta_rewrite_rule;
2006-01-31, by wenzelm
advanced translations: Context.generic;
2006-01-31, by wenzelm
advanced translations: Context.generic;
2006-01-31, by wenzelm
tidy-up of res_clause.ML, removing the "predicates" field
2006-01-30, by paulson
'setup': no list type, support implicit setup;
2006-01-30, by wenzelm
'fixes': support plain vars;
2006-01-30, by wenzelm
fixed a syntax error!
2006-01-30, by paulson
replaced gen_list by enum
2006-01-30, by haftmann
adaptions to codegen_package
2006-01-30, by haftmann
various improvements
2006-01-30, by haftmann
added three times overloaded Isar instance command
2006-01-30, by haftmann
moved instance Isar command to class_package.ML
2006-01-30, by haftmann
added map_atype, map_aterms
2006-01-30, by haftmann
tuned proof;
2006-01-29, by wenzelm
declare atomize/defn for Ball;
2006-01-29, by wenzelm
invent_fixes: merely enter body temporarily;
2006-01-29, by wenzelm
'unfolding': LocalDefs.unfold;
2006-01-29, by wenzelm
moved treatment of object-logic equalities to local_defs.ML;
2006-01-29, by wenzelm
method (un)folded: option '(raw)';
2006-01-29, by wenzelm
added attributes defn_add/del;
2006-01-29, by wenzelm
added 'defn' attribute;
2006-01-29, by wenzelm
proper order of trfuns;
2006-01-29, by wenzelm
CPure: Context.add_setup;
2006-01-29, by wenzelm
tuned proofs;
2006-01-29, by wenzelm
implicit setup;
2006-01-29, by wenzelm
default rule step: norm_hhf_tac;
2006-01-29, by wenzelm
tuned comment;
2006-01-29, by wenzelm
declare 'defn' rules;
2006-01-29, by wenzelm
LocalDefs;
2006-01-28, by wenzelm
Basic operations on local definitions.
2006-01-28, by wenzelm
removed unnecessary Syntax.fix_mixfix;
2006-01-28, by wenzelm
added axiomatization_loc, definition_loc;
2006-01-28, by wenzelm
moved local defs to local_defs.ML;
2006-01-28, by wenzelm
LocalDefs;
2006-01-28, by wenzelm
removed unatomize;
2006-01-28, by wenzelm
(un)fold: support object-level rewrites;
2006-01-28, by wenzelm
added print_consts;
2006-01-28, by wenzelm
removed obsolete keyword 'files';
2006-01-28, by wenzelm
(un)folded: support object-level rewrites;
2006-01-28, by wenzelm
added equals_cong;
2006-01-28, by wenzelm
added Isar/local_defs.ML;
2006-01-28, by wenzelm
LocalDefs.add_def;
2006-01-28, by wenzelm
LocalDefs.def_export;
2006-01-28, by wenzelm
tuned proofs;
2006-01-28, by wenzelm
Pure/Isar: (un)folded, (un)fold, unfolding support
2006-01-28, by wenzelm
interrupt_timeout for Poly replaced by stub
2006-01-27, by webertj
added atomize_iff;
2006-01-27, by wenzelm
renamed Pretty.gen_list to Pretty.enum;
2006-01-27, by wenzelm
swapped theory_context;
2006-01-27, by wenzelm
swapped Toplevel.theory_context;
2006-01-27, by wenzelm
added invent_fixes;
2006-01-27, by wenzelm
swapped Toplevel.theory_context;
2006-01-27, by wenzelm
renamed reverse_atomize to unatomize;
2006-01-27, by wenzelm
init: include view;
2006-01-27, by wenzelm
improved 'notes', including proper treatment of locale results;
2006-01-27, by wenzelm
swapped Toplevel.theory_context;
2006-01-27, by wenzelm
Locale.init;
2006-01-27, by wenzelm
renamed gen_list to enum;
2006-01-27, by wenzelm
moved theorem tags from Drule to PureThy;
2006-01-27, by wenzelm
added ProofContext.pprint_context (depends on ProofContext.debug);
2006-01-27, by wenzelm
moved theorem tags from Drule to PureThy;
2006-01-27, by wenzelm
tidying up SPASS output
2006-01-27, by paulson
tidying
2006-01-27, by paulson
better reporting
2006-01-27, by paulson
Interface to access the specification of a named locale.
2006-01-27, by ballarin
Added new file Tools/ATP/reduce_axiomsN.ML
2006-01-27, by mengj
Added in new file Tools/ATP/reduce_axiomsN.ML
2006-01-27, by mengj
Changed codes that call relevance filter.
2006-01-27, by mengj
Relevance filtering. Has replaced the previous version.
2006-01-27, by mengj
interrupt_timeout now raises Interrupt instead of SML90.Interrupt
2006-01-26, by webertj
smaller example to prevent timeout
2006-01-26, by webertj
Fixed bug in code generator for primitive definitions that
2006-01-26, by berghofe
Inductive sets with no introduction rules are now allowed as well.
2006-01-26, by berghofe
added definition(_i);
2006-01-25, by wenzelm
renamed export to export_standard (again!), because it includes Drule.local_standard';
2006-01-25, by wenzelm
ProofContext.export_standard;
2006-01-25, by wenzelm
tuned atomize_cterm;
2006-01-25, by wenzelm
turned abstract_term into ProofContext.abs_def;
2006-01-25, by wenzelm
added constant definition;
2006-01-25, by wenzelm
added 'definition';
2006-01-25, by wenzelm
tuned comment;
2006-01-25, by wenzelm
export name_multi;
2006-01-25, by wenzelm
abs_def: improved error;
2006-01-25, by wenzelm
ObjectLogic.atomize_cterm;
2006-01-25, by wenzelm
updated;
2006-01-25, by wenzelm
works with DPLL solver now
2006-01-24, by webertj
the additional freshness-condition in the one-induction
2006-01-24, by urbanc
fixed code_generate syntax;
2006-01-24, by wenzelm
renamed axiomatize(_i) to axiomatization(_i);
2006-01-24, by wenzelm
renamed inferred_type to inferred_param;
2006-01-24, by wenzelm
ProofContext.inferred_param;
2006-01-24, by wenzelm
removed the_params;
2006-01-24, by wenzelm
less
more
|
(0)
-10000
-3000
-1000
-480
+480
+1000
+3000
+10000
+30000
tip