Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-10000
-1920
+1920
+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.
removed misleading OuterLex.eq_token;
2006-12-30, by wenzelm
pretty_statement: more careful handling of name_hint;
2006-12-30, by wenzelm
added has_name_hint;
2006-12-30, by wenzelm
removed obsolete name_hint handling;
2006-12-30, by wenzelm
removed conditional combinator;
2006-12-30, by wenzelm
removed obsolete support for polyml-4.9.1;
2006-12-30, by wenzelm
* Proof General: proper undo of final 'end'; discontinued Isabelle/classic;
2006-12-30, by wenzelm
inform_file_processed: Toplevel.init_empty;
2006-12-30, by wenzelm
refined notion of empty toplevel, admits undo of 'end';
2006-12-30, by wenzelm
Toplevel.init_state;
2006-12-30, by wenzelm
removed obsolete 'clear_undos';
2006-12-30, by wenzelm
removed obsolete clear_undos_theory;
2006-12-30, by wenzelm
major restructurings
2006-12-29, by haftmann
cleanup
2006-12-29, by haftmann
improved print of constructors in OCaml
2006-12-29, by haftmann
changed syntax for axclass attach
2006-12-29, by haftmann
removed obsolete cond_add_path;
2006-12-29, by wenzelm
removed obsolete context_thy etc.;
2006-12-29, by wenzelm
removed obsolete init_pgip;
2006-12-29, by wenzelm
removed obsolete init_context;
2006-12-29, by wenzelm
obsolete (cf. ProofGeneral/proof_general_emacs.ML);
2006-12-29, by wenzelm
tuned;
2006-12-29, by wenzelm
signed_string_of_int;
2006-12-29, by wenzelm
added proper header;
2006-12-29, by wenzelm
added signed_string_of_int (pruduces proper - instead of SML's ~);
2006-12-29, by wenzelm
removed obsolete proof_general.ML;
2006-12-29, by wenzelm
minor tuning;
2006-12-29, by wenzelm
tuned specifications/proofs;
2006-12-29, by wenzelm
replaced Sign.classes by Sign.all_classes (topologically sorted);
2006-12-29, by wenzelm
renamed Graph.project to Graph.subgraph;
2006-12-29, by wenzelm
replaced Sign.classes by Sign.all_classes (topologically sorted);
2006-12-29, by wenzelm
renamed project to subgraph, improved presentation, avoided unnecessary evaluation of predicate;
2006-12-29, by wenzelm
Sorts.minimal_classes;
2006-12-29, by wenzelm
classes: more direct way to achieve topological sorting;
2006-12-29, by wenzelm
replaced classes by all_classes (topologically sorted);
2006-12-29, by wenzelm
replaced Sign.classes by Sign.all_classes (topologically sorted);
2006-12-29, by wenzelm
Enable new Proof General code again after SML/NJ compatibility fixes by Florian.
2006-12-29, by aspinall
Typo in last commit
2006-12-29, by aspinall
explicit construction of operational classes
2006-12-29, by haftmann
added handling for explicit classrel witnesses
2006-12-29, by haftmann
``classes`` now returns classes in topological order
2006-12-29, by haftmann
dropped some bookkeeping
2006-12-29, by haftmann
simplified class_package
2006-12-29, by haftmann
use_ml: reverted to simple output (Poly/ML changed);
2006-12-29, by wenzelm
removed private files
2006-12-28, by haftmann
tuned;
2006-12-28, by wenzelm
removed nospaces (Char.isSpace does not conform to Isabelle conventions);
2006-12-28, by wenzelm
tuned msg;
2006-12-28, by wenzelm
inlined nospaces (from library.ML);
2006-12-28, by wenzelm
added
2006-12-28, by haftmann
some clarifications
2006-12-27, by haftmann
different handling of type variable names
2006-12-27, by haftmann
added split
2006-12-27, by haftmann
fixed misleading error message
2006-12-27, by haftmann
dropped section header
2006-12-27, by haftmann
added OCaml code generation (without dictionaries)
2006-12-27, by haftmann
removed Haskell reserved words
2006-12-27, by haftmann
removed Main.thy
2006-12-27, by haftmann
moved code generator product setup here
2006-12-27, by haftmann
added code generator test theory
2006-12-27, by haftmann
explizit serialization for Haskell id
2006-12-27, by haftmann
removed code generation stuff belonging to other theories
2006-12-27, by haftmann
moved code generator bool setup here
2006-12-27, by haftmann
exported explicit equality on tokens
2006-12-27, by haftmann
made SML/NJ happy
2006-12-27, by haftmann
revised for new make_clauses
2006-12-22, by paulson
tidying the ATP communications
2006-12-22, by paulson
string primtives
2006-12-22, by paulson
deactivated test for the moment
2006-12-22, by haftmann
fixed typo in comment
2006-12-22, by paulson
Experimenting with interpretations of "definition".
2006-12-22, by ballarin
clarified code
2006-12-21, by haftmann
dropped superfluos code
2006-12-21, by haftmann
code clarifications
2006-12-21, by haftmann
import path made absolute
2006-12-21, by haftmann
added code lemmas for quantification over bounded nats
2006-12-21, by haftmann
Disable new Proof General code until SML/NJ compile fixed.
2006-12-21, by aspinall
Use new Proof General code by default [see comment for reverting]
2006-12-20, by aspinall
change from "Array" to "Vector"
2006-12-20, by paulson
add lemmas Standard_starfun(2)_iff
2006-12-19, by huffman
Missing elements from doc_markup_elements
2006-12-19, by aspinall
Remove obsolete prefixes from error and warning messages.
2006-12-19, by aspinall
added isatool codegen
2006-12-18, by haftmann
dropped CodegenPackage.const_of_idf
2006-12-18, by haftmann
improvements in syntax handling
2006-12-18, by haftmann
added Thyname.* and * constant expressions
2006-12-18, by haftmann
introduces "__" naming policy
2006-12-18, by haftmann
switched argument order in *.syntax lifters
2006-12-18, by haftmann
added gen_reflection_tac
2006-12-18, by haftmann
now testing executable content of nearly all HOL
2006-12-18, by haftmann
dropped debug cmd
2006-12-18, by haftmann
explicit nonfix declaration for ML "subset"
2006-12-18, by haftmann
dropped two inline directives
2006-12-18, by haftmann
introduced abstract view on number expressions in hologic.ML
2006-12-18, by haftmann
whitespace fix
2006-12-18, by haftmann
added code generation syntax for some char combinators
2006-12-18, by haftmann
infix syntax for generated code for composition
2006-12-18, by haftmann
new-style oracle setup
2006-12-18, by haftmann
added functions tutorial
2006-12-18, by haftmann
Add abstraction for objtypes and documents.
2006-12-17, by aspinall
removed Hyperreal/HyperArith.thy and Hyperreal/HyperPow.thy
2006-12-16, by huffman
moved several theorems; rearranged theory dependencies
2006-12-16, by huffman
hypreal_of_hypnat abbreviates more general of_hypnat
2006-12-16, by huffman
tracing instead of warning
2006-12-15, by webertj
updated;
2006-12-15, by wenzelm
removed obsolete assert;
2006-12-15, by wenzelm
renamed LocalTheory.assert to affirm;
2006-12-15, by wenzelm
tuned -- accomodate Alice;
2006-12-15, by wenzelm
avoid conflict with Alice keywords: renamed pack -> implode, unpack -> explode, any -> many, avoided assert;
2006-12-15, by wenzelm
remove Hyperreal/fuf.ML
2006-12-14, by huffman
remove commented section
2006-12-14, by huffman
remove ultra tactic and redundant FreeUltrafilterNat lemmas
2006-12-14, by huffman
declare insert_iff [simp]
2006-12-14, by huffman
activated improved use_ml, which captures output and reports source positions;
2006-12-14, by wenzelm
tuned;
2006-12-14, by wenzelm
prove hyperpow_realpow using transfer
2006-12-14, by huffman
remove usage of ultra tactic
2006-12-14, by huffman
add lemmas singleton and insert_iff
2006-12-14, by huffman
generalized type of hyperpow; removed hcpow
2006-12-14, by huffman
redefine hSuc as *f* Suc, and move to HyperNat.thy
2006-12-14, by huffman
proper use of IntInf instead of InfInf;
2006-12-14, by wenzelm
defs/notes: more robust transitivity reasoning;
2006-12-14, by wenzelm
added trans_terms/props;
2006-12-14, by wenzelm
locale: print context for begin;
2006-12-14, by wenzelm
remove references to star_n and FreeUltrafilterNat; new proof of NSBseq_Bseq
2006-12-14, by huffman
remove uses of star_n and FreeUltrafilterNat
2006-12-13, by huffman
remove use of FreeUltrafilterNat
2006-12-13, by huffman
added lemmas about hRe, hIm, HComplex; removed all uses of star_n
2006-12-13, by huffman
fixed type
2006-12-13, by haftmann
added stub for OCaml serializer
2006-12-13, by haftmann
cleanup
2006-12-13, by haftmann
whitespace correction
2006-12-13, by haftmann
clarifed comment
2006-12-13, by haftmann
dropped FIXME comment
2006-12-13, by haftmann
clarified character setup
2006-12-13, by haftmann
remove references to star_n
2006-12-13, by huffman
SComplex abbreviates Standard
2006-12-13, by huffman
simplified mk/dest_numeral (cf. mk/dest_binum of 1.65);
2006-12-13, by wenzelm
removed legacy ML bindings;
2006-12-13, by wenzelm
updated;
2006-12-13, by wenzelm
tuned signature;
2006-12-13, by wenzelm
internal_abbrev: observe print mode;
2006-12-13, by wenzelm
target_abbrev: internal mode for abbrevs;
2006-12-13, by wenzelm
edge: actually apply operation!
2006-12-13, by wenzelm
tuned;
2006-12-13, by wenzelm
authentic syntax for number_of
2006-12-13, by haftmann
introduced mk/dest_numeral/number for mk/dest_binum etc.
2006-12-13, by haftmann
fixed syntax for bounded quantification
2006-12-13, by haftmann
dropped superfluous header
2006-12-13, by haftmann
clarified error message
2006-12-13, by krauss
nat type now has a size functin => no longer needed as special case
2006-12-13, by krauss
simplified
2006-12-13, by krauss
local_abbrev: proper fix/declare of local entities;
2006-12-13, by wenzelm
Deleted the unused type argument of UVar
2006-12-13, by paulson
tuned comments;
2006-12-13, by wenzelm
added IsarAdvanced/Functions
2006-12-13, by krauss
generalized some lemmas; removed redundant lemmas; cleaned up some proofs
2006-12-13, by huffman
remove uses of scaleR infix syntax; add lemma Reals_number_of
2006-12-13, by huffman
tuned;
2006-12-12, by wenzelm
add_abbrev: removed Assumption.add_assms (danger of inconsistent naming);
2006-12-12, by wenzelm
updated;
2006-12-12, by wenzelm
simplified unlocalize_mixfix;
2006-12-12, by wenzelm
removed is_class -- handled internally;
2006-12-12, by wenzelm
notation: Term.equiv_types;
2006-12-12, by wenzelm
abbrev: tuned signature;
2006-12-12, by wenzelm
tuned expand_term;
2006-12-12, by wenzelm
classified show/thus as prf_asm_goal, which is usually hilited in PG;
2006-12-12, by wenzelm
tuned expand_binds;
2006-12-12, by wenzelm
tuned error messages;
2006-12-12, by wenzelm
added equiv_types;
2006-12-12, by wenzelm
add_abbrev: tuned signature;
2006-12-12, by wenzelm
added expand_term_frees;
2006-12-12, by wenzelm
abbreviate: tuned signature;
2006-12-12, by wenzelm
LocalTheory.abbrev;
2006-12-12, by wenzelm
removed redundant constants and lemmas
2006-12-12, by huffman
additions to HOL-Complex
2006-12-12, by huffman
Removal of the "keep_types" flag: we always keep types!
2006-12-12, by paulson
make SML/NJ happy;
2006-12-12, by wenzelm
made SML/NJ happy;
2006-12-12, by wenzelm
consistent naming for FreeUltrafilterNat lemmas; cleaned up
2006-12-12, by huffman
cleaned up; generalized some proofs
2006-12-12, by huffman
fix assumptions on NSDERIV_quotient
2006-12-12, by huffman
changed (ns)deriv to take functions of type 'a::real_normed_field => 'a
2006-12-12, by huffman
generalize some theorems
2006-12-12, by huffman
add type annotation
2006-12-12, by huffman
read_xnum: return leading_zeros, radix;
2006-12-12, by wenzelm
authentic syntax for Pls/Min/Bit;
2006-12-12, by wenzelm
authentic syntax for Pls/Min/Bit;
2006-12-12, by wenzelm
binary numerals: restricted to actual abstract syntax;
2006-12-12, by wenzelm
Hyperreal/FrechetDeriv.thy
2006-12-12, by huffman
theory of Frechet derivatives
2006-12-12, by huffman
specials: include single quote;
2006-12-11, by wenzelm
xstr: disallow backslashes;
2006-12-11, by wenzelm
advanced translation functions: Proof.context;
2006-12-11, by wenzelm
advanced translation functions: Proof.context;
2006-12-11, by wenzelm
added improved versions of use_text/file (still inactive);
2006-12-11, by wenzelm
added use_file;
2006-12-11, by wenzelm
load secure.ML after symbol.ML, when default output is active;
2006-12-11, by wenzelm
ordered lists instead of tables for resolving hyps; speedup
2006-12-11, by webertj
nominal_primrec now prints initial proof state.
2006-12-11, by berghofe
Abbreviations can now be specified simultaneously
2006-12-11, by berghofe
Adapted to new inductive definition package.
2006-12-11, by berghofe
added ProofGeneral settings;
2006-12-11, by wenzelm
tuned comments;
2006-12-10, by wenzelm
tuned;
2006-12-10, by wenzelm
defs: increased entropy of mixfix handling;
2006-12-10, by wenzelm
fixed term_of_list;
2006-12-10, by wenzelm
Concrete syntax for hex chars and strings.
2006-12-10, by wenzelm
renamed str_of_XXX to print_XXX;
2006-12-10, by wenzelm
HOLogic cleanup;
2006-12-10, by wenzelm
ML_Syntax.print_XXX;
2006-12-10, by wenzelm
misc cleanup -- removed non-HOL operations;
2006-12-10, by wenzelm
moved char/string syntax to Tools/string_syntax.ML;
2006-12-10, by wenzelm
added Tools/string_syntax.ML;
2006-12-10, by wenzelm
removed junk;
2006-12-10, by wenzelm
interpretation: use C_class name prefix;
2006-12-10, by wenzelm
abs/binder_tr': support printing of idtdummy;
2006-12-10, by wenzelm
respects2: tuned spacing;
2006-12-10, by wenzelm
support printing of idtdummy;
2006-12-10, by wenzelm
added is_class (approximation);
2006-12-10, by wenzelm
LocalTheory.notation/abbrev;
2006-12-10, by wenzelm
extract_case: Name.clean;
2006-12-10, by wenzelm
added target_notation/abbrev;
2006-12-10, by wenzelm
added notation/abbrev (from term_syntax.ML);
2006-12-10, by wenzelm
tuned absdummy;
2006-12-10, by wenzelm
added no_frees;
2006-12-10, by wenzelm
removed (cf. proof_context.ML and local_theory.ML);
2006-12-10, by wenzelm
removed Isar/term_syntax.ML;
2006-12-10, by wenzelm
avoid internal name O_;
2006-12-10, by wenzelm
hide const linorder.less_eq_less.max linorder.less_eq_less.min;
2006-12-10, by wenzelm
hardwired option -q;
2006-12-10, by wenzelm
added print_abbrevs;
2006-12-10, by wenzelm
renaming
2006-12-10, by nipkow
Modified lattice locale
2006-12-10, by nipkow
updated;
2006-12-09, by wenzelm
added internal_mode;
2006-12-09, by wenzelm
simplified abbrev: single argument;
2006-12-09, by wenzelm
TermSyntax.abbrev;
2006-12-09, by wenzelm
added read/pretty_term_abbrev, print_abbrevs;
2006-12-09, by wenzelm
init_context: reset naming;
2006-12-09, by wenzelm
added 'print_abbrevs';
2006-12-09, by wenzelm
added print_abbrevs;
2006-12-09, by wenzelm
added term_abbrev;
2006-12-09, by wenzelm
renamed reserved to reserved_names;
2006-12-09, by wenzelm
tuned Consts signature;
2006-12-09, by wenzelm
abbrevs: print original rhs;
2006-12-09, by wenzelm
abbreviate: always authentic, force expansion of internal abbreviations;
2006-12-09, by wenzelm
ML_Syntax.reserved(_names);
2006-12-09, by wenzelm
TermSyntax.abbrev;
2006-12-09, by wenzelm
added antiquotation abbrev;
2006-12-09, by wenzelm
added print_abbrevs;
2006-12-09, by wenzelm
tuned use_text;
2006-12-08, by wenzelm
added 'help' command (same of 'print_commands');
2006-12-08, by wenzelm
more careful evaluation of ML text, prevents spurious output;
2006-12-08, by wenzelm
date: forcing LC_ALL=C prevents funny file names;
2006-12-08, by wenzelm
root function: restore default interrupt handler;
2006-12-08, by wenzelm
patched up the proofs agsin
2006-12-08, by paulson
removed use of put_name_hint, as the ATP linkup no longer needs this
2006-12-08, by paulson
reorganized structure Tactic vs. MetaSimplifier;
2006-12-07, by wenzelm
begin/end blocks;
2006-12-07, by wenzelm
abbrevs: more careful interpretation, avoid dynamic references to local names;
2006-12-07, by wenzelm
definition/abbreviation: single argument;
2006-12-07, by wenzelm
simplified add_abbrev -- single argument;
2006-12-07, by wenzelm
removed obsolete references to ProofGeneral/isa;
2006-12-07, by wenzelm
added input_mode;
2006-12-07, by wenzelm
tuned print_locale output;
2006-12-07, by wenzelm
moved notation/abbrevs to TermSyntax;
2006-12-07, by wenzelm
expand_term: based on Envir.expand_term;
2006-12-07, by wenzelm
thms etc.: proper treatment of internal_fact with selection;
2006-12-07, by wenzelm
tuned pretty_src output;
2006-12-07, by wenzelm
simplified add_abbrevs: no mixfix;
2006-12-07, by wenzelm
added expand_term;
2006-12-07, by wenzelm
tuned;
2006-12-07, by wenzelm
Common term syntax declarations.
2006-12-07, by wenzelm
added Isar/term_syntax.ML;
2006-12-07, by wenzelm
TermSyntax.notation/abbrevs;
2006-12-07, by wenzelm
Removal of theorem tagging, which the ATP linkup no longer requires.
2006-12-07, by paulson
Removal of theorem tagging, which the ATP linkup no longer requires,
2006-12-07, by paulson
Poly/ML 5.0 setup for Isabelle2005.
2006-12-07, by wenzelm
reorganized structure Goal vs. Tactic;
2006-12-07, by wenzelm
export: added explicit term operation;
2006-12-06, by wenzelm
abbrevs: actually observe target_morphism;
2006-12-06, by wenzelm
added expand;
2006-12-06, by wenzelm
moved hidden_polymorphism to term.ML;
2006-12-06, by wenzelm
added hidden_polymorphism (from variable.ML);
2006-12-06, by wenzelm
add_abbrevs: moved common parts to consts.ML;
2006-12-06, by wenzelm
abbreviate: improved error handling, return result;
2006-12-06, by wenzelm
export: added explicit term operation;
2006-12-06, by wenzelm
LocalDefs.expand;
2006-12-06, by wenzelm
Improved tracing
2006-12-06, by paulson
no timing;
2006-12-06, by wenzelm
simplified ML bindings;
2006-12-06, by wenzelm
simplified ML bindings -- moved to HOL.thy;
2006-12-06, by wenzelm
added basic ML bindings;
2006-12-06, by wenzelm
added aliases for nat_recs/cases;
2006-12-06, by wenzelm
removed legacy ML bindings;
2006-12-06, by wenzelm
reduced to genuine legacy bindings -- others in HOL.thy;
2006-12-06, by wenzelm
removed legacy ML bindings;
2006-12-06, by wenzelm
target_name: allow qualified names;
2006-12-05, by wenzelm
add_notation: permissive about undeclared consts;
2006-12-05, by wenzelm
generic_goal: enable stmt mode;
2006-12-05, by wenzelm
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
2006-12-05, by wenzelm
notation/abbreviation: more serious handling of morphisms;
2006-12-05, by wenzelm
print_syntax etc.: plain Toplevel.context_of;
2006-12-05, by wenzelm
attribute value: morphism;
2006-12-05, by wenzelm
add_notation: permissive about undeclared consts;
2006-12-05, by wenzelm
added mapping_result;
2006-12-05, by wenzelm
added ML-Systems/polyml-5.0.ML;
2006-12-05, by wenzelm
Attrib.internal: morphism;
2006-12-05, by wenzelm
removed duplicate abbreviations (implicit inheritance);
2006-12-05, by wenzelm
restored notation for less/less_eq (observe proper order of mixfix annotations!);
2006-12-05, by wenzelm
Document structure in pgip_markup.ML. Minor fixes.
2006-12-05, by aspinall
Type alias for XML content
2006-12-05, by aspinall
setup for polyml-5.0;
2006-12-05, by wenzelm
set DYLD_LIBRARY_PATH as well;
2006-12-05, by wenzelm
Fix typo. Some cleanup for XML attributes
2006-12-05, by aspinall
Add dependency for new Emacs PG code
2006-12-05, by aspinall
Support PGIP communication for preferences in Emacs mode.
2006-12-05, by aspinall
more careful indexing of local facts;
2006-12-05, by wenzelm
* Pure: official theorem names and additional comments are now strictly separate.
2006-12-05, by wenzelm
thm/prf: separate official name vs. additional tags;
2006-12-05, by wenzelm
thm/prf: separate official name vs. additional tags;
2006-12-05, by wenzelm
notes: added non-official name;
2006-12-05, by wenzelm
note_thmss: added kind tag and non-official name;
2006-12-05, by wenzelm
Add separate PG Emacs configuration
2006-12-04, by aspinall
Include pgip markup module
2006-12-04, by aspinall
Build instructions for new Proof General module [not yet activated]
2006-12-04, by aspinall
Forward compatibility with new Proof General module.
2006-12-04, by aspinall
New files.
2006-12-04, by aspinall
Revamped Proof General interface.
2006-12-04, by aspinall
Add parse_string for attribute values and other string content
2006-12-04, by aspinall
added Ramsey.thy to Library imports, to include it in the daily builds
2006-12-04, by krauss
fixed definition syntax
2006-12-04, by krauss
theory Alloc no longer works -- quick_and_dirty;
2006-12-04, by wenzelm
converted legacy ML script;
2006-12-04, by wenzelm
Minor.
2006-12-03, by aspinall
Add output function
2006-12-03, by aspinall
Add string buffer getter. Add Rawtext constructor to allow XML-escaped strings in tree.
2006-12-03, by aspinall
Type abbreviations for element args and attributes
2006-12-03, by aspinall
meta_term_syntax: proper operation on untyped preterms;
2006-12-02, by wenzelm
generalized type signature of foldSet, fold
2006-12-02, by haftmann
added some support for embedded terms;
2006-12-02, by wenzelm
TLA: converted legacy ML scripts;
2006-12-02, by wenzelm
non-exported syntax
2006-12-01, by haftmann
made SML/NJ happy
2006-12-01, by haftmann
slight cleanup in hologic.ML
2006-12-01, by haftmann
some syntax cleanup
2006-12-01, by haftmann
stripped some legacy bindings
2006-12-01, by haftmann
Added missing "standard"
2006-12-01, by nipkow
Deleted dead code
2006-12-01, by paulson
Fixed a MAJOR BUG in clause-counting: only Boolean equalities now count as iffs
2006-12-01, by paulson
notes: proper naming of thm proof, activated import_export_proof;
2006-11-30, by wenzelm
added full_name;
2006-11-30, by wenzelm
notes: more careful treatment of Goal.close_result;
2006-11-30, by wenzelm
note_thmss: refrain from closing the derivation here;
2006-11-30, by wenzelm
notes: proper import/export of proofs (still inactive);
2006-11-30, by wenzelm
removed obsolete (export_)standard;
2006-11-30, by wenzelm
added mixfix';
2006-11-30, by wenzelm
added merge_list;
2006-11-30, by wenzelm
zero_var_indexes_inst: multiple terms;
2006-11-30, by wenzelm
Theory.merge_list;
2006-11-30, by wenzelm
qualified MetaSimplifier.norm_hhf(_protect);
2006-11-30, by wenzelm
added norm/close_result (supercede local_standard etc.);
2006-11-30, by wenzelm
added zero_var_indexes_list;
2006-11-30, by wenzelm
Goal.norm/close_result;
2006-11-30, by wenzelm
simplified syntax for 'definition', 'abbreviation';
2006-11-30, by wenzelm
*** bad commit -- reverted to previous version ***
2006-11-29, by wenzelm
removed export_standard_morphism;
2006-11-29, by wenzelm
simplified add_thmss;
2006-11-29, by wenzelm
added map/burrow_facts;
2006-11-29, by wenzelm
added INCR_COMP, COMP_INCR;
2006-11-29, by wenzelm
tuned;
2006-11-29, by wenzelm
reworked notes: towards proper import/export of proof terms;
2006-11-29, by wenzelm
removed export_standard_morphism;
2006-11-29, by wenzelm
renamed SIMPLE_METHOD' to SIMPLE_METHOD'';
2006-11-29, by wenzelm
added export;
2006-11-29, by wenzelm
tuned spaces/comments;
2006-11-29, by wenzelm
simplified method setup;
2006-11-29, by wenzelm
simplified method setup;
2006-11-29, by wenzelm
simplified method setup;
2006-11-29, by wenzelm
clauses sorted according to term order (significant speedup in some cases)
2006-11-29, by webertj
Assumption.assms_of: cterm;
2006-11-29, by wenzelm
Element.generalize_facts;
2006-11-29, by wenzelm
removed export_standard_morphism;
2006-11-29, by wenzelm
simplified add_thmss;
2006-11-29, by wenzelm
added facts_map;
2006-11-29, by wenzelm
added map/burrow_facts;
2006-11-29, by wenzelm
COMP_INCR;
2006-11-29, by wenzelm
added INCR_COMP, COMP_INCR;
2006-11-29, by wenzelm
assms_of: cterm;
2006-11-29, by wenzelm
simplified Logic.count_prems;
2006-11-29, by wenzelm
tuned proofs;
2006-11-29, by wenzelm
go back to fixed atbroy51, fix at-poly-e path settings
2006-11-28, by isatest
Removed the references for counting combinators. Instead they are counted in actual clauses.
2006-11-28, by paulson
added strict_subset
2006-11-28, by haftmann
added add_fixed;
2006-11-28, by wenzelm
simplified '?' operator;
2006-11-28, by wenzelm
simplified '?' operator;
2006-11-28, by wenzelm
simplified '?' operator;
2006-11-28, by wenzelm
added burrow_fact;
2006-11-28, by wenzelm
dest_term: strip_imp_concl;
2006-11-28, by wenzelm
simplified '?' operator;
2006-11-28, by wenzelm
Added in another function clause_name_of.
2006-11-27, by mengj
Goals in clause form are sent to the relevance filter.
2006-11-27, by mengj
Call the right inform_file_processed function on <closefile>
2006-11-27, by aspinall
Tidied code. Bool constructor is not needed.
2006-11-27, by paulson
tidied code
2006-11-27, by paulson
outermost universal quantifiers are stripped
2006-11-27, by webertj
typo fixed
2006-11-27, by webertj
added the function for free variables of a lambda-term, which is a
2006-11-27, by urbanc
outermost universal quantifiers are stripped
2006-11-27, by webertj
adapted function definitions to new syntax
2006-11-27, by urbanc
Adapted to new nominal_primrec command.
2006-11-27, by berghofe
additional bookkeeping for class target
2006-11-27, by haftmann
small syntax tuning
2006-11-27, by haftmann
introduced Simpdata structure
2006-11-27, by haftmann
added Trueprop_conv
2006-11-27, by haftmann
restructured some proofs
2006-11-27, by haftmann
tuned keyword setup for SML code generator
2006-11-27, by haftmann
moved order arities for fun and bool to Fun/Orderings
2006-11-27, by haftmann
removed HOL structure
2006-11-27, by haftmann
adjusted syntax for internal code generation
2006-11-27, by haftmann
Added nominal_primrec command.
2006-11-27, by berghofe
Adapted to new nominal_primrec command.
2006-11-27, by berghofe
Added nominal_primrec.ML
2006-11-27, by berghofe
Implemented new "nominal_primrec" command for defining
2006-11-27, by berghofe
Additional information about nominal datatypes (descriptor,
2006-11-27, by berghofe
converted legacy ML scripts;
2006-11-26, by wenzelm
Remove add_master_files which stripped paths for retracted files. Emacs PG already supports full paths here.
2006-11-26, by aspinall
* Pure: syntax constant for foo (binder) is called foo_binder;
2006-11-26, by wenzelm
extend_trtab: allow identical trfuns to be overwritten;
2006-11-26, by wenzelm
tuned;
2006-11-26, by wenzelm
Binder: syntax const is determined by binder_name, not its syntax;
2006-11-26, by wenzelm
simplified consts: no auxiliary params, sane mixfix syntax;
2006-11-26, by wenzelm
abbrevs: no result;
2006-11-26, by wenzelm
added export_(standard_)morphism;
2006-11-26, by wenzelm
Element.map_ctxt_attrib;
2006-11-26, by wenzelm
abbrevs: no result;
2006-11-26, by wenzelm
added map_ctxt_attrib;
2006-11-26, by wenzelm
abbrevs: no result;
2006-11-26, by wenzelm
added morh_result, the_inductive, add_inductive_global;
2006-11-26, by wenzelm
InductivePackage.add_inductive_global;
2006-11-26, by wenzelm
updated (binder) syntax/notation;
2006-11-26, by wenzelm
tuned morphisms;
2006-11-24, by wenzelm
added export_morphism;
2006-11-24, by wenzelm
simultaneous fact morphism;
2006-11-24, by wenzelm
added type_map;
2006-11-24, by wenzelm
added cterm_rule;
2006-11-24, by wenzelm
fake predeclaration of structure ProofContext;
2006-11-24, by wenzelm
added export_morphism;
2006-11-24, by wenzelm
ProofContext.init;
2006-11-24, by wenzelm
Comment: see RFC 2396 for relative URI syntax.
2006-11-24, by aspinall
Send full paths in PGIP version of file loaded/retracted messages
2006-11-24, by aspinall
Conversion of "equal" to "=" for TSTP format; big tidy-up
2006-11-24, by paulson
Lemma "fundef_default_value" uses predicate instead of set.
2006-11-24, by krauss
The function package declares the [code] attribute automatically again.
2006-11-24, by krauss
exported mk_base_funs for use by size-change tools
2006-11-24, by krauss
ATP linkup now generates "new TPTP" rather than "old TPTP"
2006-11-24, by paulson
more careful declaration of "inducts";
2006-11-23, by wenzelm
tuned;
2006-11-23, by wenzelm
prefer Proof.context over Context.generic;
2006-11-23, by wenzelm
prefer Proof.context over Context.generic;
2006-11-23, by wenzelm
tuned proofs;
2006-11-23, by wenzelm
Accept URLs of form file:/home... also.
2006-11-23, by aspinall
prefer antiquotations over LaTeX macros;
2006-11-23, by wenzelm
updated;
2006-11-23, by wenzelm
renamed Args.Name to Args.Text;
2006-11-23, by wenzelm
uniform interface for type_syntax/term_syntax/declaration, dependent on morphism;
2006-11-23, by wenzelm
uniform interface for type_syntax/term_syntax/declaration, dependent on morphism;
2006-11-23, by wenzelm
Morphism.thm_morphism;
2006-11-23, by wenzelm
renamed Name value to Text, which is *not* a name in terms of morphisms;
2006-11-23, by wenzelm
removed obsolete alphanum;
2006-11-23, by wenzelm
str_of_char: improved output of non-printables;
2006-11-23, by wenzelm
added head_name_of;
2006-11-23, by wenzelm
added name/var/typ/term/thm_morphism;
2006-11-23, by wenzelm
declarations: pass morphism (dummy);
2006-11-23, by wenzelm
added ISABELLE_IDENTIFIER;
2006-11-23, by wenzelm
ISABELLE_PATH/OUTPUT: append ISABELLE_IDENTIFIER if derived from ISABELLE_HOME_USER;
2006-11-23, by wenzelm
fixed some typos
2006-11-23, by urbanc
tuned the proof of the strong induction principle
2006-11-23, by urbanc
typo in comment fixed
2006-11-23, by webertj
Add retractfile to supported pgip commands
2006-11-23, by aspinall
PGIP: add retractfile. Be stricter in file open/close protocol.
2006-11-23, by aspinall
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
2006-11-23, by wenzelm
moved ML identifiers to structure ML_Syntax;
2006-11-23, by wenzelm
added morph_ctxt, morph_witness;
2006-11-23, by wenzelm
replaced map_values by morph_values;
2006-11-23, by wenzelm
moved string_of_pair/list/option to structure ML_Syntax;
2006-11-23, by wenzelm
moved ML syntax operations to structure ML_Syntax;
2006-11-23, by wenzelm
Basic ML syntax operations.
2006-11-23, by wenzelm
Abstract morphisms on formal entities.
2006-11-23, by wenzelm
added morphism.ML, General/ml_syntax.ML;
2006-11-23, by wenzelm
renamed string_of_pair/list/option to ML_Syntax.str_of_pair/list/option;
2006-11-23, by wenzelm
removed dead code;
2006-11-23, by wenzelm
Add doccomment; rename litcomment -> doccomment
2006-11-23, by aspinall
* settings: ML_IDENTIFIER includes the Isabelle version identifier;
2006-11-22, by wenzelm
Consolidation of code to "blacklist" unhelpful theorems, including record
2006-11-22, by paulson
ML_IDENTIFIER includes Isabelle version;
2006-11-22, by wenzelm
add ISABELLE_VERSION to ML_IDENTIFIER, unless this is repository or build;
2006-11-22, by wenzelm
consts: ProofContext.set_stmt true -- avoids naming of local thms;
2006-11-22, by wenzelm
init: enter inner statement mode, which prevents local notes from being named internally;
2006-11-22, by wenzelm
more careful declaration of "intros" as Pure.intro;
2006-11-22, by wenzelm
Fix to local file URI syntax. Add first part of lexicalstructure command support.
2006-11-22, by aspinall
completed class parameter handling in axclass.ML
2006-11-22, by haftmann
added Isar syntax for adding parameters to axclasses
2006-11-22, by haftmann
forced name prefix for class operations
2006-11-22, by haftmann
example tuned
2006-11-22, by haftmann
no explicit check for theory Nat
2006-11-22, by haftmann
added code lemmas
2006-11-22, by haftmann
does not import Hilber_Choice any longer
2006-11-22, by haftmann
cleanup
2006-11-22, by haftmann
incorporated structure HOList into HOLogic
2006-11-22, by haftmann
dropped eq const
2006-11-22, by haftmann
removed Extraction dependency
2006-11-22, by haftmann
final draft
2006-11-22, by haftmann
made SML/NJ happy;
2006-11-21, by wenzelm
theorem(_i): note assms of statement;
2006-11-21, by wenzelm
removed obsolete simple_note_thms;
2006-11-21, by wenzelm
added assmsN;
2006-11-21, by wenzelm
* Isar: the assumptions of a long theorem statement are available as assms;
2006-11-21, by wenzelm
activated x86_64-linux;
2006-11-21, by wenzelm
renamed Proof.put_thms_internal to Proof.put_thms;
2006-11-21, by wenzelm
simplified Proof.theorem(_i);
2006-11-21, by wenzelm
added stmt mode, which affects naming/indexing of local facts;
2006-11-21, by wenzelm
simplified theorem(_i);
2006-11-21, by wenzelm
notes: proper kind;
2006-11-21, by wenzelm
notes: proper kind;
2006-11-21, by wenzelm
removed kind attribs;
2006-11-21, by wenzelm
moved theorem kinds from PureThy to Thm;
2006-11-21, by wenzelm
moved theorem kinds from PureThy to Thm;
2006-11-21, by wenzelm
LocalTheory.notes/defs: proper kind;
2006-11-21, by wenzelm
LocalTheory.axioms/notes/defs: proper kind;
2006-11-21, by wenzelm
simplified Proof.theorem(_i);
2006-11-21, by wenzelm
LocalTheory.axioms/notes/defs: proper kind;
2006-11-21, by wenzelm
Optimized class_pairs for the common case of no subclasses
2006-11-21, by paulson
Outputs a minimal number of arity clauses. Tidying of blacklist, fixing the blacklisting of thm lists
2006-11-21, by paulson
New transformation of eliminatino rules: we simply replace the final conclusion variable by False
2006-11-21, by paulson
run poly-4.9.1 as stable and poly-4.2.0 as experimental on at
2006-11-21, by kleing
removed legacy ML setup;
2006-11-21, by wenzelm
converted legacy ML scripts;
2006-11-21, by wenzelm
converted legacy ML scripts;
2006-11-20, by wenzelm
HOL-Prolog: converted legacy ML scripts;
2006-11-20, by wenzelm
start at-sml earlier and on different machine, remove sun-sml test (takes too long)
2006-11-20, by kleing
HOL-Algebra: converted legacy ML scripts;
2006-11-19, by wenzelm
profiling disabled
2006-11-19, by webertj
code thms for classops violating type discipline ignored
2006-11-18, by haftmann
cleanup
2006-11-18, by haftmann
added instance for class size
2006-11-18, by haftmann
added combinators and lemmas
2006-11-18, by haftmann
using class instance
2006-11-18, by haftmann
dvd_def now with object equality
2006-11-18, by haftmann
op div/op mod now named without leading op
2006-11-18, by haftmann
workaround for definition violating type discipline
2006-11-18, by haftmann
moved dvd stuff to theory Divides
2006-11-18, by haftmann
re-eliminated thm trichotomy
2006-11-18, by haftmann
power is now a class
2006-11-18, by haftmann
tuned
2006-11-18, by haftmann
clarified module dependencies
2006-11-18, by haftmann
div is now a class
2006-11-18, by haftmann
reduced verbosity
2006-11-18, by haftmann
adjustments for class package
2006-11-18, by haftmann
added an intro lemma for freshness of products; set up
2006-11-17, by urbanc
more robust syntax for definition/abbreviation/notation;
2006-11-17, by wenzelm
'notation': more robust 'and' list;
2006-11-17, by wenzelm
updated;
2006-11-17, by wenzelm
added Isar.goal;
2006-11-17, by wenzelm
added where_;
2006-11-17, by wenzelm
add lemmas LIM_zero_iff, LIM_norm_zero_iff
2006-11-16, by huffman
Includes type:sort constraints in its code to collect predicates in axiom clauses.
2006-11-16, by paulson
Now includes only types used to instantiate overloaded constants in arity clauses
2006-11-16, by paulson
added General/basics.ML;
2006-11-16, by wenzelm
moved some fundamental concepts to General/basics.ML;
2006-11-16, by wenzelm
Fundamental concepts.
2006-11-16, by wenzelm
add_locale: re-init result context (avoids subtle modifications after introducing predicate views internally);
2006-11-15, by wenzelm
tuned proofs;
2006-11-15, by wenzelm
replaced NameSpace.append by NameSpace.qualified, which handles empty names as expected;
2006-11-15, by wenzelm
replaced NameSpace.append by NameSpace.qualified, which handles empty names as expected;
2006-11-15, by wenzelm
dropping accidental self-imports
2006-11-15, by haftmann
corrected polymorphism check
2006-11-15, by haftmann
clarified code for building function equation system; explicit check of type discipline
2006-11-15, by haftmann
moved evaluation to Code_Generator.thy
2006-11-15, by haftmann
added filter_set; adaptions to more strict type discipline for code lemmas
2006-11-15, by haftmann
moved transitivity rules to Orderings.thy
2006-11-15, by haftmann
added transitivity rules, reworking of min/max lemmas
2006-11-15, by haftmann
dropped dependency on sets
2006-11-15, by haftmann
reworking of min/max lemmas
2006-11-15, by haftmann
added interpretation
2006-11-15, by haftmann
removed HOL_css
2006-11-15, by haftmann
added evaluation oracle
2006-11-15, by haftmann
replaced exists_fresh lemma with a version formulated with obtains;
2006-11-15, by urbanc
updated;
2006-11-15, by wenzelm
Auxiliary antiquotations for Isabelle manuals.
2006-11-15, by wenzelm
common antiquote_setup.ML;
2006-11-15, by wenzelm
Arity clauses are now produced only for types and type classes actually used.
2006-11-15, by paulson
converted to 'inductive2';
2006-11-14, by wenzelm
added for_simple_fixes, specification;
2006-11-14, by wenzelm
replaced Variable.fix_frees by Variable.auto_fixes (depends on body mode);
2006-11-14, by wenzelm
removed fix_frees interface;
2006-11-14, by wenzelm
converted to 'inductive2';
2006-11-14, by wenzelm
inductive: canonical specification syntax (flattened result only);
2006-11-14, by wenzelm
inductive2: canonical specification syntax;
2006-11-14, by wenzelm
InductivePackage.add_inductive_i: canonical argument order;
2006-11-14, by wenzelm
inductive2: canonical specification syntax;
2006-11-14, by wenzelm
Exported some names
2006-11-14, by schirmer
simplified Proof.theorem(_i) interface -- removed target support;
2006-11-14, by wenzelm
simplified Proof.theorem(_i) interface;
2006-11-14, by wenzelm
antiquotation theory: plain Theory.requires, no peeking at ThyInfo;
2006-11-14, by wenzelm
simplified Proof.theorem(_i) interface;
2006-11-14, by wenzelm
tuned antiquotation theory;
2006-11-14, by wenzelm
value restriction
2006-11-14, by haftmann
removed old cygwin wrappers;
2006-11-14, by wenzelm
declare_constraints: reset constraint on dummyS;
2006-11-14, by wenzelm
removed Isar/isar_thy.ML;
2006-11-14, by wenzelm
added dummyS;
2006-11-14, by wenzelm
removed legacy read/cert/string_of;
2006-11-14, by wenzelm
recdef_tc(_i): local_theory interface via Specification.theorem_i;
2006-11-14, by wenzelm
incorporated IsarThy into IsarCmd;
2006-11-14, by wenzelm
removed theorem(_i);
2006-11-14, by wenzelm
upd
2006-11-13, by haftmann
atbroy51 broke down, switch to atbroy9
2006-11-13, by kleing
updated
2006-11-13, by krauss
antiquotation "theory": proper output, only check via ThyInfo.theory;
2006-11-13, by wenzelm
tuned;
2006-11-13, by wenzelm
added antiquotation @{theory name};
2006-11-13, by wenzelm
fixed comment -- oops;
2006-11-13, by wenzelm
adjusted to new fun''
2006-11-13, by haftmann
*** empty log message ***
2006-11-13, by haftmann
added antiquotation theory
2006-11-13, by haftmann
cleaned up
2006-11-13, by haftmann
added theory antiquotation
2006-11-13, by haftmann
combinator for overwriting changes with warning
2006-11-13, by haftmann
added higher-order combinators for structured results
2006-11-13, by haftmann
adjusted name in generated code
2006-11-13, by haftmann
dropped LOrder dependency
2006-11-13, by haftmann
moved upwars in HOL theory graph
2006-11-13, by haftmann
added thy dependencies
2006-11-13, by haftmann
PreList = Main - List
2006-11-13, by haftmann
introduces preorders
2006-11-13, by haftmann
dropped Inductive dependency
2006-11-13, by haftmann
dropped Typedef dependency
2006-11-13, by haftmann
added LOrder dependency
2006-11-13, by haftmann
tuned ml antiquotations
2006-11-13, by haftmann
adjusted
2006-11-13, by haftmann
tuned
2006-11-13, by haftmann
added tt tag
2006-11-13, by haftmann
auto_term => lexicographic_order
2006-11-13, by krauss
updated
2006-11-13, by krauss
replaced "auto_term" by the simpler method "relation", which does not try
2006-11-13, by krauss
added fresh_prodD, which is included fresh_prodD into mksimps setup;
2006-11-13, by wenzelm
added lexicographic_order.ML to makefile
2006-11-13, by krauss
image_constant_conv no longer [simp]
2006-11-12, by nipkow
instantiate: tuned indentity case;
2006-11-12, by wenzelm
removed dead code;
2006-11-12, by wenzelm
mk_atomize: careful matching against rules admits overloading;
2006-11-12, by wenzelm
started reorgnization of lattice theories
2006-11-12, by nipkow
Added in is_fol_thms.
2006-11-11, by mengj
level: do not account for local theory blocks (relevant for document preparation);
2006-11-11, by wenzelm
local 'end': no default tags;
2006-11-11, by wenzelm
* Local theory targets ``context/locale/class ... begin'' followed by ``end''.
2006-11-11, by wenzelm
removed obsolete context;
2006-11-11, by wenzelm
turned 'context' into plain thy_decl, discontinued thy_switch;
2006-11-11, by wenzelm
tuned proofs;
2006-11-11, by wenzelm
updated local theory targets;
2006-11-11, by wenzelm
updated local theory targets;
2006-11-11, by wenzelm
updated;
2006-11-11, by wenzelm
Update standard keyword files.
2006-11-11, by wenzelm
tuned comments;
2006-11-10, by wenzelm
tuned comments;
2006-11-10, by wenzelm
tuned names of start_timing,/end_timing/check_timer;
2006-11-10, by wenzelm
removed obsolete ML compatibility fragments;
2006-11-10, by wenzelm
avoid strange typing problem in MosML;
2006-11-10, by wenzelm
tuned names of start_timing,/end_timing/check_timer;
2006-11-10, by wenzelm
simplified local theory wrappers;
2006-11-10, by wenzelm
removed mapping;
2006-11-10, by wenzelm
simplified exit;
2006-11-10, by wenzelm
simplified LocalTheory.exit;
2006-11-10, by wenzelm
Improvement to classrel clauses: now outputs the minimum needed.
2006-11-10, by paulson
deleted all uses of sign_of as it's now the identity function
2006-11-10, by urbanc
tuned;
2006-11-10, by wenzelm
tuned Variable.trade;
2006-11-10, by wenzelm
introduces canonical AList functions for loop_tacs
2006-11-10, by haftmann
minor refinements
2006-11-10, by haftmann
redundancy checkes includes eta-expansion
2006-11-10, by haftmann
improved syntax
2006-11-10, by haftmann
added bounded_linear and bounded_bilinear locales
2006-11-10, by huffman
no special treatment for cygwin (this is supposed to be actual cygwin, not win32 polyml within cygwin);
2006-11-10, by wenzelm
tuned comments;
2006-11-10, by wenzelm
added x86-cygwin;
2006-11-09, by wenzelm
oracle raises CooperDec.COOPER instead of COOPER (this is eliminated). Erronous old behaviour due to this exception is now correcrted.
2006-11-09, by chaieb
LocalTheory.restore;
2006-11-09, by wenzelm
init: '-' refers to global context;
2006-11-09, by wenzelm
abbrevs: return result;
2006-11-09, by wenzelm
Stack.map_top;
2006-11-09, by wenzelm
abbrevs: return result;
2006-11-09, by wenzelm
separate map_top/all;
2006-11-09, by wenzelm
abbrevs: return result (use LocalTheory.abbrevs directly);
2006-11-09, by wenzelm
tuned;
2006-11-09, by wenzelm
abbrevs: return result;
2006-11-09, by wenzelm
timing/tracing code removed
2006-11-09, by webertj
interpreters for fst and snd added
2006-11-09, by webertj
new CCS-based implementation that should work with PolyML 5.0
2006-11-09, by webertj
HOL: less/less_eq on bool, modified syntax;
2006-11-09, by wenzelm
removed obsolete locale_results;
2006-11-09, by wenzelm
tuned;
2006-11-09, by wenzelm
imports Binimial;
2006-11-09, by wenzelm
updated;
2006-11-09, by wenzelm
lfp_induct_set;
2006-11-09, by wenzelm
modified less/less_eq syntax to avoid "x < y < z" etc.;
2006-11-09, by wenzelm
added lemma mult_mono'
2006-11-09, by huffman
added LIM_norm and related lemmas
2006-11-09, by huffman
moved theories Parity, GCD, Binomial to Library;
2006-11-08, by wenzelm
added profiling code, improved handling of proof terms, generation of domain
2006-11-08, by krauss
incorporated former theories Reconstruction and ResAtpMethods into ATP_Linkup;
2006-11-08, by wenzelm
case_tr': proper handling of authentic consts;
2006-11-08, by wenzelm
removed obsolete nat_case_tr' (duplicates case_tr' in datatype_package.ML);
2006-11-08, by wenzelm
renamed DatatypeHooks.invoke to all
2006-11-08, by haftmann
moved lemma eq_neq_eq_imp_neq to HOL
2006-11-08, by haftmann
renamed Lattice_Locales to Lattices
2006-11-08, by haftmann
abstract ordering theories
2006-11-08, by haftmann
obsolete (cf. ROOT.ML);
2006-11-08, by wenzelm
added structure Main (from Main.ML);
2006-11-08, by wenzelm
proper definition of add_zero_left/right;
2006-11-08, by wenzelm
removed NatArith.thy, Main.ML;
2006-11-08, by wenzelm
removed theory NatArith (now part of Nat);
2006-11-08, by wenzelm
* November 2006: Lukas Bulwahn, TUM -- HOL/function: method "lexicographic_order".
2006-11-08, by wenzelm
moved contribution note to CONTRIBUTORS;
2006-11-08, by wenzelm
Made "termination by lexicographic_order" the default for "fun" definitions.
2006-11-08, by krauss
LIM_compose -> isCont_LIM_compose;
2006-11-08, by huffman
generalized types of of_nat and of_int to work with non-commutative types
2006-11-08, by huffman
untabified
2006-11-07, by krauss
complex goal statements: misc cleanup;
2006-11-07, by wenzelm
Added datatype hook to declare all case_congs as "fundef_cong" automatically.
2006-11-07, by krauss
removed obsolete theorem statements (cf. specification.ML);
2006-11-07, by wenzelm
tuned specifications;
2006-11-07, by wenzelm
fixed locale fact references;
2006-11-07, by wenzelm
removed obsolete print_state_hook;
2006-11-07, by wenzelm
theorem statements: incorporate Obtain.statement, tuned;
2006-11-07, by wenzelm
moved statement to specification.ML;
2006-11-07, by wenzelm
removed obsolete Locale.smart_theorem;
2006-11-07, by wenzelm
avoid handling of arbitrary exceptions;
2006-11-07, by wenzelm
field-update in records is generalised to take a function on the field
2006-11-07, by schirmer
exported intro_locales_tac
2006-11-07, by schirmer
Proper theorem names at last, no fakes!!
2006-11-07, by paulson
some corrections
2006-11-07, by haftmann
adjusted title
2006-11-07, by haftmann
simplified dest_eq;
2006-11-07, by wenzelm
commented out parts which have been inactive (unintentionally) for a long time;
2006-11-07, by wenzelm
removed obsolete dest_eq_typ;
2006-11-07, by wenzelm
tuned hypsubst setup;
2006-11-07, by wenzelm
continued
2006-11-07, by haftmann
made locale partial_order compatible with axclass order; changed import order; consecutive changes
2006-11-07, by haftmann
made locale partial_order compatible with axclass order
2006-11-07, by haftmann
adjusted two lemma names due to name change in interpretation
2006-11-07, by haftmann
changed import order
2006-11-07, by haftmann
Added a (stub of a) function tutorial
2006-11-07, by krauss
Preparations for making "lexicographic_order" part of "fun"
2006-11-07, by krauss
renamed 'const_syntax' to 'notation';
2006-11-07, by wenzelm
'const_syntax' command: allow fixed variables, renamed to 'notation';
2006-11-07, by wenzelm
replaced const_syntax by notation, which operates on terms;
2006-11-07, by wenzelm
Isar.context: proper error;
2006-11-07, by wenzelm
replaced const_syntax by notation, which operates on terms;
2006-11-07, by wenzelm
read_const: include type;
2006-11-07, by wenzelm
renamed 'const_syntax' to 'notation';
2006-11-07, by wenzelm
updated;
2006-11-07, by wenzelm
Adapted to changes in FixedPoint theory.
2006-11-07, by berghofe
method exported
2006-11-07, by krauss
updated NEWS
2006-11-07, by krauss
* Added annihilation axioms ("x * 0 = 0") to axclass semiring_0.
2006-11-07, by krauss
added gfx
2006-11-07, by haftmann
dropped blastdata.ML
2006-11-06, by haftmann
(adjustions)
2006-11-06, by haftmann
two further lemmas on split
2006-11-06, by haftmann
removed dependency of ord on eq
2006-11-06, by haftmann
removed itrev as inlining theorem
2006-11-06, by haftmann
added state monad to HOL library
2006-11-06, by haftmann
code generator module naming improved
2006-11-06, by haftmann
(continued)
2006-11-06, by haftmann
(continued)
2006-11-06, by haftmann
minor cleanup
2006-11-06, by krauss
case_tr: do not intern already internal consts;
2006-11-05, by wenzelm
updated;
2006-11-05, by wenzelm
removed isactrlconst;
2006-11-05, by wenzelm
instantiate: avoid global references;
2006-11-05, by wenzelm
added const_syntax_name;
2006-11-05, by wenzelm
removed obsolete first_duplicate;
2006-11-05, by wenzelm
added syntax_name;
2006-11-05, by wenzelm
fixed print_translation for ALL/EX and <, <=, etc.; tuned syntax names;
2006-11-05, by wenzelm
Sign.const_syntax_name;
2006-11-05, by wenzelm
added gfx
2006-11-05, by haftmann
removed checkpoint interface;
2006-11-04, by wenzelm
String.compare: slow version -- performance test;
2006-11-04, by wenzelm
replaced apply_copy by apply';
2006-11-04, by wenzelm
removed is_Trueprop (use can dest_Trueprop'' instead);
2006-11-04, by wenzelm
removed is_Trueprop (use can dest_Trueprop'' instead);
2006-11-04, by wenzelm
updated;
2006-11-04, by wenzelm
HOL_USEDIR_OPTIONS: -p 1 by default;
2006-11-04, by wenzelm
tuned;
2006-11-04, by wenzelm
* October 2006: Stefan Hohe, TUM;
2006-11-04, by wenzelm
replaced Toplevel.proof_to_theory by Toplevel.end_proof;
2006-11-04, by wenzelm
optional argument for timespan (default 100);
2006-11-04, by wenzelm
added at-mac-poly-e, at64-poly-e;
2006-11-04, by wenzelm
moved DERIV stuff from Lim.thy to new Deriv.thy; cleaned up LIMSEQ_SEQ proofs
2006-11-04, by huffman
new Deriv.thy contains stuff from Lim.thy
2006-11-04, by huffman
re-added simpdata.ML
2006-11-03, by haftmann
new ML serializer
2006-11-03, by haftmann
fixed problem with eta-expansion
2006-11-03, by haftmann
tuned
2006-11-03, by haftmann
fixed problem with variable names
2006-11-03, by haftmann
tightened notion of function equations
2006-11-03, by haftmann
dropped name_mangler.ML
2006-11-03, by haftmann
some example tweaking
2006-11-03, by haftmann
added particular test for partially applied case constants
2006-11-03, by haftmann
improved evaluation setup
2006-11-03, by haftmann
adapted to changes in codegen_data.ML
2006-11-03, by haftmann
added code gen II
2006-11-03, by haftmann
simplified reasoning tools setup
2006-11-03, by haftmann
dropped prop_cs
2006-11-03, by haftmann
dropped equals_conv for nbe
2006-11-03, by haftmann
first version of style guide
2006-11-03, by haftmann
continued tutorial
2006-11-03, by haftmann
added serialization keywords
2006-11-03, by haftmann
bugfix to zipto: left and right were wrong way around.
2006-11-02, by dixon
added sum_squared
2006-11-02, by nipkow
changed a misplaced "also" to a "moreover" (caused a loop somehow)
2006-11-01, by urbanc
changed to not compile Iteration and Recursion, but Lam_Funs instead
2006-11-01, by urbanc
move DERIV_sumr from Series.thy to Lim.thy
2006-11-01, by huffman
generalize type of lemma isCont_Id
2006-11-01, by huffman
new proof of Bseq_NSbseq using transfer
2006-11-01, by huffman
changed to use Lam_Funs
2006-11-01, by urbanc
clauses for iff-introduction, unfortunately useless
2006-11-01, by paulson
tuned
2006-11-01, by urbanc
Numerous cosmetic changes.
2006-11-01, by paulson
not needed anymore
2006-11-01, by urbanc
these files are superseded by the internal recursion combinator and the file Lam_Funs.thy
2006-11-01, by urbanc
More blacklisting
2006-11-01, by paulson
added lexicographic_order tactic
2006-11-01, by bulwahn
new SML serializer
2006-10-31, by haftmann
clarified make_term interface
2006-10-31, by haftmann
introduced CodegenData.add_func_legacy
2006-10-31, by haftmann
cleaned up
2006-10-31, by haftmann
adapted seralizer syntax
2006-10-31, by haftmann
adapted to new serializer syntax
2006-10-31, by haftmann
constructing proof
2006-10-31, by haftmann
dropped constructiv `->
2006-10-31, by haftmann
new serialization syntax; experimental extensions
2006-10-31, by haftmann
refined
2006-10-31, by haftmann
refined algorithm
2006-10-31, by haftmann
simplified preprocessor framework
2006-10-31, by haftmann
cleanup
2006-10-31, by haftmann
*** empty log message ***
2006-10-31, by haftmann
fixed type signature of Type.varify
2006-10-31, by haftmann
dropped junk
2006-10-31, by haftmann
disabled some code generation (an intermeidate solution)
2006-10-31, by haftmann
adapted to new serializer syntax
2006-10-31, by haftmann
added Equals_conv
2006-10-31, by haftmann
cleaned up
2006-10-31, by haftmann
adaptions to changes in preprocessor
2006-10-31, by haftmann
dropped nth_update
2006-10-31, by haftmann
Purely cosmetic
2006-10-30, by paulson
new file for defining functions in the lambda-calculus
2006-10-30, by urbanc
Added "recdef_wf" and "simp" attribute to "wf_measures"
2006-10-26, by krauss
Removed debugging output
2006-10-26, by krauss
removed free "x" from termination goal...
2006-10-26, by krauss
Added "measures" combinator for lexicographic combinations of multiple measures.
2006-10-26, by krauss
Conversion to clause form now tolerates Boolean variables without looping.
2006-10-26, by paulson
adapted to Stefan's new inductive package
2006-10-24, by urbanc
Fixed bug in the handling of congruence rules
2006-10-23, by krauss
(added entry)
2006-10-23, by haftmann
switched merge_alists'' to AList.merge'' whenever appropriate
2006-10-23, by haftmann
new single-step proofs
2006-10-23, by paulson
meson method MUST NOT use all safe rules, only basic ones for the logical connectives.
2006-10-23, by paulson
Improved tracing
2006-10-23, by paulson
fixed two bugs
2006-10-23, by haftmann
bugfixes
2006-10-23, by haftmann
added example with split
2006-10-23, by haftmann
cleanup in ML setup code
2006-10-23, by haftmann
added option of Haskell serializer
2006-10-23, by haftmann
continued
2006-10-23, by haftmann
Added freshness context to FCBs.
2006-10-23, by berghofe
Adapted to changes in FCBs.
2006-10-23, by berghofe
Added Compile and Height examples.
2006-10-23, by berghofe
Added Compile and Height examples to Nominal directory.
2006-10-23, by berghofe
removed antisym_setup.ML
2006-10-20, by haftmann
cleaned up
2006-10-20, by haftmann
final Haskell serializer
2006-10-20, by haftmann
dropped classop shallow namespace
2006-10-20, by haftmann
added Haskell
2006-10-20, by haftmann
added reserved words for Haskell
2006-10-20, by haftmann
slight cleanup
2006-10-20, by haftmann
extended section on code generator
2006-10-20, by haftmann
small refinements
2006-10-20, by haftmann
continued
2006-10-20, by haftmann
added entries for tutorials
2006-10-20, by haftmann
Proof of "bs # fK bs us vs" no longer depends on FCBs.
2006-10-20, by berghofe
example of a single-step proof reconstruction
2006-10-20, by paulson
Fixed the "exception Empty" bug in elim2Fol
2006-10-20, by paulson
Added more debugging info
2006-10-20, by paulson
nclauses no longer requires its input to be in NNF
2006-10-20, by paulson
cleanup
2006-10-20, by haftmann
explicit change of code width possible
2006-10-20, by haftmann
code nofunc now permits theorems violating typing discipline
2006-10-20, by haftmann
abandoned foldl
2006-10-20, by haftmann
fold cleanup
2006-10-20, by haftmann
slight cleanup
2006-10-20, by haftmann
slight adaption
2006-10-20, by haftmann
added normal post setup; cleaned up "execution" constants
2006-10-20, by haftmann
added normal post setup
2006-10-20, by haftmann
added if_delayed
2006-10-20, by haftmann
started tutorial
2006-10-20, by haftmann
code_constsubst -> code_axioms
2006-10-20, by haftmann
Symtab.foldl replaced by Symtab.fold
2006-10-20, by haftmann
Induction rule for graph of recursion combinator
2006-10-19, by berghofe
Split up FCBs into separate formulae for each binder.
2006-10-19, by berghofe
cleaning up
2006-10-18, by urbanc
adapted to Stefan's new inductive package and cleaning up
2006-10-18, by urbanc
Switched function package to use the new package for inductive predicates.
2006-10-18, by krauss
More robust error handling in make_nnf and forward_res
2006-10-18, by paulson
Stylistic improvements.
2006-10-18, by ballarin
Restructured and repaired code dealing with case names
2006-10-17, by berghofe
macbroy6 still has non-standard setup
2006-10-17, by kleing
moved HOL code generator setup to Code_Generator
2006-10-16, by haftmann
slight cleanup
2006-10-16, by haftmann
fixed print translations for bounded quantification
2006-10-16, by haftmann
added explicit print translation for nat_case
2006-10-16, by haftmann
added isactrlconst
2006-10-16, by haftmann
Order and lattice structures no longer based on records.
2006-10-16, by ballarin
add experimental macbroy6 (intel-darwin)
2006-10-15, by isatest
add experimental at64 poly-4.9.1 test on atbroy101
2006-10-15, by isatest
generate devel snapshot even if experimental builds fail.
2006-10-15, by kleing
added peek;
2006-10-14, by wenzelm
added theorem(_i);
2006-10-14, by wenzelm
export map_elem;
2006-10-14, by wenzelm
added assert;
2006-10-14, by wenzelm
theorem: added local_theory version;
2006-10-14, by wenzelm
Attrib.pretty_attrib;
2006-10-14, by wenzelm
added pretty_attribs (from attrib.ML);
2006-10-14, by wenzelm
moved pretty_attribs to attrib.ML;
2006-10-14, by wenzelm
locale begin/end;
2006-10-14, by wenzelm
updated;
2006-10-13, by wenzelm
Added keywords for new inductive definition package.
2006-10-13, by berghofe
Adapted to changes in FixedPoint theory.
2006-10-13, by berghofe
Moved old inductive package to old_inductive_package.ML
2006-10-13, by berghofe
Completely rewrote inductive definition package. Now allows to
2006-10-13, by berghofe
Old version of inductive definition package (for sets).
2006-10-13, by berghofe
Moved old inductive package to old_inductive_package.ML
2006-10-13, by berghofe
Adapted to new inductive definition package.
2006-10-13, by berghofe
Adapted to changes in FixedPoint theory.
2006-10-13, by berghofe
Legacy ML bindings now refer to old inductive definition package.
2006-10-13, by berghofe
Added new package for inductive definitions, moved old package
2006-10-13, by berghofe
Generalized gfp and lfp to arbitrary complete lattices.
2006-10-13, by berghofe
Repaired strip_assums_hyp (now also works for goals not
2006-10-13, by berghofe
improved framework
2006-10-13, by haftmann
refined
2006-10-13, by haftmann
fixed bug
2006-10-13, by haftmann
tuned
2006-10-13, by haftmann
added codegen2 example
2006-10-13, by haftmann
added the missing freshness-lemmas for nat, int, char and string and
2006-10-13, by urbanc
lifted claset setup from ML to Isar level
2006-10-13, by haftmann
explicit nonfix for union and inter
2006-10-13, by haftmann
renamed enter_forward_proof to enter_proof_body;
2006-10-12, by wenzelm
added peek;
2006-10-12, by wenzelm
interpretation_in_locale: standalone goal setup;
2006-10-12, by wenzelm
tuned;
2006-10-12, by wenzelm
renamed print_lthms to print_facts, do not insist on proof state;
2006-10-12, by wenzelm
print_evaluated_term: Toplevel.context_of;
2006-10-12, by wenzelm
replaced attributes_update by map_attributes;
2006-10-12, by wenzelm
Toplevel.local_theory_to_proof: proper target;
2006-10-12, by wenzelm
Toplevel.local_theory: proper target;
2006-10-12, by wenzelm
To be consistent with "induct", I renamed "fixing" to "arbitrary".
2006-10-12, by urbanc
Extended combinators now disabled
2006-10-12, by paulson
abstraction is now turned OFF...
2006-10-12, by paulson
Logging of theorem names to the /tmp directory now works
2006-10-12, by paulson
cc: avoid space after options;
2006-10-12, by wenzelm
set DYLD_LIBRARY_PATH (for Darwin);
2006-10-12, by wenzelm
added execute/system;
2006-10-12, by wenzelm
added x86-darwin;
2006-10-12, by wenzelm
now allowing subdirectories in Doc/
2006-10-12, by haftmann
added makefile layer
2006-10-12, by haftmann
* isabelle-process: option -S (secure mode) disables some critical operations;
2006-10-11, by wenzelm
increased heap size for polyml-4.9.1;
2006-10-11, by wenzelm
tuned Toplevel.begin_local_theory;
2006-10-11, by wenzelm
exit_local_theory: pass interactive flag;
2006-10-11, by wenzelm
exit: pass interactive flag;
2006-10-11, by wenzelm
added begin parser;
2006-10-11, by wenzelm
is_sid: disallow 'begin' keyword as identifier;
2006-10-11, by wenzelm
exit: pass interactive flag, toplevel result convention;
2006-10-11, by wenzelm
add_defs: declare terms;
2006-10-11, by wenzelm
'context': demand 'begin', support local theory;
2006-10-11, by wenzelm
removed 'undo_end', recovered 'cannot_undo';
2006-10-11, by wenzelm
tuned signature;
2006-10-11, by wenzelm
minor refinements in serialization
2006-10-11, by haftmann
adapted to signature change
2006-10-11, by haftmann
slight type signature changes
2006-10-11, by haftmann
cleaned up HOL bootstrap
2006-10-11, by haftmann
abandoned findrep
2006-10-11, by haftmann
added code generator setup
2006-10-11, by haftmann
added code lemma
2006-10-11, by haftmann
Abstraction re-use code now checks that the abstraction function can be used in the current
2006-10-11, by paulson
added examples for nested let
2006-10-11, by haftmann
added tex files to CVS
2006-10-11, by haftmann
renamed body_context_node to presentation_context;
2006-10-11, by wenzelm
add_locale(_i): return actual result context;
2006-10-11, by wenzelm
class(_i): mimic Locale.add_locale(_i);
2006-10-11, by wenzelm
added type global_theory -- theory or local_theory;
2006-10-11, by wenzelm
added begin;
2006-10-11, by wenzelm
added opt_begin;
2006-10-11, by wenzelm
added raw_theory(_result);
2006-10-11, by wenzelm
Toplevel.end_proof;
2006-10-11, by wenzelm
'end': handle local theory;
2006-10-11, by wenzelm
undo_end/kill: handle local theory;
2006-10-11, by wenzelm
Toplevel: generic_theory;
2006-10-11, by wenzelm
made some proof look more like the ones in Barendregt
2006-10-10, by urbanc
A way to call the ATP linkup from ML scripts
2006-10-10, by paulson
Combinators require the theory name; added settings for SPASS
2006-10-10, by paulson
stripped pointless head
2006-10-10, by haftmann
gen_rem(s) abandoned in favour of remove / subtract
2006-10-10, by haftmann
added IsarAdvanced material
2006-10-10, by haftmann
Induction rules have schematic variables again.
2006-10-10, by krauss
initial draft
2006-10-10, by haftmann
*** empty log message ***
2006-10-10, by haftmann
initial draft
2006-10-10, by haftmann
fixed intendation
2006-10-10, by haftmann
cleanup basic HOL bootstrap
2006-10-10, by haftmann
added legacy tactic
2006-10-10, by haftmann
purged some ML legacy
2006-10-10, by haftmann
added eq_True eq_False True_implies_equals to extraction_expand
2006-10-10, by haftmann
no breaks for Haskell
2006-10-10, by haftmann
removed experimental codegen_simtype
2006-10-10, by haftmann
added keeping of funcgr
2006-10-10, by haftmann
generalized purge
2006-10-10, by haftmann
changed order
2006-10-10, by haftmann
removed quote in serialization
2006-10-10, by haftmann
added code_abstype
2006-10-10, by haftmann
added code_constsubst
2006-10-10, by haftmann
fixed typo
2006-10-10, by haftmann
added code_abstype and code_constsubst
2006-10-10, by haftmann
isabelle-process: options -S, -X;
2006-10-09, by wenzelm
tuned;
2006-10-09, by wenzelm
loop: disallow exit in secure mode;
2006-10-09, by wenzelm
Secure.commit;
2006-10-09, by wenzelm
moved Context.ml_output to Output.ml_output;
2006-10-09, by wenzelm
Secure critical operations.
2006-10-09, by wenzelm
added General/secure.ML;
2006-10-09, by wenzelm
added option -S (secure mode);
2006-10-09, by wenzelm
added nbe_post for delayed_if
2006-10-09, by nipkow
added delayed_if
2006-10-09, by nipkow
added pre/post-processor equations
2006-10-09, by nipkow
attribute "symmetric": standardized schematic variables;
2006-10-09, by wenzelm
sequential lemmas;
2006-10-09, by wenzelm
reorderd ML/lemmas (Why!?);
2006-10-09, by wenzelm
PureThy.note_thmss_i;
2006-10-09, by wenzelm
added exit;
2006-10-09, by wenzelm
added theorems(_i) -- with present_results;
2006-10-09, by wenzelm
def(_i): LocalDefs.add_defs;
2006-10-09, by wenzelm
attribute: Context.mapping;
2006-10-09, by wenzelm
removed obsolete note_thmss(_i);
2006-10-09, by wenzelm
added exit;
2006-10-09, by wenzelm
simplified derived_def;
2006-10-09, by wenzelm
removed theorems, smart_theorems etc. (cf. Specification.theorems);
2006-10-09, by wenzelm
lemmas/theorems/declare: Specification.theorems;
2006-10-09, by wenzelm
added kind attributes;
2006-10-09, by wenzelm
Drule.lhs/rhs_of;
2006-10-09, by wenzelm
added dest_equals_lhs;
2006-10-09, by wenzelm
attribute: Context.mapping;
2006-10-09, by wenzelm
replaced Drule.clhs/crhs_of by Drule.lhs/rhs_of;
2006-10-09, by wenzelm
attribute: Context.mapping;
2006-10-09, by wenzelm
standardized facts;
2006-10-09, by wenzelm
attribute symmetric: zero_var_indexes;
2006-10-09, by wenzelm
attribute symmetric: zero_var_indexes;
2006-10-09, by wenzelm
attribute: Context.mapping;
2006-10-09, by wenzelm
cleaned up interfaces
2006-10-07, by haftmann
Removed unused res_atp_setup.ML, since its functions have been put in res_atp.ML.
2006-10-07, by mengj
Common theory targets.
2006-10-07, by wenzelm
Element.export_facts;
2006-10-07, by wenzelm
refined unlocalize_mixfix;
2006-10-07, by wenzelm
TheoryTarget;
2006-10-07, by wenzelm
moved pretty_consts to proof_display.ML;
2006-10-07, by wenzelm
added pretty_consts (from specification.ML);
2006-10-07, by wenzelm
turned into abstract wrapper module, cf. theory_target.ML;
2006-10-07, by wenzelm
replaced add_def by more elaborate add_defs;
2006-10-07, by wenzelm
replaced generalize_facts by full export_(standard_)facts;
2006-10-07, by wenzelm
Thm.def_name_optional;
2006-10-07, by wenzelm
added def_name_optional;
2006-10-07, by wenzelm
removed is_equals, is_implies;
2006-10-07, by wenzelm
added the_single;
2006-10-07, by wenzelm
added term_rule;
2006-10-07, by wenzelm
added Isar/theory_target.ML;
2006-10-07, by wenzelm
improved LocalDefs.add_def;
2006-10-07, by wenzelm
mk_partial_rules_mutual: expand result terms/thms;
2006-10-07, by wenzelm
removed with_local_path -- LocalTheory.note admits qualified names;
2006-10-07, by wenzelm
moved the_single to Pure/library.ML;
2006-10-07, by wenzelm
TheoryTarget.init;
2006-10-07, by wenzelm
tuned comments;
2006-10-07, by wenzelm
tuned method syntax: polymorhic term argument;
2006-10-07, by wenzelm
tuned;
2006-10-07, by wenzelm
Fixed the printing of the used theorems by maintaining separate lists for each subgoal.
2006-10-06, by paulson
Tidied code to delete tmp files.
2006-10-06, by paulson
renamed the combinator laws
2006-10-06, by paulson
Improved detection of identical clauses, also in the conjecture
2006-10-06, by paulson
Refinements to abstraction. Seeding with combinators K, I and B.
2006-10-06, by paulson
examples for hex and bin numerals
2006-10-06, by kleing
Changed and removed some functions related to combinators, since they are Isabelle constants now.
2006-10-05, by mengj
Now the DFG output includes correct declarations of c_fequal, but not hEXTENT
2006-10-05, by paulson
improvements to abstraction, ensuring more re-use of abstraction functions
2006-10-05, by paulson
facts about combinators
2006-10-05, by paulson
a few new functions on thms and cterms
2006-10-05, by paulson
reorganize and speed up termdiffs proofs
2006-10-05, by huffman
fixed bug in linear arith
2006-10-04, by nipkow
improvements for Haskell serialization
2006-10-04, by haftmann
insert replacing ins ins_int ins_string
2006-10-04, by haftmann
cleaned up some mess
2006-10-04, by haftmann
clarified header comments
2006-10-04, by haftmann
insert replacing ins ins_int ins_string
2006-10-04, by haftmann
*** empty log message ***
2006-10-04, by haftmann
tuned
2006-10-04, by webertj
Improved error reporting
2006-10-04, by krauss
nnf_simpset built statically
2006-10-04, by webertj
rewrite proofs of powser_insidea and termdiffs_aux
2006-10-03, by huffman
generalize summability lemmas using class banach
2006-10-02, by huffman
clarified setup name
2006-10-02, by haftmann
various code refinements
2006-10-02, by haftmann
fixed some Haskell issues
2006-10-02, by haftmann
changed preprocessing framework
2006-10-02, by haftmann
clarified some things
2006-10-02, by haftmann
cleaned and extended
2006-10-02, by haftmann
added gen_primrec
2006-10-02, by haftmann
added code for insert
2006-10-02, by haftmann
improvements for code_gen
2006-10-02, by haftmann
cleaned mess
2006-10-02, by haftmann
added example for code_gen
2006-10-02, by haftmann
dropped obsolete Theory.sign_of
2006-10-02, by haftmann
tuned
2006-10-02, by haftmann
added code generator names for nat_rec and nat_case
2006-10-02, by haftmann
improved serialization for arbitrary
2006-10-02, by haftmann
normal_form now a diagnostic command
2006-10-02, by haftmann
restructured contents
2006-10-02, by haftmann
add axclass banach for complete normed vector spaces
2006-10-02, by huffman
remove unused Cauchy_Bseq lemmas
2006-10-02, by huffman
add lemmas norm_not_less_zero, norm_le_zero_iff
2006-10-02, by huffman
added is_Trueprop
2006-10-02, by paulson
tidying and simplifying
2006-10-02, by paulson
Changing the default for theory_const
2006-10-02, by paulson
extensions for Susanto
2006-10-02, by paulson
restored the "length of name > 2" check for package definitions
2006-10-02, by paulson
Now checks explicitly for Trueprop, thereby ignoring junk theorems involving OF_CLASS, etc.
2006-10-02, by paulson
exists_name: include this theory name;
2006-10-01, by wenzelm
removed obsolete Datatype_Universe.thy (cf. Datatype.thy);
2006-10-01, by wenzelm
merged with theory Datatype_Universe;
2006-10-01, by wenzelm
obsolete;
2006-10-01, by wenzelm
renamed ex/SVC_Oracle.ML to ex/svc_oracle.ML;
2006-10-01, by wenzelm
removed share_data;
2006-10-01, by wenzelm
cterm_match: avoid recalculation of maxidx;
2006-10-01, by wenzelm
reverted to revision 1.28;
2006-10-01, by wenzelm
proper use of svc_oracle.ML;
2006-10-01, by wenzelm
reactivated theory PER;
2006-10-01, by wenzelm
tuned proofs;
2006-10-01, by wenzelm
moved theory Infinite_Set to Library;
2006-10-01, by wenzelm
moved theory Infinite_Set to Library;
2006-10-01, by wenzelm
moved Infinite_Set.thy to Library;
2006-10-01, by wenzelm
tuned;
2006-10-01, by wenzelm
Removed the helper files (combinator rewrite rules, function extensionality and fequal rules).
2006-10-01, by mengj
generalize more DERIV proofs
2006-10-01, by huffman
statement: Variable.fix_frees;
2006-09-30, by wenzelm
added undo_end;
2006-09-30, by wenzelm
tuned proofs;
2006-09-30, by wenzelm
proper import of Main HOL;
2006-09-30, by wenzelm
tuned specifications and proofs;
2006-09-30, by wenzelm
hides popular names (from Datatype.thy);
2006-09-30, by wenzelm
removed obsolete sum_case_Inl/Inr;
2006-09-30, by wenzelm
renamed Variable.invent_fixes to Variable.variant_fixes;
2006-09-30, by wenzelm
generalize proofs of DERIV_isCont and DERIV_mult
2006-09-30, by huffman
generalized some DERIV proofs
2006-09-30, by huffman
add scaleR lemmas
2006-09-30, by huffman
generalize type of DERIV
2006-09-30, by huffman
add type annotations for DERIV
2006-09-30, by huffman
Combinator axioms are now from Isabelle theorems, no need to use helper files.
2006-09-30, by mengj
Added the combinator constants to the constants table.
2006-09-30, by mengj
Removed ResHolClause.LAM2COMB exception.
2006-09-30, by mengj
Reordered how files are loaded.
2006-09-30, by mengj
moved Matrix/cplex/MatrixLP.ML to Matrix/cplex/matrixlp.ML;
2006-09-29, by wenzelm
removed mixfix_content;
2006-09-29, by wenzelm
Syntax.mode;
2006-09-29, by wenzelm
Syntax.mode;
2006-09-29, by wenzelm
Sign.add_consts_authentic;
2006-09-29, by wenzelm
proper use of matrixlp.ML;
2006-09-29, by wenzelm
simplified is_package_def -- be less ambitious about B library operations;
2006-09-29, by wenzelm
obsolete;
2006-09-28, by wenzelm
added share_data;
2006-09-28, by wenzelm
Sign.add_consts_authentic;
2006-09-28, by wenzelm
consts: syntax consts only for actual syntax;
2006-09-28, by wenzelm
added share_data (dummy);
2006-09-28, by wenzelm
removed obsolete HOLCF.ML;
2006-09-28, by wenzelm
ResAtpset.get_atpset;
2006-09-28, by wenzelm
removed legacy code;
2006-09-28, by wenzelm
tuned definitions/proofs;
2006-09-28, by wenzelm
proper use of float.ML;
2006-09-28, by wenzelm
fixed translations: CONST;
2006-09-28, by wenzelm
replaced syntax/translations by abbreviation;
2006-09-28, by wenzelm
replaced syntax/translations by abbreviation;
2006-09-28, by wenzelm
removed obsolete Real/document/root.tex;
2006-09-28, by wenzelm
tuned;
2006-09-28, by wenzelm
rearranged axioms and simp rules for scaleR
2006-09-28, by huffman
added Poly/ML 4.9.1 (experimental!);
2006-09-28, by wenzelm
rearranged axioms and simp rules for scaleR
2006-09-28, by huffman
clearout of obsolete code
2006-09-28, by paulson
addition of combinators
2006-09-28, by paulson
tuned messages;
2006-09-28, by wenzelm
tuned;
2006-09-28, by wenzelm
LD_LIBRARY_PATH;
2006-09-28, by wenzelm
Definitions produced by packages are now blacklisted.
2006-09-28, by paulson
more reorganizing sections
2006-09-28, by huffman
reorganize sections
2006-09-28, by huffman
add intro/dest rules for NSLIM; rewrite equivalence proofs using transfer
2006-09-28, by huffman
add lemma hypreal_epsilon_gt_zero
2006-09-28, by huffman
generalize type of is(NS)UCont
2006-09-28, by huffman
add intro/dest rules for (NS)LIMSEQ and (NS)Cauchy; rewrite equivalence proofs using transfer
2006-09-28, by huffman
proper use of PolyML.shareCommonData;
2006-09-28, by wenzelm
add lemmas InfinitesimalI2, InfinitesimalD2
2006-09-27, by huffman
adapted to pre-5.0 versions;
2006-09-27, by wenzelm
Poly/ML startup script (for 4.9.1);
2006-09-27, by wenzelm
added ML-Systems/polyml-4.9.1.ML;
2006-09-27, by wenzelm
Compatibility wrapper for Poly/ML 4.9.1.
2006-09-27, by wenzelm
removed all references to star_n and FreeUltrafilterNat
2006-09-27, by huffman
add lemmas about hnorm, Infinitesimal
2006-09-27, by huffman
reverted to 1.58;
2006-09-27, by wenzelm
proper const_syntax for uminus, abs;
2006-09-27, by wenzelm
reorganized HNatInfinite proofs; simplified and renamed some lemmas
2006-09-27, by huffman
removed obsolete of_instream_slurp -- now already included in tty;
2006-09-27, by wenzelm
Source.tty now slurps by default;
2006-09-27, by wenzelm
of_stream/tty: slurp input eagerly;
2006-09-27, by wenzelm
tuned all_paths;
2006-09-27, by wenzelm
internal params: Vartab instead of AList;
2006-09-27, by wenzelm
removed unused serial_of, name_of;
2006-09-27, by wenzelm
removed redundant lemmas;
2006-09-27, by wenzelm
remove redundant lemmas
2006-09-27, by huffman
replaced constant 0 by HOL.zero
2006-09-27, by haftmann
hypreal_of_nat abbreviates of_nat
2006-09-27, by huffman
add lemmas of_real_eq_star_of, Reals_eq_Standard
2006-09-27, by huffman
move star_of_norm from SEQ.thy to NSA.thy
2006-09-27, by huffman
convert more proofs to transfer principle
2006-09-27, by huffman
add lemmas about Standard, real_of, scaleR
2006-09-27, by huffman
instance complex :: real_normed_field; cleaned up
2006-09-27, by huffman
add lemma stc_unique; shorten stc proofs
2006-09-27, by huffman
add lemmas approx_diff and st_unique, shorten st proofs
2006-09-27, by huffman
add lemmas about of_real and power
2006-09-27, by huffman
reorganize section headings
2006-09-27, by huffman
more lemmas about Standard and star_of
2006-09-27, by huffman
define new constant Standard = range star_of
2006-09-27, by huffman
add lemmas of_int_in_Reals, of_nat_in_Reals
2006-09-27, by huffman
add header
2006-09-26, by huffman
Changed precedence of "op O" (relation composition) from 60 to 75.
2006-09-26, by krauss
handling of \<^const> syntax for case; explicit case names for induction rules for rep_datatype
2006-09-26, by haftmann
tuned syntax for <= <
2006-09-26, by haftmann
renamed 0 and 1 to HOL.zero and HOL.one respectivly; introduced corresponding syntactic classes
2006-09-26, by haftmann
renamed 0 and 1 to HOL.zero and HOL.one respectivly
2006-09-26, by haftmann
fixed the definition of "depth"
2006-09-26, by paulson
Abstraction now handles equations where the RHS is a lambda-expression; also, strings of lambdas
2006-09-26, by paulson
some cleanup
2006-09-25, by haftmann
changed order
2006-09-25, by haftmann
inserted headings
2006-09-25, by haftmann
changed interface in codegen_package.ML
2006-09-25, by haftmann
fixed some mess
2006-09-25, by haftmann
cleaned up
2006-09-25, by haftmann
adding constants the modern way
2006-09-25, by haftmann
added examples for variable name handling
2006-09-25, by haftmann
better handling for div by zero
2006-09-25, by haftmann
updated theory description
2006-09-25, by haftmann
refinements in codegen serializer
2006-09-25, by haftmann
added 'undefined' serializer
2006-09-25, by haftmann
added code_instname
2006-09-25, by haftmann
reorganized subsection headings
2006-09-24, by huffman
moved SEQ_Infinitesimal from SEQ to HyperNat
2006-09-24, by huffman
real_norm_def [simp]
2006-09-24, by huffman
generalize types of lim and nslim
2006-09-24, by huffman
generalized types of sums, summable, and suminf
2006-09-24, by huffman
add lemma convergent_Cauchy
2006-09-24, by huffman
remove extra dependencies
2006-09-24, by huffman
add proof of summable_LIMSEQ_zero
2006-09-24, by huffman
change definitions from SOME to THE
2006-09-24, by huffman
move root and sqrt stuff from Transcendental to NthRoot
2006-09-24, by huffman
fix proof
2006-09-24, by huffman
added lemmas about LIMSEQ and norm; simplified some proofs
2006-09-22, by huffman
add lemma norm_power
2006-09-22, by huffman
added HOL-Complex-ex;
2006-09-22, by wenzelm
define constants with THE instead of SOME
2006-09-22, by huffman
Fixed bug concerning the generation of identifiers for
2006-09-22, by berghofe
Replaced irreducible_paths by all_paths.
2006-09-22, by berghofe
Added function all_paths (formerly find_paths).
2006-09-22, by berghofe
tuned proofs;
2006-09-22, by wenzelm
tuned oracle name;
2006-09-21, by wenzelm
added is_ml_reserved;
2006-09-21, by wenzelm
member (op =);
2006-09-21, by wenzelm
serial numbers for types;
2006-09-21, by wenzelm
added dest_binop;
2006-09-21, by wenzelm
member (op =);
2006-09-21, by wenzelm
member (op =);
2006-09-21, by wenzelm
tuned eta_contract;
2006-09-21, by wenzelm
added dest_equals_rhs;
2006-09-21, by wenzelm
tuned;
2006-09-21, by wenzelm
serial numbers for consts;
2006-09-21, by wenzelm
Thm.dest_binop;
2006-09-21, by wenzelm
member (op =);
2006-09-21, by wenzelm
member (op =);
2006-09-21, by wenzelm
updated timings;
2006-09-21, by wenzelm
new function hashw_int
2006-09-21, by paulson
Yet another version of fake_thm_name. "Full" hashing ensures that there are no collisions
2006-09-21, by paulson
corrected for the translation from _ to __ in c_COMBx_e
2006-09-21, by paulson
changed constants into abbreviations; shortened proofs
2006-09-21, by huffman
XML syntax for types, terms, and proofs.
2006-09-21, by berghofe
Added xml_syntax.ML
2006-09-21, by berghofe
Added Tools/xml_syntax.ML
2006-09-21, by berghofe
circumvented defect in SML/NJ type inference
2006-09-21, by haftmann
1. Function package accepts a parameter (default "some_term"), which specifies the functions
2006-09-21, by krauss
removed division_by_zero class requirements from several lemmas
2006-09-21, by huffman
added approx_hnorm theorem; removed division_by_zero class requirements from several lemmas
2006-09-21, by huffman
choose gnuplot terminal by platform
2006-09-20, by isatest
set terminal png color -- works for older versions of gnuplot;
2006-09-20, by wenzelm
added ZF-UNITY;
2006-09-20, by wenzelm
tidied
2006-09-20, by paulson
Added in combinator reduction axioms for B' C' and S'. Also split the original reduction axioms into separate files: I+K, B+C, S, B'+C', S'.
2006-09-20, by mengj
make it work on sunbroy2
2006-09-20, by isatest
Moved the functional equality axioms to helper1 files.
2006-09-20, by mengj
Introduced combinators B', C' and S'.
2006-09-20, by mengj
Removed include_min_comb and include_combS.
2006-09-20, by mengj
Add Source.of_instream_slurp to try to ensure that XML parser sees whole documents.
2006-09-20, by aspinall
improvements for codegen 2
2006-09-20, by haftmann
name shifts
2006-09-20, by haftmann
fixed bug
2006-09-20, by haftmann
Removed "induct set" attribute from total induction rules
2006-09-20, by krauss
removed debug
2006-09-20, by haftmann
Fixed error in pattern splitting algorithm
2006-09-20, by krauss
change section to subsection
2006-09-20, by huffman
add header
2006-09-20, by huffman
renamed axclass_xxxx axclasses;
2006-09-20, by wenzelm
tuned;
2006-09-19, by wenzelm
added standard;
2006-09-19, by wenzelm
added name_classrel/arities/arity;
2006-09-19, by wenzelm
pretty_full_theory: suppress internal entities by default;
2006-09-19, by wenzelm
Logic.name_classrel/arities;
2006-09-19, by wenzelm
revert to previous version;
2006-09-19, by wenzelm
added General/susp.ML;
2006-09-19, by wenzelm
removed duplicate arities;
2006-09-19, by wenzelm
sko/abs: Name.internal prevents choking of print_theory;
2006-09-19, by wenzelm
tuned method setup;
2006-09-19, by wenzelm
tuned proofs;
2006-09-19, by wenzelm
'print_theory': bang option for full verbosity;
2006-09-19, by wenzelm
* Pure: 'print_theory' now suppresses entities with internal name;
2006-09-19, by wenzelm
tuned;
2006-09-19, by wenzelm
simple html output;
2006-09-19, by wenzelm
timespan: 100 days;
2006-09-19, by wenzelm
superceded by isatest-statistics;
2006-09-19, by wenzelm
tuned;
2006-09-19, by wenzelm
target dir;
2006-09-19, by wenzelm
Standard statistics.
2006-09-19, by wenzelm
time: include year;
2006-09-19, by wenzelm
Produce statistics from isatest session logs.
2006-09-19, by wenzelm
moved Import/susp.ML to Pure/General;
2006-09-19, by wenzelm
renamed axclass_xxxx axclasses
2006-09-19, by obua
removed diagnostic messages
2006-09-19, by haftmann
Operational Equality
2006-09-19, by haftmann
this file contains a compile-challenge suggested by Adam Chlipala;
2006-09-19, by urbanc
tuned
2006-09-19, by urbanc
added auxiliary lemma for code generation 2
2006-09-19, by haftmann
removed
2006-09-19, by haftmann
moved part of normalization oracle here
2006-09-19, by haftmann
classical arity syntax
2006-09-19, by haftmann
added codegen_data
2006-09-19, by haftmann
moved base setup for evaluation oracle hier
2006-09-19, by haftmann
added OperationalEquality.thy
2006-09-19, by haftmann
code generation 2 adjustments
2006-09-19, by haftmann
(void)
2006-09-19, by haftmann
improved numeral handling for nbe
2006-09-19, by haftmann
added suspensions in Pure
2006-09-19, by haftmann
added some stuff for code generation 2
2006-09-19, by haftmann
dropped error-prone code generation 2 for wfrec
2006-09-19, by haftmann
text cleanup
2006-09-19, by haftmann
introduced syntactic classes; moved some setup to Pure/codegen, Pure/nbe or OperationalEquality.thy
2006-09-19, by haftmann
explicit divmod algorithm for code generation
2006-09-19, by haftmann
added operational equality
2006-09-19, by haftmann
added section on code generation 2
2006-09-19, by haftmann
code_gen now peek keyword
2006-09-19, by haftmann
cleanupdiff
2006-09-19, by haftmann
added classes real_div_algebra and real_field; added lemmas
2006-09-19, by huffman
add Real/RealVector.thy
2006-09-19, by huffman
* Pure: 'class_deps' command visualizes the subclass relation;
2006-09-18, by wenzelm
added class_deps;
2006-09-18, by wenzelm
added dest_arg, i.e. a tuned version of #2 o dest_comb;
2006-09-18, by wenzelm
Thm.dest_arg;
2006-09-18, by wenzelm
Present.display_graph;
2006-09-18, by wenzelm
added display_graph (from thm_deps.ML);
2006-09-18, by wenzelm
output: uninterpreted raw symbols -- these are usually LaTeX macros;
2006-09-18, by wenzelm
pretty_thm: graceful treatment of ProtoPure.thy;
2006-09-18, by wenzelm
added class_deps;
2006-09-18, by wenzelm
classes: maintain serial number;
2006-09-18, by wenzelm
tuned;
2006-09-18, by wenzelm
isatool browser: renamed option -d to -c (cf. isatool tool)
2006-09-18, by wenzelm
PRIVATE_FILE: slightly more robust way to create and dispose;
2006-09-18, by wenzelm
renamed option -d to -c (cf. isatool display);
2006-09-18, by wenzelm
updated;
2006-09-18, by wenzelm
Bug fix to prevent exception dest_Free from escaping
2006-09-18, by paulson
Added the max_new parameter, which is a cap on how many clauses may be admitted per round.
2006-09-18, by paulson
replaced implodeable_Ext by set_like
2006-09-18, by obua
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
2006-09-18, by chaieb
replace (x + - y) with (x - y)
2006-09-18, by huffman
add type constraint to otherwise looping iff rule
2006-09-17, by huffman
generalize type of (NS)LIM to work on functions with vector space domain types
2006-09-17, by huffman
norm_one is now proved from other class axioms
2006-09-17, by huffman
removed capprox, CFinite, CInfinite, CInfinitesimal, cmonad, and cgalaxy in favor of polymorphic constants
2006-09-17, by huffman
hcmod abbreviates hnorm :: hcomplex => hypreal
2006-09-17, by huffman
complex_of_real abbreviates of_real::real=>complex;
2006-09-16, by huffman
add instance for real_algebra_1 and real_normed_div_algebra
2006-09-16, by huffman
add instances for real_vector and real_algebra
2006-09-16, by huffman
define new constant of_real for class real_algebra_1;
2006-09-16, by huffman
int_diff_cases moved to Integ/IntDef.thy
2006-09-16, by huffman
generalized types of many constants to work over arbitrary vector spaces;
2006-09-16, by huffman
add theorem norm_diff_triangle_ineq
2006-09-16, by huffman
add required type annotation
2006-09-16, by huffman
removed type aliases for theory/theory_ref;
2006-09-15, by wenzelm
renamed Term.map_term_types to Term.map_types (cf. Term.fold_types);
2006-09-15, by wenzelm
tuned;
2006-09-15, by wenzelm
rrule: maintain 'extra' field for rule that contain extra vars outside elhs;
2006-09-15, by wenzelm
instantiate: omit has_duplicates check, which is irrelevant for soundness;
2006-09-15, by wenzelm
trivial whitespace change
2006-09-15, by webertj
tuned;
2006-09-15, by wenzelm
more on theorems;
2006-09-14, by wenzelm
generalized types of Infinitesimal, HFinite, and HInfinite to work over nonstandard extensions of any real normed vector space
2006-09-14, by huffman
add instance for class division_ring
2006-09-14, by huffman
removed duplicate lemmas
2006-09-14, by huffman
fixed syntax clash with Real/RealVector
2006-09-14, by huffman
*** empty log message ***
2006-09-14, by wenzelm
Function package: Outside their domain functions now return "arbitrary".
2006-09-14, by krauss
updated makefile
2006-09-14, by krauss
Fixed Subscript Exception occurring with Higher-Order recursion
2006-09-14, by krauss
remove conflicting norm syntax
2006-09-14, by huffman
made SML/NJ happy;
2006-09-14, by wenzelm
added exists_type;
2006-09-13, by wenzelm
renamed NameSpace.drop_base to NameSpace.qualifier;
2006-09-13, by wenzelm
Updated keyword file
2006-09-13, by krauss
Removed debugging code imports...
2006-09-13, by krauss
Added the "theory_const" option. Only it is OFF because it's often harmful!
2006-09-13, by paulson
Extended the blacklist with higher-order theorems. Restructured. Added checks to
2006-09-13, by paulson
bug fix to abstractions: free variables in theorem can be abstracted over.
2006-09-13, by paulson
Tweaks to is_fol_term, the first-order test. We don't count "=" as a connective
2006-09-13, by paulson
Major update to function package, including new syntax and the (only theoretical)
2006-09-13, by krauss
added instance rat :: recpower
2006-09-13, by huffman
more on theorems;
2006-09-12, by wenzelm
tuned;
2006-09-12, by wenzelm
more on terms;
2006-09-12, by wenzelm
no_syntax norm -- clash with Real/RealVector.thy;
2006-09-12, by wenzelm
simplify some proofs, remove obsolete realpow_divide
2006-09-12, by huffman
realpow_divide -> power_divide
2006-09-12, by huffman
remove extra dependency
2006-09-12, by huffman
more on terms;
2006-09-12, by wenzelm
Efficient term substitution -- avoids copying.
2006-09-12, by wenzelm
ctyp: maintain maxidx;
2006-09-12, by wenzelm
removed obsolete aconvs (use eq_list aconv);
2006-09-12, by wenzelm
tuned eq_list;
2006-09-12, by wenzelm
moved term subst functions to TermSubst;
2006-09-12, by wenzelm
intr/elim: use constant complexity thanks to tuned Thm.instantiate/implies_elim;
2006-09-12, by wenzelm
added Pure/term_subst.ML;
2006-09-12, by wenzelm
added Gentzen:1935;
2006-09-12, by wenzelm
import RealVector
2006-09-12, by huffman
formalization of vector spaces and algebras over the real numbers
2006-09-12, by huffman
induct method: renamed 'fixing' to 'arbitrary';
2006-09-11, by wenzelm
updated;
2006-09-11, by wenzelm
more rules;
2006-09-11, by wenzelm
hid succ, pred in Numeral.thy
2006-09-11, by haftmann
updated;
2006-09-11, by wenzelm
more rules;
2006-09-11, by wenzelm
tuned;
2006-09-11, by wenzelm
added axclass division_ring (like field without commutativity; includes e.g. quaternions) and generalized some theorems from field to division_ring
2006-09-10, by huffman
cleaned up
2006-09-09, by huffman
tuned;
2006-09-08, by wenzelm
tuned;
2006-09-08, by wenzelm
changed order of type classes and axclasses
2006-09-08, by haftmann
tuned;
2006-09-07, by wenzelm
updated;
2006-09-07, by wenzelm
tentative appendix C;
2006-09-07, by wenzelm
tuned;
2006-09-07, by wenzelm
read_instantiate: declare names of TVars as well (temporary workaround for no-freeze feature of type inference);
2006-09-06, by wenzelm
rawsat_thm: mk_conjunction_list replaced by Conjunction.mk_conjunction_list
2006-09-06, by webertj
got rid of Numeral.bin type
2006-09-06, by haftmann
now using TypecopyPackage
2006-09-06, by haftmann
TypedefPackage.add_typedef_* now yields name of introduced type constructor
2006-09-06, by haftmann
added Barendregt-Geuvers:2001;
2006-09-05, by wenzelm
updated;
2006-09-05, by wenzelm
more on types and type classes;
2006-09-05, by wenzelm
tuned;
2006-09-05, by wenzelm
added \isactrlvec;
2006-09-05, by wenzelm
tuned;
2006-09-05, by wenzelm
more on names;
2006-09-05, by wenzelm
tuned;
2006-09-04, by wenzelm
tuned;
2006-09-04, by wenzelm
Using Drule.local_standard to reduce the space usage
2006-09-04, by paulson
tuned;
2006-09-04, by wenzelm
updated;
2006-09-04, by wenzelm
more on variables;
2006-09-04, by wenzelm
More locale test code.
2006-09-04, by ballarin
Documented methods intro_locales and unfold_locales.
2006-09-04, by ballarin
some corrections in class section
2006-09-04, by haftmann
explicit table with constant types
2006-09-04, by haftmann
proper project_sort
2006-09-04, by haftmann
tuned
2006-09-02, by webertj
zchaff_with_proofs: proof is a reference now
2006-09-02, by webertj
signature: do not export private stuff;
2006-09-01, by wenzelm
skolem_cache_thm: Drule.close_derivation on clauses preserves some space;
2006-09-01, by wenzelm
tuned;
2006-09-01, by wenzelm
tuned;
2006-09-01, by wenzelm
explain assumptions;
2006-09-01, by wenzelm
refinements to conversion into clause form, esp for the HO case
2006-09-01, by paulson
pervasive refinements
2006-09-01, by haftmann
removed some dictionary stuff
2006-09-01, by haftmann
project_algebra yields sort projector
2006-09-01, by haftmann
final syntax for some Isar code generator keywords
2006-09-01, by haftmann
tuned;
2006-08-31, by wenzelm
misc cleanup;
2006-08-31, by wenzelm
tuned;
2006-08-31, by wenzelm
more stuff;
2006-08-31, by wenzelm
mldecls: footnotesize;
2006-08-31, by wenzelm
more on contexts;
2006-08-31, by wenzelm
String.concatWith (not available in PolyML) replaced by space_implode
2006-08-31, by webertj
improvements to abstraction generation
2006-08-31, by paulson
blacklist now handles thm lists
2006-08-31, by paulson
Empty is better than Match
2006-08-31, by paulson
term_of_prop_formula added
2006-08-31, by webertj
read_dimacs_cnf_file ignores more comment lines
2006-08-31, by webertj
faster clause representation (again): full CNF formula as a hypothesis, instead of separate clauses
2006-08-30, by webertj
code refinements
2006-08-30, by haftmann
updated;
2006-08-30, by wenzelm
tuned;
2006-08-30, by wenzelm
added yet another code generator example
2006-08-30, by haftmann
fixes
2006-08-30, by haftmann
fixed bug in wfrec appgen
2006-08-30, by haftmann
lin_arith_prover: splitting reverted because of performance loss
2006-08-30, by webertj
lin_arith_prover: splitting reverted because of performance loss
2006-08-30, by webertj
added a FIXME-comment
2006-08-29, by urbanc
tuned;
2006-08-29, by wenzelm
more on contexts;
2006-08-29, by wenzelm
refinements
2006-08-29, by haftmann
added and refined some exmples
2006-08-29, by haftmann
added typecopy_package
2006-08-29, by haftmann
added typecopy_package and some examples
2006-08-29, by haftmann
updated keywords
2006-08-29, by haftmann
minor bug fixes
2006-08-28, by paulson
removed the (apparently pointless) signature constraint
2006-08-28, by paulson
tidied
2006-08-28, by paulson
encode clauses as Isar premises, rather than as object-logic &, for faster parsing
2006-08-28, by webertj
abstraction of lambda-expressions
2006-08-25, by paulson
tidied
2006-08-25, by paulson
better skolemization, using first-order resolution rather than hoping for the right result
2006-08-25, by paulson
using inc
2006-08-25, by paulson
explicit type variables prevent empty sorts
2006-08-25, by paulson
replaced skolem declarations by automatic skolemization of everything
2006-08-25, by paulson
avoid duplicate tactics
2006-08-25, by webertj
additional list of tactics that can be added to arith
2006-08-24, by webertj
Added premises concerning finite support of recursion results to FCBs.
2006-08-24, by berghofe
speed up proof of summable_Cauchy
2006-08-23, by huffman
speed up some proofs
2006-08-23, by huffman
generalize proof of SUP_rabs_subseq
2006-08-23, by huffman
speed up some proofs
2006-08-23, by huffman
SML/NJ int type fix
2006-08-23, by haftmann
tracing
2006-08-21, by haftmann
improved preprocessing
2006-08-21, by haftmann
fixed bug in sortlookup
2006-08-21, by haftmann
more concise preprocessing of numerals for code generation
2006-08-21, by haftmann
more concise string serialization
2006-08-21, by haftmann
added some codegen examples/applications
2006-08-21, by haftmann
adapted using the characteristic equations
2006-08-18, by urbanc
modified to use the characteristic equations
2006-08-18, by urbanc
- Fixed bug that caused uniqueness proof for recursion
2006-08-18, by berghofe
used the recursion combinator for the height and substitution function
2006-08-17, by urbanc
added definition for size and substitution using the recursion
2006-08-17, by urbanc
improved thmtab
2006-08-17, by haftmann
fixed bug in sortcontext extraction
2006-08-17, by haftmann
dropped definitions_of
2006-08-17, by haftmann
added all_super_classes
2006-08-17, by haftmann
renamed module to thyname
2006-08-17, by haftmann
cleanup
2006-08-17, by haftmann
added missing supp_nat lemma
2006-08-16, by urbanc
added
2006-08-14, by haftmann
module restructuring
2006-08-14, by haftmann
code cleanup, instance_subsort now working
2006-08-14, by haftmann
added code generator packages
2006-08-14, by haftmann
adaptions to improvements
2006-08-14, by haftmann
added add_hook_bootstrap
2006-08-14, by haftmann
added new files
2006-08-14, by haftmann
simplified code generator setup
2006-08-14, by haftmann
added passage on class package
2006-08-14, by haftmann
updated code generator keywords
2006-08-14, by haftmann
Removed non-trivial definitions from calc_atm theorem list.
2006-08-14, by berghofe
Finished implementation of uniqueness proof for recursion combinator.
2006-08-14, by berghofe
*** empty log message ***
2006-08-14, by chaieb
Reification now handels binders.
2006-08-14, by chaieb
consistent prefixing for skolem functions
2006-08-09, by paulson
blacklist augmented to block some "unit" theorems that cause unsound resolution proofs
2006-08-09, by paulson
tuned: string_of_list, string_of_pair
2006-08-09, by webertj
* ProofContext.prems_limit is now -1 by default;
2006-08-09, by wenzelm
tuned proofs;
2006-08-09, by wenzelm
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
2006-08-09, by wenzelm
renamed map_theory to theory;
2006-08-09, by wenzelm
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
2006-08-09, by wenzelm
locale interpretation command: after_qed;
2006-08-09, by wenzelm
int_option: signed_string_of_int;
2006-08-09, by wenzelm
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
2006-08-09, by wenzelm
skolem declarations for built-in theorems
2006-08-08, by paulson
more explict variable names
2006-08-08, by paulson
tidying
2006-08-08, by paulson
Adapted to older logfiles containing no cpu time.
2006-08-08, by berghofe
added code_constname keyword
2006-08-08, by haftmann
fixed code generator theorem generation
2006-08-08, by haftmann
improvements for 2nd codegenerator
2006-08-08, by haftmann
cleanup code generation for Numerals
2006-08-08, by haftmann
improved & fixed code generator theorem generation
2006-08-08, by haftmann
code generator refinements
2006-08-08, by haftmann
adding code lemma now works as expected
2006-08-08, by haftmann
added more examples
2006-08-08, by haftmann
dropped duplicated line
2006-08-08, by haftmann
added Tools/typedef_codegen.ML
2006-08-08, by haftmann
abandoned equal_list in favor for eq_list
2006-08-08, by haftmann
Simple ML script for producing Gnuplot files from
2006-08-07, by berghofe
title fixed
2006-08-07, by webertj
updated;
2006-08-05, by wenzelm
avoid low-level tsig;
2006-08-05, by wenzelm
reworked read_instantiate -- separate read_insts;
2006-08-05, by wenzelm
tuned;
2006-08-05, by wenzelm
removed obsolete sign_of;
2006-08-05, by wenzelm
Amine Chaieb: experimental generic reflection and reification in HOL;
2006-08-05, by wenzelm
use atbroy101 instead of atbroy98 (freezes up)
2006-08-05, by isatest
Added Keywords: "otherwise" and "sequential", needed for function package's
2006-08-04, by krauss
*** empty log message ***
2006-08-04, by chaieb
Rule instantiations -- operations within a rule/subgoal context.
2006-08-03, by wenzelm
moved bires_inst_tac etc. to rule_insts.ML;
2006-08-03, by wenzelm
moved read_instantiate etc. to rule_insts.ML;
2006-08-03, by wenzelm
added Isar/rule_insts.ML;
2006-08-03, by wenzelm
removed obsolete commute, map_list;
2006-08-03, by wenzelm
removed obsolete add_term_tvarnames;
2006-08-03, by wenzelm
tuned;
2006-08-03, by wenzelm
tuned types_sorts, add_used;
2006-08-03, by wenzelm
RuleInsts.bires_inst_tac;
2006-08-03, by wenzelm
*** empty log message ***
2006-08-03, by chaieb
fixed generator
2006-08-03, by obua
added HOL/ex/Reflection;
2006-08-03, by wenzelm
removed True_implies (cf. True_implies_equals);
2006-08-03, by wenzelm
removed OldGoals.legacy flag (always warn);
2006-08-03, by wenzelm
removed OldGoals.legacy flag (always warn);
2006-08-03, by wenzelm
tuned;
2006-08-03, by wenzelm
removed True_implies (cf. True_implies_equals);
2006-08-03, by wenzelm
Generic reflection and reification (by Amine Chaieb).
2006-08-03, by wenzelm
Restructured algebra library, added ideals and quotient rings.
2006-08-03, by ballarin
Updated comments.
2006-08-03, by ballarin
updated;
2006-08-03, by wenzelm
tuned proofs;
2006-08-02, by wenzelm
lemma da_good_approx: adapted induction (was exploting lifted obtain result);
2006-08-02, by wenzelm
renamed Syntax.indexname to Syntax.read_indexname;
2006-08-02, by wenzelm
tuned;
2006-08-02, by wenzelm
moved debug option to proof_display.ML (again);
2006-08-02, by wenzelm
normalized Proof.context/method type aliases;
2006-08-02, by wenzelm
simplified Assumption/ProofContext.export;
2006-08-02, by wenzelm
added tactical result;
2006-08-02, by wenzelm
removed obsolete Drule.frees/vars_of etc.;
2006-08-02, by wenzelm
normalized Proof.context/method type aliases;
2006-08-02, by wenzelm
simplified Proof.end_block;
2006-08-02, by wenzelm
removed obsolete Drule.frees/vars_of etc.;
2006-08-02, by wenzelm
normalized Proof.context/method type aliases;
2006-08-02, by wenzelm
renamed Syntax.indexname to Syntax.read_indexname;
2006-08-02, by wenzelm
Variable.focus_subgoal;
2006-08-02, by wenzelm
replaced maxidx_of_proof by maxidx_proof;
2006-08-02, by wenzelm
prems-limit: int_option;
2006-08-02, by wenzelm
removed obsolete frees/vars_of etc.;
2006-08-02, by wenzelm
fake predeclaration of type Proof.context;
2006-08-02, by wenzelm
simplified export: no Seq.seq;
2006-08-02, by wenzelm
use proper RecdefPackage.get_hints;
2006-08-02, by wenzelm
removed obsolete Drule.frees/vars_of;
2006-08-02, by wenzelm
renamed thm_vars to thm_varnames;
2006-08-02, by wenzelm
removed obsolete Drule.freeze_all -- now uses legacy Drule.freeze_thaw;
2006-08-02, by wenzelm
export get_hints;
2006-08-02, by wenzelm
normalized Proof.context/method type aliases;
2006-08-02, by wenzelm
normalized Proof.context/method type aliases;
2006-08-02, by wenzelm
simplified Assumption/ProofContext.export;
2006-08-02, by wenzelm
replaced obsolete standard/freeze_all by Variable.trade;
2006-08-02, by wenzelm
removed obsolete Drule.frees/vars_of etc.;
2006-08-02, by wenzelm
Added type constraint to please sml/nj
2006-08-02, by krauss
deleted obsolete file
2006-08-02, by paulson
lin_arith_prover splits certain operators (e.g. min, max, abs)
2006-08-02, by webertj
lin_arith_prover splits certain operators (e.g. min, max, abs)
2006-08-02, by webertj
Only ignore too general axiom clauses, if the translation is partial- or constant-typed.
2006-08-02, by mengj
type annotations fixed (IntInf.int, to make SML/NJ happy)
2006-08-02, by webertj
lin_arith_prover splits certain operators (e.g. min, max, abs)
2006-08-02, by webertj
proof reconstruction now uses its own data structure to manage hyps; should be both faster and more robust
2006-08-02, by webertj
comment (timing information for last example) added
2006-08-01, by webertj
possible disagreement between proof search and proof reconstruction when eliminating inequalities over different types fixed
2006-08-01, by webertj
removed skip
2006-08-01, by obua
Added in code to check too general axiom clauses.
2006-08-01, by mengj
exported attrib;
2006-08-01, by wenzelm
lin_arith_prover splits certain operators (e.g. min, max, abs)
2006-07-31, by webertj
fixed a bug in function poly: decomposition of products
2006-07-31, by webertj
Function package can now do automatic splits of overlapping datatype patterns
2006-07-31, by krauss
Removed an "apply arith" where there are already "No Subgoals"
2006-07-31, by krauss
code reformatted
2006-07-31, by webertj
Additional freshness constraints for FCB.
2006-07-31, by berghofe
proper Element.generalize_facts;
2006-07-30, by wenzelm
add_consts: proper Sign.full_name;
2006-07-30, by wenzelm
added generalize_facts;
2006-07-30, by wenzelm
added maxidx_values;
2006-07-30, by wenzelm
export: refrain from adjusting maxidx;
2006-07-30, by wenzelm
adjust_maxidx: pass explicit lower bound;
2006-07-30, by wenzelm
Thm.adjust_maxidx;
2006-07-30, by wenzelm
removed unused add_in_order/add_once (cf. OrdList.insert);
2006-07-30, by wenzelm
demod_rule: depend on context, proper Variable.import/export;
2006-07-30, by wenzelm
tuned proofs;
2006-07-30, by wenzelm
lin_arith_prover splits certain operators (e.g. min, max, abs)
2006-07-30, by webertj
bugfix related to cancel_div_mod simproc
2006-07-30, by webertj
lin_arith_prover splits certain operators (e.g. min, max, abs)
2006-07-29, by webertj
rename legacy_pretty_thm to pretty_thm_legacy;
2006-07-29, by wenzelm
tuned comment;
2006-07-29, by wenzelm
added add_fixes_direct;
2006-07-29, by wenzelm
prove: proper assumption context, more tactic arguments;
2006-07-29, by wenzelm
added mk_conjunction_list;
2006-07-29, by wenzelm
Goal.prove: more tactic arguments;
2006-07-29, by wenzelm
Checking for unsound proofs. Tidying.
2006-07-28, by paulson
"all theorems" mode forces definition-expansion off.
2006-07-28, by paulson
title fixed
2006-07-28, by webertj
replaced extern_skolem by slightly more simplistic revert_skolems;
2006-07-27, by wenzelm
renamed ProofContext.fix_frees to Variable.fix_frees;
2006-07-27, by wenzelm
replaced ProofContext.extern_skolem by slightly more simplistic ProofContext.revert_skolems;
2006-07-27, by wenzelm
no_vars: based on Variable.import;
2006-07-27, by wenzelm
added fix_frees (from Isar/proof_context.ML);
2006-07-27, by wenzelm
declare_term_names: cover types as well;
2006-07-27, by wenzelm
eliminated obsolete freeze_thaw;
2006-07-27, by wenzelm
type annotation added to make SML/NJ happy
2006-07-27, by webertj
"moved basic assumption operations from structure ProofContext to Assumption;"
2006-07-27, by wenzelm
ProofContext.legacy_pretty_thm;
2006-07-27, by wenzelm
added legacy_pretty_thm (with fall-back on ProtoPure.thy);
2006-07-27, by wenzelm
Assumption.assume;
2006-07-27, by wenzelm
removed obsolete is_fact (cf. Thm.no_prems);
2006-07-27, by wenzelm
tuned interfaces;
2006-07-27, by wenzelm
read_def_cterms (legacy version): Consts.certify;
2006-07-27, by wenzelm
Assumption.assume;
2006-07-27, by wenzelm
moved Goal.norm_hhf(_protect) to meta_simplifier.ML (pervasive);
2006-07-27, by wenzelm
removed obsolete equal_abs_elim(_list);
2006-07-27, by wenzelm
removed obsolete pretty_thm_no_quote;
2006-07-27, by wenzelm
added Pure/assumption.ML;
2006-07-27, by wenzelm
moved basic assumption operations from structure ProofContext to Assumption;
2006-07-27, by wenzelm
tuned proofs;
2006-07-27, by wenzelm
Local assumptions, parameterized by export rules.
2006-07-27, by wenzelm
updated;
2006-07-26, by wenzelm
import(T): result includes fixed types/terms;
2006-07-26, by wenzelm
focus: result record includes (fixed) schematic variables;
2006-07-26, by wenzelm
Variable.import(T): result includes fixed types/terms;
2006-07-26, by wenzelm
linear arithmetic splits certain operators (e.g. min, max, abs)
2006-07-26, by webertj
added eval_term
2006-07-26, by haftmann
updated;
2006-07-26, by wenzelm
fixed LaTeX problem;
2006-07-26, by wenzelm
added eval_term
2006-07-26, by haftmann
Removed wrong sentence (Simon Funke)
2006-07-26, by nipkow
moved pprint functions to Isar/proof_display.ML;
2006-07-26, by wenzelm
Tactical operations depending on local subgoal structure.
2006-07-26, by wenzelm
moved pprint functions to Isar/proof_display.ML;
2006-07-26, by wenzelm
export goal_tac (was internal refine_tac);
2006-07-26, by wenzelm
added Pure/subgoal.ML;
2006-07-26, by wenzelm
updated;
2006-07-25, by wenzelm
raw symbols: disallow dot to avoid confusion in NameSpace.unpack;
2006-07-25, by wenzelm
avoid Term.is_funtype;
2006-07-25, by wenzelm
avoid structure Char;
2006-07-25, by wenzelm
added variant_abs (from term.ML);
2006-07-25, by wenzelm
added find_free (from term.ML);
2006-07-25, by wenzelm
added is/to_ascii_lower/upper;
2006-07-25, by wenzelm
is_funtype: do not export internal operation;
2006-07-25, by wenzelm
tuned;
2006-07-25, by wenzelm
use Term.add_vars instead of obsolete term_varnames;
2006-07-25, by wenzelm
renamed add_term_varnames to Term.add_varnames (cf. Term.add_vars etc.);
2006-07-25, by wenzelm
tuned ML code;
2006-07-25, by wenzelm
renamed Term.variant_abs to Syntax.variant_abs;
2006-07-25, by wenzelm
Drule.merge_rules;
2006-07-25, by wenzelm
renamed Name.give_names to Name.names and moved Name.alphanum to Symbol.alphanum
2006-07-25, by haftmann
improvements for lazy code generation
2006-07-25, by haftmann
fixed typo
2006-07-25, by haftmann
added code generator serialization for Char
2006-07-25, by haftmann
added notes on class_package.ML and codegen_package.ML
2006-07-25, by haftmann
small adjustments
2006-07-23, by haftmann
fixed bug for serialization for uminus on ints
2006-07-23, by haftmann
small improvement in serialization for wfrec
2006-07-23, by haftmann
added structure HOList
2006-07-23, by haftmann
major simplifications for integers
2006-07-23, by haftmann
tactic for prove_instance_arity now gets definition theorems as arguments
2006-07-23, by haftmann
added term_of_string function
2006-07-21, by haftmann
simplification for code generation for Integers
2006-07-21, by haftmann
adaption to argument change in primrec_package
2006-07-21, by haftmann
adaption to changes in class_package
2006-07-21, by haftmann
hooks now take string list as arguments (mutual datatypes); some nice combinators in datatype_codegen
2006-07-21, by haftmann
exported equation transformator
2006-07-21, by haftmann
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
less
more
|
(0)
-10000
-1920
+1920
+10000
+30000
tip