Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-10000
-3000
-1000
-480
+480
+1000
+3000
+10000
+30000
tip
Find changesets by keywords (author, files, the commit message), revision number or hash, or
revset expression
.
The revision graph only works with JavaScript-enabled browsers.
type local_theory;
2006-02-06, by wenzelm
norm_term: Sign.const_expansion, Envir.expand_atom;
2006-02-06, by wenzelm
TableFun: renamed xxx_multi to xxx_list;
2006-02-06, by wenzelm
type local_theory = Proof.context;
2006-02-06, by wenzelm
cert_def: use Logic.dest_def;
2006-02-06, by wenzelm
Toplevel.local_theory;
2006-02-06, by wenzelm
LocalDefs.cert_def;
2006-02-06, by wenzelm
eq_prop: Envir.beta_eta_contract;
2006-02-06, by wenzelm
renamed xxx_multi to xxx_list;
2006-02-06, by wenzelm
moved combound, rlist_abs to logic.ML;
2006-02-06, by wenzelm
union_tpairs: Library.merge;
2006-02-06, by wenzelm
moved no_vars to sign.ML;
2006-02-06, by wenzelm
lambda: abstract over any const;
2006-02-06, by wenzelm
added add_abbrevs(_i);
2006-02-06, by wenzelm
moved (beta_)eta_contract to envir.ML;
2006-02-06, by wenzelm
tuned;
2006-02-06, by wenzelm
added generic dest_def (mostly from theory.ML);
2006-02-06, by wenzelm
added (beta_)eta_contract (from pattern.ML);
2006-02-06, by wenzelm
print_theory: const abbreviations;
2006-02-06, by wenzelm
added abbreviations;
2006-02-06, by wenzelm
load envir.ML and logic.ML early;
2006-02-06, by wenzelm
Logic.rlist_abs;
2006-02-06, by wenzelm
Logic.const_of_class/class_of_const;
2006-02-06, by wenzelm
TableFun: renamed xxx_multi to xxx_list;
2006-02-06, by wenzelm
replaced Symtab.merge_multi by local merge_rules;
2006-02-06, by wenzelm
Envir.(beta_)eta_contract;
2006-02-06, by wenzelm
subsituted gen_duplicates / has_duplicates for duplicates whenever appropriate
2006-02-06, by haftmann
added strip_abs
2006-02-06, by haftmann
clarified semantics of merge
2006-02-06, by haftmann
speedup: use simproc for AC rules
2006-02-04, by huffman
UU_reorient_simproc no longer rewrites UU = numeral
2006-02-04, by huffman
removed obsolete gen_ins/mem;
2006-02-03, by wenzelm
removed add/del_rules;
2006-02-03, by wenzelm
canonical member/insert/merge;
2006-02-03, by wenzelm
removal of case analysis clauses
2006-02-03, by paulson
fix
2006-02-03, by haftmann
minor improvements
2006-02-03, by haftmann
refined signature of locale module
2006-02-03, by haftmann
no toplevel 'thy' anymore
2006-02-03, by haftmann
fix in codegen
2006-02-03, by haftmann
do not open structure;
2006-02-02, by wenzelm
reimplemented using Equiv_Relations.thy
2006-02-02, by huffman
improvement in devarifications
2006-02-02, by haftmann
alternative syntax for instances
2006-02-02, by haftmann
tuned;
2006-02-02, by wenzelm
consumes: negative argument relative to total number of prems;
2006-02-02, by wenzelm
added refine_insert;
2006-02-02, by wenzelm
Proof.refine_insert;
2006-02-02, by wenzelm
always use Attrib.src;
2006-02-02, by wenzelm
more generic type for map_specs/facts;
2006-02-02, by wenzelm
'obtains' element;
2006-02-02, by wenzelm
'obtain': optional case name;
2006-02-02, by wenzelm
index elements;
2006-02-02, by wenzelm
* Isar: 'obtains' element;
2006-02-02, by wenzelm
tuned msg;
2006-02-02, by wenzelm
theorem(_in_locale): Element.statement, Obtain.statement;
2006-02-02, by wenzelm
added parname;
2006-02-02, by wenzelm
obtain(_i): optional name for 'that';
2006-02-02, by wenzelm
tuned comments;
2006-02-02, by wenzelm
moved (general_)statement to outer_parse.ML;
2006-02-02, by wenzelm
added concluding statements: Shows/Obtains;
2006-02-02, by wenzelm
moved specific map_typ/term to sign.ML;
2006-02-02, by wenzelm
added specific map_typ/term (from term.ML);
2006-02-02, by wenzelm
Exporting recdef's hints for use by new recdef package
2006-02-02, by krauss
*_asms_of fixed.
2006-02-02, by ballarin
add 64bit atbroy98 platform
2006-02-02, by kleing
updated;
2006-02-01, by wenzelm
Added "evaluation" method and oracle.
2006-02-01, by berghofe
new and updated protocol proofs by Giamp Bella
2006-02-01, by paulson
substantial cleanup and simplifications
2006-02-01, by haftmann
name clarifications
2006-02-01, by haftmann
added map_entry_yield
2006-02-01, by haftmann
- renamed some lemmas (some had names coming from ancient
2006-02-01, by urbanc
added all constructors from PhD
2006-02-01, by urbanc
axiomatization: retrict parameters to occurrences in specs;
2006-01-31, by wenzelm
improved comments;
2006-01-31, by wenzelm
tuned LocalDefs.unfold;
2006-01-31, by wenzelm
(un)fold: removed '(raw)' option;
2006-01-31, by wenzelm
added consts_retricted;
2006-01-31, by wenzelm
(un)fold: no raw flag;
2006-01-31, by wenzelm
tuned;
2006-01-31, by wenzelm
tuned LocalTheory.pretty_consts;
2006-01-31, by wenzelm
(un)folded: removed '(raw)' option;
2006-01-31, by wenzelm
lambda: abstract over TYPE argument, too;
2006-01-31, by wenzelm
tuned comments;
2006-01-31, by wenzelm
removal of ResClause.num_of_clauses and other simplifications
2006-01-31, by paulson
working SPASS support; much tidying
2006-01-31, by paulson
added serialization for arbitrary
2006-01-31, by haftmann
minor change to CodegenPackage interface
2006-01-31, by haftmann
minor cleanups
2006-01-31, by haftmann
more coherent lookup extraction functions
2006-01-31, by haftmann
reorganization of code to support DFG otuput
2006-01-31, by paulson
* Pure: 'advanced' translation functions use Context.generic instead of just theory;
2006-01-31, by wenzelm
declare defn rules;
2006-01-31, by wenzelm
all styles now reset to defaults first, i.e. the document may switch styles back and forth;
2006-01-31, by wenzelm
export meta_rewrite_rule;
2006-01-31, by wenzelm
advanced translations: Context.generic;
2006-01-31, by wenzelm
advanced translations: Context.generic;
2006-01-31, by wenzelm
tidy-up of res_clause.ML, removing the "predicates" field
2006-01-30, by paulson
'setup': no list type, support implicit setup;
2006-01-30, by wenzelm
'fixes': support plain vars;
2006-01-30, by wenzelm
fixed a syntax error!
2006-01-30, by paulson
replaced gen_list by enum
2006-01-30, by haftmann
adaptions to codegen_package
2006-01-30, by haftmann
various improvements
2006-01-30, by haftmann
added three times overloaded Isar instance command
2006-01-30, by haftmann
moved instance Isar command to class_package.ML
2006-01-30, by haftmann
added map_atype, map_aterms
2006-01-30, by haftmann
tuned proof;
2006-01-29, by wenzelm
declare atomize/defn for Ball;
2006-01-29, by wenzelm
invent_fixes: merely enter body temporarily;
2006-01-29, by wenzelm
'unfolding': LocalDefs.unfold;
2006-01-29, by wenzelm
moved treatment of object-logic equalities to local_defs.ML;
2006-01-29, by wenzelm
method (un)folded: option '(raw)';
2006-01-29, by wenzelm
added attributes defn_add/del;
2006-01-29, by wenzelm
added 'defn' attribute;
2006-01-29, by wenzelm
proper order of trfuns;
2006-01-29, by wenzelm
CPure: Context.add_setup;
2006-01-29, by wenzelm
tuned proofs;
2006-01-29, by wenzelm
implicit setup;
2006-01-29, by wenzelm
default rule step: norm_hhf_tac;
2006-01-29, by wenzelm
tuned comment;
2006-01-29, by wenzelm
declare 'defn' rules;
2006-01-29, by wenzelm
LocalDefs;
2006-01-28, by wenzelm
Basic operations on local definitions.
2006-01-28, by wenzelm
removed unnecessary Syntax.fix_mixfix;
2006-01-28, by wenzelm
added axiomatization_loc, definition_loc;
2006-01-28, by wenzelm
moved local defs to local_defs.ML;
2006-01-28, by wenzelm
LocalDefs;
2006-01-28, by wenzelm
removed unatomize;
2006-01-28, by wenzelm
(un)fold: support object-level rewrites;
2006-01-28, by wenzelm
added print_consts;
2006-01-28, by wenzelm
removed obsolete keyword 'files';
2006-01-28, by wenzelm
(un)folded: support object-level rewrites;
2006-01-28, by wenzelm
added equals_cong;
2006-01-28, by wenzelm
added Isar/local_defs.ML;
2006-01-28, by wenzelm
LocalDefs.add_def;
2006-01-28, by wenzelm
LocalDefs.def_export;
2006-01-28, by wenzelm
tuned proofs;
2006-01-28, by wenzelm
Pure/Isar: (un)folded, (un)fold, unfolding support
2006-01-28, by wenzelm
interrupt_timeout for Poly replaced by stub
2006-01-27, by webertj
added atomize_iff;
2006-01-27, by wenzelm
renamed Pretty.gen_list to Pretty.enum;
2006-01-27, by wenzelm
swapped theory_context;
2006-01-27, by wenzelm
swapped Toplevel.theory_context;
2006-01-27, by wenzelm
added invent_fixes;
2006-01-27, by wenzelm
swapped Toplevel.theory_context;
2006-01-27, by wenzelm
renamed reverse_atomize to unatomize;
2006-01-27, by wenzelm
init: include view;
2006-01-27, by wenzelm
improved 'notes', including proper treatment of locale results;
2006-01-27, by wenzelm
swapped Toplevel.theory_context;
2006-01-27, by wenzelm
Locale.init;
2006-01-27, by wenzelm
renamed gen_list to enum;
2006-01-27, by wenzelm
moved theorem tags from Drule to PureThy;
2006-01-27, by wenzelm
added ProofContext.pprint_context (depends on ProofContext.debug);
2006-01-27, by wenzelm
moved theorem tags from Drule to PureThy;
2006-01-27, by wenzelm
tidying up SPASS output
2006-01-27, by paulson
tidying
2006-01-27, by paulson
better reporting
2006-01-27, by paulson
Interface to access the specification of a named locale.
2006-01-27, by ballarin
Added new file Tools/ATP/reduce_axiomsN.ML
2006-01-27, by mengj
Added in new file Tools/ATP/reduce_axiomsN.ML
2006-01-27, by mengj
Changed codes that call relevance filter.
2006-01-27, by mengj
Relevance filtering. Has replaced the previous version.
2006-01-27, by mengj
interrupt_timeout now raises Interrupt instead of SML90.Interrupt
2006-01-26, by webertj
smaller example to prevent timeout
2006-01-26, by webertj
Fixed bug in code generator for primitive definitions that
2006-01-26, by berghofe
Inductive sets with no introduction rules are now allowed as well.
2006-01-26, by berghofe
added definition(_i);
2006-01-25, by wenzelm
renamed export to export_standard (again!), because it includes Drule.local_standard';
2006-01-25, by wenzelm
ProofContext.export_standard;
2006-01-25, by wenzelm
tuned atomize_cterm;
2006-01-25, by wenzelm
turned abstract_term into ProofContext.abs_def;
2006-01-25, by wenzelm
added constant definition;
2006-01-25, by wenzelm
added 'definition';
2006-01-25, by wenzelm
tuned comment;
2006-01-25, by wenzelm
export name_multi;
2006-01-25, by wenzelm
abs_def: improved error;
2006-01-25, by wenzelm
ObjectLogic.atomize_cterm;
2006-01-25, by wenzelm
updated;
2006-01-25, by wenzelm
works with DPLL solver now
2006-01-24, by webertj
the additional freshness-condition in the one-induction
2006-01-24, by urbanc
fixed code_generate syntax;
2006-01-24, by wenzelm
renamed axiomatize(_i) to axiomatization(_i);
2006-01-24, by wenzelm
renamed inferred_type to inferred_param;
2006-01-24, by wenzelm
ProofContext.inferred_param;
2006-01-24, by wenzelm
removed the_params;
2006-01-24, by wenzelm
added actual operations;
2006-01-24, by wenzelm
axiomatization: optional vars;
2006-01-24, by wenzelm
LocalTheory.pretty_consts;
2006-01-24, by wenzelm
tuned;
2006-01-24, by wenzelm
add_finals: prep_consts, i.e. varify type;
2006-01-24, by wenzelm
added dest_all;
2006-01-24, by wenzelm
TimeLimit replaced by interrupt_timeout
2006-01-23, by webertj
TimeLimit replaced by interrupt_timeout
2006-01-23, by webertj
Updated to Isabelle 2006-01-23
2006-01-23, by krauss
made change for ex1
2006-01-23, by urbanc
removed problematic keyword 'atom'
2006-01-23, by haftmann
more general serializer
2006-01-23, by haftmann
slight steps forward
2006-01-23, by haftmann
exported after_qed for axclass instance
2006-01-23, by haftmann
ResClasimp.get_clasimp_lemmas now takes all subgoals rather than only the first
2006-01-23, by paulson
Clausification now handles some IFs in rewrite rules (if-split did not work)
2006-01-23, by paulson
bugfix: induct_tac no longer raises THM "dest_state"
2006-01-23, by paulson
fixed the <<= notation
2006-01-23, by paulson
replacement of bool by a datatype (making problems first-order). More lemma names
2006-01-23, by paulson
Fixed a bug.
2006-01-23, by mengj
no essential changes
2006-01-22, by urbanc
made the change for setup-functions not returning functions
2006-01-22, by urbanc
a fixme comments about abs_fun_if, which should be called perm_if
2006-01-22, by urbanc
Local theory operations, with optional target locale.
2006-01-22, by wenzelm
added restore_body;
2006-01-22, by wenzelm
added the_params;
2006-01-22, by wenzelm
tuned order;
2006-01-22, by wenzelm
added Isar/local_theory.ML;
2006-01-22, by wenzelm
Ensure dereference is delayed.
2006-01-21, by mengj
tuned;
2006-01-21, by wenzelm
* ML: simplified type attribute;
2006-01-21, by wenzelm
simplified type attribute;
2006-01-21, by wenzelm
removed duplicate type_solver (cf. Tools/typechk.ML);
2006-01-21, by wenzelm
simplified type attribute;
2006-01-21, by wenzelm
simplified type attribute;
2006-01-21, by wenzelm
simplified type attribute;
2006-01-21, by wenzelm
rename map_theory/proof to theory/proof_map;
2006-01-21, by wenzelm
tuned proofs;
2006-01-21, by wenzelm
simplified type attribute;
2006-01-21, by wenzelm
simplified type attribute;
2006-01-21, by wenzelm
type information is now also printed.
2006-01-20, by mengj
added some debugging code.
2006-01-20, by mengj
fixed a bug
2006-01-20, by mengj
quote "atom";
2006-01-19, by wenzelm
updated;
2006-01-19, by wenzelm
* ML/Isar: theory setup has type (theory -> theory);
2006-01-19, by wenzelm
use/use_thy: Output.toplevel_errors;
2006-01-19, by wenzelm
added basic syntax;
2006-01-19, by wenzelm
moved pure syntax to Syntax/syntax.ML and pure_thy.ML;
2006-01-19, by wenzelm
keep: disable Output.toplevel_errors;
2006-01-19, by wenzelm
run_thy: removed Output.toplevel_errors;
2006-01-19, by wenzelm
added ML_errors;
2006-01-19, by wenzelm
use: Output.ML_errors;
2006-01-19, by wenzelm
Syntax.basic_syn;
2006-01-19, by wenzelm
setup: theory -> theory;
2006-01-19, by wenzelm
tuned setmp;
2006-01-19, by wenzelm
setup: theory -> theory;
2006-01-19, by wenzelm
tuned comments;
2006-01-19, by wenzelm
setup: theory -> theory;
2006-01-19, by wenzelm
setup: theory -> theory;
2006-01-19, by wenzelm
Use generic Simplifier.simp_add attribute instead
2006-01-19, by berghofe
Re-inserted consts_code declaration accidentally deleted
2006-01-19, by berghofe
strengthened some lemmas; simplified some proofs
2006-01-19, by paulson
substantial improvement in serialization handling
2006-01-18, by haftmann
fixed one proof that broke because of the changes
2006-01-18, by urbanc
substantial improvements in code generator
2006-01-17, by haftmann
these hacks are no longer needed
2006-01-17, by paulson
improved SPASS support
2006-01-17, by paulson
case_result: drop_schematic, i.e. be permissive about illegal binds;
2006-01-16, by wenzelm
put_facts: do not pretend local thms were named;
2006-01-16, by wenzelm
declare the1_equality [elim?];
2006-01-16, by wenzelm
tuned;
2006-01-15, by wenzelm
tuned;
2006-01-15, by wenzelm
* Classical: optional weight for attributes;
2006-01-15, by wenzelm
guess: used fixed inferred_type of vars;
2006-01-15, by wenzelm
export add_args;
2006-01-15, by wenzelm
attributes: optional weight;
2006-01-15, by wenzelm
classical attributes: optional weight;
2006-01-15, by wenzelm
prefer ex1I over ex_ex1I in single-step reasoning;
2006-01-15, by wenzelm
generic attributes;
2006-01-14, by wenzelm
tuned;
2006-01-14, by wenzelm
* ML/Isar: simplified treatment of user-level errors;
2006-01-14, by wenzelm
sane ERROR vs. TOPLEVEL_ERROR handling;
2006-01-14, by wenzelm
added Isar.toplevel;
2006-01-14, by wenzelm
Output.error_msg;
2006-01-14, by wenzelm
removed special ERROR handling stuff (transform_error etc.);
2006-01-14, by wenzelm
added exception ERROR, error, cat_error, sys_error, assert, deny, assert_all;
2006-01-14, by wenzelm
Output.debug;
2006-01-14, by wenzelm
generated code: raise Match instead of ERROR;
2006-01-14, by wenzelm
sane ERROR handling;
2006-01-14, by wenzelm
blacklist experiments
2006-01-13, by paulson
more readable divide ops
2006-01-13, by paulson
more practical time limit
2006-01-13, by paulson
*** empty log message ***
2006-01-13, by nipkow
mixfix: added Structure;
2006-01-13, by wenzelm
uniform handling of fixes: read/cert_vars, add_fixes(_i), body flag;
2006-01-13, by wenzelm
uniform handling of fixes;
2006-01-13, by wenzelm
uniform handling of fixes;
2006-01-13, by wenzelm
uniform handling of fixes;
2006-01-13, by wenzelm
uniform handling of fixes;
2006-01-13, by wenzelm
tuned;
2006-01-13, by wenzelm
generic_setup: optional argument, defaults to Context.setup();
2006-01-13, by wenzelm
added map_theory, map_proof;
2006-01-13, by wenzelm
removed obsolete sign_of;
2006-01-13, by wenzelm
implicit setup, which admits exception_trace;
2006-01-13, by wenzelm
ProofContext.def_export;
2006-01-13, by wenzelm
updated to new induction principle
2006-01-11, by urbanc
cahges to use the new induction-principle (now proved in
2006-01-11, by urbanc
changes to make use of the new induction principle proved by
2006-01-11, by urbanc
Implemented proof of (strong) induction rule.
2006-01-11, by berghofe
Added theorem at_finite_select.
2006-01-11, by berghofe
added lemmas perm_empty, perm_insert to do with
2006-01-11, by urbanc
merged the silly lemmas into the eqvt proof of subtype
2006-01-11, by urbanc
tuned proofs
2006-01-11, by urbanc
tuned the eqvt-proof
2006-01-11, by urbanc
rolled back the last addition since these lemmas were already
2006-01-11, by urbanc
added the thms-collection "pt_id" (collection of all pt_<ak>1 lemmas)
2006-01-11, by urbanc
tuned
2006-01-11, by urbanc
tidied, and added missing thm divide_less_eq_1_neg
2006-01-11, by paulson
tidied, and giving theorems names
2006-01-11, by paulson
add transitivity rules
2006-01-11, by huffman
tuned;
2006-01-11, by wenzelm
updated;
2006-01-11, by wenzelm
tuned;
2006-01-10, by wenzelm
generic attributes;
2006-01-10, by wenzelm
* ML: generic context, data, attributes;
2006-01-10, by wenzelm
added context_of -- generic context;
2006-01-10, by wenzelm
generic attributes;
2006-01-10, by wenzelm
print rules: generic context;
2006-01-10, by wenzelm
Specification.pretty_consts ctxt;
2006-01-10, by wenzelm
generic data and attributes;
2006-01-10, by wenzelm
added rule, declaration;
2006-01-10, by wenzelm
added generic syntax;
2006-01-10, by wenzelm
tuned dependencies;
2006-01-10, by wenzelm
added declaration_attribute;
2006-01-10, by wenzelm
support for generic contexts with data;
2006-01-10, by wenzelm
fix_tac: no warning;
2006-01-10, by wenzelm
generic attributes;
2006-01-10, by wenzelm
Attrib.rule;
2006-01-10, by wenzelm
tuned
2006-01-10, by urbanc
added the lemmas supp_char and supp_string
2006-01-10, by urbanc
added some lemmas to the collection "abs_fresh"
2006-01-09, by urbanc
_E suffix for compatibility with AddIffs
2006-01-09, by paulson
tidied
2006-01-09, by paulson
simplified the special-case simprules
2006-01-09, by paulson
theorems need names
2006-01-09, by paulson
commented the transitivity and narrowing proof
2006-01-09, by urbanc
Theory specifications --- with type-inference, but no internal polymorphism.
2006-01-07, by wenzelm
added infer_type, declared_type;
2006-01-07, by wenzelm
added param, spec, named_spec;
2006-01-07, by wenzelm
added init;
2006-01-07, by wenzelm
added 'axiomatization';
2006-01-07, by wenzelm
Specification.pretty_consts;
2006-01-07, by wenzelm
gen_names: preserve empty names;
2006-01-07, by wenzelm
added Isar/specification.ML;
2006-01-07, by wenzelm
updated;
2006-01-07, by wenzelm
another change for the new induct-method
2006-01-07, by urbanc
RuleCases.make_nested;
2006-01-07, by wenzelm
support nested cases;
2006-01-07, by wenzelm
support nested cases;
2006-01-07, by wenzelm
RuleCases.make_common;
2006-01-07, by wenzelm
pretty_locale: backquote notes;
2006-01-07, by wenzelm
RuleCases.make_simple;
2006-01-07, by wenzelm
tuned order;
2006-01-07, by wenzelm
added backquote;
2006-01-07, by wenzelm
RuleCases.make_common/nested;
2006-01-07, by wenzelm
* Provers/induct: improved simultaneous goals -- nested cases;
2006-01-07, by wenzelm
added private datatype nprod (copy of prod) to be
2006-01-07, by urbanc
changed PRO_RED proof to conform with the new induction rules
2006-01-07, by urbanc
prep_meta_eq: reuse mk_rews of local simpset;
2006-01-06, by wenzelm
removed obsolete eqrule_HOL_data.ML;
2006-01-06, by wenzelm
removed obsolete eqrule_FOL_data.ML;
2006-01-06, by wenzelm
simplified EqSubst setup;
2006-01-06, by wenzelm
obsolete, reuse mk_rews of local simpset;
2006-01-06, by wenzelm
Toplevel.theory_to_proof;
2006-01-06, by wenzelm
transactions now always see quasi-functional intermediate checkpoint;
2006-01-06, by wenzelm
tuned EqSubst setup;
2006-01-06, by wenzelm
Pure/Isar: Toplevel.theory_to_proof admits transactions that modify the theory;
2006-01-06, by wenzelm
hide type datatype node;
2006-01-05, by wenzelm
tuned print_theorems_theory;
2006-01-05, by wenzelm
Toplevel.proof_position_of;
2006-01-05, by wenzelm
store_thm: transfer to current context, i.e. the target theory;
2006-01-05, by wenzelm
replaced swap by contrapos_np;
2006-01-05, by wenzelm
added setminus;
2006-01-05, by wenzelm
proper handling of simultaneous goals and mutual rules;
2006-01-05, by wenzelm
provide projections of induct_weak, induct_unsafe;
2006-01-05, by wenzelm
added strict_mutual_rule;
2006-01-05, by wenzelm
RuleCases.strict_mutual_rule;
2006-01-05, by wenzelm
changed the name of the type "nOption" to "noption".
2006-01-05, by urbanc
added "fresh_singleton" lemma
2006-01-04, by urbanc
added more documentation; will now try out a modification
2006-01-04, by urbanc
Reversed Larry's option/iff change.
2006-01-04, by nipkow
substantial additions using locales
2006-01-04, by haftmann
exported read|cert_arity interfaces
2006-01-04, by haftmann
trace_simp_depth_limit is 1 by default
2006-01-04, by nipkow
removed pointless trace msg.
2006-01-04, by nipkow
preservation of names
2006-01-04, by paulson
a few more named lemmas
2006-01-04, by paulson
fix: reintroduced pred_ctxt in gen_add_locale
2006-01-04, by haftmann
tuned;
2006-01-04, by wenzelm
* Pure/Isar: Toplevel.theory_theory_to_proof;
2006-01-04, by wenzelm
added unlocalize_mfix;
2006-01-04, by wenzelm
added unlocalize_mixfix;
2006-01-04, by wenzelm
added theory_to_theory_to_proof, which may change theory before entering the proof;
2006-01-04, by wenzelm
tuned;
2006-01-04, by wenzelm
moved forget_proof to toplevel.ML;
2006-01-04, by wenzelm
Toplevel.forget_proof;
2006-01-04, by wenzelm
adapted Toplevel.Proof;
2006-01-04, by wenzelm
removed dead code;
2006-01-04, by wenzelm
more stuff;
2006-01-04, by wenzelm
Provers/classical: stricter checks to ensure that supplied intro, dest and
2006-01-03, by paulson
added explicit paths to required theories
2006-01-03, by paulson
added implementation manual;
2006-01-03, by wenzelm
more stuff;
2006-01-03, by wenzelm
fixed LaTeX source;
2006-01-03, by wenzelm
class now a keyword
2006-01-03, by haftmann
class now an keyword, quoted where necessary
2006-01-03, by haftmann
add_local_context now yields imported and body elements seperatly; additional slight clenup in code
2006-01-03, by haftmann
rearranged burrow_split to fold_burrow to allow composition with fold_map
2006-01-03, by haftmann
added unfolding(_i);
2006-01-03, by wenzelm
unparse String/AltString: escape quotes;
2006-01-03, by wenzelm
tuned;
2006-01-03, by wenzelm
avoid hardwired Trueprop;
2006-01-03, by wenzelm
added 'using' command;
2006-01-03, by wenzelm
updated;
2006-01-03, by wenzelm
added IsarImplementation;
2006-01-03, by wenzelm
updated -- lost update!?
2006-01-03, by wenzelm
* Pure/Isar: new command 'unfolding';
2006-01-03, by wenzelm
ISABELLE_USER for remote cvs access;
2006-01-02, by wenzelm
outline;
2006-01-02, by wenzelm
"The Isabelle/Isar Implementation" manual;
2006-01-02, by wenzelm
* Provers/classical: removed obsolete classical version of elim_format;
2005-12-31, by wenzelm
tuned forall_intr_vars;
2005-12-31, by wenzelm
added classical_rule, which replaces Data.make_elim;
2005-12-31, by wenzelm
explicitly reject consts *Goal*, *False*;
2005-12-31, by wenzelm
elim rules: Classical.classical_rule;
2005-12-31, by wenzelm
removed obsolete cla_dist_concl;
2005-12-31, by wenzelm
removed classical elim_format;
2005-12-31, by wenzelm
removed obsolete Provers/make_elim.ML;
2005-12-31, by wenzelm
obsolete, see classical_rule in Provers/classical.ML;
2005-12-31, by wenzelm
more robust phantomsection;
2005-12-31, by wenzelm
require cla_dist_concl, avoid assumptions about concrete syntax;
2005-12-30, by wenzelm
avoid implicit assumptions about consts Not, op =, *Goal*, *False*;
2005-12-30, by wenzelm
provide equality_name, not_name;
2005-12-30, by wenzelm
fixed final_consts;
2005-12-30, by wenzelm
provide cla_dist_concl;
2005-12-30, by wenzelm
non-PDF: phantomsection;
2005-12-30, by wenzelm
added atom keyword
2005-12-29, by haftmann
changes in code generator keywords
2005-12-29, by haftmann
adaptions to changes in code generator
2005-12-29, by haftmann
slight improvements
2005-12-29, by haftmann
slightly improved serialization
2005-12-28, by haftmann
substantial improvements in code generating
2005-12-27, by haftmann
added map_index
2005-12-27, by haftmann
tuned proofs;
2005-12-23, by wenzelm
removed obsolete atomize_old;
2005-12-23, by wenzelm
removed obsolete induct_atomize_old;
2005-12-23, by wenzelm
the "skolem" attribute and better initialization of the clause database
2005-12-23, by paulson
blacklist of prolific theorems (must be replaced by an attribute later
2005-12-23, by paulson
tidied
2005-12-23, by paulson
tuned;
2005-12-23, by wenzelm
* Provers/induct: support simultaneous goals with mutual rules;
2005-12-23, by wenzelm
induct etc.: admit multiple rules;
2005-12-23, by wenzelm
backpatching of Substring.full;
2005-12-23, by wenzelm
goal/qed: proper treatment of two levels of conjunctions;
2005-12-23, by wenzelm
Logic.mk_conjunction_list;
2005-12-23, by wenzelm
turned bicompose_no_flatten into compose_no_flatten, without elimination;
2005-12-23, by wenzelm
CONJUNCTS: full nesting (again), PRECISE_CONJUNCTS: outer level of nesting;
2005-12-23, by wenzelm
added mk_conjunction_list2;
2005-12-23, by wenzelm
conj_elim_precise: proper treatment of nested conjunctions;
2005-12-23, by wenzelm
Thm.compose_no_flatten;
2005-12-23, by wenzelm
proper treatment of nested conjunctions, i.e. simultaneous goals and mutual rules;
2005-12-23, by wenzelm
is_prefix
2005-12-23, by haftmann
slight improvements
2005-12-22, by haftmann
more lemmas
2005-12-22, by nipkow
shorter proof
2005-12-22, by paulson
Tuned syntax for perm.
2005-12-22, by berghofe
new lemmas
2005-12-22, by nipkow
Fixed a use of an outdated Substring function
2005-12-22, by paulson
tuned;
2005-12-22, by wenzelm
exh_casedist2: norm_hhf_eq;
2005-12-22, by wenzelm
added bicompose_no_flatten, which refrains from
2005-12-22, by wenzelm
bicompose_proof: no_flatten;
2005-12-22, by wenzelm
conclude/SELECT: Thm.bicompose_no_flatten avoids unsolicited modification of result;
2005-12-22, by wenzelm
Transform mutual rule into projection.
2005-12-22, by wenzelm
added Provers/project_rule.ML
2005-12-22, by wenzelm
structure ProjectRule;
2005-12-22, by wenzelm
* induct: improved treatment of mutual goals and mutual rules;
2005-12-22, by wenzelm
updated auxiliary facts for induct method;
2005-12-22, by wenzelm
prop_tr': proper handling of aprop marked as bound;
2005-12-22, by wenzelm
consume: expand defs in prems of concls;
2005-12-22, by wenzelm
cases: main is_proper flag;
2005-12-22, by wenzelm
auto cases: marked improper;
2005-12-22, by wenzelm
less
more
|
(0)
-10000
-3000
-1000
-480
+480
+1000
+3000
+10000
+30000
tip