Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-10000
-3000
-1000
-448
+448
+1000
+3000
+10000
+30000
tip
Find changesets by keywords (author, files, the commit message), revision number or hash, or
revset expression
.
The revision graph only works with JavaScript-enabled browsers.
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
less
more
|
(0)
-10000
-3000
-1000
-448
+448
+1000
+3000
+10000
+30000
tip