Theory Eq

(*:maxLineLen=78:*)

theory Eq
imports Base
begin

chapter ‹Equational reasoning›

text ‹
  Equality is one of the most fundamental concepts of mathematics. The
  Isabelle/Pure logic (\chref{ch:logic}) provides a builtin relation ≡ :: α ⇒
  α ⇒ prop› that expresses equality of arbitrary terms (or propositions) at
  the framework level, as expressed by certain basic inference rules
  (\secref{sec:eq-rules}).

  Equational reasoning means to replace equals by equals, using reflexivity
  and transitivity to form chains of replacement steps, and congruence rules
  to access sub-structures. Conversions (\secref{sec:conv}) provide a
  convenient framework to compose basic equational steps to build specific
  equational reasoning tools.

  Higher-order matching is able to provide suitable instantiations for giving
  equality rules, which leads to the versatile concept of λ›-term rewriting
  (\secref{sec:rewriting}). Internally this is based on the general-purpose
  Simplifier engine of Isabelle, which is more specific and more efficient
  than plain conversions.

  Object-logics usually introduce specific notions of equality or equivalence,
  and relate it with the Pure equality. This enables to re-use the Pure tools
  for equational reasoning for particular object-logic connectives as well.
›


section ‹Basic equality rules \label{sec:eq-rules}›

text ‹
  Isabelle/Pure uses ≡› for equality of arbitrary terms, which includes
  equivalence of propositions of the logical framework. The conceptual
  axiomatization of the constant ≡ :: α ⇒ α ⇒ prop› is given in
  \figref{fig:pure-equality}. The inference kernel presents slightly different
  equality rules, which may be understood as derived rules from this minimal
  axiomatization. The Pure theory also provides some theorems that express the
  same reasoning schemes as theorems that can be composed like object-level
  rules as explained in \secref{sec:obj-rules}.

  For example, MLThm.symmetric as Pure inference is an ML function that
  maps a theorem th› stating t ≡ u› to one stating u ≡ t›. In contrast,
  @{thm [source] Pure.symmetric} as Pure theorem expresses the same reasoning
  in declarative form. If used like th [THEN Pure.symmetric]› in Isar source
  notation, it achieves a similar effect as the ML inference function,
  although the rule attribute @{attribute THEN} or ML operator MLop RS
  involve the full machinery of higher-order unification (modulo
  βη›-conversion) and lifting of ⋀/⟹› contexts.
›

text %mlref ‹
  \begin{mldecls}
  @{define_ML Thm.reflexive: "cterm -> thm"} \\
  @{define_ML Thm.symmetric: "thm -> thm"} \\
  @{define_ML Thm.transitive: "thm -> thm -> thm"} \\
  @{define_ML Thm.abstract_rule: "string -> cterm -> thm -> thm"} \\
  @{define_ML Thm.combination: "thm -> thm -> thm"} \\[0.5ex]
  @{define_ML Thm.equal_intr: "thm -> thm -> thm"} \\
  @{define_ML Thm.equal_elim: "thm -> thm -> thm"} \\
  \end{mldecls}

  See also 🗏‹~~/src/Pure/thm.ML› for further description of these inference
  rules, and a few more for primitive β› and η› conversions. Note that α›
  conversion is implicit due to the representation of terms with de-Bruijn
  indices (\secref{sec:terms}).
›


section ‹Conversions \label{sec:conv}›

text ‹
  The classic article cite"paulson:1983" introduces the concept of
  conversion for Cambridge LCF. This was historically important to implement
  all kinds of ``simplifiers'', but the Isabelle Simplifier is done quite
  differently, see cite‹\S9.3› in "isabelle-isar-ref".
›

text %mlref ‹
  \begin{mldecls}
  @{define_ML_structure Conv} \\
  @{define_ML_type conv} \\
  @{define_ML Simplifier.asm_full_rewrite : "Proof.context -> conv"} \\
  \end{mldecls}

   ML_structureConv is a library of combinators to build conversions,
  over type ML_typeconv (see also 🗏‹~~/src/Pure/conv.ML›). This is one
  of the few Isabelle/ML modules that are usually used with ‹open›: finding
  examples works by searching for ``‹open Conv›'' instead of ``‹Conv.›''.

   MLSimplifier.asm_full_rewrite invokes the Simplifier as a
  conversion. There are a few related operations, corresponding to the various
  modes of simplification.
›


section ‹Rewriting \label{sec:rewriting}›

text ‹
  Rewriting normalizes a given term (theorem or goal) by replacing instances
  of given equalities t ≡ u› in subterms. Rewriting continues until no
  rewrites are applicable to any subterm. This may be used to unfold simple
  definitions of the form f x1 … xn ≡ u›, but is slightly more general than
  that. ›

text %mlref ‹
  \begin{mldecls}
  @{define_ML rewrite_rule: "Proof.context -> thm list -> thm -> thm"} \\
  @{define_ML rewrite_goals_rule: "Proof.context -> thm list -> thm -> thm"} \\
  @{define_ML rewrite_goal_tac: "Proof.context -> thm list -> int -> tactic"} \\
  @{define_ML rewrite_goals_tac: "Proof.context -> thm list -> tactic"} \\
  @{define_ML fold_goals_tac: "Proof.context -> thm list -> tactic"} \\
  \end{mldecls}

   MLrewrite_rule~ctxt rules thm› rewrites the whole theorem by the
  given rules.

   MLrewrite_goals_rule~ctxt rules thm› rewrites the outer premises of
  the given theorem. Interpreting the same as a goal state
  (\secref{sec:tactical-goals}) it means to rewrite all subgoals (in the same
  manner as MLrewrite_goals_tac).

   MLrewrite_goal_tac~ctxt rules i› rewrites subgoal i› by the given
  rewrite rules.

   MLrewrite_goals_tac~ctxt rules› rewrites all subgoals by the given
  rewrite rules.

   MLfold_goals_tac~ctxt rules› essentially uses MLrewrite_goals_tac
  with the symmetric form of each member of rules›, re-ordered to fold longer
  expression first. This supports to idea to fold primitive definitions that
  appear in expended form in the proof state.
›

end