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.
corrected typo introduced by me
2007-02-06, by urbanc
now obsolete
2007-02-06, by urbanc
moved the infrastructure from the nominal_tags file to nominal_thmdecls
2007-02-06, by urbanc
Exporting curried versions of tail recursive equations instead of internal ones
2007-02-05, by krauss
proper use of NameSpace.is_qualified (avoids compatibility issues of the SML B library);
2007-02-05, by wenzelm
removed non-modular comment;
2007-02-04, by wenzelm
interpretation: attempt to be more serious about name_morphism;
2007-02-04, by wenzelm
added full_naming;
2007-02-04, by wenzelm
tuned oracle interface;
2007-02-04, by wenzelm
added print_strings;
2007-02-04, by wenzelm
old-fashioned abstype ctyp/cterm/thm prevents accidental equality tests;
2007-02-04, by wenzelm
def_simproc(_i): tuned interface;
2007-02-04, by wenzelm
added cterm interface;
2007-02-04, by wenzelm
type simproc: explicitl dependency of morphism;
2007-02-04, by wenzelm
load morphism.ML later;
2007-02-04, by wenzelm
added the two renaming functions from my PhD
2007-02-03, by urbanc
added an infrastructure that allows the user to declare lemmas to be equivariance lemmas; the intention is to use these lemmas in automated tools but also can be employed by the user
2007-02-02, by urbanc
a few additions and deletions
2007-02-02, by nipkow
tuned;
2007-02-01, by wenzelm
proper use of PureThy.has_name_hint instead of hard-wired string'';
2007-02-01, by wenzelm
removed non-modular comment;
2007-02-01, by wenzelm
new theorem int_infinite
2007-02-01, by paulson
Fix tell_thm_deps to match changse in PureThy.
2007-01-31, by aspinall
Expose hard-wired string which was changed and broke Proof General.
2007-01-31, by aspinall
clarified error message
2007-01-31, by haftmann
clarified command annotation
2007-01-31, by haftmann
changed cong alist - now using AList operations instead of overwrite_warn
2007-01-31, by haftmann
dropped Output.update_warn
2007-01-31, by haftmann
print translation for record types with empty-sorted type variables raise Match instead of producing an error
2007-01-31, by haftmann
dropped lemma duplicates in HOL.thy
2007-01-31, by haftmann
Tidying; more debugging information. New reference unwanted_types.
2007-01-31, by paulson
Tweak preferences for PGIP interfaces. Make <askids> return theory successors instead of parents (ideally should be content elements).
2007-01-30, by aspinall
Add get_succs
2007-01-30, by aspinall
Add operations on preference tables (remove, set_default).
2007-01-30, by aspinall
adjusted to new codegen_funcgr interface
2007-01-30, by haftmann
added interface for plugging in preprocessors
2007-01-30, by haftmann
additional auxiliary here
2007-01-30, by haftmann
whitespace tuning
2007-01-30, by haftmann
dropped dead code
2007-01-30, by haftmann
shifted import order
2007-01-30, by haftmann
dropped whitespace
2007-01-30, by haftmann
changed name of interpretation linorder to order
2007-01-30, by haftmann
proper simproc_setup;
2007-01-29, by wenzelm
added get_simproc, @{simproc};
2007-01-29, by wenzelm
added interface for target_naming;
2007-01-28, by wenzelm
added simproc_setup;
2007-01-28, by wenzelm
added def_simproc(_i) -- define named simprocs;
2007-01-28, by wenzelm
updated;
2007-01-28, by wenzelm
Now deals with simples cases where the input equations contain type variables
2007-01-28, by chaieb
refined algorithm
2007-01-26, by haftmann
clarified code
2007-01-26, by haftmann
exported interface for explicit error messages
2007-01-26, by haftmann
added NestedEnvironment
2007-01-26, by haftmann
Improved debugging
2007-01-26, by paulson
Streamlined and improved debugging messages
2007-01-26, by paulson
more fixes of arithmetic for min/max.
2007-01-26, by nipkow
min/max lemmas (actually unused!)
2007-01-26, by paulson
simplification of Suc/numeral combinations with min, max
2007-01-26, by paulson
Fixed long-standing, MAJOR bug in "lt"
2007-01-26, by paulson
adjusted manual to improved treatment of overloaded constants
2007-01-26, by haftmann
Allows evaluation of min/max o numerals.
2007-01-25, by nipkow
fixed bug for OCaml bigints
2007-01-25, by haftmann
tuned
2007-01-25, by haftmann
added explicit maintainance of coregular code theorems for overloaded constants
2007-01-25, by haftmann
dropped useless stuff
2007-01-25, by haftmann
clarified code
2007-01-25, by haftmann
added explicit query function for arities to subalgebra projection
2007-01-25, by haftmann
not importing NestedEnvironment
2007-01-25, by haftmann
adjusted to changes in class package
2007-01-25, by haftmann
made executable
2007-01-25, by haftmann
improved
2007-01-25, by haftmann
fxied bug for OCaml bigints
2007-01-25, by haftmann
adjusted names
2007-01-25, by haftmann
tuned eta_contract;
2007-01-24, by wenzelm
updated timing;
2007-01-24, by wenzelm
some new lemmas
2007-01-24, by paulson
Let <loadfile> execute even while a file is open interactively.
2007-01-24, by aspinall
fixes smlnj-related problem, updated signature
2007-01-23, by krauss
added a fold up and fold down as separate functions and fixed zipto to
2007-01-23, by dixon
simplified proofs
2007-01-22, by nipkow
Included ex/Fundefs.thy in HOL-ex session
2007-01-22, by krauss
* Preliminary implementation of tail recursion
2007-01-22, by krauss
Add location_of_position. Needs work elsewhere.
2007-01-22, by aspinall
Test askref
2007-01-22, by aspinall
Expose currently open file
2007-01-22, by aspinall
Sync location with pgip.rnc, fixing attribute names
2007-01-22, by aspinall
Add askrefs, setrefs, error_with_pos
2007-01-22, by aspinall
Comments
2007-01-22, by aspinall
Comment
2007-01-22, by aspinall
Add line_of, name_of destructors.
2007-01-22, by aspinall
Added lemma nat_size[simp]: "size (n::nat) = n"
2007-01-22, by krauss
tuned;
2007-01-22, by wenzelm
improved fact references: thmref;
2007-01-21, by wenzelm
added atomic, print_int;
2007-01-21, by wenzelm
tuned ML setup;
2007-01-21, by wenzelm
* ML in Isar: improved error reporting;
2007-01-21, by wenzelm
tuned;
2007-01-21, by wenzelm
*** MESSAGE REFERS TO PREVIOUS VERSION ***
2007-01-21, by wenzelm
*** MESSAGE REFERS TO PREVIOUS VERSION ***
2007-01-21, by wenzelm
tuned comments
2007-01-21, by wenzelm
simplified ML setup;
2007-01-21, by wenzelm
use_text: added name argument;
2007-01-21, by wenzelm
moved File.use to ML_Context.use;
2007-01-21, by wenzelm
use_text: added name argument;
2007-01-21, by wenzelm
Added simproc list_neq (prompted by an application)
2007-01-21, by nipkow
Added lists-as-multisets functions
2007-01-21, by nipkow
Simple and efficient binary numerals.
2007-01-20, by wenzelm
added HOL/ex/Binary.thy;
2007-01-20, by wenzelm
tuned ML setup;
2007-01-20, by wenzelm
* ML within Isar: antiquotations;
2007-01-20, by wenzelm
added @{theory};
2007-01-20, by wenzelm
added the_context_finished;
2007-01-20, by wenzelm
Toplevel.debug: coincide with Output.debugging;
2007-01-20, by wenzelm
ML tactic: proper context for compile and runtime;
2007-01-20, by wenzelm
tuned;
2007-01-20, by wenzelm
added @{simpset};
2007-01-20, by wenzelm
added is_finished_thy;
2007-01-20, by wenzelm
Output.debug: non-strict;
2007-01-20, by wenzelm
tuned ML setup;
2007-01-20, by wenzelm
added @{clasimpset};
2007-01-20, by wenzelm
added @{claset};
2007-01-20, by wenzelm
tuned;
2007-01-19, by wenzelm
tuned;
2007-01-19, by wenzelm
renamed Isar/isar_output.ML to Thy/thy_output.ML;
2007-01-19, by wenzelm
moved ML context stuff to from Context to ML_Context;
2007-01-19, by wenzelm
results: proper context;
2007-01-19, by wenzelm
tuned Scan.extend_lexicon;
2007-01-19, by wenzelm
renamed IsarOutput to ThyOutput;
2007-01-19, by wenzelm
moved parts to spec_parse.ML;
2007-01-19, by wenzelm
removed obsolete Method;
2007-01-19, by wenzelm
renamed IsarOutput to ThyOutput;
2007-01-19, by wenzelm
added various ML setup functions (from sign.ML, pure_thy.ML);
2007-01-19, by wenzelm
removed obsolete Attribute;
2007-01-19, by wenzelm
tuned signature;
2007-01-19, by wenzelm
renamed Isar/isar_output.ML to Thy/thy_output.ML;
2007-01-19, by wenzelm
tuned signature of extend_lexicon;
2007-01-19, by wenzelm
moved ML translation interfaces to isar_cmd.ML;
2007-01-19, by wenzelm
moved thm/thms to ml_context.ML;
2007-01-19, by wenzelm
moved inst from drule.ML to old_goals.ML;
2007-01-19, by wenzelm
tuned order;
2007-01-19, by wenzelm
renamed Isar/term_style.ML to Thy/term_style.ML;
2007-01-19, by wenzelm
renamed Isar/thy_header.ML to Thy/thy_header.ML;
2007-01-19, by wenzelm
ML context and antiquotations (material from context.ML);
2007-01-19, by wenzelm
Parsers for complex specifications (material from outer_parse.ML);
2007-01-19, by wenzelm
renamed Isar/isar_output.ML to Thy/thy_output.ML;
2007-01-19, by wenzelm
moved parts of OuterParse to SpecParse;
2007-01-19, by wenzelm
moved parts of OuterParse to SpecParse;
2007-01-19, by wenzelm
HOL-Lambda: usedir -m no_brackets;
2007-01-19, by wenzelm
simplified ML setup;
2007-01-19, by wenzelm
tuned;
2007-01-19, by wenzelm
renamed IsarOutput to ThyOutput;
2007-01-19, by wenzelm
updated;
2007-01-19, by wenzelm
moved ML context stuff to from Context to ML_Context;
2007-01-19, by wenzelm
renamed IsarOutput to ThyOutput;
2007-01-19, by wenzelm
interpreter for Finite_Set.finite added
2007-01-19, by webertj
reformatted to 80 chars/line
2007-01-19, by webertj
Theorem "(x::int) dvd 1 = ( ¦x¦ = 1)" added to default simpset.
2007-01-19, by chaieb
adapted ML context operations;
2007-01-19, by wenzelm
added generic_theory_of;
2007-01-19, by wenzelm
added 'declaration' command;
2007-01-19, by wenzelm
added 'declaration' command;
2007-01-19, by wenzelm
adapted ML context operations;
2007-01-19, by wenzelm
ML context: full generic context, tuned signature;
2007-01-19, by wenzelm
updated
2007-01-19, by wenzelm
Fix pgmlsymbolsoff
2007-01-18, by aspinall
tuned a bit the proofs
2007-01-17, by urbanc
correctled left/right following of another context in zipto.
2007-01-17, by dixon
induction rules for trancl/rtrancl expressed using subsets
2007-01-17, by paulson
Deleted mk_fol_type, since the constructors can be used directly
2007-01-17, by paulson
Streamlining: removing the type argument of CombApp; abbreviating ResClause as RC
2007-01-17, by paulson
fixed typo introduced by me
2007-01-16, by urbanc
changed dictionary representation to explicit classrel witnesses
2007-01-16, by haftmann
reverted order of classrels
2007-01-16, by haftmann
cleanup
2007-01-16, by haftmann
formalisation of Crary's chapter on logical relations
2007-01-16, by urbanc
added capabilities to handle mutual inductions
2007-01-16, by urbanc
refined and added example for ExecutableRat
2007-01-16, by haftmann
introduced binding concept
2007-01-16, by haftmann
slight cleanup
2007-01-16, by haftmann
renamed locale partial_order to order
2007-01-16, by haftmann
refined and added example for ExecutableRat
2007-01-16, by haftmann
updated keywords
2007-01-16, by haftmann
added sections on mutual induction and patterns
2007-01-15, by krauss
optimized translation of HO problems
2007-01-14, by paulson
Reverted to structure representation with records.
2007-01-12, by ballarin
more term inspection
2007-01-12, by haftmann
introduced binding concept
2007-01-12, by haftmann
adjusted manual
2007-01-12, by haftmann
well-founded relations for the integers
2007-01-11, by paulson
updated to mention the automatic unfolding of constants
2007-01-11, by webertj
removed NameSpace.split -- use qualifier/base instead;
2007-01-10, by wenzelm
fixed exit: proper type check of state;
2007-01-10, by wenzelm
tuned
2007-01-10, by webertj
minor comment change
2007-01-10, by webertj
no unfolding necessary anymore (refute does that automatically now)
2007-01-10, by webertj
improved case patterns
2007-01-10, by haftmann
added undefined in cases
2007-01-10, by haftmann
named preprocessorts
2007-01-09, by haftmann
cleanup
2007-01-09, by haftmann
activated new class code
2007-01-09, by haftmann
handling for "undefined" in case expressions
2007-01-09, by haftmann
named preprocessors
2007-01-09, by haftmann
The "of 1, simplified" stopped working some time ago, leaving these simprules
2007-01-09, by paulson
More compact proof reconstruction: lines having fewer than !min_deps dependences are folded
2007-01-09, by paulson
simplified the resoution proofs
2007-01-09, by paulson
Cleanup message model: add info fatality level. Add informfileoutdated and some use of completed flag.
2007-01-09, by aspinall
Add info fatality for error messages.
2007-01-09, by aspinall
Add informfileoutdated and completed flag. This makes the PGIP messages match the Broker states.
2007-01-09, by aspinall
slight cleanups
2007-01-09, by haftmann
improved names
2007-01-09, by haftmann
proper node names
2007-01-09, by haftmann
slight cleanup
2007-01-09, by haftmann
improved variable name handling
2007-01-09, by haftmann
moved variable environments here
2007-01-09, by haftmann
moved a lot to codegen_func.ML
2007-01-09, by haftmann
typo
2007-01-09, by haftmann
added map_abs_vars
2007-01-09, by haftmann
tuned signature;
2007-01-08, by wenzelm
print functions for typs and terms added
2007-01-07, by webertj
Be more chatty in PGIP file operations.
2007-01-07, by aspinall
A few lemmas about relative primes when dividing trough gcd
2007-01-06, by chaieb
A few theorems on integer divisibily.
2007-01-06, by chaieb
Introduction of a bound on DEPTH_ITER, to prevent the meson method from running forever
2007-01-05, by paulson
reverted to v1.60 (PolyML 4.1.3 still has the wrong signature for Array.modifyi)
2007-01-05, by webertj
added codegen_func.ML
2007-01-05, by haftmann
non-layout-sensitive syntax for Haskell
2007-01-05, by haftmann
some cleanup
2007-01-05, by haftmann
primitive definitions are always eta-expanded
2007-01-05, by haftmann
added block_enclose
2007-01-05, by haftmann
added CodeEval
2007-01-05, by haftmann
dealing with ml_string and char instances
2007-01-05, by haftmann
dealing with ml_string combinators
2007-01-05, by haftmann
adaptions
2007-01-05, by haftmann
removed Toplevel.print_exn hook -- existing error_msg_fn does the job;
2007-01-05, by wenzelm
RAW-ProofGeneral: more dependencies;
2007-01-05, by wenzelm
Proof.context now sent to watcher and used in type inference step of proof reconstruction
2007-01-05, by paulson
tuned msg;
2007-01-04, by wenzelm
removed obsolete ProofGeneral/syntax_standalone.ML;
2007-01-04, by wenzelm
approximate Syntax.read_int/nat by Int.fromString -- avoids dependency on Syntax module;
2007-01-04, by wenzelm
added mk_simproc': tuned interface;
2007-01-04, by wenzelm
clarification
2007-01-04, by haftmann
dropped function theorems are considered as deleted
2007-01-04, by haftmann
examples for evaluation oracle
2007-01-04, by haftmann
fixed eval oracle
2007-01-04, by haftmann
Be more chatty in PGIP file operations.proof_general_pgip.ML
2007-01-04, by aspinall
broken error handling for command syntax -- reverted to revision 1.9;
2007-01-04, by wenzelm
Use warning fatality
2007-01-04, by aspinall
Add warning fatality
2007-01-04, by aspinall
improvements to proof reconstruction. Some files loaded in a different order
2007-01-04, by paulson
using Array.modifyi (no functional change)
2007-01-04, by webertj
run as RAW session;
2007-01-04, by wenzelm
removed obsolete option -C;
2007-01-04, by wenzelm
removed obsolete Pure-copied target;
2007-01-04, by wenzelm
updated manual
2007-01-04, by haftmann
updated manual
2007-01-04, by haftmann
obsolete sign_of calls removed
2007-01-04, by webertj
fixed output
2007-01-04, by haftmann
different handling of eta expansion
2007-01-04, by haftmann
eta-expansion now only to common maximum number of arguments
2007-01-04, by haftmann
clarified code
2007-01-04, by haftmann
more term examples
2007-01-04, by haftmann
eliminated Option.app
2007-01-04, by haftmann
constants are unfolded, universal quantifiers are stripped, some minor changes
2007-01-04, by webertj
Fix error reporting in Emacs to also match Isar command failure exactly.
2007-01-03, by aspinall
Use Isar toplevel print_exn_fn for generating error responses instead of Output.error_msg.
2007-01-03, by aspinall
Expose command failure recovery code for top level.
2007-01-03, by aspinall
Selected functions from syntax module
2007-01-03, by aspinall
x-symbol is no longer switched off in the ATP linkup
2007-01-03, by paulson
Improvements to proof reconstruction. Now "fixes" is inserted
2007-01-03, by paulson
Contains old Tools/ATP/AtpCommunication.ML, plus proof reconstruction
2007-01-03, by paulson
first version of structured proof reconstruction
2007-01-03, by paulson
Morphism.fact;
2007-01-02, by wenzelm
Term.lambda: abstract over arbitrary closed terms;
2007-01-02, by wenzelm
Add standalone file to help porters
2006-12-31, by aspinall
Quote arguments in PGIP exceptions. Tune comment.
2006-12-31, by aspinall
Initialise parser at startup. Remove some obsolete ProofGeneral.XXX outer syntax, mapping PGIP commands directly to Isar.
2006-12-31, by aspinall
Fix diagnostic kind (*are* spuriouscmd). Add init to get right table for logic at startup. Use theoryitem as default for unrecognised command.
2006-12-31, by aspinall
removed dead code;
2006-12-30, by wenzelm
removed conditional combinator;
2006-12-30, by wenzelm
removed conditional combinator;
2006-12-30, by wenzelm
refrain from setting ml_prompts again;
2006-12-30, by wenzelm
removed misleading OuterLex.eq_token;
2006-12-30, by wenzelm
pretty_statement: more careful handling of name_hint;
2006-12-30, by wenzelm
added has_name_hint;
2006-12-30, by wenzelm
removed obsolete name_hint handling;
2006-12-30, by wenzelm
removed conditional combinator;
2006-12-30, by wenzelm
removed obsolete support for polyml-4.9.1;
2006-12-30, by wenzelm
* Proof General: proper undo of final 'end'; discontinued Isabelle/classic;
2006-12-30, by wenzelm
inform_file_processed: Toplevel.init_empty;
2006-12-30, by wenzelm
refined notion of empty toplevel, admits undo of 'end';
2006-12-30, by wenzelm
Toplevel.init_state;
2006-12-30, by wenzelm
removed obsolete 'clear_undos';
2006-12-30, by wenzelm
removed obsolete clear_undos_theory;
2006-12-30, by wenzelm
major restructurings
2006-12-29, by haftmann
cleanup
2006-12-29, by haftmann
improved print of constructors in OCaml
2006-12-29, by haftmann
changed syntax for axclass attach
2006-12-29, by haftmann
removed obsolete cond_add_path;
2006-12-29, by wenzelm
removed obsolete context_thy etc.;
2006-12-29, by wenzelm
removed obsolete init_pgip;
2006-12-29, by wenzelm
removed obsolete init_context;
2006-12-29, by wenzelm
obsolete (cf. ProofGeneral/proof_general_emacs.ML);
2006-12-29, by wenzelm
tuned;
2006-12-29, by wenzelm
signed_string_of_int;
2006-12-29, by wenzelm
added proper header;
2006-12-29, by wenzelm
added signed_string_of_int (pruduces proper - instead of SML's ~);
2006-12-29, by wenzelm
removed obsolete proof_general.ML;
2006-12-29, by wenzelm
minor tuning;
2006-12-29, by wenzelm
tuned specifications/proofs;
2006-12-29, by wenzelm
replaced Sign.classes by Sign.all_classes (topologically sorted);
2006-12-29, by wenzelm
renamed Graph.project to Graph.subgraph;
2006-12-29, by wenzelm
replaced Sign.classes by Sign.all_classes (topologically sorted);
2006-12-29, by wenzelm
renamed project to subgraph, improved presentation, avoided unnecessary evaluation of predicate;
2006-12-29, by wenzelm
Sorts.minimal_classes;
2006-12-29, by wenzelm
classes: more direct way to achieve topological sorting;
2006-12-29, by wenzelm
replaced classes by all_classes (topologically sorted);
2006-12-29, by wenzelm
replaced Sign.classes by Sign.all_classes (topologically sorted);
2006-12-29, by wenzelm
Enable new Proof General code again after SML/NJ compatibility fixes by Florian.
2006-12-29, by aspinall
Typo in last commit
2006-12-29, by aspinall
explicit construction of operational classes
2006-12-29, by haftmann
added handling for explicit classrel witnesses
2006-12-29, by haftmann
``classes`` now returns classes in topological order
2006-12-29, by haftmann
dropped some bookkeeping
2006-12-29, by haftmann
simplified class_package
2006-12-29, by haftmann
use_ml: reverted to simple output (Poly/ML changed);
2006-12-29, by wenzelm
removed private files
2006-12-28, by haftmann
tuned;
2006-12-28, by wenzelm
removed nospaces (Char.isSpace does not conform to Isabelle conventions);
2006-12-28, by wenzelm
tuned msg;
2006-12-28, by wenzelm
inlined nospaces (from library.ML);
2006-12-28, by wenzelm
added
2006-12-28, by haftmann
some clarifications
2006-12-27, by haftmann
different handling of type variable names
2006-12-27, by haftmann
added split
2006-12-27, by haftmann
fixed misleading error message
2006-12-27, by haftmann
dropped section header
2006-12-27, by haftmann
added OCaml code generation (without dictionaries)
2006-12-27, by haftmann
removed Haskell reserved words
2006-12-27, by haftmann
removed Main.thy
2006-12-27, by haftmann
moved code generator product setup here
2006-12-27, by haftmann
added code generator test theory
2006-12-27, by haftmann
explizit serialization for Haskell id
2006-12-27, by haftmann
removed code generation stuff belonging to other theories
2006-12-27, by haftmann
moved code generator bool setup here
2006-12-27, by haftmann
exported explicit equality on tokens
2006-12-27, by haftmann
made SML/NJ happy
2006-12-27, by haftmann
revised for new make_clauses
2006-12-22, by paulson
tidying the ATP communications
2006-12-22, by paulson
string primtives
2006-12-22, by paulson
deactivated test for the moment
2006-12-22, by haftmann
fixed typo in comment
2006-12-22, by paulson
Experimenting with interpretations of "definition".
2006-12-22, by ballarin
clarified code
2006-12-21, by haftmann
dropped superfluos code
2006-12-21, by haftmann
code clarifications
2006-12-21, by haftmann
import path made absolute
2006-12-21, by haftmann
added code lemmas for quantification over bounded nats
2006-12-21, by haftmann
Disable new Proof General code until SML/NJ compile fixed.
2006-12-21, by aspinall
Use new Proof General code by default [see comment for reverting]
2006-12-20, by aspinall
change from "Array" to "Vector"
2006-12-20, by paulson
add lemmas Standard_starfun(2)_iff
2006-12-19, by huffman
Missing elements from doc_markup_elements
2006-12-19, by aspinall
Remove obsolete prefixes from error and warning messages.
2006-12-19, by aspinall
added isatool codegen
2006-12-18, by haftmann
dropped CodegenPackage.const_of_idf
2006-12-18, by haftmann
improvements in syntax handling
2006-12-18, by haftmann
added Thyname.* and * constant expressions
2006-12-18, by haftmann
introduces "__" naming policy
2006-12-18, by haftmann
switched argument order in *.syntax lifters
2006-12-18, by haftmann
added gen_reflection_tac
2006-12-18, by haftmann
now testing executable content of nearly all HOL
2006-12-18, by haftmann
dropped debug cmd
2006-12-18, by haftmann
explicit nonfix declaration for ML "subset"
2006-12-18, by haftmann
dropped two inline directives
2006-12-18, by haftmann
introduced abstract view on number expressions in hologic.ML
2006-12-18, by haftmann
whitespace fix
2006-12-18, by haftmann
added code generation syntax for some char combinators
2006-12-18, by haftmann
infix syntax for generated code for composition
2006-12-18, by haftmann
new-style oracle setup
2006-12-18, by haftmann
added functions tutorial
2006-12-18, by haftmann
Add abstraction for objtypes and documents.
2006-12-17, by aspinall
removed Hyperreal/HyperArith.thy and Hyperreal/HyperPow.thy
2006-12-16, by huffman
moved several theorems; rearranged theory dependencies
2006-12-16, by huffman
hypreal_of_hypnat abbreviates more general of_hypnat
2006-12-16, by huffman
tracing instead of warning
2006-12-15, by webertj
updated;
2006-12-15, by wenzelm
removed obsolete assert;
2006-12-15, by wenzelm
renamed LocalTheory.assert to affirm;
2006-12-15, by wenzelm
tuned -- accomodate Alice;
2006-12-15, by wenzelm
avoid conflict with Alice keywords: renamed pack -> implode, unpack -> explode, any -> many, avoided assert;
2006-12-15, by wenzelm
remove Hyperreal/fuf.ML
2006-12-14, by huffman
remove commented section
2006-12-14, by huffman
remove ultra tactic and redundant FreeUltrafilterNat lemmas
2006-12-14, by huffman
declare insert_iff [simp]
2006-12-14, by huffman
activated improved use_ml, which captures output and reports source positions;
2006-12-14, by wenzelm
tuned;
2006-12-14, by wenzelm
prove hyperpow_realpow using transfer
2006-12-14, by huffman
remove usage of ultra tactic
2006-12-14, by huffman
add lemmas singleton and insert_iff
2006-12-14, by huffman
generalized type of hyperpow; removed hcpow
2006-12-14, by huffman
redefine hSuc as *f* Suc, and move to HyperNat.thy
2006-12-14, by huffman
proper use of IntInf instead of InfInf;
2006-12-14, by wenzelm
defs/notes: more robust transitivity reasoning;
2006-12-14, by wenzelm
added trans_terms/props;
2006-12-14, by wenzelm
locale: print context for begin;
2006-12-14, by wenzelm
remove references to star_n and FreeUltrafilterNat; new proof of NSBseq_Bseq
2006-12-14, by huffman
remove uses of star_n and FreeUltrafilterNat
2006-12-13, by huffman
remove use of FreeUltrafilterNat
2006-12-13, by huffman
added lemmas about hRe, hIm, HComplex; removed all uses of star_n
2006-12-13, by huffman
fixed type
2006-12-13, by haftmann
added stub for OCaml serializer
2006-12-13, by haftmann
cleanup
2006-12-13, by haftmann
whitespace correction
2006-12-13, by haftmann
clarifed comment
2006-12-13, by haftmann
dropped FIXME comment
2006-12-13, by haftmann
clarified character setup
2006-12-13, by haftmann
remove references to star_n
2006-12-13, by huffman
SComplex abbreviates Standard
2006-12-13, by huffman
simplified mk/dest_numeral (cf. mk/dest_binum of 1.65);
2006-12-13, by wenzelm
removed legacy ML bindings;
2006-12-13, by wenzelm
updated;
2006-12-13, by wenzelm
tuned signature;
2006-12-13, by wenzelm
internal_abbrev: observe print mode;
2006-12-13, by wenzelm
target_abbrev: internal mode for abbrevs;
2006-12-13, by wenzelm
edge: actually apply operation!
2006-12-13, by wenzelm
tuned;
2006-12-13, by wenzelm
authentic syntax for number_of
2006-12-13, by haftmann
introduced mk/dest_numeral/number for mk/dest_binum etc.
2006-12-13, by haftmann
fixed syntax for bounded quantification
2006-12-13, by haftmann
dropped superfluous header
2006-12-13, by haftmann
clarified error message
2006-12-13, by krauss
nat type now has a size functin => no longer needed as special case
2006-12-13, by krauss
simplified
2006-12-13, by krauss
local_abbrev: proper fix/declare of local entities;
2006-12-13, by wenzelm
Deleted the unused type argument of UVar
2006-12-13, by paulson
tuned comments;
2006-12-13, by wenzelm
added IsarAdvanced/Functions
2006-12-13, by krauss
generalized some lemmas; removed redundant lemmas; cleaned up some proofs
2006-12-13, by huffman
remove uses of scaleR infix syntax; add lemma Reals_number_of
2006-12-13, by huffman
tuned;
2006-12-12, by wenzelm
add_abbrev: removed Assumption.add_assms (danger of inconsistent naming);
2006-12-12, by wenzelm
updated;
2006-12-12, by wenzelm
simplified unlocalize_mixfix;
2006-12-12, by wenzelm
removed is_class -- handled internally;
2006-12-12, by wenzelm
notation: Term.equiv_types;
2006-12-12, by wenzelm
abbrev: tuned signature;
2006-12-12, by wenzelm
tuned expand_term;
2006-12-12, by wenzelm
classified show/thus as prf_asm_goal, which is usually hilited in PG;
2006-12-12, by wenzelm
tuned expand_binds;
2006-12-12, by wenzelm
tuned error messages;
2006-12-12, by wenzelm
added equiv_types;
2006-12-12, by wenzelm
add_abbrev: tuned signature;
2006-12-12, by wenzelm
added expand_term_frees;
2006-12-12, by wenzelm
abbreviate: tuned signature;
2006-12-12, by wenzelm
LocalTheory.abbrev;
2006-12-12, by wenzelm
removed redundant constants and lemmas
2006-12-12, by huffman
additions to HOL-Complex
2006-12-12, by huffman
Removal of the "keep_types" flag: we always keep types!
2006-12-12, by paulson
make SML/NJ happy;
2006-12-12, by wenzelm
made SML/NJ happy;
2006-12-12, by wenzelm
consistent naming for FreeUltrafilterNat lemmas; cleaned up
2006-12-12, by huffman
cleaned up; generalized some proofs
2006-12-12, by huffman
fix assumptions on NSDERIV_quotient
2006-12-12, by huffman
changed (ns)deriv to take functions of type 'a::real_normed_field => 'a
2006-12-12, by huffman
generalize some theorems
2006-12-12, by huffman
add type annotation
2006-12-12, by huffman
read_xnum: return leading_zeros, radix;
2006-12-12, by wenzelm
authentic syntax for Pls/Min/Bit;
2006-12-12, by wenzelm
authentic syntax for Pls/Min/Bit;
2006-12-12, by wenzelm
binary numerals: restricted to actual abstract syntax;
2006-12-12, by wenzelm
Hyperreal/FrechetDeriv.thy
2006-12-12, by huffman
theory of Frechet derivatives
2006-12-12, by huffman
specials: include single quote;
2006-12-11, by wenzelm
xstr: disallow backslashes;
2006-12-11, by wenzelm
advanced translation functions: Proof.context;
2006-12-11, by wenzelm
advanced translation functions: Proof.context;
2006-12-11, by wenzelm
added improved versions of use_text/file (still inactive);
2006-12-11, by wenzelm
added use_file;
2006-12-11, by wenzelm
load secure.ML after symbol.ML, when default output is active;
2006-12-11, by wenzelm
ordered lists instead of tables for resolving hyps; speedup
2006-12-11, by webertj
less
more
|
(0)
-10000
-3000
-1000
-480
+480
+1000
+3000
+10000
+30000
tip