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.
Thm.add_cterm_frees;
2007-06-25, by wenzelm
made type conv pervasive;
2007-06-25, by wenzelm
made type conv pervasive;
2007-06-25, by wenzelm
tex problem fixed
2007-06-24, by nipkow
tuned and used field_simps
2007-06-24, by nipkow
*** empty log message ***
2007-06-24, by nipkow
*** empty log message ***
2007-06-24, by nipkow
new lemmas
2007-06-24, by nipkow
*** empty log message ***
2007-06-24, by nipkow
tuned and renamed group_eq_simps and ring_eq_simps
2007-06-23, by nipkow
fix looping simp rule
2007-06-22, by huffman
reinstate real_root_less_iff [simp]
2007-06-22, by huffman
merge is now identity
2007-06-22, by chaieb
new method "elim_to_cases" provides ad-hoc conversion of obtain-style
2007-06-22, by krauss
section headings
2007-06-21, by huffman
add thm antiquotations
2007-06-21, by huffman
spelling
2007-06-21, by huffman
add thm antiquotations
2007-06-21, by huffman
changed simp rules for of_nat
2007-06-21, by huffman
tuned proofs -- avoid implicit prems;
2007-06-21, by wenzelm
moved quantifier elimination tools to Tools/Qelim/;
2007-06-21, by wenzelm
moved Presburger setup back to Presburger.thy;
2007-06-21, by wenzelm
tuned proofs -- avoid implicit prems;
2007-06-21, by wenzelm
tuned proofs -- avoid implicit prems;
2007-06-21, by wenzelm
renamed NatSimprocs.thy to Arith_Tools.thy;
2007-06-21, by wenzelm
tuned;
2007-06-21, by wenzelm
adapted tool setup;
2007-06-21, by wenzelm
added Ferrante-Rackoff setup;
2007-06-21, by wenzelm
tuned comments;
2007-06-21, by wenzelm
moved HOL/Tools/Presburger/qelim.ML to HOL/Tools/qelim.ML;
2007-06-21, by wenzelm
Ferrante-Rackoff quantifier elimination.
2007-06-21, by wenzelm
Context data for Ferrante-Rackoff quantifier elimination.
2007-06-21, by wenzelm
replaced Real/Ferrante-Rackoff tool by generic version in Main HOL;
2007-06-21, by wenzelm
Dense linear order witout endpoints
2007-06-21, by wenzelm
renamed metis-env.ML to metis_env.ML;
2007-06-21, by wenzelm
added Id;
2007-06-21, by wenzelm
fine tune automatic generation of inversion lemmas
2007-06-21, by narboux
integration of Metis prover
2007-06-21, by paulson
renamed metis-env to metis-env.ML;
2007-06-21, by wenzelm
tuned comments;
2007-06-20, by wenzelm
obsolete (cf. ATP_Linkup.thy);
2007-06-20, by wenzelm
added Tools/metis_tools.ML;
2007-06-20, by wenzelm
added Metis setup (from Metis.thy);
2007-06-20, by wenzelm
added HOL-Nominal-Examples;
2007-06-20, by wenzelm
The Metis prover (slightly modified version from Larry);
2007-06-20, by wenzelm
avoid using implicit prems in assumption
2007-06-20, by huffman
Added flexflex_first_order and tidied first_order_resolution
2007-06-20, by paulson
A more robust flexflex_unique
2007-06-20, by paulson
remove simp attribute from of_nat_diff, for backward compatibility with zdiff_int
2007-06-20, by huffman
tuned error msg
2007-06-20, by krauss
Remove dedicated flag setting elements in favour of setproverflag.
2007-06-20, by aspinall
Remove dedicated flag setting elements in favour of setproverflag. Restore displayconfig response in askpgip.
2007-06-20, by aspinall
Synchronize schema with current version
2007-06-20, by aspinall
added lemmas
2007-06-20, by nipkow
added meta_impE
2007-06-20, by nipkow
change simp rules for of_nat to work like int did previously (reorient of_nat_Suc, remove of_nat_mult [simp]); preserve original variable names in legacy int theorems
2007-06-20, by huffman
section headings
2007-06-20, by huffman
simplify some proofs
2007-06-20, by huffman
oops -- fixed profiling;
2007-06-19, by wenzelm
Balanced binary trees (material from library.ML);
2007-06-19, by wenzelm
profiling: observe no_timing;
2007-06-19, by wenzelm
added raw_tactic;
2007-06-19, by wenzelm
moved balanced tree operations to General/balanced_tree.ML;
2007-06-19, by wenzelm
added with_subgoal;
2007-06-19, by wenzelm
balanced conjunctions;
2007-06-19, by wenzelm
balanced conjunctions;
2007-06-19, by wenzelm
added General/balanced_tree.ML;
2007-06-19, by wenzelm
BalancedTree;
2007-06-19, by wenzelm
balanced conjunctions;
2007-06-19, by wenzelm
tuned;
2007-06-19, by wenzelm
generalized proofs so that call graphs can have any node type.
2007-06-19, by krauss
macbroy5: trying -j 2;
2007-06-19, by wenzelm
tuned conjunction tactics: slightly smaller proof terms;
2007-06-18, by wenzelm
tuned laws for cancellation in divisions for fields.
2007-06-17, by nipkow
moved nonzero_mult_divide_cancel_right to Ring_and_Field as nonzero_mult_divide_cancel_right'; tuned proofs
2007-06-17, by chaieb
Added eta_conv and eta-expansion conversion: waiting for it to be in thm.ML; exported is_refl
2007-06-17, by chaieb
gen_qelim_conv now reduces the universal quatifier to the existential one; Now also deals with Ex f for eta-contracted f;
2007-06-17, by chaieb
thin_prems_tac first max-scopes universal quantifiers; eta_conv moved to Pure/conv.ML
2007-06-17, by chaieb
Tuned error messages; tuned;
2007-06-17, by chaieb
normalizer conversions depend on the proof context; added functions for conversion and wrapper that sill depend on the variable ordering (_ord)
2007-06-17, by chaieb
added theorems nonzero_mult_divide_cancel_right' nonzero_mult_divide_cancel_left' ordered_field_no_lb ordered_field_no_ub
2007-06-17, by chaieb
moved lemma all_not_ex to HOL.thy ; tuned proofs
2007-06-17, by chaieb
Tuned instantiation of Groebner bases to fields
2007-06-17, by chaieb
added Theorem all_not_ex
2007-06-17, by chaieb
renamed vars in zle_trans for compatibility
2007-06-17, by nipkow
tuned
2007-06-16, by nipkow
The simprocs "divide_cancel_factor" and "ring_eq_cancel_factor" no
2007-06-16, by nipkow
Locally added definition of "int :: nat => int" again to make
2007-06-15, by berghofe
made divide_self a simp rule
2007-06-15, by nipkow
Removed thunk from Fun
2007-06-15, by nipkow
Church numerals added
2007-06-15, by nipkow
method assumption: uniform treatment of prems as legacy feature;
2007-06-14, by wenzelm
tuned proofs;
2007-06-14, by wenzelm
tuned proofs: avoid implicit prems;
2007-06-14, by wenzelm
fixed term_constants (impact on is_relevant); terms in generalize_tac are sorted before we abstract over them (to *try* to avoid the case when a term to be abstracted over already occurs in an other)
2007-06-14, by chaieb
no computation rules in the pre-simplifiaction set
2007-06-14, by chaieb
Added some lemmas to default presburger simpset; tuned proofs
2007-06-14, by chaieb
tuned proofs: avoid implicit prems;
2007-06-14, by wenzelm
tuned proofs: avoid implicit prems;
2007-06-14, by wenzelm
Now ResHolClause also does first-order problems!
2007-06-14, by paulson
Now also handles FO problems
2007-06-14, by paulson
Deleted unused code
2007-06-14, by paulson
tidied
2007-06-14, by paulson
tuned proofs: avoid implicit prems;
2007-06-14, by wenzelm
clarified who we consider to be a contributor
2007-06-14, by kleing
Fixed Problem with ML-bindings for thm names;
2007-06-14, by chaieb
fixed filter syntax
2007-06-14, by nipkow
updated 'find_theorems' -- moved ProofGeneral specifics to ProofGeneral/CHANGES;
2007-06-14, by wenzelm
tuned proofs: avoid implicit prems;
2007-06-14, by wenzelm
int abbreviates of_nat
2007-06-13, by huffman
tuned proofs: avoid implicit prems;
2007-06-13, by wenzelm
tuned proofs: avoid implicit prems;
2007-06-13, by wenzelm
tuned comments;
2007-06-13, by wenzelm
tuned proofs: avoid implicit prems;
2007-06-13, by wenzelm
clean up instance proofs; reorganize section headings
2007-06-13, by huffman
reactivated theory Class;
2007-06-13, by wenzelm
added the Q_Unit rule (was missing) and adjusted the proof accordingly
2007-06-13, by urbanc
* Isar: method "assumption" (implicit closing of subproofs) takes non-atomic goal assumptions into account;
2007-06-13, by wenzelm
generate_fresh works even if there is no free variable in the goal
2007-06-13, by narboux
tuned;
2007-06-13, by wenzelm
tuned proofs: avoid implicit prems;
2007-06-13, by wenzelm
removed constant int :: nat => int;
2007-06-13, by huffman
thm antiquotations
2007-06-13, by huffman
transaction: context_position (non-destructive only);
2007-06-13, by wenzelm
added map_current;
2007-06-13, by wenzelm
tuned msg;
2007-06-13, by wenzelm
apply_method/end_proof: pass position;
2007-06-13, by wenzelm
renamed map to map_current;
2007-06-13, by wenzelm
tuned;
2007-06-13, by wenzelm
removed unused is_atomic;
2007-06-13, by wenzelm
renamed prove_raw to prove_internal;
2007-06-13, by wenzelm
merge/merge_refs: plain error instead of exception TERM;
2007-06-13, by wenzelm
Context positions.
2007-06-13, by wenzelm
added context_position.ML;
2007-06-13, by wenzelm
renamed Goal.prove_raw to Goal.prove_internal;
2007-06-13, by wenzelm
Method.Basic: include position;
2007-06-13, by wenzelm
tuned proofs: avoid implicit prems;
2007-06-13, by wenzelm
Basic text: include position;
2007-06-13, by wenzelm
thm antiquotations
2007-06-12, by huffman
add lemma inj_of_nat
2007-06-12, by huffman
thm antiquotations
2007-06-12, by huffman
Unfortunately needed patch due to incompatibility with SML -- oo is infix and hence can not appear on the left handside of patterns
2007-06-12, by chaieb
changed int stuff into integer for SMLNJ compatibility
2007-06-12, by chaieb
more of_rat lemmas
2007-06-12, by huffman
add function of_rat and related lemmas
2007-06-12, by huffman
turned curry (op opr) into curry op opr --- because of smlnj
2007-06-12, by chaieb
De-overloaded operations for int and real.
2007-06-12, by wenzelm
SML basis with type int representing proper integers, not machine words.
2007-06-12, by wenzelm
Tuned proofs : now use 'algebra ad: ...'
2007-06-12, by chaieb
cooper_tac takes now two lists of theorems to be added/deleted from the simpset dor pre-simplification
2007-06-12, by chaieb
changed val restriction to local due to smlnj
2007-06-12, by chaieb
Changed normalizer Data to contain a simpset besides the list of instances; Before the method starts, it simplifies with this simpset; Added attribute 'algebra' to add and delete theorems from the simpset above;
2007-06-12, by chaieb
Added algebra_tac; tuned;
2007-06-12, by chaieb
Method now takes theorems to be added or deleted from a simpset for simplificatio before the core method starts
2007-06-12, by chaieb
algebra_tac moved to file Tools/Groebner_Basis/groebner.ML; Method now takes theorems to be added or deleted from a simpset for simplificatio *before* the core method starts
2007-06-12, by chaieb
nex example
2007-06-11, by nipkow
Conversion for computation on constants now depends on the context
2007-06-11, by chaieb
tuned setup for the fields instantiation for Groebner Bases;
2007-06-11, by chaieb
Added dependency on file Groebner_Basis.thy
2007-06-11, by chaieb
Added instantiation of algebra method to fields
2007-06-11, by chaieb
hid constant "dom"
2007-06-11, by nipkow
Removed from CVS, since obselete in the new Presburger Method;
2007-06-11, by chaieb
Generated reflected QE procedure for Presburger Arithmetic-- Cooper's Algorithm -- see HOL/ex/Reflected_Presburger.thy
2007-06-11, by chaieb
Added more examples
2007-06-11, by chaieb
Now only contains generic conversion for quantifier elimination in HOL
2007-06-11, by chaieb
A new tactic for Presburger;
2007-06-11, by chaieb
tuned
2007-06-11, by chaieb
Temporarily added theorems for QE that were in old Presburger.thy ; This will diseappear with the new Ferrante and Rackoff shortly;
2007-06-11, by chaieb
tuned tactic
2007-06-11, by chaieb
Temporarily use int instead of IntInf.int but Code generator should map HOL's int to ML's IntInf.int --- To be fixed
2007-06-11, by chaieb
tuned Proof and Document
2007-06-11, by chaieb
tuned Proof
2007-06-11, by chaieb
A new and cleaned up Theory for QE. for Presburger arithmetic
2007-06-11, by chaieb
Added new files for Presburger (cooper_data.ML, cooper.ML) and deleted old unused ones cooper_dec, cooper_proof, reflected_cooper etc..
2007-06-11, by chaieb
explicitely depends on file groebner.ML
2007-06-11, by chaieb
Context Data for the new presburger Method
2007-06-11, by chaieb
A new simpler and cleaner implementation of proof Synthesis for Presburger Arithmetic --- Cooper's Algorithm
2007-06-11, by chaieb
remove references to constant int::nat=>int
2007-06-11, by huffman
simplify int proofs
2007-06-11, by huffman
modify proofs to avoid referring to int::nat=>int
2007-06-11, by huffman
add int_of_nat versions of lemmas about int::nat=>int
2007-06-11, by huffman
add lemma of_nat_power
2007-06-11, by huffman
add int_of_nat versions of lemmas about int::nat=>int
2007-06-11, by huffman
add abbreviation int_of_nat for of_nat::nat=>int;
2007-06-11, by huffman
disabled theory "Reflected_Presburger" for smlnj (temporarily);
2007-06-10, by wenzelm
disabled theories MIR and ReflectedFerrack for smlnj (temporarily);
2007-06-10, by wenzelm
*** empty log message ***
2007-06-10, by nipkow
remove dependencies of proofs on constant int::nat=>int, preparing to remove it
2007-06-09, by huffman
eqtype int -- explicitly encourage overloaded equality;
2007-06-09, by wenzelm
simplified type integer;
2007-06-09, by wenzelm
Adapted Proofterm.bicompose_proof to Larry's changes in
2007-06-08, by berghofe
Method "algebra" solves polynomial equations over (semi)rings
2007-06-08, by chaieb
generalize zpower_number_of_{even,odd} lemmas
2007-06-08, by huffman
deleted comments
2007-06-07, by obua
deleted legacy lemmas
2007-06-07, by obua
somebody elses problem fixed
2007-06-07, by nipkow
filter syntax change
2007-06-07, by nipkow
remove redundant lemmas
2007-06-07, by huffman
remove references to preal-specific theorems
2007-06-07, by huffman
define (1::preal); clean up instance declarations
2007-06-07, by huffman
tuned
2007-06-07, by huffman
instance preal :: ordered_cancel_ab_semigroup_add
2007-06-07, by huffman
use new-style class for sq_ord; rename op << to sq_le
2007-06-06, by huffman
take out Class.thy again, because it does not yet compile cleanly
2007-06-06, by urbanc
add axclass semiring_char_0 for types where of_nat is injective
2007-06-06, by huffman
changed filter syntax from : to <-
2007-06-06, by nipkow
hide filter
2007-06-06, by nipkow
tuned list comprehension, changed filter syntax from : to <-
2007-06-06, by nipkow
clean up proofs of exp_zero, sin_zero, cos_zero
2007-06-06, by huffman
generalize class constraints on some lemmas
2007-06-06, by huffman
generalize of_nat and related constants to class semiring_1
2007-06-06, by huffman
declare complex_diff as simp rule
2007-06-06, by huffman
New Reflected Presburger added to HOL/ex
2007-06-06, by chaieb
Groebner Basis Examples.
2007-06-05, by wenzelm
print_antiquotations: sort_strings;
2007-06-05, by wenzelm
tuned document;
2007-06-05, by wenzelm
tuned source deps;
2007-06-05, by wenzelm
simplified/renamed add_numerals;
2007-06-05, by wenzelm
renamed ex/Eval_Examples.thy;
2007-06-05, by wenzelm
added ex/Groebner_Examples.thy;
2007-06-05, by wenzelm
tuned document;
2007-06-05, by wenzelm
Added two examples in Complex/ex :Reflected QE for linear real arith and QE for mixed integer real linear arithmetic
2007-06-05, by chaieb
Added twe Examples for Quantifier elimination ofer linear real arithmetic and over the mixed theory of linear real artihmetic with integers
2007-06-05, by chaieb
tuned boostrap
2007-06-05, by haftmann
eliminated Code_Generator.thy
2007-06-05, by haftmann
tuned integers
2007-06-05, by haftmann
tuned;
2007-06-05, by wenzelm
fixed type int vs. integer;
2007-06-05, by wenzelm
renamed locale ring/semiring to gb_ring/gb_semiring to avoid clash with Ring_and_Field versions;
2007-06-05, by wenzelm
add new lemmas
2007-06-05, by huffman
Polynomials now only depend on Deriv; Definition of degree changed
2007-06-05, by chaieb
lemma lemma_DERIV_subst moved to Deriv.thy
2007-06-05, by chaieb
tuned proofs;
2007-06-05, by wenzelm
tuned comments;
2007-06-05, by wenzelm
Semiring normalization and Groebner Bases.
2007-06-05, by wenzelm
moved generic algebra modules
2007-06-05, by haftmann
updated documentation
2007-06-05, by haftmann
fixed broken execption handling
2007-06-05, by haftmann
simplified notion of "operational classes"
2007-06-05, by haftmann
merged Code_Generator.thy into HOL.thy
2007-06-05, by haftmann
added a function partition and a few lemmas
2007-06-05, by chaieb
added a few theorems about foldl and set
2007-06-05, by chaieb
added lcm, ilcm (lcm for integers) and some lemmas about them;
2007-06-05, by chaieb
included Class.thy in the compiling process for Nominal/Examples
2007-06-05, by urbanc
remove simp attribute from lemma_STAR theorems
2007-06-05, by huffman
add lemma exp_of_real
2007-06-05, by huffman
tuned list comprehension
2007-06-04, by nipkow
tuned;
2007-06-04, by wenzelm
added is_atomic;
2007-06-04, by wenzelm
added assume_rule_tac;
2007-06-04, by wenzelm
reverted appnd to append
2007-06-04, by haftmann
authentic syntax for List.append
2007-06-04, by haftmann
tuned comments
2007-06-04, by haftmann
added a few comments to the proofs
2007-06-04, by urbanc
removed fixmes
2007-06-04, by chaieb
opaque-constraint removed
2007-06-04, by chaieb
tuned;
2007-06-04, by chaieb
monomorphic equality: let ML work out the details;
2007-06-03, by wenzelm
added gen_merge_lists/merge_lists/merge_alists (legacy operations from library.ML);
2007-06-03, by wenzelm
tuned Tactic signature;
2007-06-03, by wenzelm
removed obsolete Library.seq;
2007-06-03, by wenzelm
moved flip to library.ML;
2007-06-03, by wenzelm
added CSUBGOAL;
2007-06-03, by wenzelm
cleaned up signature;
2007-06-03, by wenzelm
added downto0 (from library.ML);
2007-06-03, by wenzelm
merge_ss: plain merge of prems;
2007-06-03, by wenzelm
added flip (from General/basics.ML);
2007-06-03, by wenzelm
tuned document;
2007-06-03, by wenzelm
use antiquotations instead of raw TeX code;
2007-06-03, by wenzelm
name_of_fqgar: precise type;
2007-06-03, by wenzelm
added plural (from Pure/library.ML);
2007-06-03, by wenzelm
local open FundefLib;
2007-06-03, by wenzelm
renamed gen_submultiset to submultiset;
2007-06-03, by wenzelm
HOL-ex: tuned deps;
2007-06-03, by wenzelm
tuned list comprehension, added lemma
2007-06-03, by nipkow
fixed tex error
2007-06-03, by nipkow
*** empty log message ***
2007-06-03, by nipkow
*** empty log message ***
2007-06-03, by nipkow
extended
2007-06-02, by webertj
cosmetic
2007-06-02, by webertj
made SML/NJ happy;
2007-06-02, by wenzelm
added target/local_abbrev (from proof_context.ML);
2007-06-02, by wenzelm
moved specific target/local_abbrev to theory_target.ML;
2007-06-02, by wenzelm
"function (sequential)" and "fun" now handle incomplete patterns silently by adding "undefined" cases.
2007-06-02, by krauss
added "plural : 'a -> 'a -> 'b list -> 'a" for convenient error msg construction
2007-06-02, by krauss
proper handling of Tools;
2007-06-02, by wenzelm
cosmetic
2007-06-02, by webertj
refute_tac made more deterministic
2007-06-02, by webertj
extended
2007-06-02, by webertj
cosmetic
2007-06-02, by webertj
tracing disabled
2007-06-02, by webertj
additional tracing information
2007-06-01, by webertj
tuned
2007-06-01, by webertj
some tests for arith added
2007-06-01, by webertj
Moved list comprehension into List
2007-06-01, by nipkow
MiniSAT mentioned in comment
2007-06-01, by webertj
fixed handling of meta-logic propositions
2007-06-01, by webertj
simplified interfaces, some restructuring
2007-06-01, by krauss
updated
2007-06-01, by krauss
added some bibtex entries
2007-06-01, by krauss
Added "merge-lemma" about wellfoundedness of unions (useful for some termination proofs)
2007-06-01, by krauss
Added simp-rules: "R O {} = {}" and "{} O R = {}"
2007-06-01, by krauss
rudimenary
2007-06-01, by haftmann
tuned
2007-06-01, by haftmann
dropped superfluous name bindings
2007-06-01, by haftmann
localized
2007-06-01, by haftmann
fixed typo
2007-06-01, by haftmann
insert: canonical argument order;
2007-05-31, by wenzelm
simplified/unified list fold;
2007-05-31, by wenzelm
replace (- 1) with -1
2007-05-31, by huffman
simplify some proofs
2007-05-31, by huffman
tuned headers -- adapted to usual conventions;
2007-05-31, by wenzelm
moved Compute_Oracle from Pure/Tools to Tools;
2007-05-31, by wenzelm
proper theory setup for compute oracle (based on CPure);
2007-05-31, by wenzelm
moved IsaPlanner from Provers to Tools;
2007-05-31, by wenzelm
moved IsaPlanner from Provers to Tools;
2007-05-31, by wenzelm
made aconvc pervasive;
2007-05-31, by wenzelm
moved aconvc to more_thm.ML;
2007-05-31, by wenzelm
tuned ML setup;
2007-05-31, by wenzelm
decode_term: force qualified name into Const;
2007-05-31, by wenzelm
proper loading of ML files (in HOL.thy);
2007-05-31, by wenzelm
HOL_proofs;
2007-05-31, by wenzelm
moved Integ files to canonical place;
2007-05-31, by wenzelm
proper loading of ML files;
2007-05-31, by wenzelm
removed dead code;
2007-05-31, by wenzelm
tuned header;
2007-05-31, by wenzelm
doc: exclude isabelle_isar.pdf;
2007-05-31, by wenzelm
tuned the proof
2007-05-31, by urbanc
introduced symmetric variants of the lemmas for alpha-equivalence
2007-05-31, by urbanc
proper loading of ML files;
2007-05-31, by wenzelm
removed obsolete IFOL.thy/FOL.thy values;
2007-05-31, by wenzelm
proper loading of ML files;
2007-05-31, by wenzelm
tuned header;
2007-05-31, by wenzelm
tuned oracle setup;
2007-05-31, by wenzelm
moved HOLCF tools to canonical place;
2007-05-31, by wenzelm
moved TFL files to canonical place;
2007-05-31, by wenzelm
moved TFL files to canonical place;
2007-05-31, by wenzelm
added src/Tools;
2007-05-31, by wenzelm
fixed title;
2007-05-31, by wenzelm
Tools: generic tools outside of Pure.
2007-05-31, by wenzelm
moved Integ files to canonical place;
2007-05-31, by wenzelm
fixed use_thy "LocalWeakening";
2007-05-31, by wenzelm
included new example in the compiling process
2007-05-31, by urbanc
a theory using locally nameless terms and strong induction principles
2007-05-31, by urbanc
tuned the proof
2007-05-31, by urbanc
emulate later version of TextIO.inputLine;
2007-05-31, by wenzelm
reversed SML B library patches;
2007-05-31, by wenzelm
TextIO.inputLine: use present SML B library version;
2007-05-31, by wenzelm
tuned USEDIR_OPTIONS;
2007-05-30, by wenzelm
removed HOL4 image, which seldom works;
2007-05-30, by wenzelm
simplified data setup
2007-05-30, by haftmann
instance: always print sorts on failure
2007-05-30, by haftmann
more example
2007-05-30, by haftmann
fixed typo
2007-05-30, by haftmann
updated
2007-05-30, by haftmann
generalized lemmas
2007-05-30, by haftmann
eliminated strings
2007-05-30, by haftmann
tuned
2007-05-30, by haftmann
clarified error message
2007-05-30, by krauss
simplify names of locale interpretations
2007-05-30, by huffman
renamed some lemmas in Complex.thy
2007-05-30, by huffman
cleaned up proofs; reorganized sections; removed redundant lemmas
2007-05-30, by huffman
use new-style instance declarations
2007-05-29, by huffman
instance complex :: banach
2007-05-29, by huffman
add lemma real_sqrt_sum_squares_less
2007-05-29, by huffman
cleaned up some proofs
2007-05-29, by huffman
interpretation bounded_linear_divide
2007-05-29, by huffman
add bounded_linear lemmas
2007-05-29, by huffman
add isUCont lemmas
2007-05-29, by huffman
updated examples to include an instance of (lexicographic_order simp:...)
2007-05-29, by krauss
Complex: generalized type of exp
2007-05-28, by huffman
generalized exp to work over any complete field; new proof of exp_add
2007-05-28, by huffman
add type annotations for exp
2007-05-28, by huffman
interpretations additive_scaleR_left, additive_scaleR_right
2007-05-28, by huffman
remove division_by_zero requirement from termdiffs lemmas; cleaned up some proofs
2007-05-28, by huffman
new proof of Cauchy product formula for series
2007-05-27, by huffman
What it says
2007-05-26, by nipkow
improved error handling
2007-05-25, by haftmann
using rudimentary class target mechanism
2007-05-25, by haftmann
*** empty log message ***
2007-05-25, by haftmann
fixed typo
2007-05-25, by haftmann
fix typos
2007-05-25, by huffman
*** empty log message ***
2007-05-25, by nipkow
*** empty log message ***
2007-05-25, by nipkow
*** empty log message ***
2007-05-25, by nipkow
tuned
2007-05-25, by nipkow
Added List_Comprehension
2007-05-25, by nipkow
adapted to fix for fresh_fun_simp
2007-05-25, by urbanc
took out Class.thy from the compiling process until memory problems are solved
2007-05-25, by urbanc
simplify some proofs
2007-05-25, by huffman
*** empty log message ***
2007-05-24, by nipkow
Squared things out.
2007-05-24, by obua
fix a bug : the semantics of no_asm was the opposite
2007-05-24, by narboux
temporary fix for a bug in fresh_fun_simp
2007-05-24, by urbanc
formalisation of my PhD (the result was correct, but the proof needed several corrections)
2007-05-24, by urbanc
add an option in fresh_fun_simp to prevent rewriting in assumptions
2007-05-24, by narboux
fixes tvar issue in type inference
2007-05-24, by haftmann
tuned
2007-05-24, by haftmann
tuned warning
2007-05-24, by haftmann
rudimentary class target implementation
2007-05-24, by haftmann
tuned Pure/General/name_space.ML
2007-05-24, by haftmann
Introduced new classes monoid_add and group_add
2007-05-24, by nipkow
add lemma complete_algebra_summable_geometric
2007-05-23, by huffman
formatting
2007-05-23, by paulson
generalize powerseries and termdiffs lemmas using axclasses
2007-05-23, by huffman
remove unused simproc definition
2007-05-23, by huffman
remove redundant simproc; remove legacy ML bindings
2007-05-23, by huffman
remove redundant simproc
2007-05-23, by huffman
new simp rule Infinitesimal_of_hypreal_iff
2007-05-22, by huffman
removed redundant lemmas
2007-05-22, by huffman
generalize uniqueness of limits to class real_normed_algebra_1
2007-05-22, by huffman
Some hacks for SPASS format
2007-05-22, by paulson
some optimizations, cleanup
2007-05-22, by krauss
add missing instance declarations
2007-05-22, by huffman
adjusted to change in Provers/Arith/combine_numerals.ML
2007-05-22, by haftmann
adjusted to change in Provers/Arith/combine_numerals.ML
2007-05-22, by haftmann
regression tests: send failure reports to krauss@in.tum.de, too
2007-05-22, by krauss
rename lemmas LIM_ident, isCont_ident, DERIV_ident
2007-05-22, by huffman
remove obsolete CSeries.thy
2007-05-22, by huffman
generalized ring_eq_cancel simprocs to class idom; removed redundant field_eq_cancel simprocs
2007-05-22, by huffman
new field_combine_numerals simproc, which uses fractions as coefficients
2007-05-21, by huffman
search bottom up to get the inner fresh fun
2007-05-21, by narboux
add a bottom up search function
2007-05-21, by narboux
tuned
2007-05-21, by haftmann
evaluation for integers
2007-05-21, by haftmann
added lemma divAlg_div_mof
2007-05-21, by haftmann
improved code for rev
2007-05-21, by haftmann
min/max
2007-05-21, by haftmann
generalize CombineNumerals functor to allow coefficients with types other than IntInf.int
2007-05-21, by huffman
add lemmas divide_numeral_1 and inverse_numeral_1
2007-05-21, by huffman
fixed signature
2007-05-21, by krauss
Method "lexicographic_order" now takes the same arguments as "auto"
2007-05-21, by krauss
change fresh_fun_simp to treat occurences in assumptions and try to solve the generated subgoals
2007-05-21, by narboux
define pi with THE instead of SOME; cleaned up
2007-05-20, by huffman
add lemmas for sin,cos,tan of 30,45,60 degrees; cleaned up
2007-05-20, by huffman
add lemma power2_eq_imp_eq
2007-05-20, by huffman
added lemma for permutations on strings
2007-05-20, by urbanc
moved sqrt lemmas from Transcendental.thy to NthRoot.thy
2007-05-20, by huffman
remove obsolete DERIV_ln lemmas
2007-05-20, by huffman
add realpow_pos_nth2 back in
2007-05-20, by huffman
add odd_real_root lemmas
2007-05-20, by huffman
add lemmas about inverse functions; cleaned up proof of polar_ex
2007-05-20, by huffman
change premises of DERIV_inverse_function lemma
2007-05-20, by huffman
rearranged sections
2007-05-20, by huffman
add lemmas about continuity and derivatives of roots
2007-05-20, by huffman
add lemma DERIV_inverse_function
2007-05-20, by huffman
add lemmas LIM_compose2, isCont_LIM_compose2
2007-05-20, by huffman
improved aliassing
2007-05-19, by haftmann
more robust thm handling
2007-05-19, by haftmann
added a set of NNF normalization lemmas and nnf_conv
2007-05-19, by chaieb
added lt and some other infix operation analogous to Ocaml's num library
2007-05-19, by chaieb
added a generic conversion for quantifier elimination and a special useful instance
2007-05-19, by chaieb
added binop_conv, aconvc
2007-05-19, by chaieb
added cpat antiquotation for reading certified patterns
2007-05-19, by chaieb
unfold min/max in Stefans code generator
2007-05-19, by nipkow
added code generation based on Isabelle's rat type.
2007-05-19, by nipkow
Disabled Stefancs code generator - already enabled in RealDef.
2007-05-19, by nipkow
constant op @ now named append
2007-05-19, by haftmann
fixed comment
2007-05-19, by haftmann
dropped legacy
2007-05-19, by haftmann
improved eta expansion
2007-05-19, by haftmann
dropped nonsense comment
2007-05-19, by haftmann
fixed text
2007-05-19, by haftmann
eliminated name clash with List.append
2007-05-19, by haftmann
added qualification for ambiguous definition names
2007-05-19, by haftmann
tuned
2007-05-19, by haftmann
typ_of instance for int
2007-05-19, by haftmann
hide locale predicate "field" from HOL library
2007-05-19, by haftmann
no special treatment in naming of locale predicates stemming form classes
2007-05-19, by haftmann
uniform module names for code generation
2007-05-19, by haftmann
added Executable_Real
2007-05-19, by haftmann
updated
2007-05-19, by haftmann
Had to replace "case 1/2" by "case base/step". No idea why.
2007-05-19, by nipkow
*** empty log message ***
2007-05-19, by nipkow
remove dependence on Hilbert_Choice.thy
2007-05-19, by huffman
use THE instead of SOME
2007-05-19, by huffman
minimize imports
2007-05-18, by huffman
Prove existence of nth roots using Intermediate Value Theorem
2007-05-18, by huffman
avoid using real_mult_inverse_left; cleaned up
2007-05-18, by huffman
use mult_strict_mono instead of real_mult_less_mono
2007-05-18, by huffman
less
more
|
(0)
-10000
-3000
-1000
-480
+480
+1000
+3000
+10000
+30000
tip