Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-10000
-3000
-1000
-384
+384
+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.
added lemma fresh_right, which is useful
2006-05-03, by urbanc
added the_theory;
2006-05-02, by wenzelm
extend/remove_syntax: observe inout flag for translations, too;
2006-05-02, by wenzelm
handle exception SYS_ERROR;
2006-05-02, by wenzelm
abbreviation: observe local syntax mode;
2006-05-02, by wenzelm
added set_syntax_mode, restore_syntax_mode;
2006-05-02, by wenzelm
sys_error: exception SYS_ERROR;
2006-05-02, by wenzelm
maintain implicit syntax mode;
2006-05-02, by wenzelm
ThyInfo.the_theory;
2006-05-02, by wenzelm
ThyInfo.the_theory;
2006-05-02, by wenzelm
actually removed old stuff;
2006-05-02, by wenzelm
replaced syntax/translations by abbreviation;
2006-05-02, by wenzelm
replaced syntax/translations by abbreviation;
2006-05-02, by wenzelm
replaced syntax/translations by abbreviation;
2006-05-02, by wenzelm
beta_eta_conversion added to pre_cnf_tac
2006-05-02, by webertj
added obfuscation for mails
2006-05-02, by haftmann
tidied and harmonized "params_of_state"
2006-05-02, by paulson
tuned;
2006-05-02, by wenzelm
tuned;
2006-05-02, by wenzelm
added domain_error;
2006-05-02, by wenzelm
of_sort: option;
2006-05-02, by wenzelm
some facts about min, max and add, diff
2006-05-01, by paulson
a few more examples
2006-05-01, by paulson
class_triv: Sign.certify_class;
2006-05-01, by wenzelm
arities: maintain original codomain;
2006-05-01, by wenzelm
added sort_triv;
2006-05-01, by wenzelm
of_sort: simplified derivation;
2006-05-01, by wenzelm
adapted arities;
2006-05-01, by wenzelm
add theorem flift2_defined_iff
2006-05-01, by huffman
add theorem typdef_flat
2006-05-01, by huffman
AxClass.define_class_i, AxClass.get_definition;
2006-04-30, by wenzelm
tuned;
2006-04-30, by wenzelm
AxClass.define_class;
2006-04-30, by wenzelm
build classes/arities: refer to operations in sorts.ML;
2006-04-30, by wenzelm
moved certify_class/sort to type.ML;
2006-04-30, by wenzelm
removed add_classes/classrel/arities (superceded by AxClass.axiomatize_class/classrel/arity);
2006-04-30, by wenzelm
added serial_string;
2006-04-30, by wenzelm
renamed add_axclass(_i) to define_axclass(_i);
2006-04-30, by wenzelm
AxClass.axiomatize_arity_i;
2006-04-30, by wenzelm
AxClass.define_class_i;
2006-04-30, by wenzelm
* Pure: axclasses now purely definitional;
2006-04-30, by wenzelm
reduced code duplication;
2006-04-29, by wenzelm
added insert_list;
2006-04-29, by wenzelm
added unconstrainT;
2006-04-29, by wenzelm
added unconstrainTs;
2006-04-29, by wenzelm
instances data: mutable cache;
2006-04-29, by wenzelm
tuned;
2006-04-29, by wenzelm
Capitalized theory names.
2006-04-28, by berghofe
Removed broken proof.
2006-04-28, by berghofe
Added Class, Fsub, and Lambda_mu examples for nominal datatypes.
2006-04-28, by berghofe
New keyword file for HOL nominal datatype package.
2006-04-28, by berghofe
Added new targets for nominal datatype package.
2006-04-28, by berghofe
Capitalized theory names.
2006-04-28, by berghofe
New ROOT file for nominal datatype examples.
2006-04-28, by berghofe
Renamed "nominal" theory to "Nominal".
2006-04-28, by berghofe
New ROOT file for nominal datatype package.
2006-04-28, by berghofe
added some helper files for HOL goals/lemmas. Clauses have TPTP format.
2006-04-28, by mengj
changed the functions for getting HOL helper clauses.
2006-04-28, by mengj
removed the functions for getting HOL helper paths.
2006-04-28, by mengj
SplitAt -> chop
2006-04-27, by berghofe
Adapted to new interface of add_axclass_i.
2006-04-27, by berghofe
added zip/take/drop lemmas
2006-04-27, by nipkow
tuned;
2006-04-27, by wenzelm
renamed Source.mapfilter to Source.map_filter;
2006-04-27, by wenzelm
added map_filter;
2006-04-27, by wenzelm
renamed mapfilter to map_filter, made pervasive (again);
2006-04-27, by wenzelm
tuned basic list operators (flat, maps, map_filter);
2006-04-27, by wenzelm
renamed HOLogic.mk_bin to mk_binum for consistency with dest_binum
2006-04-27, by paulson
slight shortening of blacklist
2006-04-27, by paulson
cosmetic changes
2006-04-27, by paulson
some new functions
2006-04-27, by paulson
isar-keywords.el
2006-04-27, by urbanc
*** empty log message ***
2006-04-26, by wenzelm
curried Seq.cons;
2006-04-26, by wenzelm
removed splitAt (superceded by chop);
2006-04-26, by wenzelm
tuned;
2006-04-26, by wenzelm
removed obsolete expand_case_tac;
2006-04-26, by wenzelm
fixed silly symlink bug
2006-04-26, by haftmann
added Ben Porter's stuff
2006-04-26, by kleing
moved arithmetic series to geometric series in SetInterval
2006-04-26, by kleing
Sign.arity_sorts;
2006-04-25, by wenzelm
unlocalize_mixfix: fallback on NoSyn;
2006-04-25, by wenzelm
tuned;
2006-04-25, by wenzelm
refer to structure Type instead of Sorts;
2006-04-25, by wenzelm
added inter_sort;
2006-04-25, by wenzelm
added remove_sort;
2006-04-25, by wenzelm
added arity_number/sorts;
2006-04-25, by wenzelm
made 'flat' pervasive (again);
2006-04-25, by wenzelm
get_info: removed 'super' field;
2006-04-25, by wenzelm
seperated typedef codegen from main code
2006-04-24, by haftmann
more precise tactics
2006-04-24, by haftmann
fixed typo
2006-04-24, by haftmann
more precise data structure
2006-04-24, by haftmann
cleaned up some diagnostic mathom
2006-04-24, by haftmann
moved coalesce to AList, added equality predicates to library
2006-04-24, by haftmann
added LP.thy
2006-04-23, by obua
Changed the treatment of equalities.
2006-04-22, by mengj
Changed the logic detection method.
2006-04-20, by mengj
exported linkup_logic_mode and changed the default setting
2006-04-19, by paulson
fix to spacing in switches, for Vampire under SML/NJ
2006-04-19, by paulson
definition expansion checks for excess variables
2006-04-19, by paulson
the "th" field of type "clause"
2006-04-19, by paulson
tidying and reformatting
2006-04-19, by paulson
tidying; ATP options including CASC mode for Vampire
2006-04-19, by paulson
Take conjectures and axioms as thms when convert them to ResHolClause.clause format.
2006-04-18, by mengj
Take conjectures and axioms as thms when convert them to ResClause.clause format.
2006-04-18, by mengj
Tidied up some programs.
2006-04-18, by mengj
fixed typo
2006-04-16, by haftmann
add lemma less_UU_iff as default simp rule
2006-04-13, by huffman
hide common name of constant 'run'
2006-04-13, by huffman
early test of Classpackage, Codegenerator;
2006-04-13, by wenzelm
fixed typo in method invocation;
2006-04-13, by wenzelm
ignore sort constraints of consts declarations;
2006-04-13, by wenzelm
ignore sort constraints of consts declarations;
2006-04-13, by wenzelm
add_axclass(_i): canonical specification format;
2006-04-13, by wenzelm
certify: ignore sort constraints of declarations (MAJOR CHANGE);
2006-04-13, by wenzelm
added print_theorems/theory, print_theorems_diff (from pure_thy.ML);
2006-04-13, by wenzelm
axclass: old-style concrete syntax for canonical specification format;
2006-04-13, by wenzelm
ProofDisplay.print_theorems/theory;
2006-04-13, by wenzelm
added maxidx_of;
2006-04-13, by wenzelm
tuned;
2006-04-13, by wenzelm
added typ_equiv;
2006-04-13, by wenzelm
moved print_theorems/theory to Isar/proof_display.ML;
2006-04-13, by wenzelm
added dest_conjunction_list;
2006-04-13, by wenzelm
export unflat (again);
2006-04-13, by wenzelm
use conjunction stuff from conjunction.ML;
2006-04-13, by wenzelm
expand_atom: Type.raw_match;
2006-04-13, by wenzelm
added equal_elim_rule2;
2006-04-13, by wenzelm
tuned comment;
2006-04-13, by wenzelm
ignore sorts of consts declarations;
2006-04-13, by wenzelm
reworded add_axclass(_i): canonical specification format,
2006-04-13, by wenzelm
added conjunction.ML;
2006-04-13, by wenzelm
Meta-level conjunction.
2006-04-13, by wenzelm
added conjunction.ML;
2006-04-13, by wenzelm
Sign.typ_equiv;
2006-04-13, by wenzelm
added subversion treatment
2006-04-13, by haftmann
classes: prefer thy operations;
2006-04-11, by wenzelm
export pretty_classrel/arity;
2006-04-11, by wenzelm
'axclass': no parameters;
2006-04-11, by wenzelm
tuned;
2006-04-11, by wenzelm
removed superclasses (see sign.ML);
2006-04-11, by wenzelm
added super_classes (from sorts.ML);
2006-04-11, by wenzelm
added mk_classrel, dest_classrel, mk_arities, dest_arity (from axclass.ML);
2006-04-11, by wenzelm
moved abstract syntax operations to logic.ML;
2006-04-11, by wenzelm
Moved stuff from Ring_and_Field to Matrix
2006-04-10, by obua
Adapted to changed type of add_typedef_i.
2006-04-10, by berghofe
Hoare(Parallel) dependencies on document/*
2006-04-10, by nipkow
added references
2006-04-10, by nipkow
Minimal doc
2006-04-10, by nipkow
Included cyclic list examples
2006-04-10, by nipkow
fixed value restriction
2006-04-10, by haftmann
Added splicing algorithm.
2006-04-10, by nipkow
hide (open) const;
2006-04-10, by wenzelm
simplified AxClass.add_axclass interface;
2006-04-10, by wenzelm
added aT (from axclass.ML);
2006-04-10, by wenzelm
removed unused class_le_path, sort_less;
2006-04-10, by wenzelm
add_axclass(_i): return class name only;
2006-04-10, by wenzelm
Term.itselfT;
2006-04-10, by wenzelm
Added function "splice"
2006-04-09, by nipkow
Even/Odd: avoid clash with even/odd of Main HOL;
2006-04-09, by wenzelm
results: smart_pretty_thm uses adhoc proof context if possible;
2006-04-09, by wenzelm
added full_name;
2006-04-09, by wenzelm
add_syntax: actually observe print mode;
2006-04-09, by wenzelm
print_term etc.: actually observe print mode in final output;
2006-04-09, by wenzelm
abbrevs: mode does not affect name space;
2006-04-09, by wenzelm
added coalesce;
2006-04-09, by wenzelm
moved theory presentation to Isar/ROOT.ML;
2006-04-09, by wenzelm
hide consts in Numeral.thy;
2006-04-09, by wenzelm
tuned syntax/abbreviations;
2006-04-09, by wenzelm
unfold(ed): not necessrily meta equations;
2006-04-09, by wenzelm
Made "empty" an abbreviation.
2006-04-09, by nipkow
*** empty log message ***
2006-04-09, by nipkow
Removed old set interval syntax.
2006-04-09, by nipkow
pretty_term: late externing of consts (support authentic syntax);
2006-04-08, by wenzelm
pretty: late externing of consts (support authentic syntax);
2006-04-08, by wenzelm
removed fix_mixfix;
2006-04-08, by wenzelm
abbreviation(_i): do not expand abbreviations, do not use derived_def;
2006-04-08, by wenzelm
add_abbrevs(_i): support print mode;
2006-04-08, by wenzelm
abbrevs: support print mode;
2006-04-08, by wenzelm
simplified handling of authentic syntax (cf. early externing in consts.ML);
2006-04-08, by wenzelm
'abbreviation': optional print mode;
2006-04-08, by wenzelm
tuned;
2006-04-08, by wenzelm
pretty_term': early vs. late externing (support authentic syntax);
2006-04-08, by wenzelm
print_theory: print abbreviations nicely;
2006-04-08, by wenzelm
added intern/extern/extern_early;
2006-04-08, by wenzelm
refined 'abbreviation';
2006-04-08, by wenzelm
made symlink relative
2006-04-08, by haftmann
made symlink relative
2006-04-08, by haftmann
converted Müller to Mueller to make smlnj 110.58 work
2006-04-08, by kleing
Fixed bug that caused proof of induction rule to fail
2006-04-07, by berghofe
remame ASeries to Arithmetic_Series
2006-04-07, by kleing
Added alternative version of thms_of_proof that does not recursively
2006-04-07, by berghofe
hash table now stores thm and get_clasimp_atp_lemmas returns thm rather than term.
2006-04-07, by mengj
filter now accepts axioms as thm, instead of term.
2006-04-07, by mengj
tptp_write_file accepts axioms as thm.
2006-04-07, by mengj
added another function for CNF.
2006-04-07, by mengj
lemmas returned from ResClasimp.get_clasimp_atp_lemmas are thm rather than term.
2006-04-07, by mengj
renamed ASeries to Arithmetic_Series, removed the ^M
2006-04-07, by kleing
modified the perm_compose rule such that it
2006-04-06, by urbanc
cleanup in typedef/datatype package
2006-04-06, by haftmann
added explicit serialization for int equality
2006-04-06, by haftmann
adapted for definitional code generation
2006-04-06, by haftmann
cleanup in datatype package
2006-04-06, by haftmann
small type annotation fix
2006-04-06, by haftmann
added hook for codegen_theorems.ML
2006-04-06, by haftmann
adaptions to change in typedef_package.ML
2006-04-06, by haftmann
added functions for definitional code generation
2006-04-06, by haftmann
added definitional code generator module: codegen_theorems.ML
2006-04-06, by haftmann
minor changes
2006-04-06, by haftmann
exported specification names
2006-04-06, by haftmann
minor extensions
2006-04-05, by haftmann
pool of constants; definition expansion; current best settings
2006-04-05, by paulson
removed some illegal characters: they were crashing SML/NJ
2006-03-31, by paulson
Removal of unused code
2006-03-31, by paulson
Simplified version of Jia's filter. Now all constants are pooled, rather than
2006-03-28, by paulson
renamed map_val to map_ran
2006-03-28, by schirmer
added map_val, superseding map_at and substitute
2006-03-28, by schirmer
some internal cleanup
2006-03-28, by haftmann
removed illegal character codes
2006-03-27, by paulson
simplified the proof at_fin_set_supp
2006-03-26, by urbanc
changed abbreviation for "infinite" back to translation because
2006-03-25, by nipkow
lazy patterns in lambda abstractions
2006-03-24, by huffman
changed the it_prm proof to work for recursion
2006-03-24, by urbanc
tuned some proofs
2006-03-24, by urbanc
Removed occurrences of makestring, which does not
2006-03-24, by berghofe
Converted translations to abbbreviations.
2006-03-23, by nipkow
Replaced iteration combinator by recursion combinator.
2006-03-23, by berghofe
detection of definitions of relevant constants
2006-03-23, by paulson
Only display atpset theorems if Output.show_debug_msgs is true.
2006-03-23, by mengj
added the first two simple proofs of the recursion
2006-03-22, by urbanc
comment fixed
2006-03-22, by webertj
Introduction of "whitelist": theorems forced past the relevance filter
2006-03-22, by paulson
Slight simplification of proofs
2006-03-22, by paulson
Removal of obsolete strategies. Initial support for locales: Frees and Consts
2006-03-22, by paulson
comment for conjI added
2006-03-22, by webertj
translations -> abbreviations (a cool feature)
2006-03-22, by nipkow
fixed example;
2006-03-21, by wenzelm
mark_boundT: produce well-typed term;
2006-03-21, by wenzelm
subtract (op =);
2006-03-21, by wenzelm
avoid polymorphic equality;
2006-03-21, by wenzelm
avoid polymorphic equality;
2006-03-21, by wenzelm
moved gen_eq_set to library.ML;
2006-03-21, by wenzelm
added ~$$ (negative literal);
2006-03-21, by wenzelm
avoid polymorphic equality;
2006-03-21, by wenzelm
remove (op =);
2006-03-21, by wenzelm
gen_eq_set, remove (op =);
2006-03-21, by wenzelm
abbreviation upto, length;
2006-03-21, by wenzelm
added subtract;
2006-03-21, by wenzelm
subtract (op =);
2006-03-21, by wenzelm
remove (op =);
2006-03-21, by wenzelm
Now SML/NJ-friendly (IntInf)
2006-03-21, by paulson
Removal of unnecessary simprules: simproc cancel_numerals now works without
2006-03-21, by paulson
interpret: Proof.assert_forward_or_chain;
2006-03-20, by wenzelm
subsetI is often necessary
2006-03-20, by paulson
Now the setup for cancel_numerals accepts mixed Sucs/+ where the Sucs no longer
2006-03-20, by paulson
Tuned signature of Locale.add_locale(_i).
2006-03-20, by ballarin
simplified mg_domain (use Sign.classes/arities_of);
2006-03-18, by wenzelm
made $$ and "this" monomorphic (string);
2006-03-18, by wenzelm
tuned;
2006-03-18, by wenzelm
export arities_of instead of classes_arities_of;
2006-03-18, by wenzelm
updated;
2006-03-18, by wenzelm
renamed const less to lt;
2006-03-18, by wenzelm
renamed constant less in lattice
2006-03-18, by haftmann
fixed problem with proof reconstruction by adding add_Suc to arith-simpset.
2006-03-17, by nipkow
added parser locale_expr_unless
2006-03-17, by schirmer
fixed clsvar bug
2006-03-17, by haftmann
add_locale(_i) returns internal locale name.
2006-03-17, by ballarin
added example for operational classes and code generator
2006-03-17, by haftmann
slight improvement in serializer, stub for code generator theorems added
2006-03-17, by haftmann
Renamed setsum_mult to setsum_right_distrib.
2006-03-17, by ballarin
Internal restructuring: local parameters.
2006-03-17, by ballarin
renamed op < <= to Orderings.less(_eq)
2006-03-17, by haftmann
New interface function parameters_of_expr.
2006-03-16, by ballarin
add_inst_arity_i renamed to prove_arity.
2006-03-15, by berghofe
rename_frees: treat trivial names;
2006-03-15, by wenzelm
added singleton;
2006-03-14, by wenzelm
updated;
2006-03-14, by wenzelm
turned string_of_mixfix into pretty_mixfix;
2006-03-14, by wenzelm
added monomorphic;
2006-03-14, by wenzelm
added 'print_statement' command;
2006-03-14, by wenzelm
added print_stmts;
2006-03-14, by wenzelm
added pretty_statement;
2006-03-14, by wenzelm
added command, keyword;
2006-03-14, by wenzelm
Output.add_mode: keyword component;
2006-03-14, by wenzelm
string_of_mixfix;
2006-03-14, by wenzelm
print_statement;
2006-03-14, by wenzelm
added remove_trrules(_i);
2006-03-14, by wenzelm
added is_elim (from Provers/classical.ML);
2006-03-14, by wenzelm
added 'no_translations';
2006-03-14, by wenzelm
added pretty_stmt;
2006-03-14, by wenzelm
declared_const: check for type constraint only, i.e. admit abbreviations as well;
2006-03-14, by wenzelm
ObjectLogic.is_elim;
2006-03-14, by wenzelm
tuned constdecl;
2006-03-14, by wenzelm
updated;
2006-03-14, by wenzelm
Pure: no_translations;
2006-03-14, by wenzelm
refined representation of instance dictionaries
2006-03-14, by haftmann
entry for Library/AssocList
2006-03-13, by schirmer
First version of function for defining graph of iteration combinator.
2006-03-13, by berghofe
got rid of type Sign.sg;
2006-03-11, by wenzelm
renamed plus to add;
2006-03-11, by wenzelm
renamed const minus to subtract;
2006-03-11, by wenzelm
simplified AxClass interfaces;
2006-03-11, by wenzelm
added axclass_instance_XXX (from axclass.ML);
2006-03-11, by wenzelm
*** empty log message ***
2006-03-11, by wenzelm
added read_class, read/cert_classrel/arity (from axclass.ML);
2006-03-11, by wenzelm
moved read_class, read/cert_classrel/arity to sign.ML;
2006-03-11, by wenzelm
use axclass.ML earlier (in Isar/ROOT.ML);
2006-03-11, by wenzelm
nbe: no_document;
2006-03-11, by wenzelm
tuned;
2006-03-10, by wenzelm
exporting reapAll and killChild
2006-03-10, by paulson
text delimiter fixed
2006-03-10, by webertj
comment delimiter fixed
2006-03-10, by webertj
clauses now use (meta-)hyps instead of (meta-)implications; significant speedup
2006-03-10, by webertj
fix for document preparation
2006-03-10, by haftmann
Added Library/AssocList.thy
2006-03-10, by schirmer
renamed HOL + - * etc. to HOL.plus HOL.minus HOL.times etc.
2006-03-10, by haftmann
Changed some warnings to debug messages
2006-03-10, by paulson
Frequency analysis of constants (with types).
2006-03-10, by paulson
Shortened the exception messages from assume.
2006-03-10, by mengj
METAHYPS catches THM assume exception and prints out the terms containing schematic vars.
2006-03-10, by mengj
added many simple lemmas
2006-03-10, by huffman
Added more functions to the signature and tidied up some functions.
2006-03-09, by mengj
tuned;
2006-03-08, by wenzelm
tuned some proofs
2006-03-08, by urbanc
select_goals: split original conjunctions;
2006-03-08, by wenzelm
method: goal restriction defaults to [1];
2006-03-08, by wenzelm
infer_derivs: avoid allocating empty MinProof;
2006-03-08, by wenzelm
tuned;
2006-03-08, by wenzelm
Isar/method: goal restriction;
2006-03-08, by wenzelm
constdecl: always allow 'where';
2006-03-08, by wenzelm
deleted some proofs "on comment"
2006-03-08, by urbanc
tuned some proofs
2006-03-08, by urbanc
tuned some of the proofs about fresh_fun
2006-03-08, by urbanc
first running version of type classes
2006-03-08, by haftmann
first running version of type classes
2006-03-08, by haftmann
first running version of type classes
2006-03-08, by haftmann
Frequency strategy. Revised indentation, etc.
2006-03-08, by paulson
*** empty log message ***
2006-03-08, by nipkow
added ROOT.ML
2006-03-07, by obua
Indentation
2006-03-07, by paulson
Tidying and restructuring.
2006-03-07, by paulson
Tidying and tracing. Handling exn CLAUSE so that errors don't reach top-level.
2006-03-07, by paulson
Tidying. clausify_rules_pairs_abs now returns clauses in the same order as before.
2006-03-07, by paulson
Tidying. New invoke_atp_ml for top-level debugging. Flag to force FOL mode.
2006-03-07, by paulson
Tidying, and getting rid of SELECT_GOAL (as it does something different now)
2006-03-07, by paulson
Added HOL-ZF to Isabelle.
2006-03-07, by obua
substantial improvement in codegen iml
2006-03-07, by haftmann
Function get_clasimp_atp_lemmas gets all lemmas from claset, simpet and atpset.
2006-03-07, by mengj
relevance_filter takes input axioms as Term.term.
2006-03-07, by mengj
Proof reconstruction now only takes names of theorems as input.
2006-03-07, by mengj
Added tptp_write_file to write all necessary ATP input clauses to one file.
2006-03-07, by mengj
tptp_write_file now takes goals and axioms as Term.term and writes them to a file.
2006-03-07, by mengj
Added functions to retrieve local and global atpset rules.
2006-03-07, by mengj
Moved the settings for ATP time limit to res_atp.ML
2006-03-07, by mengj
Merged res_atp_setup.ML into res_atp.ML.
2006-03-07, by mengj
When ATP methods call ATPs, all input clauses from one subgoal are written to one file.
2006-03-07, by mengj
Merged res_atp_setup.ML into res_atp.ML.
2006-03-07, by mengj
SELECT_GOAL: fixed trivial case;
2006-03-05, by wenzelm
fixed a typo in a comment
2006-03-05, by webertj
tuned;
2006-03-04, by wenzelm
method: SelectGoals;
2006-03-04, by wenzelm
method: syntax for SelectGoals;
2006-03-04, by wenzelm
text: added SelectGoals;
2006-03-04, by wenzelm
tuned conj_curry;
2006-03-04, by wenzelm
added extract, retrofit;
2006-03-04, by wenzelm
added mk_conjunction;
2006-03-04, by wenzelm
method: restriction to first n sub-goals;
2006-03-04, by wenzelm
minor changes
2006-03-03, by nipkow
more examples
2006-03-03, by nipkow
changed and retracted change of location of code lemmas.
2006-03-03, by nipkow
ignore repeated vars on lhs, cleanup
2006-03-03, by nipkow
improvements for nbe
2006-03-03, by haftmann
reformatting
2006-03-02, by paulson
subset_refl now included using the atp attribute
2006-03-02, by paulson
moved the "use" directive
2006-03-02, by paulson
fixed the bugs itroduced by the previous commit
2006-03-02, by urbanc
made some small changes to generate nicer latex-output
2006-03-02, by urbanc
split the files
2006-03-02, by urbanc
Added in a signature.
2006-03-02, by mengj
fixed a problem where a permutation is not analysed
2006-03-01, by urbanc
streamlined the proof
2006-03-01, by urbanc
refined representation of codegen intermediate language
2006-03-01, by haftmann
some small tunings
2006-03-01, by urbanc
added fresh_fun_eqvt theorem to the theorem collection
2006-03-01, by urbanc
less
more
|
(0)
-10000
-3000
-1000
-384
+384
+1000
+3000
+10000
+30000
tip