Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-10000
-3000
-1000
-192
+192
+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.
exported customized syntax interface
2005-11-29, by haftmann
Corrected atom class constraints in strong induction rule.
2005-11-29, by berghofe
made some of the theorem look-ups static (by using
2005-11-29, by urbanc
added (curried) fold2
2005-11-28, by haftmann
added proof of measure_induct_rule;
2005-11-28, by wenzelm
Added flags for setting and detecting whether a problem needs combinators.
2005-11-28, by mengj
Only output types if !keep_types is true.
2005-11-28, by mengj
Added two functions for CNF translation, used by other files.
2005-11-28, by mengj
Added in four control flags for HOL and FOL translations.
2005-11-28, by mengj
Slight modification to trace information.
2005-11-28, by mengj
Added two methods "vampire" and "eprover" that handle both HOL and FOL proofs.
2005-11-28, by mengj
Only output arities and class relations if !ResClause.keep_types is true.
2005-11-28, by mengj
some small tuning
2005-11-28, by urbanc
ISAR-fied two proofs about equality for abstraction functions.
2005-11-28, by urbanc
* Provers/induct: obtain pattern;
2005-11-27, by wenzelm
added an authors section (please let me know if somebody is left out or unhappy)
2005-11-27, by urbanc
some minor tunings
2005-11-27, by urbanc
added the version of nominal.thy that contains
2005-11-27, by urbanc
cleaned up all examples so that they work with the
2005-11-27, by urbanc
finished cleaning up the parts that collect
2005-11-27, by urbanc
Corrected treatment of non-recursive abstraction types.
2005-11-26, by berghofe
tuned induct proofs;
2005-11-25, by wenzelm
induct: insert defs in object-logic form;
2005-11-25, by wenzelm
tuned induct proofs;
2005-11-25, by wenzelm
tuned induct proofs;
2005-11-25, by wenzelm
consume: unfold defs in all major prems;
2005-11-25, by wenzelm
revert_skolem: fall back on Syntax.deskolem;
2005-11-25, by wenzelm
forall_conv ~1;
2005-11-25, by wenzelm
added dummy_pattern;
2005-11-25, by wenzelm
tuned names;
2005-11-25, by wenzelm
forall_conv: limit prefix;
2005-11-25, by wenzelm
fix_tac: proper treatment of major premises in goal;
2005-11-25, by wenzelm
removed obsolete dummy paragraphs;
2005-11-25, by wenzelm
tuned;
2005-11-25, by wenzelm
code generator: case expressions, improved name resolving
2005-11-25, by haftmann
added fsub.thy (poplmark challenge) to the examples
2005-11-25, by urbanc
Fixed problem with strong induction theorem for datatypes containing
2005-11-25, by berghofe
send more information with test-takes-too-long message
2005-11-25, by kleing
fixed spelling of 'case_conclusion';
2005-11-24, by wenzelm
tuned induct proofs;
2005-11-24, by wenzelm
tuned induction proofs;
2005-11-23, by wenzelm
more robust revert_skolem;
2005-11-23, by wenzelm
tuned;
2005-11-23, by wenzelm
Provers/induct: definitional insts and fixing;
2005-11-23, by wenzelm
consume: proper treatment of defs;
2005-11-23, by wenzelm
added case_conclusion attribute;
2005-11-23, by wenzelm
(co)induct: taking;
2005-11-23, by wenzelm
RuleCases.case_conclusion;
2005-11-23, by wenzelm
tuned;
2005-11-23, by wenzelm
added case_conclusion attribute;
2005-11-23, by wenzelm
improved failure tracking
2005-11-23, by haftmann
Datatype_Universe: hide base names only;
2005-11-22, by wenzelm
added type cases/cases_tactic, and CASES, SUBGOAL_CASES;
2005-11-22, by wenzelm
cases_tactic;
2005-11-22, by wenzelm
moved multi_resolve(s) to drule.ML;
2005-11-22, by wenzelm
find_xxxS: term instead of thm;
2005-11-22, by wenzelm
export map_tags;
2005-11-22, by wenzelm
make coinduct actually work;
2005-11-22, by wenzelm
Drule.multi_resolves;
2005-11-22, by wenzelm
declare coinduct rule;
2005-11-22, by wenzelm
added code generator syntax
2005-11-22, by haftmann
added codegenerator
2005-11-22, by haftmann
added code generator syntax
2005-11-22, by haftmann
new treatment of polymorphic types, using Sign.const_typargs
2005-11-22, by paulson
added codegen package
2005-11-21, by haftmann
added serializer
2005-11-21, by haftmann
tweak
2005-11-21, by paulson
fixed some inconveniencies in website
2005-11-21, by haftmann
CONJUNCTS;
2005-11-19, by wenzelm
tuned;
2005-11-19, by wenzelm
Goal.norm_hhf_protected;
2005-11-19, by wenzelm
added coinduct attribute;
2005-11-19, by wenzelm
added CONJUNCTS: treat conjunction as separate sub-goals;
2005-11-19, by wenzelm
simpset: added reorient field, set_reorient;
2005-11-19, by wenzelm
tuned norm_hhf_protected;
2005-11-19, by wenzelm
removed conj_mono;
2005-11-19, by wenzelm
induct: CONJUNCTS for multiple goals;
2005-11-19, by wenzelm
tuned induct syntax;
2005-11-19, by wenzelm
FOL: -p 2;
2005-11-19, by wenzelm
presburger method updated to deal better with mod and div, tweo lemmas added to Divides.thy
2005-11-18, by chaieb
-- changed the interface of functions vampire_oracle and eprover_oracle.
2005-11-18, by mengj
-- terms are fully typed.
2005-11-18, by mengj
-- before converting axiom and conjecture clauses into ResClause.clause format, perform "check_is_fol_term" first.
2005-11-18, by mengj
-- combined common CNF functions used by HOL and FOL axioms, the difference between conversion of HOL and FOL theorems only comes in when theorems are converted to ResClause.clause or ResHolClause.clause format.
2005-11-18, by mengj
-- added combinator reduction axioms (typed and untyped) for HOL goals.
2005-11-18, by mengj
-- split up inputs to ATPs into two groups: temporary files (axioms and goals) and permanent helper files (e.g. combinator reduction axioms).
2005-11-18, by mengj
-- combined "make_nnf" functions for both FOL and HOL vampire/eprover methods.
2005-11-18, by mengj
-- removed "check_is_fol" from "make_nnf" so that the NNF procedure doesn't check whether a thm is FOL.
2005-11-18, by mengj
tuned document;
2005-11-16, by wenzelm
tuned;
2005-11-16, by wenzelm
improved induction proof: local defs/fixes;
2005-11-16, by wenzelm
tuned Pattern.match/unify;
2005-11-16, by wenzelm
added deskolem;
2005-11-16, by wenzelm
added THEN_ALL_NEW_CASES;
2005-11-16, by wenzelm
added revert_skolem, mk_def, add_def;
2005-11-16, by wenzelm
ProofContext.mk_def;
2005-11-16, by wenzelm
Term.betapplys;
2005-11-16, by wenzelm
tuned Pattern.match/unify;
2005-11-16, by wenzelm
added betapplys;
2005-11-16, by wenzelm
tuned interfaces to support incremental match/unify (cf. versions in type.ML);
2005-11-16, by wenzelm
tuned;
2005-11-16, by wenzelm
norm_hhf: no normalization of protected props;
2005-11-16, by wenzelm
added protect_cong, cong_mono_thm;
2005-11-16, by wenzelm
induct: support local definitions to be passed through the induction;
2005-11-16, by wenzelm
Trueprop: use ObjectLogic.judgment etc.;
2005-11-16, by wenzelm
Term.betapply;
2005-11-16, by wenzelm
new version of "tryres" allowing multiple unifiers (apparently needed for
2005-11-16, by paulson
pgmlsymbolson: append Symbol.xsymbolsN at end!
2005-11-16, by wenzelm
better no -d option;
2005-11-15, by wenzelm
added generic transformators
2005-11-15, by haftmann
removal of is_hol
2005-11-14, by paulson
added module system
2005-11-14, by haftmann
added modules for code generator generation two, not operational yet
2005-11-14, by haftmann
class_package - operational view on type classes
2005-11-14, by haftmann
string_of_alist - convenient q'n'd printout function
2005-11-14, by haftmann
support for polyml-4.2.0;
2005-11-14, by wenzelm
new syntax for class_package
2005-11-14, by haftmann
added const_instance;
2005-11-14, by wenzelm
added instance;
2005-11-14, by wenzelm
added ML-Systems/polyml-4.1.4-patch.ML, ML-Systems/polyml-4.2.0.ML;
2005-11-14, by wenzelm
Compatibility wrapper for Poly/ML 4.2.0.
2005-11-14, by wenzelm
tuned;
2005-11-14, by wenzelm
added a few equivariance lemmas (they need to be automated
2005-11-14, by urbanc
changed the HOL_basic_ss back and selectively added
2005-11-13, by urbanc
exchanged HOL_ss for HOL_basic_ss in the simplification
2005-11-13, by urbanc
a proof step corrected due to the changement in the presburger method.
2005-11-11, by chaieb
old argument "abs" is replaced by "no_abs". Abstraction is turned on by default.
2005-11-11, by chaieb
add header
2005-11-11, by huffman
tuned proofs;
2005-11-10, by wenzelm
moved find_free to term.ML;
2005-11-10, by wenzelm
guess: Seq.hd;
2005-11-10, by wenzelm
guess: Toplevel.proof;
2005-11-10, by wenzelm
added find_free (from Isar/proof_context.ML);
2005-11-10, by wenzelm
curried multiply;
2005-11-10, by wenzelm
induct method: fixes;
2005-11-10, by wenzelm
uncurried Consts.typargs;
2005-11-10, by wenzelm
renamed Thm.cgoal_of to Thm.cprem_of;
2005-11-10, by wenzelm
duplicate axioms in ATP linkup, and general fixes
2005-11-10, by paulson
tidying
2005-11-10, by paulson
called the induction principle "unsafe" instead of "test".
2005-11-10, by urbanc
Skolemization by inference, but not quite finished
2005-11-09, by paulson
Explicit data structures for some Isar language elements.
2005-11-09, by wenzelm
tuned;
2005-11-09, by wenzelm
tvars_intr_list: natural argument order;
2005-11-09, by wenzelm
moved datatype elem to element.ML;
2005-11-09, by wenzelm
P.context_element, P.locale_element;
2005-11-09, by wenzelm
Element.context;
2005-11-09, by wenzelm
use existing exeption Empty;
2005-11-09, by wenzelm
avoid code redundancy;
2005-11-09, by wenzelm
tuned comments;
2005-11-09, by wenzelm
removed obsolete term set operations;
2005-11-09, by wenzelm
P.locale_element;
2005-11-09, by wenzelm
added fold_terms;
2005-11-09, by wenzelm
added Isar/element.ML;
2005-11-09, by wenzelm
Thm.varifyT': natural argument order;
2005-11-09, by wenzelm
added join function
2005-11-09, by haftmann
allowing indentation of 'theory' keyword
2005-11-08, by haftmann
simplified after_qed;
2005-11-08, by wenzelm
avoid prove_plain, export_plain, simplified after_qed;
2005-11-08, by wenzelm
removed export_plain;
2005-11-08, by wenzelm
renamed assert_prop to ensure_prop;
2005-11-08, by wenzelm
renamed goals.ML to old_goals.ML;
2005-11-08, by wenzelm
export compose_hhf;
2005-11-08, by wenzelm
removed impose_hyps, satisfy_hyps;
2005-11-08, by wenzelm
const args: do not store variable names (unused);
2005-11-08, by wenzelm
renamed goals.ML to old_goals.ML;
2005-11-08, by wenzelm
(fix for accidental commit)
2005-11-08, by haftmann
(codegen)
2005-11-08, by haftmann
generate pattern combinators for new datatypes
2005-11-08, by huffman
reimplemented Case syntax using print/parse translations; moved as-patterns to separate section
2005-11-07, by huffman
add case syntax for type one
2005-11-07, by huffman
remove syntax for as-patterns
2005-11-07, by huffman
avoid 'as' as identifier;
2005-11-07, by wenzelm
avoid 'as' as identifier;
2005-11-07, by wenzelm
Added strong induction theorem (currently only axiomatized!).
2005-11-07, by berghofe
Initial commit.
2005-11-07, by urbanc
Initial commit of the theory "Weakening".
2005-11-07, by urbanc
added thms perm, distinct and fresh to the simplifier.
2005-11-07, by urbanc
added proper fillin_mixfix
2005-11-07, by haftmann
added fillin_mixfix, replace_quote
2005-11-07, by haftmann
New function store_thmss_atts.
2005-11-07, by berghofe
used the function Library.product for the cprod from Stefan
2005-11-07, by urbanc
fixed bug with nominal induct
2005-11-07, by urbanc
added fillin_mixfix' needed by serializer
2005-11-07, by haftmann
add case syntax stuff
2005-11-06, by huffman
use consts for infix syntax
2005-11-06, by huffman
add proof of Bekic's theorem: fix_cprod
2005-11-06, by huffman
simplify definitions
2005-11-05, by huffman
put iterate and fix in separate sections; added Letrec
2005-11-05, by huffman
renamed and added ch2ch, cont2cont, mono2mono theorems ending in _fun, _lambda, _LAM
2005-11-05, by huffman
add line breaks to Rep_CFun syntax
2005-11-05, by huffman
moved adm_chfindom from Fix.thy to Cfun.thy; moved admw-related stuff to its own section
2005-11-04, by huffman
less
more
|
(0)
-10000
-3000
-1000
-192
+192
+1000
+3000
+10000
+30000
tip